Documentation

Mathlib.AlgebraicTopology.SimplicialSet.KanComplex.MulStruct

Pointed simplices #

Given a simplicial set X, n : ℕ and x : X _⦋0⦌, we introduce the type X.PtSimplex n x of morphisms Δ[n] ⟶ X which send ∂Δ[n] to x. We introduce structures PtSimplex.RelStruct and PtSimplex.MulStruct which will be used in the definition of homotopy groups of Kan complexes.

@[reducible, inline]
abbrev SSet.PtSimplex (X : SSet) (n : ) (x : X.obj (Opposite.op (SimplexCategory.mk 0))) :

Given a simplicial set X, n : ℕ and x : X _⦋0⦌, this is the type of morphisms Δ[n] ⟶ X which are constant with value x on the boundary.

Equations
Instances For
    structure SSet.PtSimplex.RelStruct {X : SSet} {n : } {x : X.obj (Opposite.op (SimplexCategory.mk 0))} (f g : X.PtSimplex n x) (i : Fin (n + 1)) :

    For each i : Fin (n + 1), this is a variant of the homotopy relation on n-simplices that are constant on the boundary. Simplices f and g are related if they appear respectively as the i.castSucc and i.succ faces of a n + 1-simplex such that all the other faces are constant.

    Instances For
      structure SSet.PtSimplex.MulStruct {X : SSet} {n : } {x : X.obj (Opposite.op (SimplexCategory.mk 0))} (f g fg : X.PtSimplex n x) (i : Fin n) :

      For each i : Fin n, this structure is a candidate for the relation saying that fg is the product of f and g in the homotopy group (of a Kan complex). It is so if g, fg and f are respectively the i.castSucc.castSucc, i.castSucc.succ and i.succ.succ faces of a n + 1-simplex such that all the other faces are constant. (The multiplication on homotopy groups will be defined using i := Fin.last _, but in general, this structure is useful in order to obtain properties of RelStruct.)

      Instances For