Construction of the projection P_infty
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 the projection P_infty : K[X] ⟶ K[X]
by passing
to the limit the projections P q
defined in projections.lean
. This
projection is a critical tool in this formalisation of the Dold-Kan correspondence,
because in the case of abelian categories, P_infty
corresponds to the
projection on the normalized Moore subcomplex, with kernel the degenerate subcomplex.
(See equivalence.lean
for the general strategy of proof of the Dold-Kan equivalence.)
The endomorphism P_infty : K[X] ⟶ K[X]
obtained from the P q
by passing to the limit.
Equations
- algebraic_topology.dold_kan.P_infty = chain_complex.of_hom (λ (n : ℕ), X.obj (opposite.op (simplex_category.mk n))) (algebraic_topology.alternating_face_map_complex.obj_d X) _ (λ (n : ℕ), X.obj (opposite.op (simplex_category.mk n))) (algebraic_topology.alternating_face_map_complex.obj_d X) _ (λ (n : ℕ), (algebraic_topology.dold_kan.P n).f n) algebraic_topology.dold_kan.P_infty._proof_1
The endomorphism Q_infty : K[X] ⟶ K[X]
obtained from the Q q
by passing to the limit.
P_infty
induces a natural transformation, i.e. an endomorphism of
the functor alternating_face_map_complex C
.
Equations
The natural transformation in each degree that is induced by nat_trans_P_infty
.
Given an object Y : karoubi (simplicial_object C)
, this lemma
computes P_infty
for the associated object in simplicial_object (karoubi C)
in terms of P_infty
for Y.X : simplicial_object C
and Y.p
.