Documentation
ConNF
.
Model
.
Hailperin
Search
return to top
source
Imports
Init
ConNF.Model.TTT
Imported by
ConNF
.
TSet
.
exists_inter
ConNF
.
TSet
.
exists_compl
ConNF
.
TSet
.
exists_up
ConNF
.
TSet
.
up
ConNF
.
TSet
.
mem_up_iff
ConNF
.
TSet
.
op
ConNF
.
TSet
.
up_injective
ConNF
.
TSet
.
up_inj
ConNF
.
TSet
.
up_self
ConNF
.
TSet
.
up_eq_singleton_iff
ConNF
.
TSet
.
singleton_eq_up_iff
ConNF
.
TSet
.
op_injective
ConNF
.
TSet
.
op_inj
ConNF
.
TSet
.
op_eq_singleton_iff
ConNF
.
TSet
.
smul_up
ConNF
.
TSet
.
smul_op
ConNF
.
TSet
.
exists_singletonImage
ConNF
.
TSet
.
exists_insertion2
ConNF
.
TSet
.
exists_insertion3
ConNF
.
TSet
.
exists_cross
ConNF
.
TSet
.
exists_typeLower
ConNF
.
TSet
.
exists_converse
ConNF
.
TSet
.
exists_cardinalOne
ConNF
.
TSet
.
exists_subset
New file
#
In this file...
Main declarations
#
ConNF.foo
: Something new.
source
theorem
ConNF
.
TSet
.
exists_inter
[
Params
]
{
α
β
:
Λ
}
(
hβ
:
↑
β
<
↑
α
)
(
x
y
:
TSet
↑
α
)
:
∃ (
w
:
TSet
↑
α
),
∀ (
z
:
TSet
↑
β
),
z
∈[
hβ
]
w
↔
z
∈[
hβ
]
x
∧
z
∈[
hβ
]
y
source
theorem
ConNF
.
TSet
.
exists_compl
[
Params
]
{
α
β
:
Λ
}
(
hβ
:
↑
β
<
↑
α
)
(
x
:
TSet
↑
α
)
:
∃ (
y
:
TSet
↑
α
),
∀ (
z
:
TSet
↑
β
),
z
∈[
hβ
]
y
↔
¬
z
∈[
hβ
]
x
source
theorem
ConNF
.
TSet
.
exists_up
[
Params
]
{
α
β
:
Λ
}
(
hβ
:
↑
β
<
↑
α
)
(
x
y
:
TSet
↑
β
)
:
∃ (
w
:
TSet
↑
α
),
∀ (
z
:
TSet
↑
β
),
z
∈[
hβ
]
w
↔
z
=
x
∨
z
=
y
source
def
ConNF
.
TSet
.
up
[
Params
]
{
α
β
:
Λ
}
(
hβ
:
↑
β
<
↑
α
)
(
x
y
:
TSet
↑
β
)
:
TSet
↑
α
The unordered pair.
Equations
ConNF.TSet.up
hβ
x
y
=
⋯
.
choose
Instances For
source
@[simp]
theorem
ConNF
.
TSet
.
mem_up_iff
[
Params
]
{
α
β
:
Λ
}
(
hβ
:
↑
β
<
↑
α
)
(
x
y
z
:
TSet
↑
β
)
:
z
∈[
hβ
]
up
hβ
x
y
↔
z
=
x
∨
z
=
y
source
def
ConNF
.
TSet
.
op
[
Params
]
{
α
β
γ
:
Λ
}
(
hβ
:
↑
β
<
↑
α
)
(
hγ
:
↑
γ
<
↑
β
)
(
x
y
:
TSet
↑
γ
)
:
TSet
↑
α
The Kuratowski ordered pair.
Equations
ConNF.TSet.op
hβ
hγ
x
y
=
ConNF.TSet.up
hβ
(
ConNF.singleton
hγ
x
)
(
ConNF.TSet.up
hγ
x
y
)
Instances For
source
theorem
ConNF
.
TSet
.
up_injective
[
Params
]
{
α
β
:
Λ
}
(
hβ
:
↑
β
<
↑
α
)
{
x
y
z
w
:
TSet
↑
β
}
(
h
:
up
hβ
x
y
=
up
hβ
z
w
)
:
x
=
z
∧
y
=
w
∨
x
=
w
∧
y
=
z
source
@[simp]
theorem
ConNF
.
TSet
.
up_inj
[
Params
]
{
α
β
:
Λ
}
(
hβ
:
↑
β
<
↑
α
)
(
x
y
z
w
:
TSet
↑
β
)
:
up
hβ
x
y
=
up
hβ
z
w
↔
x
=
z
∧
y
=
w
∨
x
=
w
∧
y
=
z
source
@[simp]
theorem
ConNF
.
TSet
.
up_self
[
Params
]
{
α
β
:
Λ
}
(
hβ
:
↑
β
<
↑
α
)
{
x
:
TSet
↑
β
}
:
up
hβ
x
x
=
ConNF.singleton
hβ
x
source
@[simp]
theorem
ConNF
.
TSet
.
up_eq_singleton_iff
[
Params
]
{
α
β
:
Λ
}
(
hβ
:
↑
β
<
↑
α
)
(
x
y
z
:
TSet
↑
β
)
:
up
hβ
x
y
=
ConNF.singleton
hβ
z
↔
x
=
z
∧
y
=
z
source
@[simp]
theorem
ConNF
.
TSet
.
singleton_eq_up_iff
[
Params
]
{
α
β
:
Λ
}
(
hβ
:
↑
β
<
↑
α
)
(
x
y
z
:
TSet
↑
β
)
:
ConNF.singleton
hβ
z
=
up
hβ
x
y
↔
x
=
z
∧
y
=
z
source
theorem
ConNF
.
TSet
.
op_injective
[
Params
]
{
α
β
γ
:
Λ
}
(
hβ
:
↑
β
<
↑
α
)
(
hγ
:
↑
γ
<
↑
β
)
{
x
y
z
w
:
TSet
↑
γ
}
(
h
:
op
hβ
hγ
x
y
=
op
hβ
hγ
z
w
)
:
x
=
z
∧
y
=
w
source
@[simp]
theorem
ConNF
.
TSet
.
op_inj
[
Params
]
{
α
β
γ
:
Λ
}
(
hβ
:
↑
β
<
↑
α
)
(
hγ
:
↑
γ
<
↑
β
)
(
x
y
z
w
:
TSet
↑
γ
)
:
op
hβ
hγ
x
y
=
op
hβ
hγ
z
w
↔
x
=
z
∧
y
=
w
source
@[simp]
theorem
ConNF
.
TSet
.
op_eq_singleton_iff
[
Params
]
{
α
β
γ
:
Λ
}
(
hβ
:
↑
β
<
↑
α
)
(
hγ
:
↑
γ
<
↑
β
)
(
x
y
:
TSet
↑
γ
)
(
z
:
TSet
↑
β
)
:
op
hβ
hγ
x
y
=
ConNF.singleton
hβ
z
↔
ConNF.singleton
hγ
x
=
z
∧
ConNF.singleton
hγ
y
=
z
source
@[simp]
theorem
ConNF
.
TSet
.
smul_up
[
Params
]
{
α
β
:
Λ
}
(
hβ
:
↑
β
<
↑
α
)
(
x
y
:
TSet
↑
β
)
(
ρ
:
AllPerm
↑
α
)
:
ρ
•
up
hβ
x
y
=
up
hβ
(
ρ
↘
hβ
•
x
) (
ρ
↘
hβ
•
y
)
source
@[simp]
theorem
ConNF
.
TSet
.
smul_op
[
Params
]
{
α
β
γ
:
Λ
}
(
hβ
:
↑
β
<
↑
α
)
(
hγ
:
↑
γ
<
↑
β
)
(
x
y
:
TSet
↑
γ
)
(
ρ
:
AllPerm
↑
α
)
:
ρ
•
op
hβ
hγ
x
y
=
op
hβ
hγ
(
ρ
↘
hβ
↘
hγ
•
x
) (
ρ
↘
hβ
↘
hγ
•
y
)
source
theorem
ConNF
.
TSet
.
exists_singletonImage
[
Params
]
{
α
β
γ
δ
ε
:
Λ
}
(
hβ
:
↑
β
<
↑
α
)
(
hγ
:
↑
γ
<
↑
β
)
(
hδ
:
↑
δ
<
↑
γ
)
(
hε
:
↑
ε
<
↑
δ
)
(
x
:
TSet
↑
β
)
:
∃ (
y
:
TSet
↑
α
),
∀ (
z
w
:
TSet
↑
ε
),
op
hγ
hδ
(
ConNF.singleton
hε
z
)
(
ConNF.singleton
hε
w
)
∈[
hβ
]
y
↔
op
hδ
hε
z
w
∈[
hγ
]
x
source
theorem
ConNF
.
TSet
.
exists_insertion2
[
Params
]
{
α
β
γ
δ
ε
ζ
:
Λ
}
(
hβ
:
↑
β
<
↑
α
)
(
hγ
:
↑
γ
<
↑
β
)
(
hδ
:
↑
δ
<
↑
γ
)
(
hε
:
↑
ε
<
↑
δ
)
(
hζ
:
↑
ζ
<
↑
ε
)
(
x
:
TSet
↑
γ
)
:
∃ (
y
:
TSet
↑
α
),
∀ (
a
b
c
:
TSet
↑
ζ
),
op
hγ
hδ
(
ConNF.singleton
hε
(
ConNF.singleton
hζ
a
)
)
(
op
hε
hζ
b
c
)
∈[
hβ
]
y
↔
op
hε
hζ
a
c
∈[
hδ
]
x
source
theorem
ConNF
.
TSet
.
exists_insertion3
[
Params
]
{
α
β
γ
δ
ε
ζ
:
Λ
}
(
hβ
:
↑
β
<
↑
α
)
(
hγ
:
↑
γ
<
↑
β
)
(
hδ
:
↑
δ
<
↑
γ
)
(
hε
:
↑
ε
<
↑
δ
)
(
hζ
:
↑
ζ
<
↑
ε
)
(
x
:
TSet
↑
γ
)
:
∃ (
y
:
TSet
↑
α
),
∀ (
a
b
c
:
TSet
↑
ζ
),
op
hγ
hδ
(
ConNF.singleton
hε
(
ConNF.singleton
hζ
a
)
)
(
op
hε
hζ
b
c
)
∈[
hβ
]
y
↔
op
hε
hζ
a
b
∈[
hδ
]
x
source
theorem
ConNF
.
TSet
.
exists_cross
[
Params
]
{
α
β
γ
δ
:
Λ
}
(
hβ
:
↑
β
<
↑
α
)
(
hγ
:
↑
γ
<
↑
β
)
(
hδ
:
↑
δ
<
↑
γ
)
(
x
:
TSet
↑
γ
)
:
∃ (
y
:
TSet
↑
α
),
∀ (
a
:
TSet
↑
β
),
a
∈[
hβ
]
y
↔
∃ (
b
:
TSet
↑
δ
) (
c
:
TSet
↑
δ
),
a
=
op
hγ
hδ
b
c
∧
c
∈[
hδ
]
x
source
theorem
ConNF
.
TSet
.
exists_typeLower
[
Params
]
{
α
β
γ
δ
ε
:
Λ
}
(
hβ
:
↑
β
<
↑
α
)
(
hγ
:
↑
γ
<
↑
β
)
(
hδ
:
↑
δ
<
↑
γ
)
(
hε
:
↑
ε
<
↑
δ
)
(
x
:
TSet
↑
α
)
:
∃ (
y
:
TSet
↑
δ
),
∀ (
a
:
TSet
↑
ε
),
a
∈[
hε
]
y
↔
∀ (
b
:
TSet
↑
δ
),
op
hγ
hδ
b
(
ConNF.singleton
hε
a
)
∈[
hβ
]
x
source
theorem
ConNF
.
TSet
.
exists_converse
[
Params
]
{
α
β
γ
δ
:
Λ
}
(
hβ
:
↑
β
<
↑
α
)
(
hγ
:
↑
γ
<
↑
β
)
(
hδ
:
↑
δ
<
↑
γ
)
(
x
:
TSet
↑
α
)
:
∃ (
y
:
TSet
↑
α
),
∀ (
a
b
:
TSet
↑
δ
),
op
hγ
hδ
a
b
∈[
hβ
]
y
↔
op
hγ
hδ
b
a
∈[
hβ
]
x
source
theorem
ConNF
.
TSet
.
exists_cardinalOne
[
Params
]
{
α
β
γ
:
Λ
}
(
hβ
:
↑
β
<
↑
α
)
(
hγ
:
↑
γ
<
↑
β
)
:
∃ (
x
:
TSet
↑
α
),
∀ (
a
:
TSet
↑
β
),
a
∈[
hβ
]
x
↔
∃ (
b
:
TSet
↑
γ
),
a
=
ConNF.singleton
hγ
b
source
theorem
ConNF
.
TSet
.
exists_subset
[
Params
]
{
α
β
γ
δ
ε
:
Λ
}
(
hβ
:
↑
β
<
↑
α
)
(
hγ
:
↑
γ
<
↑
β
)
(
hδ
:
↑
δ
<
↑
γ
)
(
hε
:
↑
ε
<
↑
δ
)
:
∃ (
x
:
TSet
↑
α
),
∀ (
a
b
:
TSet
↑
δ
),
op
hγ
hδ
a
b
∈[
hβ
]
x
↔
∀ (
c
:
TSet
↑
ε
),
c
∈[
hε
]
a
→
c
∈[
hε
]
b