Documentation

Mathlib.AlgebraicTopology.DoldKan.NCompGamma

The unit isomorphism of the Dold-Kan equivalence

In order to construct the unit isomorphism of the Dold-Kan equivalence, we first construct natural transformations Γ₂N₁.natTrans : N₁ ⋙ Γ₂ ⟶ toKaroubi (SimplicialObject C) and Γ₂N₂.natTrans : N₂ ⋙ Γ₂ ⟶ 𝟭 (SimplicialObject C). It is then shown that Γ₂N₂.natTrans is an isomorphism by using that it becomes an isomorphism after the application of the functor N₂ : Karoubi (SimplicialObject C) ⥤ Karoubi (ChainComplex C ℕ) which reflects isomorphisms.

(See Equivalence.lean for the general strategy of proof of the Dold-Kan equivalence.)

@[irreducible]

The natural transformation N₁ ⋙ Γ₂ ⟶ toKaroubi (SimplicialObject C).

Equations
  • One or more equations did not get rendered due to their size.
Instances For
    @[irreducible]

    The compatibility isomorphism relating N₂ ⋙ Γ₂ and N₁ ⋙ Γ₂.

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      @[simp]
      theorem AlgebraicTopology.DoldKan.Γ₂N₂ToKaroubiIso_hom_app {C : Type u_1} [CategoryTheory.Category.{u_2, u_1} C] [CategoryTheory.Preadditive C] [CategoryTheory.Limits.HasFiniteCoproducts C] (X : CategoryTheory.SimplicialObject C) :
      AlgebraicTopology.DoldKan.Γ₂N₂ToKaroubiIso.hom.app X = AlgebraicTopology.DoldKan.Γ₂.map (AlgebraicTopology.DoldKan.toKaroubiCompN₂IsoN₁.hom.app X)
      @[simp]
      theorem AlgebraicTopology.DoldKan.Γ₂N₂ToKaroubiIso_inv_app {C : Type u_1} [CategoryTheory.Category.{u_2, u_1} C] [CategoryTheory.Preadditive C] [CategoryTheory.Limits.HasFiniteCoproducts C] (X : CategoryTheory.SimplicialObject C) :
      AlgebraicTopology.DoldKan.Γ₂N₂ToKaroubiIso.inv.app X = AlgebraicTopology.DoldKan.Γ₂.map (AlgebraicTopology.DoldKan.toKaroubiCompN₂IsoN₁.inv.app X)
      @[irreducible]

      The natural transformation N₂ ⋙ Γ₂ ⟶ 𝟭 (SimplicialObject C).

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        theorem AlgebraicTopology.DoldKan.compatibility_Γ₂N₁_Γ₂N₂_natTrans {C : Type u_1} [CategoryTheory.Category.{u_2, u_1} C] [CategoryTheory.Preadditive C] [CategoryTheory.Limits.HasFiniteCoproducts C] (X : CategoryTheory.SimplicialObject C) :
        AlgebraicTopology.DoldKan.Γ₂N₁.natTrans.app X = CategoryTheory.CategoryStruct.comp (AlgebraicTopology.DoldKan.Γ₂N₂ToKaroubiIso.app X).inv (AlgebraicTopology.DoldKan.Γ₂N₂.natTrans.app ((CategoryTheory.Idempotents.toKaroubi (CategoryTheory.SimplicialObject C)).obj X))
        theorem AlgebraicTopology.DoldKan.identity_N₂_objectwise {C : Type u_1} [CategoryTheory.Category.{u_2, u_1} C] [CategoryTheory.Preadditive C] [CategoryTheory.Limits.HasFiniteCoproducts C] (P : CategoryTheory.Idempotents.Karoubi (CategoryTheory.SimplicialObject C)) :
        CategoryTheory.CategoryStruct.comp (AlgebraicTopology.DoldKan.N₂Γ₂.inv.app (AlgebraicTopology.DoldKan.N₂.obj P)) (AlgebraicTopology.DoldKan.N₂.map (AlgebraicTopology.DoldKan.Γ₂N₂.natTrans.app P)) = CategoryTheory.CategoryStruct.id (AlgebraicTopology.DoldKan.N₂.obj P)
        theorem AlgebraicTopology.DoldKan.identity_N₂ {C : Type u_1} [CategoryTheory.Category.{u_2, u_1} C] [CategoryTheory.Preadditive C] [CategoryTheory.Limits.HasFiniteCoproducts C] :
        CategoryTheory.CategoryStruct.comp (CategoryTheory.CategoryStruct.id AlgebraicTopology.DoldKan.N₂ AlgebraicTopology.DoldKan.N₂Γ₂.inv) (CategoryTheory.CategoryStruct.comp (CategoryTheory.Functor.associator AlgebraicTopology.DoldKan.N₂ AlgebraicTopology.DoldKan.Γ₂ AlgebraicTopology.DoldKan.N₂).inv (AlgebraicTopology.DoldKan.Γ₂N₂.natTrans CategoryTheory.CategoryStruct.id AlgebraicTopology.DoldKan.N₂)) = CategoryTheory.CategoryStruct.id AlgebraicTopology.DoldKan.N₂
        @[simp]
        theorem AlgebraicTopology.DoldKan.Γ₂N₂_inv {C : Type u_1} [CategoryTheory.Category.{u_2, u_1} C] [CategoryTheory.Preadditive C] [CategoryTheory.Limits.HasFiniteCoproducts C] :
        AlgebraicTopology.DoldKan.Γ₂N₂.inv = AlgebraicTopology.DoldKan.Γ₂N₂.natTrans

        The unit isomorphism of the Dold-Kan equivalence.

        Equations
        • AlgebraicTopology.DoldKan.Γ₂N₂ = (CategoryTheory.asIso AlgebraicTopology.DoldKan.Γ₂N₂.natTrans).symm
        Instances For
          @[simp]
          theorem AlgebraicTopology.DoldKan.Γ₂N₁_inv {C : Type u_1} [CategoryTheory.Category.{u_2, u_1} C] [CategoryTheory.Preadditive C] [CategoryTheory.Limits.HasFiniteCoproducts C] :
          AlgebraicTopology.DoldKan.Γ₂N₁.inv = AlgebraicTopology.DoldKan.Γ₂N₁.natTrans

          The natural isomorphism toKaroubi (SimplicialObject C) ≅ N₁ ⋙ Γ₂.

          Equations
          • AlgebraicTopology.DoldKan.Γ₂N₁ = (CategoryTheory.asIso AlgebraicTopology.DoldKan.Γ₂N₁.natTrans).symm
          Instances For