Documentation

Mathlib.AlgebraicTopology.SimplicialSet.HomotopyCat

The homotopy category of a simplicial set #

The homotopy category of a simplicial set is defined as a quotient of the free category on its underlying reflexive quiver (equivalently its one truncation). The quotient imposes an additional hom relation on this free category, asserting that f ≫ g = h whenever f, g, and h are respectively the 2nd, 0th, and 1st faces of a 2-simplex.

In fact, the associated functor

SSet.hoFunctor : SSet.{u} ⥤ Cat.{u, u} := SSet.truncation 2 ⋙ SSet.hoFunctor₂

is defined by first restricting from simplicial sets to 2-truncated simplicial sets (throwing away the data that is not used for the construction of the homotopy category) and then composing with an analogously defined SSet.hoFunctor₂ : SSet.Truncated.{u} 2 ⥤ Cat.{u,u} implemented relative to the syntax of the 2-truncated simplex category.

TODO: Future work will show the functor SSet.hoFunctor to be left adjoint to the nerve by providing an analogous decomposition of the nerve functor, made by possible by the fact that nerves of categories are 2-coskeletal, and then composing a pair of adjunctions, which factor through the category of 2-truncated simplicial sets.

A 2-truncated simplicial set S has an underlying refl quiver with S _[0]₂ as its underlying type.

