Documentation

Mathlib.CategoryTheory.Limits.FullSubcategory

Limits in full subcategories #

We introduce the notion of a property closed under taking limits and show that if P is closed under taking limits, then limits in FullSubcategory P can be constructed from limits in C. More precisely, the inclusion creates such limits.

We say that a property is closed under limits of shape J if whenever all objects in a J-shaped diagram have the property, any limit of this diagram also has the property.

Equations
Instances For

    We say that a property is closed under colimits of shape J if whenever all objects in a J-shaped diagram have the property, any colimit of this diagram also has the property.

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      theorem CategoryTheory.Limits.closedUnderLimitsOfShape_of_limit {C : Type u} [Category.{v, u} C] {J : Type w} [Category.{w', w} J] {P : CProp} [ClosedUnderIsomorphisms P] (h : ∀ {F : Functor J C} [inst : HasLimit F], (∀ (j : J), P (F.obj j))P (limit F)) :
      theorem CategoryTheory.Limits.closedUnderColimitsOfShape_of_colimit {C : Type u} [Category.{v, u} C] {J : Type w} [Category.{w', w} J] {P : CProp} [ClosedUnderIsomorphisms P] (h : ∀ {F : Functor J C} [inst : HasColimit F], (∀ (j : J), P (F.obj j))P (colimit F)) :
      theorem CategoryTheory.Limits.ClosedUnderLimitsOfShape.limit {C : Type u} [Category.{v, u} C] {J : Type w} [Category.{w', w} J] {P : CProp} (h : ClosedUnderLimitsOfShape J P) {F : Functor J C} [HasLimit F] :
      (∀ (j : J), P (F.obj j))P (Limits.limit F)
      theorem CategoryTheory.Limits.ClosedUnderColimitsOfShape.colimit {C : Type u} [Category.{v, u} C] {J : Type w} [Category.{w', w} J] {P : CProp} (h : ClosedUnderColimitsOfShape J P) {F : Functor J C} [HasColimit F] :
      (∀ (j : J), P (F.obj j))P (Limits.colimit F)

      If a J-shaped diagram in FullSubcategory P has a limit cone in C whose cone point lives in the full subcategory, then this defines a limit in the full subcategory.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For

        If a J-shaped diagram in FullSubcategory P has a limit in C whose cone point lives in the full subcategory, then this defines a limit in the full subcategory.

        Equations
        • One or more equations did not get rendered due to their size.
        Instances For

          If a J-shaped diagram in FullSubcategory P has a colimit cocone in C whose cocone point lives in the full subcategory, then this defines a colimit in the full subcategory.

          Equations
          • One or more equations did not get rendered due to their size.
          Instances For

            If a J-shaped diagram in FullSubcategory P has a colimit in C whose cocone point lives in the full subcategory, then this defines a colimit in the full subcategory.

            Equations
            • One or more equations did not get rendered due to their size.
            Instances For

              If P is closed under limits of shape J, then the inclusion creates such limits.

              Equations
              • One or more equations did not get rendered due to their size.
              Instances For

                If P is closed under colimits of shape J, then the inclusion creates such colimits.

                Equations
                • One or more equations did not get rendered due to their size.
                Instances For