Documentation

Mathlib.AlgebraicTopology.SimplicialSet.StdSimplex

The standard simplex #

We define the standard simplices Δ[n] as simplicial sets. See files SimplicialSet.Boundary and SimplicialSet.Horn for their boundaries∂Δ[n] and horns Λ[n, i]. (The notations are available via open Simplicial.)

The functor SimplexCategorySSet which sends ⦋n⦌ to the standard simplex Δ[n] is a cosimplicial object in the category of simplicial sets. (This functor is essentially given by the Yoneda embedding).

Equations
Instances For

    The functor SimplexCategorySSet which sends ⦋n⦌ to the standard simplex Δ[n] is a cosimplicial object in the category of simplicial sets. (This functor is essentially given by the Yoneda embedding).

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

      Pretty printer defined by notation3 command.

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

        Simplices of the standard simplex identify to morphisms in SimplexCategory.

        Equations
        Instances For

          If x : Δ[n] _⦋d⦌ and i : Fin (d + 1), we may evaluate x i : Fin (n + 1).

          Equations
          • One or more equations did not get rendered due to their size.
          theorem SSet.stdSimplex.ext {n d : } (x y : (stdSimplex.obj (SimplexCategory.mk n)).obj (Opposite.op (SimplexCategory.mk d))) (h : ∀ (i : Fin (d + 1)), x i = y i) :
          x = y
          theorem SSet.stdSimplex.ext_iff {n d : } {x y : (stdSimplex.obj (SimplexCategory.mk n)).obj (Opposite.op (SimplexCategory.mk d))} :
          x = y ∀ (i : Fin (d + 1)), x i = y i
          @[reducible, inline]

          Constructor for simplices of the standard simplex which takes a OrderHom as an input.

          Equations
          Instances For
            @[simp]
            theorem SSet.stdSimplex.objMk_apply {n m : } (f : Fin (m + 1) →o Fin (n + 1)) (i : Fin (m + 1)) :
            (objMk f) i = f i

            The m-simplices of the n-th standard simplex are the monotone maps from Fin (m+1) to Fin (n+1).

            Equations
            Instances For

              The canonical bijection (stdSimplex.obj n ⟶ X) ≃ X.obj (op n).

              Equations
              Instances For

                The (degenerate) m-simplex in the standard simplex concentrated in vertex k.

                Equations
                Instances For

                  The 0-simplices of Δ[n] identify to the elements in Fin (n + 1).

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

                    The edge of the standard simplex with endpoints a and b.

                    Equations
                    Instances For
                      theorem SSet.stdSimplex.coe_edge_down_toOrderHom (n : ) (a b : Fin (n + 1)) (hab : a b) :
                      def SSet.stdSimplex.triangle {n : } (a b c : Fin (n + 1)) (hab : a b) (hbc : b c) :

                      The triangle in the standard simplex with vertices a, b, and c.

                      Equations
                      Instances For
                        theorem SSet.stdSimplex.coe_triangle_down_toOrderHom {n : } (a b c : Fin (n + 1)) (hab : a b) (hbc : b c) :

                        Given S : Finset (Fin (n + 1)), this is the corresponding face of Δ[n], as a subcomplex.

                        Equations
                        • One or more equations did not get rendered due to their size.
                        Instances For
                          @[simp]
                          theorem SSet.stdSimplex.mem_face_iff {n : } (S : Finset (Fin (n + 1))) {d : } (x : (stdSimplex.obj (SimplexCategory.mk n)).obj (Opposite.op (SimplexCategory.mk d))) :
                          x (face S).obj (Opposite.op (SimplexCategory.mk d)) ∀ (i : Fin (d + 1)), x i S
                          theorem SSet.stdSimplex.face_inter_face {n : } (S₁ S₂ : Finset (Fin (n + 1))) :
                          face S₁face S₂ = face (S₁S₂)
                          @[reducible, inline]

                          The subcomplex of a simplicial set that is generated by a simplex.

                          Equations
                          Instances For
                            theorem SSet.stdSimplex.face_eq_ofSimplex {n : } (S : Finset (Fin (n + 1))) (m : ) (e : Fin (m + 1) ≃o { x : Fin (n + 1) // x S }) :

                            If S : Finset (Fin (n + 1)) is order isomorphic to Fin (m + 1), then the face face S of Δ[n] is representable by m, i.e. face S is isomorphic to Δ[m], see stdSimplex.isoOfRepresentableBy.

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

                              If a simplicial set X is representable by ⦋m⦌ for some m : ℕ, then this is the corresponding isomorphism Δ[m] ≅ X.

                              Equations
                              Instances For

                                The functor which sends ⦋n⦌ to the simplicial set Δ[n] equipped by the obvious augmentation towards the terminal object of the category of sets.

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