Skip to content

Commit

Permalink
chore: rename lemmas involving closedUnder{Co}limits (#11608)
Browse files Browse the repository at this point in the history
They contain a hypothesis `ClosedUnder{Co}Limits`, hence should be named accordingly.
  • Loading branch information
grunweg committed Mar 24, 2024
1 parent 0865637 commit ffd4025
Showing 1 changed file with 15 additions and 10 deletions.
25 changes: 15 additions & 10 deletions Mathlib/CategoryTheory/Limits/FullSubcategory.lean
Expand Up @@ -105,17 +105,18 @@ def createsLimitsOfShapeFullSubcategoryInclusion (h : ClosedUnderLimitsOfShape J
CreatesLimit := @fun F => createsLimitFullSubcategoryInclusionOfClosed h F
#align category_theory.limits.creates_limits_of_shape_full_subcategory_inclusion CategoryTheory.Limits.createsLimitsOfShapeFullSubcategoryInclusion

theorem hasLimit_of_closed_under_limits (h : ClosedUnderLimitsOfShape J P)
theorem hasLimit_of_closedUnderLimits (h : ClosedUnderLimitsOfShape J P)
(F : J ⥤ FullSubcategory P) [HasLimit (F ⋙ fullSubcategoryInclusion P)] : HasLimit F :=
have : CreatesLimit F (fullSubcategoryInclusion P) :=
createsLimitFullSubcategoryInclusionOfClosed h F
hasLimit_of_created F (fullSubcategoryInclusion P)
#align category_theory.limits.has_limit_of_closed_under_limits CategoryTheory.Limits.hasLimit_of_closed_under_limits
#align category_theory.limits.has_limit_of_closed_under_limits CategoryTheory.Limits.hasLimit_of_closedUnderLimits
@[deprecated] alias hasLimit_of_closed_under_limits := hasLimit_of_closedUnderLimits -- 2024-03-23

theorem hasLimitsOfShape_of_closed_under_limits (h : ClosedUnderLimitsOfShape J P)
theorem hasLimitsOfShape_of_closedUnderLimits (h : ClosedUnderLimitsOfShape J P)
[HasLimitsOfShape J C] : HasLimitsOfShape J (FullSubcategory P) :=
{ has_limit := fun F => hasLimit_of_closed_under_limits h F }
#align category_theory.limits.has_limits_of_shape_of_closed_under_limits CategoryTheory.Limits.hasLimitsOfShape_of_closed_under_limits
{ has_limit := fun F => hasLimit_of_closedUnderLimits h F }
#align category_theory.limits.has_limits_of_shape_of_closed_under_limits CategoryTheory.Limits.hasLimitsOfShape_of_closedUnderLimits

/-- If `P` is closed under colimits of shape `J`, then the inclusion creates such colimits. -/
def createsColimitFullSubcategoryInclusionOfClosed (h : ClosedUnderColimitsOfShape J P)
Expand All @@ -130,17 +131,21 @@ def createsColimitsOfShapeFullSubcategoryInclusion (h : ClosedUnderColimitsOfSha
CreatesColimit := @fun F => createsColimitFullSubcategoryInclusionOfClosed h F
#align category_theory.limits.creates_colimits_of_shape_full_subcategory_inclusion CategoryTheory.Limits.createsColimitsOfShapeFullSubcategoryInclusion

theorem hasColimit_of_closed_under_colimits (h : ClosedUnderColimitsOfShape J P)
theorem hasColimit_of_closedUnderColimits (h : ClosedUnderColimitsOfShape J P)
(F : J ⥤ FullSubcategory P) [HasColimit (F ⋙ fullSubcategoryInclusion P)] : HasColimit F :=
have : CreatesColimit F (fullSubcategoryInclusion P) :=
createsColimitFullSubcategoryInclusionOfClosed h F
hasColimit_of_created F (fullSubcategoryInclusion P)
#align category_theory.limits.has_colimit_of_closed_under_colimits CategoryTheory.Limits.hasColimit_of_closed_under_colimits
#align category_theory.limits.has_colimit_of_closed_under_colimits CategoryTheory.Limits.hasColimit_of_closedUnderColimits
@[deprecated] alias hasColimit_of_closed_under_colimits :=
hasColimit_of_closedUnderColimits -- 2024-03-23

theorem hasColimitsOfShape_of_closed_under_colimits (h : ClosedUnderColimitsOfShape J P)
theorem hasColimitsOfShape_of_closedUnderColimits (h : ClosedUnderColimitsOfShape J P)
[HasColimitsOfShape J C] : HasColimitsOfShape J (FullSubcategory P) :=
{ has_colimit := fun F => hasColimit_of_closed_under_colimits h F }
#align category_theory.limits.has_colimits_of_shape_of_closed_under_colimits CategoryTheory.Limits.hasColimitsOfShape_of_closed_under_colimits
{ has_colimit := fun F => hasColimit_of_closedUnderColimits h F }
#align category_theory.limits.has_colimits_of_shape_of_closed_under_colimits CategoryTheory.Limits.hasColimitsOfShape_of_closedUnderColimits
@[deprecated] alias hasColimitsOfShape_of_closed_under_colimits :=
hasColimitsOfShape_of_closedUnderColimits -- 2024-03-23

end

Expand Down

0 comments on commit ffd4025

Please sign in to comment.