Edge x₀ x₁ is a wrapper around a 1-simplex in a 2-truncated simplicial set
with source x₀ and target x₁.
- simplex : X.obj (Opposite.op { obj := SimplexCategory.mk 1, property := ⋯ })
Instances For
Equations
Instances For
CompStruct e₀₁ e₁₂ e₀₂ is a wrapper around a 2-simplex in a 2-truncated simplicial set
with edges e₀₁, e₁₂, e₀₂ in the obvious configuration.
- simplex : X.obj (Opposite.op { obj := SimplexCategory.mk 2, property := ⋯ })
- h₀₁ : X.map (SimplexCategory.Truncated.Hom.tr (SimplexCategory.δ 2) ⋯ ⋯).op self.simplex = e₀₁.simplex
- h₁₂ : X.map (SimplexCategory.Truncated.Hom.tr (SimplexCategory.δ 0) ⋯ ⋯).op self.simplex = e₁₂.simplex
- h₀₂ : X.map (SimplexCategory.Truncated.Hom.tr (SimplexCategory.δ 1) ⋯ ⋯).op self.simplex = e₀₂.simplex
Instances For
A 2-truncated quasicategory is a 2-truncated simplicial set with 3 properties: (2, 1)-filling: any path of length 2 in may be filled to a 2-simplex whose spine equals the given path. (3, 1)-filling: given any path f of length 3, 2-simplices σ₃ and σ₀ filling the restricted paths f₀₁₂ and f₁₂₃ respectively, and a 2-simplex σ₂ filling the path formed by f₀₁ and the diagonal of σ₀, there is a 2-simplex σ₁ filling the path formed by the diagonal of σ₃ and f₂₃ and whose diagonal is the diagonal of σ₂. (3, 2)-filling: given any path f of length 3, 2-simplices σ₃ and σ₀ filling the restricted paths f₀₁₂ and f₁₂₃ respectively, and a 2-simplex σ₁ filling the path formed by f₂₃ and the diagonal of σ₃, there is a 2-simplex σ₂ filling the path formed by f₀₁ and the diagonal of σ₀ and whose diagonal is the diagonal of σ₁.
- fill21 {x₀ x₁ x₂ : X.obj (Opposite.op { obj := SimplexCategory.mk 0, property := ⋯ })} (e₀₁ : Edge x₀ x₁) (e₁₂ : Edge x₁ x₂) : Nonempty ((e₀₂ : Edge x₀ x₂) × CompStruct e₀₁ e₁₂ e₀₂)
- fill31 {x₀ x₁ x₂ x₃ : X.obj (Opposite.op { obj := SimplexCategory.mk 0, property := ⋯ })} {e₀₁ : Edge x₀ x₁} {e₁₂ : Edge x₁ x₂} {e₂₃ : Edge x₂ x₃} {e₀₂ : Edge x₀ x₂} {e₁₃ : Edge x₁ x₃} {e₀₃ : Edge x₀ x₃} (f₃ : CompStruct e₀₁ e₁₂ e₀₂) (f₀ : CompStruct e₁₂ e₂₃ e₁₃) (f₂ : CompStruct e₀₁ e₁₃ e₀₃) : Nonempty (CompStruct e₀₂ e₂₃ e₀₃)
- fill32 {x₀ x₁ x₂ x₃ : X.obj (Opposite.op { obj := SimplexCategory.mk 0, property := ⋯ })} {e₀₁ : Edge x₀ x₁} {e₁₂ : Edge x₁ x₂} {e₂₃ : Edge x₂ x₃} {e₀₂ : Edge x₀ x₂} {e₁₃ : Edge x₁ x₃} {e₀₃ : Edge x₀ x₃} (f₃ : CompStruct e₀₁ e₁₂ e₀₂) (f₀ : CompStruct e₁₂ e₂₃ e₁₃) (f₁ : CompStruct e₀₂ e₂₃ e₀₃) : Nonempty (CompStruct e₀₁ e₁₃ e₀₃)
Instances
Given the data of two consecutive edges e₀₁ and e₁₂, construct a map
Λ[2, 1].toSSet ⟶ S which restricts to maps Δ[1] ⟶ S corresponding
to the two edges (this is made precise in the lemmas horn_from_edges_restr₀ and
horn_from_edges_restr₁).
Equations
Instances For
See horn_from_edges for details.
See horn_from_edges for details.
Given a map Δ[2] ⟶ S extending the horn given by horn_from_edges, construct
and edge e₀₂ such that e₀₁, e₁₂, e₀₂ bound a 2-simplex of S (this is witnessed
by CompStruct e₀₁ e₁₂ e₀₂).
Equations
- One or more equations did not get rendered due to their size.
Instances For
Choose the i-th face from the given faces, where i is represented by a : horn₃₁.R,
i.e. a is 0, 2 or 3
Equations
- SSet.horn₃₁.chooseFace f₃ f₀ f₂ SSet.horn₃₁.R.f₀ = SSet.yonedaEquiv.symm f₀.simplex
- SSet.horn₃₁.chooseFace f₃ f₀ f₂ SSet.horn₃₁.R.f₂ = SSet.yonedaEquiv.symm f₂.simplex
- SSet.horn₃₁.chooseFace f₃ f₀ f₂ SSet.horn₃₁.R.f₃ = SSet.yonedaEquiv.symm f₃.simplex
Instances For
Equations
- SSet.horn₃₁.chooseFace' f₃ f₀ f₂ SSet.horn₃₁.R.f₀ = f₀.simplex
- SSet.horn₃₁.chooseFace' f₃ f₀ f₂ SSet.horn₃₁.R.f₂ = f₂.simplex
- SSet.horn₃₁.chooseFace' f₃ f₀ f₂ SSet.horn₃₁.R.f₃ = f₃.simplex
Instances For
Equations
Instances For
Use the fact that Λ[3, 1] is the coequalizer of multicoforkFromFaces allows the
construction of a map Λ[3, 1].toSSet ⟶ S.
Equations
- SSet.horn₃₁.fromFaces f₃ f₀ f₂ = SSet.horn₃₁.isMulticoeq.desc (SSet.horn₃₁.multicoforkFromFaces f₃ f₀ f₂)
Instances For
Given a map Δ[3] ⟶ S extending the horn given by fromFaces, obtain a
2-simplex bounded by edges e₀₂, e₂₃ and e₀₃. See also Quasicategory₂.fill31.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Choose the i-th face from the given faces, where i is represented by a : horn₃₂.R,
i.e. a is 0, 1 or 3
Equations
- SSet.horn₃₂.chooseFace f₃ f₀ f₁ SSet.horn₃₂.R.f₀ = SSet.yonedaEquiv.symm f₀.simplex
- SSet.horn₃₂.chooseFace f₃ f₀ f₁ SSet.horn₃₂.R.f₁ = SSet.yonedaEquiv.symm f₁.simplex
- SSet.horn₃₂.chooseFace f₃ f₀ f₁ SSet.horn₃₂.R.f₃ = SSet.yonedaEquiv.symm f₃.simplex
Instances For
Equations
- SSet.horn₃₂.chooseFace' f₃ f₀ f₁ SSet.horn₃₂.R.f₀ = f₀.simplex
- SSet.horn₃₂.chooseFace' f₃ f₀ f₁ SSet.horn₃₂.R.f₁ = f₁.simplex
- SSet.horn₃₂.chooseFace' f₃ f₀ f₁ SSet.horn₃₂.R.f₃ = f₃.simplex
Instances For
Equations
Instances For
Use the fact that Λ[3, 2] is the coequalizer of multicoforkFromFaces allows the
construction of a map Λ[3, 2].toSSet ⟶ S.
Equations
- SSet.horn₃₂.fromFaces f₃ f₀ f₁ = SSet.horn₃₂.multicoforkIsMulticoeq.desc (SSet.horn₃₂.multicoforkFromFaces f₃ f₀ f₁)
Instances For
Given a map Δ[3] ⟶ S extending the horn given by fromFaces, obtain a
2-simplex bounded by edges e₀₁, e₁₃ and e₀₃. See also Quasicategory₂.fill32.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The 2-truncation of a quasi-category is a 2-truncated quasi-category.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
Instances For
Two edges f and g are left homotopic if there is a 2-simplex with
(0, 1)-edge f, (0, 2)-edge g and (1, 2)-edge id. We use Nonempty to
have a Prop valued HomotopicL.
Equations
Instances For
See HomotopicL.
Equations
Instances For
Left homotopy relation is reflexive
Equations
- ⋯ = ⋯
Instances For
Left homotopy relation is symmetric
Equations
- ⋯ = ⋯
Instances For
Left homotopy relation is transitive
Equations
- ⋯ = ⋯
Instances For
Right homotopy relation is reflexive
Equations
- ⋯ = ⋯
Instances For
Right homotopy relation is symmetric
Equations
- ⋯ = ⋯
Instances For
Right homotopy relation is transitive
Equations
- ⋯ = ⋯
Instances For
The right and left homotopy relations coincide
The homotopy category of a 2-truncated quasicategory A has as objects the 0-simplices of A
Equations
- SSet.Quasicategory₂.HomotopyCategory₂ A = A.obj (Opposite.op { obj := SimplexCategory.mk 0, property := SSet.Truncated.edgeMap._proof_1 })
Instances For
Equations
- SSet.Quasicategory₂.instSetoidEdge x₀ x₁ = { r := SSet.Truncated.HomotopicL, iseqv := ⋯ }
The morphisms between two vertices x₀, x₁ in HomotopyCategory₂ A are homotopy classes
of 1-simplices between x₀ and x₁.
Equations
- SSet.Quasicategory₂.HEdge x₀ x₁ = Quotient (SSet.Quasicategory₂.instSetoidEdge x₀ x₁)
Instances For
Given two consecutive edges f, g in a 2-truncated quasicategory, nonconstructively choose
an edge that is the diagonal of a 2-simplex with spine given by f and g.
Equations
Instances For
Equations
Instances For
The edge composeEdges f g is the unique edge up to homotopy such that there is
a 2-simplex with spine given by f and g.
The compositions of homotopic edges are homotopic
Composition of morphisms in HomotopyCategory₂ A is given by lifting composeEdges.
Equations
- SSet.Quasicategory₂.composeHEdges f g = Quotient.lift₂ (fun (f : SSet.Truncated.Edge x₀ x₁) (g : SSet.Truncated.Edge x₁ x₂) => ⟦SSet.Quasicategory₂.composeEdges f g⟧) ⋯ f g
Instances For
Equations
- One or more equations did not get rendered due to their size.
Equations
- SSet.Quasicategory₂.instCategoryHomotopyCategory₂ = { toCategoryStruct := SSet.Quasicategory₂.instCategoryStructHomotopyCategory₂, id_comp := ⋯, comp_id := ⋯, assoc := ⋯ }
The reflexive prefunctor sending edges (in the 1-truncation) of A to their homotopy class.
Equations
- SSet.Quasicategory₂.quotientReflPrefunctor₂ = { obj := id, map := fun {X Y : SSet.OneTruncation₂ A} (f : X ⟶ Y) => Quotient.mk' { simplex := f.edge, h₀ := ⋯, h₁ := ⋯ }, map_id := ⋯ }
Instances For
By the adjunction ReflQuiv.adj, we obtain a functor from the free category on the reflexive
quiver underlying A to the homotopy category corresponding to quotientReflPrefunctor₂.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The adjoint relation between quotientReflPrefunctor₂ and quotientFunctor₂ expressed
on the level of functors.
quotientFunctor₂ respects the hom relation HoRel₂.
An edge from x₀ to x₁ in a 2-truncated simplicial set defines an arrow in the refl quiver
OneTruncation₂.{u} A) from x₀ to x₁.
Equations
- SSet.Quasicategory₂.edgeToHom f = { edge := f.simplex, src_eq := ⋯, tgt_eq := ⋯ }
Instances For
An edge from x₀ to x₁ in a 2-truncated simplicial set defines an arrow in the free category
generated from the refl quiver OneTruncation₂.{u} A) from x₀ to x₁.
Equations
Instances For
Two (left) homotopic edges f, g are equivalent under the hom-relation HoRel₂
generated by 2-simplices.
If a reflexive prefunctor F : FreeRefl (OneTruncation₂ A) ⥤rq C respects
the hom-relation HoRel₂, then it can be lifted to HomotopyCategory₂ A.
Equations
- One or more equations did not get rendered due to their size.
Instances For
If a functor F : FreeRefl (OneTruncation₂ A) ⥤ C respects the hom-relation HoRel₂,
then it can be lifted to HomotopyCategory₂ A (see the weaker statement liftRq₂).
Equations
- One or more equations did not get rendered due to their size.
Instances For
Lifts to the homotopy category are unique.
Since both HomotopyCategory A and HomotopyCategory₂ A satisfy the same universal property,
they are isomorphic.
Equations
- One or more equations did not get rendered due to their size.