Documentation

Mathlib.Algebra.Homology.HomologicalComplexLimits

Limits and colimits in the category of homological complexes #

In this file, it is shown that if a category C has (co)limits of shape J, then it is also the case of the categories HomologicalComplex C c, and the evaluation functors eval C c i : HomologicalComplex C c ⥤ C commute to these.

A cone in HomologicalComplex C c is limit if the induced cones obtained by applying eval C c i : HomologicalComplex C c ⥤ C for all i are limit.

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

    A cone for a functor F : J ⥤ HomologicalComplex C c which is given in degree n by the limit F ⋙ eval C c n.

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      @[simp]
      theorem HomologicalComplex.coneOfHasLimitEval_pt_d {C : Type u_1} {ι : Type u_2} {J : Type u_3} [CategoryTheory.Category.{u_4, u_1} C] [CategoryTheory.Category.{u_5, u_3} J] {c : ComplexShape ι} [CategoryTheory.Limits.HasZeroMorphisms C] (F : CategoryTheory.Functor J (HomologicalComplex C c)) [∀ (n : ι), CategoryTheory.Limits.HasLimit (F.comp (eval C c n))] (n m : ι) :
      (coneOfHasLimitEval F).pt.d n m = CategoryTheory.Limits.limMap { app := fun (j : J) => (F.obj j).d n m, naturality := }

      The cone coneOfHasLimitEval F is limit.

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

        A cocone in HomologicalComplex C c is colimit if the induced cocones obtained by applying eval C c i : HomologicalComplex C c ⥤ C for all i are colimit.

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

          A cocone for a functor F : J ⥤ HomologicalComplex C c which is given in degree n by the colimit of F ⋙ eval C c n.

          Equations
          • One or more equations did not get rendered due to their size.
          Instances For
            @[simp]
            theorem HomologicalComplex.coconeOfHasColimitEval_pt_d {C : Type u_1} {ι : Type u_2} {J : Type u_3} [CategoryTheory.Category.{u_4, u_1} C] [CategoryTheory.Category.{u_5, u_3} J] {c : ComplexShape ι} [CategoryTheory.Limits.HasZeroMorphisms C] (F : CategoryTheory.Functor J (HomologicalComplex C c)) [∀ (n : ι), CategoryTheory.Limits.HasColimit (F.comp (eval C c n))] (n m : ι) :
            (coconeOfHasColimitEval F).pt.d n m = CategoryTheory.Limits.colimMap { app := fun (j : J) => (F.obj j).d n m, naturality := }

            The cocone coconeOfHasLimitEval F is colimit.

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