Documentation

Mathlib.Algebra.Homology.ShortComplex.Limits

Limits and colimits in the category of short complexes #

In this file, it is shown if a category C with zero morphisms has limits of a certain shape J, then it is also the case of the category ShortComplex C.

TODO (@rioujoel): Do the same for colimits.

def CategoryTheory.ShortComplex.isLimitOfIsLimitπ {J : Type u_1} {C : Type u_2} [CategoryTheory.Category.{u_3, u_1} J] [CategoryTheory.Category.{u_4, u_2} C] [CategoryTheory.Limits.HasZeroMorphisms C] {F : CategoryTheory.Functor J (CategoryTheory.ShortComplex C)} (c : CategoryTheory.Limits.Cone F) (h₁ : CategoryTheory.Limits.IsLimit (CategoryTheory.ShortComplex.π₁.mapCone c)) (h₂ : CategoryTheory.Limits.IsLimit (CategoryTheory.ShortComplex.π₂.mapCone c)) (h₃ : CategoryTheory.Limits.IsLimit (CategoryTheory.ShortComplex.π₃.mapCone c)) :

If a cone with values in ShortComplex C is such that it becomes limit when we apply the three projections ShortComplex C ⥤ C, then it is limit.

Equations
  • One or more equations did not get rendered due to their size.
