Split simplicial objects in preadditive categories #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
In this file we define a functor nondeg_complex : simplicial_object.split C ⥤ chain_complex C ℕ
when C
is a preadditive category with finite coproducts, and get an isomorphism
to_karoubi_nondeg_complex_iso_N₁ : nondeg_complex ⋙ to_karoubi _ ≅ forget C ⋙ dold_kan.N₁
.
(See equivalence.lean
for the general strategy of proof of the Dold-Kan equivalence.)
The projection on a summand of the coproduct decomposition given by a splitting of a simplicial object.
Equations
- s.π_summand A = (s.iso Δ).inv ≫ category_theory.limits.sigma.desc (λ (B : simplicial_object.splitting.index_set Δ), dite (B = A) (λ (h : B = A), category_theory.eq_to_hom _) (λ (h : ¬B = A), 0))
If a simplicial object X
in an additive category is split,
then P_infty
vanishes on all the summands of X _[n]
which do
not correspond to the identity of [n]
.
The differentials s.d i j : s.N i ⟶ s.N j
on nondegenerate simplices of a split
simplicial object are induced by the differentials on the alternating face map complex.
Equations
If s
is a splitting of a simplicial object X
in a preadditive category,
s.nondeg_complex
is a chain complex which is given in degree n
by
the nondegenerate n
-simplices of X
.
The chain complex s.nondeg_complex
attached to a splitting of a simplicial object X
becomes isomorphic to the normalized Moore complex N₁.obj X
defined as a formal direct
factor in the category karoubi (chain_complex C ℕ)
.
Equations
- s.to_karoubi_nondeg_complex_iso_N₁ = {hom := {f := {f := λ (n : ℕ), s.ι_summand (simplicial_object.splitting.index_set.id (opposite.op (simplex_category.mk n))) ≫ algebraic_topology.dold_kan.P_infty.f n, comm' := _}, comm := _}, inv := {f := {f := λ (n : ℕ), s.π_summand (simplicial_object.splitting.index_set.id (opposite.op (simplex_category.mk n))), comm' := _}, comm := _}, hom_inv_id' := _, inv_hom_id' := _}
The functor which sends a split simplicial object in a preadditive category to the chain complex which consists of nondegenerate simplices.
Equations
- simplicial_object.split.nondeg_complex_functor = {obj := λ (S : simplicial_object.split C), S.s.nondeg_complex, map := λ (S₁ S₂ : simplicial_object.split C) (Φ : S₁ ⟶ S₂), {f := Φ.f, comm' := _}, map_id' := _, map_comp' := _}
The natural isomorphism (in karoubi (chain_complex C ℕ)
) between the chain complex
of nondegenerate simplices of a split simplicial object and the normalized Moore complex
defined as a formal direct factor of the alternating face map complex.
Equations
- simplicial_object.split.to_karoubi_nondeg_complex_functor_iso_N₁ = category_theory.nat_iso.of_components (λ (S : simplicial_object.split C), S.s.to_karoubi_nondeg_complex_iso_N₁) simplicial_object.split.to_karoubi_nondeg_complex_functor_iso_N₁._proof_1