Projective resolutions #
A projective resolution P : ProjectiveResolution Z
of an object Z : C
consists of
an ℕ
-indexed chain complex P.complex
of projective objects,
along with a chain map P.π
from C
to the chain complex consisting just of Z
in degree zero,
so that the augmented chain complex is exact.
When C
is abelian, this exactness condition is equivalent to π
being a quasi-isomorphism.
It turns out that this formulation allows us to set up the basic theory of derived functors
without even assuming C
is abelian.
(Typically, however, to show HasProjectiveResolutions C
one will assume EnoughProjectives C
and Abelian C
.
This construction appears in CategoryTheory.Abelian.Projective
.)
We show that given P : ProjectiveResolution X
and Q : ProjectiveResolution Y
,
any morphism X ⟶ Y
admits a lift to a chain map P.complex ⟶ Q.complex
.
(It is a lift in the sense that
the projection maps P.π
and Q.π
intertwine the lift and the original morphism.)
Moreover, we show that any two such lifts are homotopic.
As a consequence, if every object admits a projective resolution,
we can construct a functor projectiveResolutions C : C ⥤ HomotopyCategory C
.
- complex : ChainComplex C ℕ
- π : s.complex ⟶ (ChainComplex.single₀ C).obj Z
- projective : ∀ (n : ℕ), CategoryTheory.Projective (HomologicalComplex.X s.complex n)
- exact₀ : CategoryTheory.Exact (HomologicalComplex.d s.complex 1 0) (HomologicalComplex.Hom.f s.π 0)
- exact : ∀ (n : ℕ), CategoryTheory.Exact (HomologicalComplex.d s.complex (n + 2) (n + 1)) (HomologicalComplex.d s.complex (n + 1) n)
- epi : CategoryTheory.Epi (HomologicalComplex.Hom.f s.π 0)
A ProjectiveResolution Z
consists of a bundled ℕ
-indexed chain complex of projective objects,
along with a quasi-isomorphism to the complex consisting of just Z
supported in degree 0
.
(We don't actually ask here that the chain map is a quasi-iso, just exactness everywhere:
that π
is a quasi-iso is a lemma when the category is abelian.
Should we just ask for it here?)
Except in situations where you want to provide a particular projective resolution (for example to compute a derived functor), you will not typically need to use this bundled object, and will instead use
ProjectiveResolution Z
: theℕ
-indexed chain complex (equipped withProjective
andExact
instances)ProjectiveResolution.π Z
: the chain map fromProjectiveResolution Z
to(ChainComplex.single₀ C).obj Z
(all the components are equipped withEpi
instances, and when the category isAbelian
we will showπ
is a quasi-iso).
Instances For
- out : Nonempty (CategoryTheory.ProjectiveResolution Z)
An object admits a projective resolution.
Instances
- out : ∀ (Z : C), CategoryTheory.HasProjectiveResolution Z
You will rarely use this typeclass directly: it is implied by the combination
[EnoughProjectives C]
and [Abelian C]
.
By itself it's enough to set up the basic theory of derived functors.
Instances
A projective object admits a trivial projective resolution: itself in degree 0.
Instances For
Auxiliary construction for lift
.
Instances For
Auxiliary construction for lift
.
Instances For
Auxiliary lemma for lift
.
Auxiliary construction for lift
.
Instances For
A morphism in C
lifts to a chain map between projective resolutions.
Instances For
The resolution maps intertwine the lift of a morphism and that morphism.
An auxiliary definition for liftHomotopyZero
.
Instances For
An auxiliary definition for liftHomotopyZero
.
Instances For
An auxiliary definition for liftHomotopyZero
.
Instances For
Any lift of the zero morphism is homotopic to zero.
Instances For
Two lifts of the same morphism are homotopic.
Instances For
The lift of the identity morphism is homotopic to the identity chain map.
Instances For
The lift of a composition is homotopic to the composition of the lifts.
Instances For
Any two projective resolutions are homotopy equivalent.
Instances For
Instances For
An arbitrarily chosen projective resolution of an object.
Instances For
The chain map from the arbitrarily chosen projective resolution
projectiveResolution.complex Z
back to the chain complex consisting
of Z
supported in degree 0
.
Instances For
The lift of a morphism to a chain map between the arbitrarily chosen projective resolutions.
Instances For
Taking projective resolutions is functorial,
if considered with target the homotopy category
(ℕ
-indexed chain complexes and chain maps up to homotopy).