Documentation

ConNF.External.Counting

New file #

In this file...

We are roughly following Scott Fenton's development of NF: https://us.metamath.org/nfeuni/mmnf.html.

Main declarations #

def ConNF.disjoint [Params] {α β γ δ ε : Λ} ( : β < α) ( : γ < β) ( : δ < γ) ( : ε < δ) :
TSet α

The set {⟨x, y⟩ | x ∩ y = ∅} (or rather, a set that contains only these Kuratowski pairs).

Equations
  • One or more equations did not get rendered due to their size.
Instances For
    theorem ConNF.mem_disjoint_iff' [Params] {α β γ δ ε : Λ} ( : β < α) ( : γ < β) ( : δ < γ) ( : ε < δ) (x y : TSet δ) :
    x, y⟩[, ] ∈[] disjoint ∀ (z : TSet ε), ¬z ∈[] x ⊓[] y
    @[simp]
    theorem ConNF.mem_disjoint_iff [Params] {α β γ δ ε : Λ} ( : β < α) ( : γ < β) ( : δ < γ) ( : ε < δ) (x y : TSet δ) :
    x, y⟩[, ] ∈[] disjoint x ⊓[] y = empty
    def ConNF.unionEq [Params] {α β γ δ ε ζ η : Λ} ( : β < α) ( : γ < β) ( : δ < γ) ( : ε < δ) ( : ζ < ε) ( : η < ζ) :
    TSet α

    The set {⟨{{z}}, ⟨y, x⟩ | y ∪ z = x} (or rather, again, a set that contains only these pairs).

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      theorem ConNF.mem_unionEq_iff' [Params] {α β γ δ ε ζ η : Λ} ( : β < α) ( : γ < β) ( : δ < γ) ( : ε < δ) ( : ζ < ε) ( : η < ζ) (x y z : TSet ζ) :
      {{z}[]}[], y, x⟩[, ]⟩[, ] ∈[] unionEq ∀ (a : TSet η), ¬(a ∈[] x ¬a ∈[] y ¬a ∈[] z)
      @[simp]
      theorem ConNF.mem_unionEq_iff [Params] {α β γ δ ε ζ η : Λ} ( : β < α) ( : γ < β) ( : δ < γ) ( : ε < δ) ( : ζ < ε) ( : η < ζ) (x y z : TSet ζ) :
      {{z}[]}[], y, x⟩[, ]⟩[, ] ∈[] unionEq y ⊔[] z = x
      def ConNF.cardAdd [Params] {α β γ : Λ} ( : β < α) ( : γ < β) (x y : TSet α) :
      TSet α

      The sum of two cardinals: x + y = {a ∪ b | a ∈ x ∧ b ∈ y ∧ a ∩ b = ∅}.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        @[simp]
        theorem ConNF.mem_cardAdd_iff [Params] {α β γ : Λ} ( : β < α) ( : γ < β) (x y : TSet α) (z : TSet β) :
        z ∈[] cardAdd x y ∃ (a : TSet β) (b : TSet β), a ∈[] x b ∈[] y a ⊓[] b = empty a ⊔[] b = z
        def ConNF.succ [Params] {α β γ : Λ} ( : β < α) ( : γ < β) (x : TSet α) :
        TSet α

        The successor of a cardinal: x + 1 = {a ∪ {b} | a ∈ x, b ∉ a}.

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