Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- ConNF.«term_⊓'_» = Lean.ParserDescr.trailingNode `ConNF.«term_⊓'_» 69 69 (Lean.ParserDescr.binary `andthen (Lean.ParserDescr.symbol " ⊓' ") (Lean.ParserDescr.cat `term 69))
Instances For
@[simp]
theorem
ConNF.mem_inter_iff
[ConNF.Params]
{α β : ConNF.Λ}
(hβ : ↑β < ↑α)
(x y : ConNF.TSet ↑α)
(z : ConNF.TSet ↑β)
:
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- ConNF.«term_ᶜ'» = Lean.ParserDescr.trailingNode `ConNF.«term_ᶜ'» 1024 1024 (Lean.ParserDescr.symbol " ᶜ'")
Instances For
@[simp]
theorem
ConNF.mem_compl_iff
[ConNF.Params]
{α β : ConNF.Λ}
(hβ : ↑β < ↑α)
(x : ConNF.TSet ↑α)
(z : ConNF.TSet ↑β)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
@[simp]
theorem
ConNF.mem_singleton_iff
[ConNF.Params]
{α β : ConNF.Λ}
(hβ : ↑β < ↑α)
(x y : ConNF.TSet ↑β)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
ConNF.singletonImage'
[ConNF.Params]
{α β γ δ ε : ConNF.Λ}
(hβ : ↑β < ↑α)
(hγ : ↑γ < ↑β)
(hδ : ↑δ < ↑γ)
(hε : ↑ε < ↑δ)
(x : ConNF.TSet ↑β)
:
ConNF.TSet ↑α
Equations
- ConNF.singletonImage' hβ hγ hδ hε x = ⋯.choose
Instances For
def
ConNF.insertion2'
[ConNF.Params]
{α β γ δ ε ζ : ConNF.Λ}
(hβ : ↑β < ↑α)
(hγ : ↑γ < ↑β)
(hδ : ↑δ < ↑γ)
(hε : ↑ε < ↑δ)
(hζ : ↑ζ < ↑ε)
(x : ConNF.TSet ↑γ)
:
ConNF.TSet ↑α
Equations
- ConNF.insertion2' hβ hγ hδ hε hζ x = ⋯.choose
Instances For
@[simp]
def
ConNF.insertion3'
[ConNF.Params]
{α β γ δ ε ζ : ConNF.Λ}
(hβ : ↑β < ↑α)
(hγ : ↑γ < ↑β)
(hδ : ↑δ < ↑γ)
(hε : ↑ε < ↑δ)
(hζ : ↑ζ < ↑ε)
(x : ConNF.TSet ↑γ)
:
ConNF.TSet ↑α
Equations
- ConNF.insertion3' hβ hγ hδ hε hζ x = ⋯.choose
Instances For
def
ConNF.vCross
[ConNF.Params]
{α β γ δ : ConNF.Λ}
(hβ : ↑β < ↑α)
(hγ : ↑γ < ↑β)
(hδ : ↑δ < ↑γ)
(x : ConNF.TSet ↑γ)
:
ConNF.TSet ↑α
Equations
- ConNF.vCross hβ hγ hδ x = ⋯.choose
Instances For
@[simp]
theorem
ConNF.mem_vCross_iff
[ConNF.Params]
{α β γ δ : ConNF.Λ}
(hβ : ↑β < ↑α)
(hγ : ↑γ < ↑β)
(hδ : ↑δ < ↑γ)
(x : ConNF.TSet ↑γ)
(a : ConNF.TSet ↑β)
:
a ∈[hβ] ConNF.vCross hβ hγ hδ x ↔ ∃ (b : ConNF.TSet ↑δ) (c : ConNF.TSet ↑δ), a = ⟨b, c⟩[hγ, hδ] ∧ c ∈[hδ] x
def
ConNF.typeLower
[ConNF.Params]
{α β γ δ ε : ConNF.Λ}
(hβ : ↑β < ↑α)
(hγ : ↑γ < ↑β)
(hδ : ↑δ < ↑γ)
(hε : ↑ε < ↑δ)
(x : ConNF.TSet ↑α)
:
ConNF.TSet ↑δ
Equations
- ConNF.typeLower hβ hγ hδ hε x = ⋯.choose
Instances For
@[simp]
theorem
ConNF.mem_typeLower_iff
[ConNF.Params]
{α β γ δ ε : ConNF.Λ}
(hβ : ↑β < ↑α)
(hγ : ↑γ < ↑β)
(hδ : ↑δ < ↑γ)
(hε : ↑ε < ↑δ)
(x : ConNF.TSet ↑α)
(a : ConNF.TSet ↑ε)
:
def
ConNF.converse'
[ConNF.Params]
{α β γ δ : ConNF.Λ}
(hβ : ↑β < ↑α)
(hγ : ↑γ < ↑β)
(hδ : ↑δ < ↑γ)
(x : ConNF.TSet ↑α)
:
ConNF.TSet ↑α
Equations
- ConNF.converse' hβ hγ hδ x = ⋯.choose
Instances For
@[simp]
theorem
ConNF.converse'_spec
[ConNF.Params]
{α β γ δ : ConNF.Λ}
(hβ : ↑β < ↑α)
(hγ : ↑γ < ↑β)
(hδ : ↑δ < ↑γ)
(x : ConNF.TSet ↑α)
(a b : ConNF.TSet ↑δ)
:
Equations
- ConNF.cardinalOne hβ hγ = ⋯.choose
Instances For
@[simp]
theorem
ConNF.mem_cardinalOne_iff
[ConNF.Params]
{α β γ : ConNF.Λ}
(hβ : ↑β < ↑α)
(hγ : ↑γ < ↑β)
(a : ConNF.TSet ↑β)
:
a ∈[hβ] ConNF.cardinalOne hβ hγ ↔ ∃ (b : ConNF.TSet ↑γ), a = {b}[hγ]
def
ConNF.subset'
[ConNF.Params]
{α β γ δ ε : ConNF.Λ}
(hβ : ↑β < ↑α)
(hγ : ↑γ < ↑β)
(hδ : ↑δ < ↑γ)
(hε : ↑ε < ↑δ)
:
ConNF.TSet ↑α
Equations
- ConNF.subset' hβ hγ hδ hε = ⋯.choose
Instances For
theorem
ConNF.subset'_spec
[ConNF.Params]
{α β γ δ ε : ConNF.Λ}
(hβ : ↑β < ↑α)
(hγ : ↑γ < ↑β)
(hδ : ↑δ < ↑γ)
(hε : ↑ε < ↑δ)
(a b : ConNF.TSet ↑δ)
: