Documentation

Mathlib.AlgebraicTopology.SimplicialSet.Basic

Simplicial sets #

A simplicial set is just a simplicial object in Type, i.e. a Type-valued presheaf on the simplex category.

(One might be tempted to call these "simplicial types" when working in type-theoretic foundations, but this would be unnecessarily confusing given the existing notion of a simplicial type in homotopy type theory.)

def SSet :
Type (u + 1)

The category of simplicial sets. This is the category of contravariant functors from SimplexCategory to Type u.

Equations
Instances For
    theorem SSet.hom_ext {X Y : SSet} {f g : X Y} (w : ∀ (n : SimplexCategoryᵒᵖ), f.app n = g.app n) :
    f = g

    The ulift functor SSet.{u} ⥤ SSet.{max u v} on simplicial sets.

    Equations
    Instances For
      def SSet.Truncated (n : ) :
      Type (u + 1)

      Truncated simplicial sets.

      Equations
      Instances For

        The ulift functor SSet.Truncated.{u} ⥤ SSet.Truncated.{max u v} on truncated simplicial sets.

        Equations
        Instances For
          theorem SSet.Truncated.hom_ext {n : } {X Y : Truncated n} {f g : X Y} (w : ∀ (n_1 : (SimplexCategory.Truncated n)ᵒᵖ), f.app n_1 = g.app n_1) :
          f = g
          @[reducible, inline]

          The truncation functor on simplicial sets.

          Equations
          Instances For
            @[reducible, inline]

            The n-skeleton as a functor SSet.Truncated n ⥤ SSet.

            Equations
            Instances For
              @[reducible, inline]

              The n-coskeleton as a functor SSet.Truncated n ⥤ SSet.

              Equations
              Instances For
                @[reducible, inline]

                The n-skeleton as an endofunctor on SSet.

                Equations
                Instances For
                  @[reducible, inline]

                  The n-coskeleton as an endofunctor on SSet.

                  Equations
                  Instances For
                    noncomputable def SSet.skAdj (n : ) :

                    The adjunction between the n-skeleton and n-truncation.

                    Equations
                    Instances For
                      noncomputable def SSet.coskAdj (n : ) :

                      The adjunction between n-truncation and the n-coskeleton.

                      Equations
                      Instances For

                        Since Truncated.inclusion is fully faithful, so is right Kan extension along it.

                        Equations
                        Instances For

                          Since Truncated.inclusion is fully faithful, so is left Kan extension along it.

                          Equations
                          Instances For
                            @[reducible, inline]
                            abbrev SSet.Augmented :
                            Type (u + 1)

                            The category of augmented simplicial sets, as a particular case of augmented simplicial objects.

                            Equations
                            Instances For