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
- SSet.OneTruncation₂ S = S.obj (Opposite.op { obj := SimplexCategory.mk 0, property := SSet.OneTruncation₂.proof_1 })
Instances For
Abbreviations for face maps in the 2-truncated simplex category.
Equations
- SSet.δ₂ i hn hn' = SimplexCategory.δ i
Instances For
Abbreviations for degeneracy maps in the 2-truncated simplex category.
Equations
- SSet.σ₂ i hn hn' = SimplexCategory.σ i
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.
- edge : S.obj (Opposite.op { obj := SimplexCategory.mk 1, property := ⋯ })
An arrow in
OneTruncation₂.Hom X Y
includes the data of a 1-simplex. An arrow in
OneTruncation₂.Hom X Y
includes a source equality.An arrow in
OneTruncation₂.Hom X Y
includes a target equality.
Instances For
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
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
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
- SSet.OneTruncation₂.ofNerve₂ C = CategoryTheory.ReflQuiv.isoOfEquiv SSet.OneTruncation₂.nerveEquiv SSet.OneTruncation₂.nerveHomEquiv ⋯
Instances For
The refl quiver underlying a nerve is naturally isomorphic to the refl quiver underlying the category.
Equations
Instances For
The map that picks up the initial vertex of a 2-simplex, as a morphism in the 2-truncated simplex category.
Equations
Instances For
The map that picks up the middle vertex of a 2-simplex, as a morphism in the 2-truncated simplex category.
Equations
Instances For
The map that picks up the final vertex of a 2-simplex, as a morphism in the 2-truncated simplex category.
Equations
Instances For
The initial vertex of a 2-simplex in a 2-truncated simplicial set.
Equations
- SSet.Truncated.ev0₂ φ = V.map SSet.Truncated.ι0₂.op φ
Instances For
The middle vertex of a 2-simplex in a 2-truncated simplicial set.
Equations
- SSet.Truncated.ev1₂ φ = V.map SSet.Truncated.ι1₂.op φ
Instances For
The final vertex of a 2-simplex in a 2-truncated simplicial set.
Equations
- SSet.Truncated.ev2₂ φ = V.map SSet.Truncated.ι2₂.op φ
Instances For
The 0th face of a 2-simplex, as a morphism in the 2-truncated simplex category.
Instances For
The 1st face of a 2-simplex, as a morphism in the 2-truncated simplex category.
Instances For
The 2nd face of a 2-simplex, as a morphism in the 2-truncated simplex category.
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
- SSet.Truncated.ev12₂ φ = { edge := V.map SSet.Truncated.δ0₂.op φ, src_eq := ⋯, tgt_eq := ⋯ }
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
- SSet.Truncated.ev02₂ φ = { edge := V.map SSet.Truncated.δ1₂.op φ, src_eq := ⋯, tgt_eq := ⋯ }
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
- SSet.Truncated.ev01₂ φ = { edge := V.map SSet.Truncated.δ2₂.op φ, src_eq := ⋯, tgt_eq := ⋯ }
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
.
- mk {V : SSet.Truncated 2} (φ : V.obj (Opposite.op { obj := SimplexCategory.mk 2, property := ⋯ })) : SSet.Truncated.HoRel₂ { as := V.toPrefunctor.2 SSet.Truncated.ι0₂.op φ } { as := V.toPrefunctor.2 SSet.Truncated.ι2₂.op φ } (Quot.mk (CategoryTheory.Quotient.CompClosure CategoryTheory.Cat.FreeReflRel) (SSet.Truncated.ev02₂ φ).toPath) (Quot.mk (CategoryTheory.Quotient.CompClosure CategoryTheory.Cat.FreeReflRel) ((SSet.Truncated.ev01₂ φ).toPath.comp (SSet.Truncated.ev12₂ φ).toPath))
Instances For
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
- V.HomotopyCategory = CategoryTheory.Quotient SSet.Truncated.HoRel₂
Instances For
Equations
- V.instCategoryHomotopyCategory = inferInstanceAs (CategoryTheory.Category.{?u.12, ?u.12} (CategoryTheory.Quotient SSet.Truncated.HoRel₂))
A canonical functor from the free category on the refl quiver underlying a 2-truncated
simplicial set V
to its homotopy category.
Equations
- SSet.Truncated.HomotopyCategory.quotientFunctor V = CategoryTheory.Quotient.functor SSet.Truncated.HoRel₂
Instances For
By Quotient.lift_unique'
(not Quotient.lift
) we have that quotientFunctor V
is an
epimorphism.
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.