Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- ConNF.«term_⊔'_» = Lean.ParserDescr.trailingNode `ConNF.«term_⊔'_» 68 68 (Lean.ParserDescr.binary `andthen (Lean.ParserDescr.symbol " ⊔' ") (Lean.ParserDescr.cat `term 68))
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_∆'_» 100 100 (Lean.ParserDescr.binary `andthen (Lean.ParserDescr.symbol " ∆' ") (Lean.ParserDescr.cat `term 100))
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_\'_» 70 70 (Lean.ParserDescr.binary `andthen (Lean.ParserDescr.symbol " \\' ") (Lean.ParserDescr.cat `term 70))
Instances For
A short name is chosen because of its frequency of use.
Equations
- ConNF.univ hβ = (ConNF.empty hβ) ᶜ[hβ]
Instances For
The set of all ordered pairs.
Equations
- ConNF.orderedPairs hβ hγ hδ = ConNF.vCross hβ hγ hδ (ConNF.univ hδ)
Instances For
def
ConNF.converse
[Params]
{α β γ δ : Λ}
(hβ : ↑β < ↑α)
(hγ : ↑γ < ↑β)
(hδ : ↑δ < ↑γ)
(x : TSet ↑α)
:
TSet ↑α
Equations
- ConNF.converse hβ hγ hδ x = ConNF.converse' hβ hγ hδ x ⊓[hβ] ConNF.orderedPairs hβ hγ hδ
Instances For
def
ConNF.cross
[Params]
{α β γ δ : Λ}
(hβ : ↑β < ↑α)
(hγ : ↑γ < ↑β)
(hδ : ↑δ < ↑γ)
(x y : TSet ↑γ)
:
TSet ↑α
Equations
- ConNF.cross hβ hγ hδ x y = ConNF.converse hβ hγ hδ (ConNF.vCross hβ hγ hδ x) ⊓[hβ] ConNF.vCross hβ hγ hδ y
Instances For
def
ConNF.singletonImage
[Params]
{α β γ δ ε : Λ}
(hβ : ↑β < ↑α)
(hγ : ↑γ < ↑β)
(hδ : ↑δ < ↑γ)
(hε : ↑ε < ↑δ)
(x : TSet ↑β)
:
TSet ↑α
Equations
- ConNF.singletonImage hβ hγ hδ hε x = ConNF.singletonImage' hβ hγ hδ hε x ⊓[hβ] ConNF.cross hβ hγ hδ (ConNF.cardinalOne hδ hε) (ConNF.cardinalOne hδ hε)
Instances For
def
ConNF.codom
[Params]
{α β γ δ : Λ}
(hβ : ↑β < ↑α)
(hγ : ↑γ < ↑β)
(hδ : ↑δ < ↑γ)
(r : TSet ↑α)
:
TSet ↑γ
The codomain of a relation.
Equations
- ConNF.codom hβ hγ hδ r = (ConNF.typeLower ⋯ hβ hγ hδ (ConNF.singletonImage ⋯ hβ hγ hδ r) ᶜ[⋯]) ᶜ[hδ]
Instances For
def
ConNF.field
[Params]
{α β γ δ : Λ}
(hβ : ↑β < ↑α)
(hγ : ↑γ < ↑β)
(hδ : ↑δ < ↑γ)
(r : TSet ↑α)
:
TSet ↑γ
The field of a relation.
Equations
- ConNF.field hβ hγ hδ r = ConNF.dom hβ hγ hδ r ⊔[hδ] ConNF.codom hβ hγ hδ r
Instances For
def
ConNF.subset
[Params]
{α β γ δ ε : Λ}
(hβ : ↑β < ↑α)
(hγ : ↑γ < ↑β)
(hδ : ↑δ < ↑γ)
(hε : ↑ε < ↑δ)
:
TSet ↑α
Equations
- ConNF.subset hβ hγ hδ hε = ConNF.subset' hβ hγ hδ hε ⊓[hβ] ConNF.orderedPairs hβ hγ hδ
Instances For
def
ConNF.membership
[Params]
{α β γ δ ε : Λ}
(hβ : ↑β < ↑α)
(hγ : ↑γ < ↑β)
(hδ : ↑δ < ↑γ)
(hε : ↑ε < ↑δ)
:
TSet ↑α
Equations
- ConNF.membership hβ hγ hδ hε = ConNF.subset hβ hγ hδ hε ⊓[hβ] ConNF.cross hβ hγ hδ (ConNF.cardinalOne hδ hε) (ConNF.univ hδ)
Instances For
Equations
- ConNF.powerset hβ hγ x = ConNF.dom ⋯ ⋯ hβ (ConNF.subset ⋯ ⋯ hβ hγ ⊓[⋯] ConNF.vCross ⋯ ⋯ hβ {x}[hβ])
Instances For
def
ConNF.doubleSingletons
[Params]
{α β γ δ : Λ}
(hβ : ↑β < ↑α)
(hγ : ↑γ < ↑β)
(hδ : ↑δ < ↑γ)
(x : TSet ↑γ)
:
TSet ↑α
The set ι²''x = {{{a}} | a ∈ x}
.
Equations
- ConNF.doubleSingletons hβ hγ hδ x = ConNF.cross hβ hγ hδ x x ⊓[hβ] ConNF.cardinalOne hβ hγ
Instances For
The union of a set of singletons: ι⁻¹''x = {a | {a} ∈ x}
.
Scott Fenton calls this the "unit union".
Equations
- ConNF.singletonUnion hβ hγ x = ConNF.typeLower ⋯ ⋯ hβ hγ (ConNF.vCross ⋯ ⋯ hβ x)
Instances For
The set of singletons of a set: ι''x = {{a} | a ∈ x}
.
Scott Fenton calls this the "unit powerset".
Equations
- ConNF.singletons hβ hγ x = ConNF.singletonUnion ⋯ hβ (ConNF.doubleSingletons ⋯ hβ hγ x)
Instances For
The union of a set of sets.
⋃ x =
{a | a ∈ b ∧ b ∈ x} =
singletonUnion {{a} | a ∈ b ∧ b ∈ x} =
singletonUnion dom {⟨{a}, b⟩ | a ∈ b ∧ b ∈ x} =
singletonUnion dom ({⟨{a}, b⟩ | a ∈ b} ∩ (1 × x))
Equations
- ConNF.sUnion hβ hγ x = ConNF.singletonUnion hβ hγ (ConNF.dom ⋯ ⋯ hβ (ConNF.membership ⋯ ⋯ hβ hγ ⊓[⋯] ConNF.cross ⋯ ⋯ hβ (ConNF.cardinalOne hβ hγ) x))
Instances For
def
ConNF.orderedTriples
[Params]
{α β γ δ ε ζ : Λ}
(hβ : ↑β < ↑α)
(hγ : ↑γ < ↑β)
(hδ : ↑δ < ↑γ)
(hε : ↑ε < ↑δ)
(hζ : ↑ζ < ↑ε)
:
TSet ↑α
The set of all ordered triples.
Equations
- ConNF.orderedTriples hβ hγ hδ hε hζ = ConNF.cross hβ hγ hδ (ConNF.doubleSingletons hδ hε hζ (ConNF.univ hζ)) (ConNF.vCross hδ hε hζ (ConNF.univ hζ))
Instances For
def
ConNF.insertion2
[Params]
{α β γ δ ε ζ : Λ}
(hβ : ↑β < ↑α)
(hγ : ↑γ < ↑β)
(hδ : ↑δ < ↑γ)
(hε : ↑ε < ↑δ)
(hζ : ↑ζ < ↑ε)
(x : TSet ↑γ)
:
TSet ↑α
Equations
- ConNF.insertion2 hβ hγ hδ hε hζ x = ConNF.insertion2' hβ hγ hδ hε hζ x ⊓[hβ] ConNF.orderedTriples hβ hγ hδ hε hζ
Instances For
def
ConNF.insertion3
[Params]
{α β γ δ ε ζ : Λ}
(hβ : ↑β < ↑α)
(hγ : ↑γ < ↑β)
(hδ : ↑δ < ↑γ)
(hε : ↑ε < ↑δ)
(hζ : ↑ζ < ↑ε)
(x : TSet ↑γ)
:
TSet ↑α
Equations
- ConNF.insertion3 hβ hγ hδ hε hζ x = ConNF.insertion3' hβ hγ hδ hε hζ x ⊓[hβ] ConNF.orderedTriples hβ hγ hδ hε hζ
Instances For
def
ConNF.image
[Params]
{α β γ δ : Λ}
(hβ : ↑β < ↑α)
(hγ : ↑γ < ↑β)
(hδ : ↑δ < ↑γ)
(r : TSet ↑α)
(x : TSet ↑γ)
:
TSet ↑γ
The image of a set under a relation.
Equations
- ConNF.image hβ hγ hδ r x = ConNF.preimage hβ hγ hδ (ConNF.converse hβ hγ hδ r) x