Construction of projections for the Dold-Kan correspondence #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
TODO (@joelriou) continue adding the various files referenced below
In this file, we construct endomorphisms P q : K[X] ⟶ K[X]
for all
q : ℕ
. We study how they behave with respect to face maps with the lemmas
higher_faces_vanish.of_P
, higher_faces_vanish.comp_P_eq_self
and
comp_P_eq_self_iff
.
Then, we show that they are projections (see P_f_idem
and P_idem
). They are natural transformations (see nat_trans_P
and P_f_naturality
) and are compatible with the application
of additive functors (see map_P
).
By passing to the limit, these endomorphisms P q
shall be used in p_infty.lean
in order to define P_infty : K[X] ⟶ K[X]
, see equivalence.lean
for the general
strategy of proof of the Dold-Kan equivalence.
(See equivalence.lean
for the general strategy of proof of the Dold-Kan equivalence.)
This is the inductive definition of the projections P q : K[X] ⟶ K[X]
,
with P 0 := 𝟙 _
and P (q+1) := P q ≫ (𝟙 _ + Hσ q)
.
All the P q
coincide with 𝟙 _
in degree 0.
Q q
is the complement projection associated to P q
All the Q q
coincide with 0
in degree 0.
This lemma expresses the vanishing of
(P q).f (n+1) ≫ X.δ k : X _[n+1] ⟶ X _[n]
when k≠0
and k≥n-q+2
For each q
, P q
is a natural transformation.
Equations
- algebraic_topology.dold_kan.nat_trans_P q = {app := λ (X : category_theory.simplicial_object C), algebraic_topology.dold_kan.P q, naturality' := _}
For each q
, Q q
is a natural transformation.
Equations
- algebraic_topology.dold_kan.nat_trans_Q q = {app := λ (X : category_theory.simplicial_object C), algebraic_topology.dold_kan.Q q, naturality' := _}