Documentation

ConNF.Background.Ordinal

def Ordinal.withBotOrderIso {α : Type u} [Preorder α] [IsWellOrder α fun (x1 x2 : α) => x1 < x2] :
(fun (x1 x2 : WithBot α) => x1 < x2) ≃r Sum.Lex EmptyRelation fun (x1 x2 : α) => x1 < x2
Equations
  • One or more equations did not get rendered due to their size.
Instances For
    @[simp]
    theorem Ordinal.type_withBot {α : Type u} [Preorder α] [IsWellOrder α fun (x1 x2 : α) => x1 < x2] :
    (type fun (x1 x2 : WithBot α) => x1 < x2) = 1 + type fun (x1 x2 : α) => x1 < x2
    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 α) :
    (type fun (x1 x2 : α) => x1 < x2).IsLimit
    theorem Ordinal.isLimit_iff_noMaxOrder {α : Type u} [Nonempty α] [Preorder α] [IsWellOrder α fun (x1 x2 : α) => x1 < x2] :
    (type fun (x1 x2 : α) => x1 < x2).IsLimit NoMaxOrder α
    theorem Ordinal.type_Iio_lt {α : Type u} [LtWellOrder α] (x : α) :
    type (Subrel (fun (x1 x2 : α) => x1 < x2) (Set.Iio x)) < type fun (x1 x2 : α) => x1 < x2
    def Ordinal.iicOrderIso {α : Type u} [LtWellOrder α] (x : α) :
    Subrel (fun (x1 x2 : α) => x1 < x2) (Set.Iic x) ≃r Sum.Lex (Subrel (fun (x1 x2 : α) => x1 < x2) (Set.Iio x)) EmptyRelation
    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      theorem Ordinal.type_Iic_eq {α : Type u} [LtWellOrder α] (x : α) :
      type (Subrel (fun (x1 x2 : α) => x1 < x2) (Set.Iic x)) = type (Subrel (fun (x1 x2 : α) => x1 < x2) (Set.Iio x)) + 1
      theorem Ordinal.type_Iic_lt {α : Type u} [LtWellOrder α] [NoMaxOrder α] (x : α) :
      type (Subrel (fun (x1 x2 : α) => x1 < x2) (Set.Iic x)) < type fun (x1 x2 : α) => x1 < x2

      Lifting ordinals #

      instance Ordinal.ULift.isTrans {α : Type u} {r : ααProp} [IsTrans α r] :
      instance Ordinal.ULift.isWellOrder {α : Type u} {r : ααProp} [IsWellOrder α r] :
      theorem Ordinal.lift_typein_apply {α : Type u} {β : Type v} {r : ααProp} {s : ββProp} [IsWellOrder α r] [IsWellOrder β s] (f : r ≼i s) (a : α) :

      The additive structure on the set of ordinals below a cardinal #

      theorem Ordinal.type_Iio (o : Ordinal.{u}) :
      (type fun (x1 x2 : (Set.Iio o)) => x1 < x2) = lift.{u + 1, u} o
      @[simp]
      theorem Ordinal.typein_Iio {o : Ordinal.{u}} (x : (Set.Iio o)) :
      (typein fun (x1 x2 : (Set.Iio o)) => x1 < x2).toRelEmbedding x = lift.{u + 1, u} x
      theorem Ordinal.add_lt_ord {c : Cardinal.{u}} (h : Cardinal.aleph0 c) {x y : Ordinal.{u}} (hx : x < c.ord) (hy : y < c.ord) :
      x + y < c.ord
      Equations
      Instances For
        Equations
        Instances For
          Equations
          Instances For
            @[simp]
            theorem Ordinal.iioAdd_def {c : Cardinal.{u}} (h : Cardinal.aleph0 c) (x y : (Set.Iio c.ord)) :
            ↑(x + y) = x + y
            theorem Ordinal.nat_lt_ord {c : Cardinal.{u}} (h : Cardinal.aleph0 c) (n : ) :
            n < c.ord
            def Ordinal.iioOfNat {c : Cardinal.{u}} (h : Cardinal.aleph0 c) (n : ) :
            OfNat (↑(Set.Iio c.ord)) n
            Equations
            Instances For