X-Git-Url: http://git.megacz.com/?p=coq-categories.git;a=blobdiff_plain;f=src%2FRepresentableStructure_ch7_2.v;h=f318c7c3e849758b21db040abcf564dea263057d;hp=da3f519e76c7f9a629535569f63d9aed9ddc0b64;hb=21607813788d83fb58ce128df442a4ee3edfbdaf;hpb=00b060e4854e5a1ba01746be44ac9deb49d7fbf5 diff --git a/src/RepresentableStructure_ch7_2.v b/src/RepresentableStructure_ch7_2.v index da3f519..f318c7c 100644 --- a/src/RepresentableStructure_ch7_2.v +++ b/src/RepresentableStructure_ch7_2.v @@ -16,6 +16,9 @@ Require Import NaturalTransformations_ch7_4. Require Import NaturalIsomorphisms_ch7_5. Require Import MonoidalCategories_ch7_8. Require Import Coherence_ch7_8. +Require Import BinoidalCategories. +Require Import PreMonoidalCategories. +Require Import MonoidalCategories_ch7_8. Section RepresentableStructure. Context `(ec:ECategory(mn:=mn)(V:=V)). @@ -106,6 +109,7 @@ Section RepresentableStructure. apply hom_covariant_distributes. Defined. + (* Lemma undo_homfunctor `(f:a~~{ec}~~>b) : f ~~ eid _ >>> (HomFunctor a \ f). simpl. setoid_rewrite <- associativity. @@ -143,7 +147,7 @@ Section RepresentableStructure. set (@eqv_equivalence) as qmt. apply qmt. Qed. - + *) End RepresentableStructure. Opaque HomFunctor.