Equations
Instances For
    @[reducible, inline]
    abbrev SSet.δ₂ {n : } (i : Fin (n + 2)) (hn : (SimplexCategory.mk n).len 2 := by decide) (hn' : (SimplexCategory.mk (n + 1)).len 2 := by decide) :
    { obj := SimplexCategory.mk n, property := hn } { obj := SimplexCategory.mk (n + 1), property := hn' }

    Abbreviations for face maps in the 2-truncated simplex category.

    Equations
    Instances For
      @[reducible, inline]
      abbrev SSet.σ₂ {n : } (i : Fin (n + 1)) (hn : (SimplexCategory.mk (n + 1)).len 2 := by decide) (hn' : (SimplexCategory.mk n).len 2 := by decide) :
      { obj := SimplexCategory.mk (n + 1), property := hn } { obj := SimplexCategory.mk n, property := hn' }

      Abbreviations for degeneracy maps in the 2-truncated simplex category.

      Equations
      Instances For

        The hom-types of the refl quiver underlying a simplicial set S are types of edges in S _[1]₂ together with source and target equalities.

        Instances For
          theorem SSet.OneTruncation₂.Hom.ext {S : SSet.Truncated 2} {X Y : SSet.OneTruncation₂ S} {x y : X.Hom Y} (edge : x.edge = y.edge) :
          x = y

          A 2-truncated simplicial set S has an underlying refl quiver SSet.OneTruncation₂ S.

          Equations
          • One or more equations did not get rendered due to their size.

          The functor that carries a 2-truncated simplicial set to its underlying refl quiver.

          Equations
          • One or more equations did not get rendered due to their size.
          Instances For
            @[simp]
            theorem SSet.oneTruncation₂_map_obj {S T : SSet.Truncated 2} (F : S T) (a✝ : S.obj (Opposite.op { obj := SimplexCategory.mk 0, property := SSet.oneTruncation₂.proof_1 })) :
            (SSet.oneTruncation₂.map F).obj a✝ = F.app (Opposite.op { obj := SimplexCategory.mk 0, property := SSet.oneTruncation₂.proof_1 }) a✝
            @[simp]
            theorem SSet.oneTruncation₂_map_map_edge {S T : SSet.Truncated 2} (F : S T) {X✝ Y✝ : ((fun (S : SSet.Truncated 2) => CategoryTheory.ReflQuiv.of (SSet.OneTruncation₂ S)) S)} (f : X✝ Y✝) :
            ((SSet.oneTruncation₂.map F).map f).edge = F.app (Opposite.op { obj := SimplexCategory.mk 1, property := SSet.oneTruncation₂.proof_2 }) f.edge
            theorem SSet.OneTruncation₂.hom_ext {S : SSet.Truncated 2} {x y : SSet.OneTruncation₂ S} {f g : x y} :
            f.edge = g.edgef = g

            An equivalence between the type of objects underlying a category and the type of 0-simplices in the 2-truncated nerve.

            Equations
            • One or more equations did not get rendered due to their size.
            Instances For
              @[simp]
              def SSet.OneTruncation₂.nerveHomEquiv {C : Type u} [CategoryTheory.Category.{v, u} C] (X Y : SSet.OneTruncation₂ ((SSet.truncation 2).obj (CategoryTheory.nerve C))) :
              (X Y) (SSet.OneTruncation₂.nerveEquiv X SSet.OneTruncation₂.nerveEquiv Y)

              A hom equivalence over the function OneTruncation₂.nerveEquiv.

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

                The refl quiver underlying a nerve is isomorphic to the refl quiver underlying the category.

                Equations
                Instances For
                  def SSet.Truncated.ι0₂ :
                  { obj := SimplexCategory.mk 0, property := } { obj := SimplexCategory.mk 2, property := }

                  The map that picks up the initial vertex of a 2-simplex, as a morphism in the 2-truncated simplex category.

                  Equations
                  Instances For
                    def SSet.Truncated.ι1₂ :
                    { obj := SimplexCategory.mk 0, property := } { obj := SimplexCategory.mk 2, property := }

                    The map that picks up the middle vertex of a 2-simplex, as a morphism in the 2-truncated simplex category.

                    Equations
                    Instances For
                      def SSet.Truncated.ι2₂ :
                      { obj := SimplexCategory.mk 0, property := } { obj := SimplexCategory.mk 2, property := }

                      The map that picks up the final vertex of a 2-simplex, as a morphism in the 2-truncated simplex category.

                      Equations
                      Instances For
                        def SSet.Truncated.ev0₂ {V : SSet.Truncated 2} (φ : V.obj (Opposite.op { obj := SimplexCategory.mk 2, property := })) :

                        The initial vertex of a 2-simplex in a 2-truncated simplicial set.

                        Equations
                        Instances For
                          def SSet.Truncated.ev1₂ {V : SSet.Truncated 2} (φ : V.obj (Opposite.op { obj := SimplexCategory.mk 2, property := })) :

                          The middle vertex of a 2-simplex in a 2-truncated simplicial set.

                          Equations
                          Instances For
                            def SSet.Truncated.ev2₂ {V : SSet.Truncated 2} (φ : V.obj (Opposite.op { obj := SimplexCategory.mk 2, property := })) :

                            The final vertex of a 2-simplex in a 2-truncated simplicial set.

                            Equations
                            Instances For
                              def SSet.Truncated.δ0₂ :
                              { obj := SimplexCategory.mk 1, property := } { obj := SimplexCategory.mk 2, property := }

                              The 0th face of a 2-simplex, as a morphism in the 2-truncated simplex category.

                              Equations
                              Instances For
                                def SSet.Truncated.δ1₂ :
                                { obj := SimplexCategory.mk 1, property := } { obj := SimplexCategory.mk 2, property := }

                                The 1st face of a 2-simplex, as a morphism in the 2-truncated simplex category.

                                Equations
                                Instances For
                                  def SSet.Truncated.δ2₂ :
                                  { obj := SimplexCategory.mk 1, property := } { obj := SimplexCategory.mk 2, property := }

                                  The 2nd face of a 2-simplex, as a morphism in the 2-truncated simplex category.

                                  Equations
                                  Instances For

                                    The arrow in the ReflQuiver OneTruncation₂ V of a 2-truncated simplicial set arising from the 0th face of a 2-simplex.

                                    Equations
                                    Instances For

                                      The arrow in the ReflQuiver OneTruncation₂ V of a 2-truncated simplicial set arising from the 1st face of a 2-simplex.

                                      Equations
                                      Instances For

                                        The arrow in the ReflQuiver OneTruncation₂ V of a 2-truncated simplicial set arising from the 2nd face of a 2-simplex.

                                        Equations
                                        Instances For

                                          The 2-simplices in a 2-truncated simplicial set V generate a hom relation on the free category on the underlying refl quiver of V.

                                          Instances For
                                            theorem SSet.Truncated.HoRel₂.mk' {V : SSet.Truncated 2} (φ : V.obj (Opposite.op { obj := SimplexCategory.mk 2, property := })) {X₀ X₁ X₂ : SSet.OneTruncation₂ V} (f₀₁ : X₀ X₁) (f₁₂ : X₁ X₂) (f₀₂ : X₀ X₂) (h₀₁ : f₀₁.edge = V.map (SSet.δ₂ 2 ).op φ) (h₁₂ : f₁₂.edge = V.map (SSet.δ₂ 0 ).op φ) (h₀₂ : f₀₂.edge = V.map (SSet.δ₂ 1 ).op φ) :
                                            SSet.Truncated.HoRel₂ { as := X₀ } { as := X₂ } (Quot.mk (CategoryTheory.Quotient.CompClosure CategoryTheory.Cat.FreeReflRel) f₀₂.toPath) (Quot.mk (CategoryTheory.Quotient.CompClosure CategoryTheory.Cat.FreeReflRel) (f₀₁.toPath.comp f₁₂.toPath))

                                            A 2-simplex whose faces are identified with certain arrows in OneTruncation₂ V defines a term of type HoRel₂ between those arrows.

                                            The type underlying the homotopy category of a 2-truncated simplicial set V.

                                            Equations
                                            Instances For

                                              A canonical functor from the free category on the refl quiver underlying a 2-truncated simplicial set V to its homotopy category.

                                              Equations
                                              Instances For
                                                def SSet.Truncated.mapHomotopyCategory {V W : SSet.Truncated 2} (F : V W) :
                                                CategoryTheory.Functor V.HomotopyCategory W.HomotopyCategory

                                                A map of 2-truncated simplicial sets induces a functor between homotopy categories.

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

                                                  The functor that takes a 2-truncated simplicial set to its homotopy category.

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

                                                    The functor that takes a simplicial set to its homotopy category by passing through the 2-truncation.

                                                    Equations
                                                    Instances For