mathlib3 documentation

category_theory.adjunction.limits

Adjunctions and limits #

THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.

A left adjoint preserves colimits (category_theory.adjunction.left_adjoint_preserves_colimits), and a right adjoint preserves limits (category_theory.adjunction.right_adjoint_preserves_limits).

Equivalences create and reflect (co)limits. (category_theory.adjunction.is_equivalence_creates_limits, category_theory.adjunction.is_equivalence_creates_colimits, category_theory.adjunction.is_equivalence_reflects_limits, category_theory.adjunction.is_equivalence_reflects_colimits,)

In category_theory.adjunction.cocones_iso we show that when F ⊣ G, the functor associating to each Y the cocones over K ⋙ F with cone point Y is naturally isomorphic to the functor associating to each Y the cocones over K with cone point G.obj Y.

The right adjoint of cocones.functoriality K F : cocone K ⥤ cocone (K ⋙ F).

Auxiliary definition for functoriality_is_left_adjoint.

Equations

The unit for the adjunction for cocones.functoriality K F : cocone K ⥤ cocone (K ⋙ F).

Auxiliary definition for functoriality_is_left_adjoint.

Equations
@[simp]
theorem category_theory.adjunction.functoriality_unit_app_hom {C : Type u₁} [category_theory.category C] {D : Type u₂} [category_theory.category D] {F : C D} {G : D C} (adj : F G) {J : Type u} [category_theory.category J] (K : J C) (c : category_theory.limits.cocone K) :
((adj.functoriality_unit K).app c).hom = adj.unit.app c.X

The counit for the adjunction for cocones.functoriality K F : cocone K ⥤ cocone (K ⋙ F).

Auxiliary definition for functoriality_is_left_adjoint.

Equations
@[simp]

The left adjoint of cones.functoriality K G : cone K ⥤ cone (K ⋙ G).

Auxiliary definition for functoriality_is_right_adjoint.

Equations
@[simp]
theorem category_theory.adjunction.functoriality_unit'_app_hom {C : Type u₁} [category_theory.category C] {D : Type u₂} [category_theory.category D] {F : C D} {G : D C} (adj : F G) {J : Type u} [category_theory.category J] (K : J D) (c : category_theory.limits.cone (K G)) :
((adj.functoriality_unit' K).app c).hom = adj.unit.app c.X

The unit for the adjunction forcones.functoriality K G : cone K ⥤ cone (K ⋙ G).

Auxiliary definition for functoriality_is_right_adjoint.

Equations

The counit for the adjunction forcones.functoriality K G : cone K ⥤ cone (K ⋙ G).

Auxiliary definition for functoriality_is_right_adjoint.

Equations
@[simp]
def category_theory.adjunction.cocones_iso_component_hom {C : Type u₁} [category_theory.category C] {D : Type u₂} [category_theory.category D] {F : C D} {G : D C} (adj : F G) {J : Type u} [category_theory.category J] {K : J C} (Y : D) (t : ((category_theory.cocones J D).obj (opposite.op (K F))).obj Y) :

auxiliary construction for cocones_iso

Equations
@[simp]
theorem category_theory.adjunction.cocones_iso_component_hom_app {C : Type u₁} [category_theory.category C] {D : Type u₂} [category_theory.category D] {F : C D} {G : D C} (adj : F G) {J : Type u} [category_theory.category J] {K : J C} (Y : D) (t : ((category_theory.cocones J D).obj (opposite.op (K F))).obj Y) (j : J) :
(adj.cocones_iso_component_hom Y t).app j = (adj.hom_equiv (K.obj j) Y) (t.app j)
def category_theory.adjunction.cocones_iso_component_inv {C : Type u₁} [category_theory.category C] {D : Type u₂} [category_theory.category D] {F : C D} {G : D C} (adj : F G) {J : Type u} [category_theory.category J] {K : J C} (Y : D) (t : (G (category_theory.cocones J C).obj (opposite.op K)).obj Y) :

auxiliary construction for cocones_iso

Equations
@[simp]
theorem category_theory.adjunction.cocones_iso_component_inv_app {C : Type u₁} [category_theory.category C] {D : Type u₂} [category_theory.category D] {F : C D} {G : D C} (adj : F G) {J : Type u} [category_theory.category J] {K : J C} (Y : D) (t : (G (category_theory.cocones J C).obj (opposite.op K)).obj Y) (j : J) :
(adj.cocones_iso_component_inv Y t).app j = ((adj.hom_equiv (K.obj j) Y).symm) (t.app j)
def category_theory.adjunction.cones_iso_component_hom {C : Type u₁} [category_theory.category C] {D : Type u₂} [category_theory.category D] {F : C D} {G : D C} (adj : F G) {J : Type u} [category_theory.category J] {K : J D} (X : Cᵒᵖ) (t : (F.op (category_theory.cones J D).obj K).obj X) :

auxiliary construction for cones_iso

Equations
@[simp]
theorem category_theory.adjunction.cones_iso_component_hom_app {C : Type u₁} [category_theory.category C] {D : Type u₂} [category_theory.category D] {F : C D} {G : D C} (adj : F G) {J : Type u} [category_theory.category J] {K : J D} (X : Cᵒᵖ) (t : (F.op (category_theory.cones J D).obj K).obj X) (j : J) :
(adj.cones_iso_component_hom X t).app j = (adj.hom_equiv (opposite.unop X) (K.obj j)) (t.app j)
@[simp]
theorem category_theory.adjunction.cones_iso_component_inv_app {C : Type u₁} [category_theory.category C] {D : Type u₂} [category_theory.category D] {F : C D} {G : D C} (adj : F G) {J : Type u} [category_theory.category J] {K : J D} (X : Cᵒᵖ) (t : ((category_theory.cones J C).obj (K G)).obj X) (j : J) :
(adj.cones_iso_component_inv X t).app j = ((adj.hom_equiv (opposite.unop X) (K.obj j)).symm) (t.app j)
def category_theory.adjunction.cones_iso_component_inv {C : Type u₁} [category_theory.category C] {D : Type u₂} [category_theory.category D] {F : C D} {G : D C} (adj : F G) {J : Type u} [category_theory.category J] {K : J D} (X : Cᵒᵖ) (t : ((category_theory.cones J C).obj (K G)).obj X) :

auxiliary construction for cones_iso

Equations

When F ⊣ G, the functor associating to each Y the cocones over K ⋙ F with cone point Y is naturally isomorphic to the functor associating to each Y the cocones over K with cone point G.obj Y.

Equations
def category_theory.adjunction.cones_iso {C : Type u₁} [category_theory.category C] {D : Type u₂} [category_theory.category D] {F : C D} {G : D C} (adj : F G) {J : Type u} [category_theory.category J] {K : J D} :

When F ⊣ G, the functor associating to each X the cones over K with cone point F.op.obj X is naturally isomorphic to the functor associating to each X the cones over K ⋙ G with cone point X.

Equations