Documentation

Mathlib.AlgebraicTopology.SimplexCategory

The simplex category #

We construct a skeletal model of the simplex category, with objects and the morphism n ⟶ m being the monotone maps from Fin (n+1) to Fin (m+1).

We show that this category is equivalent to NonemptyFinLinOrd.

Remarks #

The definitions SimplexCategory and SimplexCategory.Hom are marked as irreducible.

We provide the following functions to work with these objects:

  1. SimplexCategory.mk creates an object of SimplexCategory out of a natural number. Use the notation [n] in the Simplicial locale.
  2. SimplexCategory.len gives the "length" of an object of SimplexCategory, as a natural.
  3. SimplexCategory.Hom.mk makes a morphism out of a monotone map between Fin's.
  4. SimplexCategory.Hom.toOrderHom gives the underlying monotone map associated to a term of SimplexCategory.Hom.
@[irreducible]

The simplex category:

  • objects are natural numbers n : ℕ
  • morphisms from n to m are monotone functions Fin (n+1) → Fin (m+1)
Instances For

    Interpret a natural number as an object of the simplex category.

    Instances For

      the n-dimensional simplex can be denoted [n]

      Instances For

        The length of an object of SimplexCategory.

        Instances For
          def SimplexCategory.rec {F : SimplexCategorySort u_1} (h : (n : ) → F (SimplexCategory.mk n)) (X : SimplexCategory) :
          F X

          A recursor for SimplexCategory. Use it as induction Δ using SimplexCategory.rec.

          Instances For
            @[irreducible]

            Morphisms in the SimplexCategory.

            Instances For

              Make a moprhism in SimplexCategory from a monotone map of Fin's.

              Instances For

                Recover the monotone map from a morphism in the simplex category.

                Instances For

                  Identity morphisms of SimplexCategory.

                  Instances For

                    The constant morphism from [0].

                    Instances For

                      Make a morphism [n] ⟶ [m] from a monotone map between fin's. This is useful for constructing morphisms between [n] directly without identifying n with [n].len.

                      Instances For

                        Generating maps for the simplex category #

                        TODO: prove that the simplex category is equivalent to one given by the following generators and relations.

                        The i-th face map from [n] to [n+1]

                        Instances For

                          The i-th degeneracy map from [n+1] to [n]

                          Instances For
                            @[simp]
                            theorem SimplexCategory.skeletalFunctor_map :
                            ∀ {X Y : SimplexCategory} (f : X Y), SimplexCategory.skeletalFunctor.map f = { toFun := fun i => { down := ↑(SimplexCategory.Hom.toOrderHom f) i.down }, monotone' := (_ : ∀ (i j : ↑((fun a => NonemptyFinLinOrd.of (ULift.{v, 0} (Fin (SimplexCategory.len a + 1)))) X)), i j↑(SimplexCategory.Hom.toOrderHom f) i.down ↑(SimplexCategory.Hom.toOrderHom f) j.down) }

                            The equivalence that exhibits SimplexCategory as skeleton of NonemptyFinLinOrd

                            Instances For

                              The truncated simplex category.

                              Instances For

                                The fully faithful inclusion of the truncated simplex category into the usual simplex category.

                                Instances For

                                  A morphism in SimplexCategory is a monomorphism precisely when it is an injective function

                                  A morphism in SimplexCategory is an epimorphism if and only if it is a surjective function

                                  This functor SimplexCategory ⥤ Cat sends [n] (for n : ℕ) to the category attached to the ordered set {0, 1, ..., n}

                                  Instances For