Instances For
    noncomputable def CategoryTheory.ShortComplex.limitCone {J : Type u_1} {C : Type u_2} [CategoryTheory.Category.{u_3, u_1} J] [CategoryTheory.Category.{u_4, u_2} C] [CategoryTheory.Limits.HasZeroMorphisms C] (F : CategoryTheory.Functor J (CategoryTheory.ShortComplex C)) [CategoryTheory.Limits.HasLimit (F.comp CategoryTheory.ShortComplex.π₁)] [CategoryTheory.Limits.HasLimit (F.comp CategoryTheory.ShortComplex.π₂)] [CategoryTheory.Limits.HasLimit (F.comp CategoryTheory.ShortComplex.π₃)] :

    Construction of a limit cone for a functor J ⥤ ShortComplex C using the limits of the three components J ⥤ C.

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      noncomputable def CategoryTheory.ShortComplex.isLimitπ₁MapConeLimitCone {J : Type u_1} {C : Type u_2} [CategoryTheory.Category.{u_3, u_1} J] [CategoryTheory.Category.{u_4, u_2} C] [CategoryTheory.Limits.HasZeroMorphisms C] (F : CategoryTheory.Functor J (CategoryTheory.ShortComplex C)) [CategoryTheory.Limits.HasLimit (F.comp CategoryTheory.ShortComplex.π₁)] [CategoryTheory.Limits.HasLimit (F.comp CategoryTheory.ShortComplex.π₂)] [CategoryTheory.Limits.HasLimit (F.comp CategoryTheory.ShortComplex.π₃)] :
      CategoryTheory.Limits.IsLimit (CategoryTheory.ShortComplex.π₁.mapCone (CategoryTheory.ShortComplex.limitCone F))

      limitCone F becomes limit after the application of π₁ : ShortComplex C ⥤ C.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        noncomputable def CategoryTheory.ShortComplex.isLimitπ₂MapConeLimitCone {J : Type u_1} {C : Type u_2} [CategoryTheory.Category.{u_3, u_1} J] [CategoryTheory.Category.{u_4, u_2} C] [CategoryTheory.Limits.HasZeroMorphisms C] (F : CategoryTheory.Functor J (CategoryTheory.ShortComplex C)) [CategoryTheory.Limits.HasLimit (F.comp CategoryTheory.ShortComplex.π₁)] [CategoryTheory.Limits.HasLimit (F.comp CategoryTheory.ShortComplex.π₂)] [CategoryTheory.Limits.HasLimit (F.comp CategoryTheory.ShortComplex.π₃)] :
        CategoryTheory.Limits.IsLimit (CategoryTheory.ShortComplex.π₂.mapCone (CategoryTheory.ShortComplex.limitCone F))

        limitCone F becomes limit after the application of π₂ : ShortComplex C ⥤ C.

        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          noncomputable def CategoryTheory.ShortComplex.isLimitπ₃MapConeLimitCone {J : Type u_1} {C : Type u_2} [CategoryTheory.Category.{u_3, u_1} J] [CategoryTheory.Category.{u_4, u_2} C] [CategoryTheory.Limits.HasZeroMorphisms C] (F : CategoryTheory.Functor J (CategoryTheory.ShortComplex C)) [CategoryTheory.Limits.HasLimit (F.comp CategoryTheory.ShortComplex.π₁)] [CategoryTheory.Limits.HasLimit (F.comp CategoryTheory.ShortComplex.π₂)] [CategoryTheory.Limits.HasLimit (F.comp CategoryTheory.ShortComplex.π₃)] :
          CategoryTheory.Limits.IsLimit (CategoryTheory.ShortComplex.π₃.mapCone (CategoryTheory.ShortComplex.limitCone F))

          limitCone F becomes limit after the application of π₃ : ShortComplex C ⥤ C.

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

            limitCone F is limit.

            Equations
            • One or more equations did not get rendered due to their size.
            Instances For
              noncomputable instance CategoryTheory.ShortComplex.instPreservesLimitπ₁ {J : Type u_1} {C : Type u_2} [CategoryTheory.Category.{u_3, u_1} J] [CategoryTheory.Category.{u_4, u_2} C] [CategoryTheory.Limits.HasZeroMorphisms C] (F : CategoryTheory.Functor J (CategoryTheory.ShortComplex C)) [CategoryTheory.Limits.HasLimit (F.comp CategoryTheory.ShortComplex.π₁)] [CategoryTheory.Limits.HasLimit (F.comp CategoryTheory.ShortComplex.π₂)] [CategoryTheory.Limits.HasLimit (F.comp CategoryTheory.ShortComplex.π₃)] :
              CategoryTheory.Limits.PreservesLimit F CategoryTheory.ShortComplex.π₁
              Equations
              • One or more equations did not get rendered due to their size.
              noncomputable instance CategoryTheory.ShortComplex.instPreservesLimitπ₂ {J : Type u_1} {C : Type u_2} [CategoryTheory.Category.{u_3, u_1} J] [CategoryTheory.Category.{u_4, u_2} C] [CategoryTheory.Limits.HasZeroMorphisms C] (F : CategoryTheory.Functor J (CategoryTheory.ShortComplex C)) [CategoryTheory.Limits.HasLimit (F.comp CategoryTheory.ShortComplex.π₁)] [CategoryTheory.Limits.HasLimit (F.comp CategoryTheory.ShortComplex.π₂)] [CategoryTheory.Limits.HasLimit (F.comp CategoryTheory.ShortComplex.π₃)] :
              CategoryTheory.Limits.PreservesLimit F CategoryTheory.ShortComplex.π₂
              Equations
              • One or more equations did not get rendered due to their size.
              noncomputable instance CategoryTheory.ShortComplex.instPreservesLimitπ₃ {J : Type u_1} {C : Type u_2} [CategoryTheory.Category.{u_3, u_1} J] [CategoryTheory.Category.{u_4, u_2} C] [CategoryTheory.Limits.HasZeroMorphisms C] (F : CategoryTheory.Functor J (CategoryTheory.ShortComplex C)) [CategoryTheory.Limits.HasLimit (F.comp CategoryTheory.ShortComplex.π₁)] [CategoryTheory.Limits.HasLimit (F.comp CategoryTheory.ShortComplex.π₂)] [CategoryTheory.Limits.HasLimit (F.comp CategoryTheory.ShortComplex.π₃)] :
              CategoryTheory.Limits.PreservesLimit F CategoryTheory.ShortComplex.π₃
              Equations
              • One or more equations did not get rendered due to their size.
              Equations
              Equations
              Equations
              Equations
              • One or more equations did not get rendered due to their size.
              Equations
              • One or more equations did not get rendered due to their size.
              Equations
              • One or more equations did not get rendered due to their size.

              If a cocone with values in ShortComplex C is such that it becomes colimit when we apply the three projections ShortComplex C ⥤ C, then it is colimit.

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

                Construction of a colimit cocone for a functor J ⥤ ShortComplex C using the colimits of the three components J ⥤ C.

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

                  colimitCocone F becomes colimit after the application of π₁ : ShortComplex C ⥤ C.

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

                    colimitCocone F becomes colimit after the application of π₂ : ShortComplex C ⥤ C.

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

                      colimitCocone F becomes colimit after the application of π₃ : ShortComplex C ⥤ C.

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

                        colimitCocone F is colimit.

                        Equations
                        • One or more equations did not get rendered due to their size.
                        Instances For
                          noncomputable instance CategoryTheory.ShortComplex.instPreservesColimitπ₁ {J : Type u_1} {C : Type u_2} [CategoryTheory.Category.{u_3, u_1} J] [CategoryTheory.Category.{u_4, u_2} C] [CategoryTheory.Limits.HasZeroMorphisms C] (F : CategoryTheory.Functor J (CategoryTheory.ShortComplex C)) [CategoryTheory.Limits.HasColimit (F.comp CategoryTheory.ShortComplex.π₁)] [CategoryTheory.Limits.HasColimit (F.comp CategoryTheory.ShortComplex.π₂)] [CategoryTheory.Limits.HasColimit (F.comp CategoryTheory.ShortComplex.π₃)] :
                          CategoryTheory.Limits.PreservesColimit F CategoryTheory.ShortComplex.π₁
                          Equations
                          • One or more equations did not get rendered due to their size.
                          noncomputable instance CategoryTheory.ShortComplex.instPreservesColimitπ₂ {J : Type u_1} {C : Type u_2} [CategoryTheory.Category.{u_3, u_1} J] [CategoryTheory.Category.{u_4, u_2} C] [CategoryTheory.Limits.HasZeroMorphisms C] (F : CategoryTheory.Functor J (CategoryTheory.ShortComplex C)) [CategoryTheory.Limits.HasColimit (F.comp CategoryTheory.ShortComplex.π₁)] [CategoryTheory.Limits.HasColimit (F.comp CategoryTheory.ShortComplex.π₂)] [CategoryTheory.Limits.HasColimit (F.comp CategoryTheory.ShortComplex.π₃)] :
                          CategoryTheory.Limits.PreservesColimit F CategoryTheory.ShortComplex.π₂
                          Equations
                          • One or more equations did not get rendered due to their size.
                          noncomputable instance CategoryTheory.ShortComplex.instPreservesColimitπ₃ {J : Type u_1} {C : Type u_2} [CategoryTheory.Category.{u_3, u_1} J] [CategoryTheory.Category.{u_4, u_2} C] [CategoryTheory.Limits.HasZeroMorphisms C] (F : CategoryTheory.Functor J (CategoryTheory.ShortComplex C)) [CategoryTheory.Limits.HasColimit (F.comp CategoryTheory.ShortComplex.π₁)] [CategoryTheory.Limits.HasColimit (F.comp CategoryTheory.ShortComplex.π₂)] [CategoryTheory.Limits.HasColimit (F.comp CategoryTheory.ShortComplex.π₃)] :
                          CategoryTheory.Limits.PreservesColimit F CategoryTheory.ShortComplex.π₃
                          Equations
                          • One or more equations did not get rendered due to their size.
                          Equations
                          Equations
                          Equations
                          Equations
                          • One or more equations did not get rendered due to their size.
                          Equations
                          • One or more equations did not get rendered due to their size.
                          Equations
                          • One or more equations did not get rendered due to their size.