Ordinal ranks of PSet and ZFSet #
In this file, we define the ordinal ranks of PSet
and ZFSet
. These ranks are the same as
IsWellFounded.rank
over ∈
, but are defined in a way that the universe levels of ranks are the
same as the indexing types.
Definitions #
PSet.rank
: Ordinal rank of a pre-set.ZFSet.rank
: Ordinal rank of a ZFC set.
PSet rank #
The ordinal rank of a pre-set
Equations
- (PSet.mk α A).rank = ⨆ (a : α), Order.succ (A a).rank
Instances For
theorem
PSet.rank_le_iff
{o : Ordinal.{u_1}}
{x : PSet.{u_1}}
:
x.rank ≤ o ↔ ∀ ⦃y : PSet.{u_1}⦄, y ∈ x → y.rank < o
@[simp]
For the rank of ⋃₀ x
, we only have rank (⋃₀ x) ≤ rank x ≤ rank (⋃₀ x) + 1
.
This inequality is split into rank_sUnion_le
and le_succ_rank_sUnion
.
theorem
PSet.rank_eq_wfRank
{x : PSet.{u}}
:
Ordinal.lift.{u + 1, u} x.rank = IsWellFounded.rank (fun (x1 x2 : PSet.{u}) => x1 ∈ x2) x
PSet.rank
is equal to the IsWellFounded.rank
over ∈
.
ZFSet rank #
The ordinal rank of a ZFC set
Equations
Instances For
@[simp]
For the rank of ⋃₀ x
, we only have rank (⋃₀ x) ≤ rank x ≤ rank (⋃₀ x) + 1
.
This inequality is split into rank_sUnion_le
and le_succ_rank_sUnion
.
@[simp]
theorem
ZFSet.rank_range
{α : Type u_1}
[Small.{u, u_1} α]
(f : α → ZFSet.{u})
:
(ZFSet.range f).rank = ⨆ (i : α), Order.succ (f i).rank
theorem
ZFSet.rank_eq_wfRank
{x : ZFSet.{u}}
:
Ordinal.lift.{u + 1, u} x.rank = IsWellFounded.rank (fun (x1 x2 : ZFSet.{u}) => x1 ∈ x2) x
ZFSet.rank
is equal to the IsWellFounded.rank
over ∈
.