Documentation

Mathlib.Algebra.Homology.Factorizations.Basic

Basic definitions for factorizations lemmas #

We define the class of morphisms degreewiseEpiWithInjectiveKernel : MorphismProperty (CochainComplex C ℤ) in the category of cochain complexes in an abelian category C.

When restricted to the full subcategory of bounded below cochain complexes in an abelian category C that has enough injectives, this is the class of fibrations for a model category structure on the bounded below category of cochain complexes in C. In this folder, we intend to prove two factorization lemmas in the category of bounded below cochain complexes (TODO):

The difficult part is CM5a (whose proof uses CM5b). These lemmas shall be essential ingredients in the proof that the bounded below derived category of an abelian category C with enough injectives identifies to the bounded below homotopy category of complexes of injective objects in C. This will be used in the construction of total derived functors (and a refactor of the sequence of derived functors).

A morphism of cochain complexes φ in an abelian category satisfies degreewiseEpiWithInjectiveKernel φ if for any i : ℤ, the morphism φ.f i is an epimorphism with an injective kernel.

Equations
Instances For
    instance CochainComplex.instIsMultiplicativeIntDegreewiseEpiWithInjectiveKernel {C : Type u_1} [CategoryTheory.Category.{u_2, u_1} C] [CategoryTheory.Abelian C] :
    CochainComplex.degreewiseEpiWithInjectiveKernel.IsMultiplicative
    Equations
    • =