X-Git-Url: http://git.megacz.com/?p=coq-categories.git;a=blobdiff_plain;f=src%2FFreydCategories.v;h=8b921dfb79f7a14d2083c9226e3f3450697d359a;hp=c269e5064cf970e22bc0970ddf1e995dd5676c5a;hb=658181bed516646957267b055341d9d4b197ed0d;hpb=e928451c4c45cdbdd975bbfb229e8cc2616b8194 diff --git a/src/FreydCategories.v b/src/FreydCategories.v index c269e50..8b921df 100644 --- a/src/FreydCategories.v +++ b/src/FreydCategories.v @@ -3,8 +3,7 @@ (*******************************************************************************) Generalizable All Variables. -Require Import Preamble. -Require Import General. +Require Import Notations. Require Import Categories_ch1_3. Require Import Functors_ch1_4. Require Import Isomorphisms_ch1_5. @@ -26,7 +25,7 @@ Class FreydCategory `(C:CartesianCat(Ob:=Ob)(C:=C1)(bin_obj':=bobj)) (* a premonoidal category K with the same objects (its unit object is 1 because the functor is both IIO and strict) *) - `(K:PreMonoidalCat(Ob:=Ob)(bin_obj':=bobj)(I:=@one _ _ _ C)) + `(K:PreMonoidalCat(Ob:=Ob)(bin_obj':=bobj)(I:=pmon_I C)) (* an identity-on-objects functor J:C->Z(K) *) := { fc_J : Functor C (Center_is_Monoidal K) (fun x => x) @@ -36,7 +35,7 @@ Class FreydCategory (* and strict (meaning the functor's coherence maps are identities) *) ; fc_strict_first : forall a b, #(mf_first(PreMonoidalFunctor:=fc_mf_J) a b) ~~ id _ (* mf_consistent gives us mf_second *) -(* ; fc_strict_id : #(mf_i(PreMonoidalFunctor:=fc_mf_J)) ~~ id _*) + ; fc_strict_id : #(mf_i(PreMonoidalFunctor:=fc_mf_J)) ~~ id _ ; fc_C := C ; fc_K := K