Factorization lemma #
Let C be an abelian category with enough injectives. We show that
any morphism f : K ⟶ L between bounded below cochain complexes in C
can be factored as i ≫ p where i : K ⟶ L' is a monomorphism (with
L' bounded below) and p : L' ⟶ L a quasi-isomorphism that is an epimorphism
with a degreewise injective kernel. (This is part of the factorization axiom CM5
for a model category structure on bounded below cochain complexes (TODO @joelriou).)
Given a cochain complex K, this is a cochain complex I K with
zero differentials which in degree n consists of the injective
object Injective.under (K.X n).
Equations
- CochainComplex.cm5b.I K = { X := fun (n : ℤ) => CategoryTheory.Injective.under (K.X n), d := fun (x x_1 : ℤ) => 0, shape := ⋯, d_comp_d' := ⋯ }
Instances For
The second projection mappingCone (𝟙 (I K)) ⊞ L ⟶ L.
Equations
Instances For
A lift of a morphism f : K ⟶ L between bounded below cochain complexes
as a monomorphism K ⟶ mappingCone (𝟙 (I K)) ⊞ L.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The second projection p K L : mappingCone (𝟙 (I K)) ⊞ L ⟶ L is a homotopy equivalence.
Equations
- One or more equations did not get rendered due to their size.