Documentation

Mathlib.CategoryTheory.Abelian.ProjectiveResolution

Abelian categories with enough projectives have projective resolutions #

Main results #

When the underlying category is abelian:

Auxiliary construction for lift.

Equations
Instances For
    noncomputable def CategoryTheory.ProjectiveResolution.liftFSucc {C : Type u} [CategoryTheory.Category.{v, u} C] [CategoryTheory.Abelian C] {Y : C} {Z : C} (P : CategoryTheory.ProjectiveResolution Y) (Q : CategoryTheory.ProjectiveResolution Z) (n : ) (g : P.complex.X n Q.complex.X n) (g' : P.complex.X (n + 1) Q.complex.X (n + 1)) (w : CategoryTheory.CategoryStruct.comp g' (Q.complex.d (n + 1) n) = CategoryTheory.CategoryStruct.comp (P.complex.d (n + 1) n) g) :
    (g'' : P.complex.X (n + 2) Q.complex.X (n + 2)) ×' CategoryTheory.CategoryStruct.comp g'' (Q.complex.d (n + 2) (n + 1)) = CategoryTheory.CategoryStruct.comp (P.complex.d (n + 2) (n + 1)) g'

    Auxiliary construction for lift.

    Equations
    Instances For

      A morphism in C lift to a chain map between projective resolutions.

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

        An auxiliary definition for liftHomotopyZero.

        Equations
        Instances For
          noncomputable def CategoryTheory.ProjectiveResolution.liftHomotopyZeroOne {C : Type u} [CategoryTheory.Category.{v, u} C] [CategoryTheory.Abelian C] {Y : C} {Z : C} {P : CategoryTheory.ProjectiveResolution Y} {Q : CategoryTheory.ProjectiveResolution Z} (f : P.complex Q.complex) (comm : CategoryTheory.CategoryStruct.comp f Q = 0) :
          P.complex.X 1 Q.complex.X 2

          An auxiliary definition for liftHomotopyZero.

          Equations
          • One or more equations did not get rendered due to their size.
          Instances For
            noncomputable def CategoryTheory.ProjectiveResolution.liftHomotopyZeroSucc {C : Type u} [CategoryTheory.Category.{v, u} C] [CategoryTheory.Abelian C] {Y : C} {Z : C} {P : CategoryTheory.ProjectiveResolution Y} {Q : CategoryTheory.ProjectiveResolution Z} (f : P.complex Q.complex) (n : ) (g : P.complex.X n Q.complex.X (n + 1)) (g' : P.complex.X (n + 1) Q.complex.X (n + 2)) (w : f.f (n + 1) = CategoryTheory.CategoryStruct.comp (P.complex.d (n + 1) n) g + CategoryTheory.CategoryStruct.comp g' (Q.complex.d (n + 2) (n + 1))) :
            P.complex.X (n + 2) Q.complex.X (n + 3)

            An auxiliary definition for liftHomotopyZero.

            Equations
            Instances For
              @[simp]
              theorem CategoryTheory.ProjectiveResolution.liftHomotopyZeroSucc_comp_assoc {C : Type u} [CategoryTheory.Category.{v, u} C] [CategoryTheory.Abelian C] {Y : C} {Z : C} {P : CategoryTheory.ProjectiveResolution Y} {Q : CategoryTheory.ProjectiveResolution Z✝} (f : P.complex Q.complex) (n : ) (g : P.complex.X n Q.complex.X (n + 1)) (g' : P.complex.X (n + 1) Q.complex.X (n + 2)) (w : f.f (n + 1) = CategoryTheory.CategoryStruct.comp (P.complex.d (n + 1) n) g + CategoryTheory.CategoryStruct.comp g' (Q.complex.d (n + 2) (n + 1))) {Z : C} (h : Q.complex.X (n + 2) Z) :
              @[simp]
              theorem CategoryTheory.ProjectiveResolution.liftHomotopyZeroSucc_comp {C : Type u} [CategoryTheory.Category.{v, u} C] [CategoryTheory.Abelian C] {Y : C} {Z : C} {P : CategoryTheory.ProjectiveResolution Y} {Q : CategoryTheory.ProjectiveResolution Z} (f : P.complex Q.complex) (n : ) (g : P.complex.X n Q.complex.X (n + 1)) (g' : P.complex.X (n + 1) Q.complex.X (n + 2)) (w : f.f (n + 1) = CategoryTheory.CategoryStruct.comp (P.complex.d (n + 1) n) g + CategoryTheory.CategoryStruct.comp g' (Q.complex.d (n + 2) (n + 1))) :

              Any lift of the zero morphism is homotopic to zero.

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

                Two lifts of the same morphism are homotopic.

                Equations
                Instances For

                  The lift of the identity morphism is homotopic to the identity chain map.

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

                    The lift of a composition is homotopic to the composition of the lifts.

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

                      Any two projective resolutions are homotopy equivalent.

                      Equations
                      • One or more equations did not get rendered due to their size.
                      Instances For
                        @[reducible, inline]

                        An arbitrarily chosen projective resolution of an object.

                        Equations
                        Instances For

                          Taking projective resolutions is functorial, if considered with target the homotopy category (-indexed chain complexes and chain maps up to homotopy).

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

                            If P : ProjectiveResolution X, then the chosen (projectiveResolutions C).obj X is isomorphic (in the homotopy category) to P.complex.

                            Equations
                            Instances For

                              Our goal is to define ProjectiveResolution.of Z : ProjectiveResolution Z. The 0-th object in this resolution will just be Projective.over Z, i.e. an arbitrarily chosen projective object with a map to Z. After that, we build the n+1-st object as Projective.syzygies applied to the previously constructed morphism, and the map from the n-th object as Projective.d.

                              Auxiliary definition for ProjectiveResolution.of.

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

                                In any abelian category with enough projectives, ProjectiveResolution.of Z constructs an projective resolution of the object Z.

                                Equations
                                Instances For