Skip to content

Commit

Permalink
chore(category_theory/limits/limits): Add missing lemmas
Browse files Browse the repository at this point in the history
  • Loading branch information
jcommelin committed Dec 17, 2018
1 parent 9506e6c commit 4b9f9a6
Showing 1 changed file with 17 additions and 0 deletions.
17 changes: 17 additions & 0 deletions category_theory/limits/limits.lean
Expand Up @@ -5,6 +5,7 @@
import category_theory.whiskering
import category_theory.yoneda
import category_theory.limits.cones
import tactic.squeeze

open category_theory category_theory.category category_theory.functor

Expand Down Expand Up @@ -362,6 +363,14 @@ lemma limit.map_pre {K : Type v} [small_category K] [has_limits_of_shape K C] (E
lim.map α ≫ limit.pre G E = limit.pre F E ≫ lim.map (whisker_left E α) :=
by ext; rw [assoc, limit.pre_π, lim.map_π, assoc, lim.map_π, ←assoc, limit.pre_π]; refl

lemma limit.map_pre' {K : Type v} [small_category K] [has_limits_of_shape.{u v} K C]
(F : J ⥤ C) {E₁ E₂ : K ⥤ J} (α : E₁ ⟹ E₂) :
limit.pre F E₂ = limit.pre F E₁ ≫ lim.map (whisker_right α F) :=
by ext1; simp [(category.assoc _ _ _ _).symm]

lemma limit.id_pre (F : J ⥤ C) :
limit.pre F (functor.id _) = lim.map (functor.left_unitor F).inv := by tidy

lemma limit.map_post {D : Type u'} [category.{u' v} D] [has_limits_of_shape J D] (H : C ⥤ D) :
/- H (limit F) ⟶ H (limit G) ⟶ limit (G ⋙ H) vs
H (limit F) ⟶ limit (F ⋙ H) ⟶ limit (G ⋙ H) -/
Expand Down Expand Up @@ -567,6 +576,14 @@ lemma colimit.pre_map {K : Type v} [small_category K] [has_colimits_of_shape K C
colimit.pre F E ≫ colim.map α = colim.map (whisker_left E α) ≫ colimit.pre G E :=
by ext; rw [←assoc, colimit.ι_pre, colim.ι_map, ←assoc, colim.ι_map, assoc, colimit.ι_pre]; refl

lemma colimit.pre_map' {K : Type v} [small_category K] [has_colimits_of_shape.{u v} K C]
(F : J ⥤ C) {E₁ E₂ : K ⥤ J} (α : E₁ ⟹ E₂) :
colimit.pre F E₁ = colim.map (whisker_right α F) ≫ colimit.pre F E₂ :=
by ext1; simp [(category.assoc _ _ _ _).symm]

lemma colimit.pre_id (F : J ⥤ C) :
colimit.pre F (functor.id _) = colim.map (functor.left_unitor F).hom := by tidy

lemma colimit.map_post {D : Type u'} [category.{u' v} D] [has_colimits_of_shape J D] (H : C ⥤ D) :
/- H (colimit F) ⟶ H (colimit G) ⟶ colimit (G ⋙ H) vs
H (colimit F) ⟶ colimit (F ⋙ H) ⟶ colimit (G ⋙ H) -/
Expand Down

0 comments on commit 4b9f9a6

Please sign in to comment.