Documentation

Mathlib.AlgebraicTopology.SimplicialSet.ProdStdSimplex

Binary product of standard simplices #

In this file, we show that Δ[p] ⊗ Δ[q] identifies to the nerve of ULift (Fin (p + 1) × Fin (q + 1)). We relate the n-simplices of Δ[p] ⊗ Δ[q] to order preserving maps Fin (n + 1) →o Fin (p + 1) × Fin (q + 1), Via this bijection, a simplex in Δ[p] ⊗ Δ[q] is nondegenerate iff the corresponding monotone map Fin (n + 1) →o Fin (p + 1) × Fin (q + 1) is injective (or a strict mono).

We also show that the dimension of Δ[p] ⊗ Δ[q] is ≤ p + q.

n-simplices in Δ[p] ⊗ Δ[q] identify to order preserving maps Fin (n + 1) →o Fin (p + 1) × Fin (q + 1).

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

    The binary product Δ[p] ⊗ Δ[q] identifies to the nerve of ULift (Fin (p + 1) × Fin (q + 1)).

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

      Given a n-simplex x in Δ[p] ⊗ Δ[q], this is the order preserving map Fin (n + 1) →o Fin (m + 1) (with p + q = m) which corresponds to the sum of the two components of objEquiv x : Fin (n + 1) →o Fin (p + 1) × Fin (q + 1).

      Equations
      Instances For