Documentation

Mathlib.CategoryTheory.Abelian.Projective.Extend

Projective resolutions as cochain complexes indexed by the integers #

Given a projective resolution R of an object X in an abelian category C, we define R.cochainComplex : CochainComplex C ℤ, which is the extension of R.complex : ChainComplex C ℕ, and the quasi-isomorphism R.π' : R.cochainComplex ⟶ (CochainComplex.singleFunctor C 0).obj X.

If R : ProjectiveResolution X, this is the cochain complex indexed by obtained by extending by zero the chain complex R.complex indexed by .

Equations
Instances For
    noncomputable def CategoryTheory.ProjectiveResolution.cochainComplexXIso {C : Type u} [Category.{v, u} C] [Limits.HasZeroObject C] [Preadditive C] {X : C} (R : ProjectiveResolution X) (n : ) (k : ) (h : -k = n := by lia) :

    If R : ProjectiveResolution X, then R.chainComplex.X n (with n : ℕ) is isomorphic to R.complex.X k (with k : ℕ) when k = n.

    Equations
    Instances For
      theorem CategoryTheory.ProjectiveResolution.cochainComplex_d {C : Type u} [Category.{v, u} C] [Limits.HasZeroObject C] [Preadditive C] {X : C} (R : ProjectiveResolution X) (n₁ n₂ : ) (k₁ k₂ : ) (h₁ : -k₁ = n₁ := by lia) (h₂ : -k₂ = n₂ := by lia) :
      R.cochainComplex.d n₁ n₂ = CategoryStruct.comp (R.cochainComplexXIso n₁ k₁ ).hom (CategoryStruct.comp (R.complex.d k₁ k₂) (R.cochainComplexXIso n₂ k₂ ).inv)
      theorem CategoryTheory.ProjectiveResolution.cochainComplex_d_assoc {C : Type u} [Category.{v, u} C] [Limits.HasZeroObject C] [Preadditive C] {X : C} (R : ProjectiveResolution X) (n₁ n₂ : ) (k₁ k₂ : ) (h₁ : -k₁ = n₁ := by lia) (h₂ : -k₂ = n₂ := by lia) {Z : C} (h : R.cochainComplex.X n₂ Z) :

      The quasi-isomorphism R.cochainComplex ⟶ (CochainComplex.singleFunctor C 0).obj X in CochainComplex C ℤ when R is a projective resolution of X.

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