Comparison with the normalized Moore complex functor #
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 show that when the category A
is abelian,
there is an isomorphism N₁_iso_normalized_Moore_complex_comp_to_karoubi
between
the functor N₁ : simplicial_object A ⥤ karoubi (chain_complex A ℕ)
defined in functor_n.lean
and the composition of
normalized_Moore_complex A
with the inclusion
chain_complex A ℕ ⥤ karoubi (chain_complex A ℕ)
.
This isomorphism shall be used in equivalence.lean
in order to obtain
the Dold-Kan equivalence
category_theory.abelian.dold_kan.equivalence : simplicial_object A ≌ chain_complex A ℕ
with a functor (definitionally) equal to normalized_Moore_complex A
.
(See equivalence.lean
for the general strategy of proof of the Dold-Kan equivalence.)
P_infty factors through the normalized Moore complex
Equations
- algebraic_topology.dold_kan.P_infty_to_normalized_Moore_complex X = chain_complex.of_hom (λ (n : ℕ), X.obj (opposite.op (simplex_category.mk n))) (algebraic_topology.alternating_face_map_complex.obj_d X) _ (λ (n : ℕ), ↑(algebraic_topology.normalized_Moore_complex.obj_X X n)) (algebraic_topology.normalized_Moore_complex.obj_d X) _ (λ (n : ℕ), (algebraic_topology.normalized_Moore_complex.obj_X X n).factor_thru (algebraic_topology.dold_kan.P_infty.f n) _) _
inclusion_of_Moore_complex_map X
is a split mono.
When the category A
is abelian,
the functor N₁ : simplicial_object A ⥤ karoubi (chain_complex A ℕ)
defined
using P_infty
identifies to the composition of the normalized Moore complex functor
and the inclusion in the Karoubi envelope.
Equations
- algebraic_topology.dold_kan.N₁_iso_normalized_Moore_complex_comp_to_karoubi A = {hom := {app := λ (X : category_theory.simplicial_object A), {f := algebraic_topology.dold_kan.P_infty_to_normalized_Moore_complex X, comm := _}, naturality' := _}, inv := {app := λ (X : category_theory.simplicial_object A), {f := algebraic_topology.inclusion_of_Moore_complex_map X, comm := _}, naturality' := _}, hom_inv_id' := _, inv_hom_id' := _}