Moore complex #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
We construct the normalized Moore complex, as a functor
simplicial_object C ⥤ chain_complex C ℕ
,
for any abelian category C
.
The n
-th object is intersection of
the kernels of X.δ i : X.obj n ⟶ X.obj (n-1)
, for i = 1, ..., n
.
The differentials are induced from X.δ 0
,
which maps each of these intersections of kernels to the next.
This functor is one direction of the Dold-Kan equivalence, which we're still working towards.
References #
The definitions in this namespace are all auxiliary definitions for normalized_Moore_complex
and should usually only be accessed via that.
The normalized Moore complex in degree n
, as a subobject of X n
.
Equations
- algebraic_topology.normalized_Moore_complex.obj_X X (n + 1) = finset.univ.inf (λ (k : fin (n + 1)), category_theory.limits.kernel_subobject (X.δ k.succ))
- algebraic_topology.normalized_Moore_complex.obj_X X 0 = ⊤
The differentials in the normalized Moore complex.
Equations
- algebraic_topology.normalized_Moore_complex.obj_d X (n + 1) = (algebraic_topology.normalized_Moore_complex.obj_X X (n + 1)).factor_thru ((algebraic_topology.normalized_Moore_complex.obj_X X (n + 1 + 1)).arrow ≫ X.δ 0) _
- algebraic_topology.normalized_Moore_complex.obj_d X 0 = (algebraic_topology.normalized_Moore_complex.obj_X X (0 + 1)).arrow ≫ X.δ 0 ≫ category_theory.inv ⊤.arrow
The normalized Moore complex functor, on objects.
The normalized Moore complex functor, on morphisms.
Equations
- algebraic_topology.normalized_Moore_complex.map f = chain_complex.of_hom (λ (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 Y n)) (algebraic_topology.normalized_Moore_complex.obj_d Y) _ (λ (n : ℕ), (algebraic_topology.normalized_Moore_complex.obj_X Y n).factor_thru ((algebraic_topology.normalized_Moore_complex.obj_X X n).arrow ≫ f.app (opposite.op (simplex_category.mk n))) _) _
The (normalized) Moore complex of a simplicial object X
in an abelian category C
.
The n
-th object is intersection of
the kernels of X.δ i : X.obj n ⟶ X.obj (n-1)
, for i = 1, ..., n
.
The differentials are induced from X.δ 0
,
which maps each of these intersections of kernels to the next.
Equations
- algebraic_topology.normalized_Moore_complex C = {obj := algebraic_topology.normalized_Moore_complex.obj _inst_2, map := λ (X Y : category_theory.simplicial_object C) (f : X ⟶ Y), algebraic_topology.normalized_Moore_complex.map f, map_id' := _, map_comp' := _}