Equations
- One or more equations did not get rendered due to their size.
Instances For
theorem
Ordinal.noMaxOrder_of_isLimit
{α : Type u}
[Preorder α]
[IsWellOrder α fun (x1 x2 : α) => x1 < x2]
(h : (type fun (x1 x2 : α) => x1 < x2).IsLimit)
:
theorem
Ordinal.isLimit_of_noMaxOrder
{α : Type u}
[Nonempty α]
[Preorder α]
[IsWellOrder α fun (x1 x2 : α) => x1 < x2]
(h : NoMaxOrder α)
:
theorem
Ordinal.isLimit_iff_noMaxOrder
{α : Type u}
[Nonempty α]
[Preorder α]
[IsWellOrder α fun (x1 x2 : α) => x1 < x2]
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
Lifting ordinals #
instance
Ordinal.ULift.isTrichotomous
{α : Type u}
{r : α → α → Prop}
[IsTrichotomous α r]
:
IsTrichotomous (ULift.{v, u} α) (InvImage r ULift.down)
instance
Ordinal.ULift.isTrans
{α : Type u}
{r : α → α → Prop}
[IsTrans α r]
:
IsTrans (ULift.{v, u} α) (InvImage r ULift.down)
instance
Ordinal.ULift.isWellOrder
{α : Type u}
{r : α → α → Prop}
[IsWellOrder α r]
:
IsWellOrder (ULift.{v, u} α) (InvImage r ULift.down)
theorem
Ordinal.lift_typein_apply
{α : Type u}
{β : Type v}
{r : α → α → Prop}
{s : β → β → Prop}
[IsWellOrder α r]
[IsWellOrder β s]
(f : r ≼i s)
(a : α)
:
lift.{max u v, v} ((typein s).toRelEmbedding (f a)) = lift.{max u v, u} ((typein r).toRelEmbedding a)
The additive structure on the set of ordinals below a cardinal #
@[simp]
theorem
Ordinal.add_lt_ord
{c : Cardinal.{u}}
(h : Cardinal.aleph0 ≤ c)
{x y : Ordinal.{u}}
(hx : x < c.ord)
(hy : y < c.ord)
:
Equations
- Ordinal.iioAdd h = { add := fun (x y : ↑(Set.Iio c.ord)) => ⟨↑x + ↑y, ⋯⟩ }
Instances For
Instances For
Equations
- Ordinal.iioZero h = { zero := ⟨0, ⋯⟩ }
Instances For
@[simp]
Equations
- Ordinal.iioAddMonoid h = AddMonoid.mk ⋯ ⋯ nsmulRec ⋯ ⋯
Instances For
Equations
- Ordinal.iioOfNat h n = { ofNat := ⟨↑n, ⋯⟩ }
Instances For
theorem
Ordinal.iio_noMaxOrder
{c : Cardinal.{u}}
(h : Cardinal.aleph0 ≤ c)
:
NoMaxOrder ↑(Set.Iio c.ord)