Documentation

ConNF.Base.Position

Position functions #

In this file, we define what it means for a type to have a position function.

Main declarations #

class ConNF.Position [ConNF.Params] (X : Type u_1) :
Type (max u u_1)
  • pos : X ConNF.μ
Instances
    def ConNF.pos_induction [ConNF.Params] {X : Type u_1} [ConNF.Position X] {C : XProp} (x : X) (h : ∀ (x : X), (∀ (y : X), ConNF.pos y < ConNF.pos xC y)C x) :
    C x
    Equations
    • =
    Instances For