Documentation

ConNF.External.Counting

New file #

In this file...

Main declarations #

def ConNF.insert [ConNF.Params] {α : ConNF.Λ} (x : ConNF.TSet α) :

The set {z ∪ {a} | z ∈ x}.

Equations
Instances For
    def ConNF.cardinalNat [ConNF.Params] {α β γ : ConNF.Λ} (hβ : β < α) (hγ : γ < β) (n : ) :
    Equations
    Instances For
      @[simp]
      theorem ConNF.mem_cardinalNat_iff [ConNF.Params] {α β γ : ConNF.Λ} (hβ : β < α) (hγ : γ < β) (n : ) (a : ConNF.TSet β) :
      a ∈[] ConNF.cardinalNat n ∃ (s : Finset (ConNF.TSet γ)), s.card = n ∀ (b : ConNF.TSet γ), b ∈[] a b s