Documentation

Mathlib.AlgebraicTopology.SimplicialSet.AnodyneExtensions.Rank

Rank functions for pairings #

We introduce types of (weak) rank functions for a pairing P of a subcomplex A of a simplicial set X. These are functions f : P.II → α such that P.AncestralRel x y implies f x < f y (in the weak case, we require this only under the additional condition that x and y are of the same dimension). Such rank functions are used in order to show that the ancestrality relation on P.II is well founded, i.e. that P is regular (when we already know P is proper). Conversely, we shall show that if P is regular, then P.RankFunction is non empty (TODO @joelriou).

(We also introduce similar definitions for the structure PairingCore.)

References #

structure SSet.Subcomplex.Pairing.RankFunction {X : SSet} {A : X.Subcomplex} (P : A.Pairing) (α : Type v) [PartialOrder α] :
Type (max u v)

A rank function for a pairing is a function from the type (II) simplices to a partially ordered type which maps ancestrality relations to strict inequalities.

Instances For
    structure SSet.Subcomplex.Pairing.WeakRankFunction {X : SSet} {A : X.Subcomplex} (P : A.Pairing) (α : Type v) [PartialOrder α] :
    Type (max u v)

    A weak rank function for a pairing is a function from the type (II) simplices to a partially ordered type which maps an ancestrality relation between simplices of the same dimension to a strict inequality.

    Instances For

      The weak rank function attached to a rank function.

      Equations
      Instances For
        @[simp]
        theorem SSet.Subcomplex.Pairing.RankFunction.toWeakRankFunction_rank {X : SSet} {A : X.Subcomplex} (P : A.Pairing) (α : Type v) [PartialOrder α] (f : P.RankFunction α) (a✝ : P.II) :
        (toWeakRankFunction P α f).rank a✝ = f.rank a✝
        structure SSet.Subcomplex.PairingCore.RankFunction {X : SSet} {A : X.Subcomplex} (h : A.PairingCore) (α : Type v) [PartialOrder α] :
        Type (max u_1 v)

        A rank function for h : A.PairingCore is a function from the index type h.ι to a partially ordered type which maps the ancestrality relations to strict inequalities.

        Instances For
          structure SSet.Subcomplex.PairingCore.WeakRankFunction {X : SSet} {A : X.Subcomplex} (h : A.PairingCore) (α : Type v) [PartialOrder α] :
          Type (max u_1 v)

          A weak rank function h : A.PairingCore is a function from the index type h.ι to a partially ordered type which maps an ancestrality relation between indices of the same dimension to a strict inequality.

          Instances For

            Rank functions for h : A.PairingCore correspond to rank functions for h.pairing : A.Pairing.

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

              Weak rank functions for h : A.PairingCore correspond to weak rank functions for h.pairing : A.Pairing.

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