X-Git-Url: http://git.megacz.com/?a=blobdiff_plain;ds=sidebyside;f=src%2FAdjoints_ch9.v;h=b4361ef9f2f0948084cdb2c55cf917c8ed629f6d;hb=422dab8d300548c294b95c0f4bbf27aecadbd745;hp=df870eb947210f3aa79789acd6a7b4e772ace464;hpb=ff3003c261295c60d367580b6700396102eb5a9c;p=coq-categories.git diff --git a/src/Adjoints_ch9.v b/src/Adjoints_ch9.v index df870eb..b4361ef 100644 --- a/src/Adjoints_ch9.v +++ b/src/Adjoints_ch9.v @@ -1,5 +1,5 @@ Generalizable All Variables. -Require Import Preamble. +Require Import Notations. Require Import Categories_ch1_3. Require Import Functors_ch1_4. Require Import Isomorphisms_ch1_5. @@ -26,8 +26,8 @@ Notation "'η'" := (adj_unit _). (* Lemma homset_adjunction `(C:ECategory(V:=V))`(D:ECategory(V:=V))(L:Func C D)(R:Func D C) : (L -| R) - -> RepresentableFunctorºᑭ _ _ >>>> YonedaBiFunctor D ≃ - RepresentableFunctorºᑭ _ _ >>>> YonedaBiFunctor C. + -> HomFunctorºᑭ _ _ >>>> YonedaBiFunctor D ≃ + HomFunctorºᑭ _ _ >>>> YonedaBiFunctor C. *) (* adjuncts are unique up to natural iso *) (* adjuncts compose *)