Rank in a well-founded relation #
For r
a well-founded relation, IsWellFounded.rank r a
is recursively defined as the least
ordinal greater than the ranks of all elements below a
.
Rank of an accessible value #
The rank of an element a
accessible under a relation r
is defined recursively as the
smallest ordinal greater than the ranks of all elements below it (i.e. elements b
such that
r b a
).
Equations
- h.rank = Acc.recOn h fun (a : α) (_h : ∀ (y : α), r y a → Acc r y) (ih : (y : α) → r y a → Ordinal.{?u.43}) => ⨆ (b : { b : α // r b a }), Order.succ (ih ↑b ⋯)
Instances For
Rank in a well-founded relation #
noncomputable def
IsWellFounded.rank
{α : Type u}
(r : α → α → Prop)
[hwf : IsWellFounded α r]
(a : α)
:
The rank of an element a
under a well-founded relation r
is defined recursively as the
smallest ordinal greater than the ranks of all elements below it (i.e. elements b
such that
r b a
).
Equations
- IsWellFounded.rank r a = ⋯.rank
Instances For
theorem
IsWellFounded.rank_lt_of_rel
{α : Type u}
{a b : α}
{r : α → α → Prop}
[hwf : IsWellFounded α r]
(h : r a b)
:
theorem
IsWellFounded.mem_range_rank_of_le
{α : Type u}
{a : α}
{r : α → α → Prop}
[hwf : IsWellFounded α r]
{o : Ordinal.{u}}
(h : o ≤ rank r a)
:
theorem
WellFoundedLT.rank_strictMono
{α : Type u}
[Preorder α]
[WellFoundedLT α]
:
StrictMono (IsWellFounded.rank fun (x1 x2 : α) => x1 < x2)
theorem
WellFoundedGT.rank_strictAnti
{α : Type u}
[Preorder α]
[WellFoundedGT α]
:
StrictAnti (IsWellFounded.rank fun (x1 x2 : α) => x1 > x2)
@[simp]
@[deprecated IsWellFounded.rank (since := "2024-09-07")]
The rank of an element a
under a well-founded relation r
is defined inductively as the
smallest ordinal greater than the ranks of all elements below it (i.e. elements b
such that
r b a
).
Instances For
@[deprecated IsWellFounded.rank_eq (since := "2024-09-07")]
@[deprecated IsWellFounded.rank_lt_of_rel (since := "2024-09-07")]
theorem
WellFounded.rank_lt_of_rel
{α : Type u}
{a b : α}
{r : α → α → Prop}
(hwf : WellFounded r)
(h : r a b)
:
@[deprecated WellFoundedLT.rank_strictMono (since := "2024-09-07")]
@[deprecated WellFoundedGT.rank_strictAnti (since := "2024-09-07")]