formal
stringlengths
41
427k
informal
stringclasses
1 value
Ordinal.le_sub_of_le ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b c : Ordinal.{u_4} h : b ≤ a ⊢ c ≤ a - b ↔ b + c ≤ a ** rw [← add_le_add_iff_left b, Ordinal.add_sub_cancel_of_le h] ** Qed
Ordinal.sub_zero ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a : Ordinal.{u_4} ⊢ a - 0 = a ** simpa only [zero_add] using add_sub_cancel 0 a ** Qed
Ordinal.zero_sub ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a : Ordinal.{u_4} ⊢ 0 - a = 0 ** rw [← Ordinal.le_zero] ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a : Ordinal.{u_4} ⊢ 0 - a ≤ 0 ** apply sub_le_self ** Qed
Ordinal.sub_self ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a : Ordinal.{u_4} ⊢ a - a = 0 ** simpa only [add_zero] using add_sub_cancel a 0 ** Qed
Ordinal.sub_eq_zero_iff_le ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} h : a - b = 0 ⊢ a ≤ b ** simpa only [h, add_zero] using le_add_sub a b ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} h : a ≤ b ⊢ a - b = 0 ** rwa [← Ordinal.le_zero, sub_le, add_zero] ** Qed
Ordinal.sub_sub ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b c d : Ordinal.{u_4} ⊢ a - b - c ≤ d ↔ a - (b + c) ≤ d ** rw [sub_le, sub_le, sub_le, add_assoc] ** Qed
Ordinal.add_sub_add_cancel ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b c : Ordinal.{u_4} ⊢ a + b - (a + c) = b - c ** rw [← sub_sub, add_sub_cancel] ** Qed
Ordinal.sub_isLimit ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} l : IsLimit a h : b < a ⊢ b + 0 < a ** rwa [add_zero] ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} l : IsLimit a h✝ : b < a c : Ordinal.{u_4} h : c < a - b ⊢ succ c < a - b ** rw [lt_sub, add_succ] ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} l : IsLimit a h✝ : b < a c : Ordinal.{u_4} h : c < a - b ⊢ succ (b + c) < a ** exact l.2 _ (lt_sub.1 h) ** Qed
Ordinal.one_add_omega ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ⊢ 1 + ω = ω ** refine' le_antisymm _ (le_add_left _ _) ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ⊢ 1 + ω ≤ ω ** rw [omega, ← lift_one.{_, 0}, ← lift_add, lift_le, ← type_unit, ← type_sum_lex] ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ⊢ type (Sum.Lex EmptyRelation fun x x_1 => x < x_1) ≤ type fun x x_1 => x < x_1 ** refine' ⟨RelEmbedding.collapse (RelEmbedding.ofMonotone _ _)⟩ ** case refine'_1 α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ⊢ Unit ⊕ ℕ → ℕ ** apply Sum.rec ** case refine'_1.inl α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ⊢ Unit → ℕ case refine'_1.inr α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ⊢ ℕ → ℕ ** exact fun _ => 0 ** case refine'_1.inr α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ⊢ ℕ → ℕ ** exact Nat.succ ** case refine'_2 α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ⊢ ∀ (a b : Unit ⊕ ℕ), Sum.Lex EmptyRelation (fun x x_1 => x < x_1) a b → Sum.rec (fun x => 0) Nat.succ a < Sum.rec (fun x => 0) Nat.succ b ** intro a b ** case refine'_2 α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Unit ⊕ ℕ ⊢ Sum.Lex EmptyRelation (fun x x_1 => x < x_1) a b → Sum.rec (fun x => 0) Nat.succ a < Sum.rec (fun x => 0) Nat.succ b ** cases a <;> cases b <;> intro H <;> cases' H with _ _ H _ _ H <;> [exact H.elim; exact Nat.succ_pos _; exact Nat.succ_lt_succ H] ** Qed
Ordinal.one_add_of_omega_le ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u_4} h : ω ≤ o ⊢ 1 + o = o ** rw [← Ordinal.add_sub_cancel_of_le h, ← add_assoc, one_add_omega] ** Qed
Ordinal.mul_eq_zero' ** α✝ : Type u_1 β✝ : Type u_2 γ : Type u_3 r : α✝ → α✝ → Prop s : β✝ → β✝ → Prop t : γ → γ → Prop a b : Ordinal.{u_4} α : Type u_4 x✝³ : α → α → Prop x✝² : IsWellOrder α x✝³ β : Type u_4 x✝¹ : β → β → Prop x✝ : IsWellOrder β x✝¹ ⊢ type x✝³ * type x✝¹ = 0 ↔ type x✝³ = 0 ∨ type x✝¹ = 0 ** simp_rw [← type_prod_lex, type_eq_zero_iff_isEmpty] ** α✝ : Type u_1 β✝ : Type u_2 γ : Type u_3 r : α✝ → α✝ → Prop s : β✝ → β✝ → Prop t : γ → γ → Prop a b : Ordinal.{u_4} α : Type u_4 x✝³ : α → α → Prop x✝² : IsWellOrder α x✝³ β : Type u_4 x✝¹ : β → β → Prop x✝ : IsWellOrder β x✝¹ ⊢ IsEmpty (β × α) ↔ IsEmpty α ∨ IsEmpty β ** rw [or_comm] ** α✝ : Type u_1 β✝ : Type u_2 γ : Type u_3 r : α✝ → α✝ → Prop s : β✝ → β✝ → Prop t : γ → γ → Prop a b : Ordinal.{u_4} α : Type u_4 x✝³ : α → α → Prop x✝² : IsWellOrder α x✝³ β : Type u_4 x✝¹ : β → β → Prop x✝ : IsWellOrder β x✝¹ ⊢ IsEmpty (β × α) ↔ IsEmpty β ∨ IsEmpty α ** exact isEmpty_prod ** Qed
Ordinal.le_mul_left ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} hb : 0 < b ⊢ a ≤ a * b ** convert mul_le_mul_left' (one_le_iff_pos.2 hb) a ** case h.e'_3 α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} hb : 0 < b ⊢ a = a * 1 ** rw [mul_one a] ** Qed
Ordinal.le_mul_right ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} hb : 0 < b ⊢ a ≤ b * a ** convert mul_le_mul_right' (one_le_iff_pos.2 hb) a ** case h.e'_3 α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} hb : 0 < b ⊢ a = 1 * a ** rw [one_mul a] ** Qed
Ordinal.mul_le_of_limit_aux ** α✝ : Type u_1 β✝ : Type u_2 γ : Type u_3 r✝ : α✝ → α✝ → Prop s✝ : β✝ → β✝ → Prop t : γ → γ → Prop α β : Type u_4 r : α → α → Prop s : β → β → Prop inst✝¹ : IsWellOrder α r inst✝ : IsWellOrder β s c : Ordinal.{u_4} h : IsLimit (type s) H : ∀ (b' : Ordinal.{u_4}), b' < type s → type r * b' ≤ c l : c < type r * type s ⊢ False ** suffices ∀ a b, Prod.Lex s r (b, a) (enum _ _ l) by cases' enum _ _ l with b a exact irrefl _ (this _ _) ** α✝ : Type u_1 β✝ : Type u_2 γ : Type u_3 r✝ : α✝ → α✝ → Prop s✝ : β✝ → β✝ → Prop t : γ → γ → Prop α β : Type u_4 r : α → α → Prop s : β → β → Prop inst✝¹ : IsWellOrder α r inst✝ : IsWellOrder β s c : Ordinal.{u_4} h : IsLimit (type s) H : ∀ (b' : Ordinal.{u_4}), b' < type s → type r * b' ≤ c l : c < type r * type s ⊢ ∀ (a : α) (b : β), Prod.Lex s r (b, a) (enum (Prod.Lex s r) c l) ** intro a b ** α✝ : Type u_1 β✝ : Type u_2 γ : Type u_3 r✝ : α✝ → α✝ → Prop s✝ : β✝ → β✝ → Prop t : γ → γ → Prop α β : Type u_4 r : α → α → Prop s : β → β → Prop inst✝¹ : IsWellOrder α r inst✝ : IsWellOrder β s c : Ordinal.{u_4} h : IsLimit (type s) H : ∀ (b' : Ordinal.{u_4}), b' < type s → type r * b' ≤ c l : c < type r * type s a : α b : β ⊢ Prod.Lex s r (b, a) (enum (Prod.Lex s r) c l) ** rw [← typein_lt_typein (Prod.Lex s r), typein_enum] ** α✝ : Type u_1 β✝ : Type u_2 γ : Type u_3 r✝ : α✝ → α✝ → Prop s✝ : β✝ → β✝ → Prop t : γ → γ → Prop α β : Type u_4 r : α → α → Prop s : β → β → Prop inst✝¹ : IsWellOrder α r inst✝ : IsWellOrder β s c : Ordinal.{u_4} h : IsLimit (type s) H : ∀ (b' : Ordinal.{u_4}), b' < type s → type r * b' ≤ c l : c < type r * type s a : α b : β ⊢ typein (Prod.Lex s r) (b, a) < c ** have := H _ (h.2 _ (typein_lt_type s b)) ** α✝ : Type u_1 β✝ : Type u_2 γ : Type u_3 r✝ : α✝ → α✝ → Prop s✝ : β✝ → β✝ → Prop t : γ → γ → Prop α β : Type u_4 r : α → α → Prop s : β → β → Prop inst✝¹ : IsWellOrder α r inst✝ : IsWellOrder β s c : Ordinal.{u_4} h : IsLimit (type s) H : ∀ (b' : Ordinal.{u_4}), b' < type s → type r * b' ≤ c l : c < type r * type s a : α b : β this : type r * succ (typein s b) ≤ c ⊢ typein (Prod.Lex s r) (b, a) < c ** rw [mul_succ] at this ** α✝ : Type u_1 β✝ : Type u_2 γ : Type u_3 r✝ : α✝ → α✝ → Prop s✝ : β✝ → β✝ → Prop t : γ → γ → Prop α β : Type u_4 r : α → α → Prop s : β → β → Prop inst✝¹ : IsWellOrder α r inst✝ : IsWellOrder β s c : Ordinal.{u_4} h : IsLimit (type s) H : ∀ (b' : Ordinal.{u_4}), b' < type s → type r * b' ≤ c l : c < type r * type s a : α b : β this : type r * typein s b + type r ≤ c ⊢ typein (Prod.Lex s r) (b, a) < c ** have := ((add_lt_add_iff_left _).2 (typein_lt_type _ a)).trans_le this ** α✝ : Type u_1 β✝ : Type u_2 γ : Type u_3 r✝ : α✝ → α✝ → Prop s✝ : β✝ → β✝ → Prop t : γ → γ → Prop α β : Type u_4 r : α → α → Prop s : β → β → Prop inst✝¹ : IsWellOrder α r inst✝ : IsWellOrder β s c : Ordinal.{u_4} h : IsLimit (type s) H : ∀ (b' : Ordinal.{u_4}), b' < type s → type r * b' ≤ c l : c < type r * type s a : α b : β this✝ : type r * typein s b + type r ≤ c this : type r * typein s b + typein r a < c ⊢ typein (Prod.Lex s r) (b, a) < c ** refine' (RelEmbedding.ofMonotone (fun a => _) fun a b => _).ordinal_type_le.trans_lt this ** α✝ : Type u_1 β✝ : Type u_2 γ : Type u_3 r✝ : α✝ → α✝ → Prop s✝ : β✝ → β✝ → Prop t : γ → γ → Prop α β : Type u_4 r : α → α → Prop s : β → β → Prop inst✝¹ : IsWellOrder α r inst✝ : IsWellOrder β s c : Ordinal.{u_4} h : IsLimit (type s) H : ∀ (b' : Ordinal.{u_4}), b' < type s → type r * b' ≤ c l : c < type r * type s this : ∀ (a : α) (b : β), Prod.Lex s r (b, a) (enum (Prod.Lex s r) c l) ⊢ False ** cases' enum _ _ l with b a ** case mk α✝ : Type u_1 β✝ : Type u_2 γ : Type u_3 r✝ : α✝ → α✝ → Prop s✝ : β✝ → β✝ → Prop t : γ → γ → Prop α β : Type u_4 r : α → α → Prop s : β → β → Prop inst✝¹ : IsWellOrder α r inst✝ : IsWellOrder β s c : Ordinal.{u_4} h : IsLimit (type s) H : ∀ (b' : Ordinal.{u_4}), b' < type s → type r * b' ≤ c l : c < type r * type s this : ∀ (a : α) (b : β), Prod.Lex s r (b, a) (enum (Prod.Lex s r) c l) b : β a : α ⊢ False ** exact irrefl _ (this _ _) ** case refine'_1 α✝ : Type u_1 β✝ : Type u_2 γ : Type u_3 r✝ : α✝ → α✝ → Prop s✝ : β✝ → β✝ → Prop t : γ → γ → Prop α β : Type u_4 r : α → α → Prop s : β → β → Prop inst✝¹ : IsWellOrder α r inst✝ : IsWellOrder β s c : Ordinal.{u_4} h : IsLimit (type s) H : ∀ (b' : Ordinal.{u_4}), b' < type s → type r * b' ≤ c l : c < type r * type s a✝ : α b : β this✝ : type r * typein s b + type r ≤ c this : type r * typein s b + typein r a✝ < c a : ↑{b_1 | Prod.Lex s r b_1 (b, a✝)} ⊢ ↑{b_1 | s b_1 b} × α ⊕ ↑{b | r b a✝} ** rcases a with ⟨⟨b', a'⟩, h⟩ ** case refine'_1.mk.mk α✝ : Type u_1 β✝ : Type u_2 γ : Type u_3 r✝ : α✝ → α✝ → Prop s✝ : β✝ → β✝ → Prop t : γ → γ → Prop α β : Type u_4 r : α → α → Prop s : β → β → Prop inst✝¹ : IsWellOrder α r inst✝ : IsWellOrder β s c : Ordinal.{u_4} h✝ : IsLimit (type s) H : ∀ (b' : Ordinal.{u_4}), b' < type s → type r * b' ≤ c l : c < type r * type s a : α b : β this✝ : type r * typein s b + type r ≤ c this : type r * typein s b + typein r a < c b' : β a' : α h : (b', a') ∈ {b_1 | Prod.Lex s r b_1 (b, a)} ⊢ ↑{b_1 | s b_1 b} × α ⊕ ↑{b | r b a} ** by_cases e : b = b' ** case pos α✝ : Type u_1 β✝ : Type u_2 γ : Type u_3 r✝ : α✝ → α✝ → Prop s✝ : β✝ → β✝ → Prop t : γ → γ → Prop α β : Type u_4 r : α → α → Prop s : β → β → Prop inst✝¹ : IsWellOrder α r inst✝ : IsWellOrder β s c : Ordinal.{u_4} h✝ : IsLimit (type s) H : ∀ (b' : Ordinal.{u_4}), b' < type s → type r * b' ≤ c l : c < type r * type s a : α b : β this✝ : type r * typein s b + type r ≤ c this : type r * typein s b + typein r a < c b' : β a' : α h : (b', a') ∈ {b_1 | Prod.Lex s r b_1 (b, a)} e : b = b' ⊢ ↑{b_1 | s b_1 b} × α ⊕ ↑{b | r b a} ** refine' Sum.inr ⟨a', _⟩ ** case pos α✝ : Type u_1 β✝ : Type u_2 γ : Type u_3 r✝ : α✝ → α✝ → Prop s✝ : β✝ → β✝ → Prop t : γ → γ → Prop α β : Type u_4 r : α → α → Prop s : β → β → Prop inst✝¹ : IsWellOrder α r inst✝ : IsWellOrder β s c : Ordinal.{u_4} h✝ : IsLimit (type s) H : ∀ (b' : Ordinal.{u_4}), b' < type s → type r * b' ≤ c l : c < type r * type s a : α b : β this✝ : type r * typein s b + type r ≤ c this : type r * typein s b + typein r a < c b' : β a' : α h : (b', a') ∈ {b_1 | Prod.Lex s r b_1 (b, a)} e : b = b' ⊢ a' ∈ {b | r b a} ** subst e ** case pos α✝ : Type u_1 β✝ : Type u_2 γ : Type u_3 r✝ : α✝ → α✝ → Prop s✝ : β✝ → β✝ → Prop t : γ → γ → Prop α β : Type u_4 r : α → α → Prop s : β → β → Prop inst✝¹ : IsWellOrder α r inst✝ : IsWellOrder β s c : Ordinal.{u_4} h✝ : IsLimit (type s) H : ∀ (b' : Ordinal.{u_4}), b' < type s → type r * b' ≤ c l : c < type r * type s a : α b : β this✝ : type r * typein s b + type r ≤ c this : type r * typein s b + typein r a < c a' : α h : (b, a') ∈ {b_1 | Prod.Lex s r b_1 (b, a)} ⊢ a' ∈ {b | r b a} ** cases' h with _ _ _ _ h _ _ _ h ** case pos.left α✝ : Type u_1 β✝ : Type u_2 γ : Type u_3 r✝ : α✝ → α✝ → Prop s✝ : β✝ → β✝ → Prop t : γ → γ → Prop α β : Type u_4 r : α → α → Prop s : β → β → Prop inst✝¹ : IsWellOrder α r inst✝ : IsWellOrder β s c : Ordinal.{u_4} h✝ : IsLimit (type s) H : ∀ (b' : Ordinal.{u_4}), b' < type s → type r * b' ≤ c l : c < type r * type s a : α b : β this✝ : type r * typein s b + type r ≤ c this : type r * typein s b + typein r a < c a' : α h : s b b ⊢ a' ∈ {b | r b a} ** exact (irrefl _ h).elim ** case pos.right α✝ : Type u_1 β✝ : Type u_2 γ : Type u_3 r✝ : α✝ → α✝ → Prop s✝ : β✝ → β✝ → Prop t : γ → γ → Prop α β : Type u_4 r : α → α → Prop s : β → β → Prop inst✝¹ : IsWellOrder α r inst✝ : IsWellOrder β s c : Ordinal.{u_4} h✝ : IsLimit (type s) H : ∀ (b' : Ordinal.{u_4}), b' < type s → type r * b' ≤ c l : c < type r * type s a : α b : β this✝ : type r * typein s b + type r ≤ c this : type r * typein s b + typein r a < c a' : α h : r a' a ⊢ a' ∈ {b | r b a} ** exact h ** case neg α✝ : Type u_1 β✝ : Type u_2 γ : Type u_3 r✝ : α✝ → α✝ → Prop s✝ : β✝ → β✝ → Prop t : γ → γ → Prop α β : Type u_4 r : α → α → Prop s : β → β → Prop inst✝¹ : IsWellOrder α r inst✝ : IsWellOrder β s c : Ordinal.{u_4} h✝ : IsLimit (type s) H : ∀ (b' : Ordinal.{u_4}), b' < type s → type r * b' ≤ c l : c < type r * type s a : α b : β this✝ : type r * typein s b + type r ≤ c this : type r * typein s b + typein r a < c b' : β a' : α h : (b', a') ∈ {b_1 | Prod.Lex s r b_1 (b, a)} e : ¬b = b' ⊢ ↑{b_1 | s b_1 b} × α ⊕ ↑{b | r b a} ** refine' Sum.inl (⟨b', _⟩, a') ** case neg α✝ : Type u_1 β✝ : Type u_2 γ : Type u_3 r✝ : α✝ → α✝ → Prop s✝ : β✝ → β✝ → Prop t : γ → γ → Prop α β : Type u_4 r : α → α → Prop s : β → β → Prop inst✝¹ : IsWellOrder α r inst✝ : IsWellOrder β s c : Ordinal.{u_4} h✝ : IsLimit (type s) H : ∀ (b' : Ordinal.{u_4}), b' < type s → type r * b' ≤ c l : c < type r * type s a : α b : β this✝ : type r * typein s b + type r ≤ c this : type r * typein s b + typein r a < c b' : β a' : α h : (b', a') ∈ {b_1 | Prod.Lex s r b_1 (b, a)} e : ¬b = b' ⊢ b' ∈ {b_1 | s b_1 b} ** cases' h with _ _ _ _ h _ _ _ h ** case neg.left α✝ : Type u_1 β✝ : Type u_2 γ : Type u_3 r✝ : α✝ → α✝ → Prop s✝ : β✝ → β✝ → Prop t : γ → γ → Prop α β : Type u_4 r : α → α → Prop s : β → β → Prop inst✝¹ : IsWellOrder α r inst✝ : IsWellOrder β s c : Ordinal.{u_4} h✝ : IsLimit (type s) H : ∀ (b' : Ordinal.{u_4}), b' < type s → type r * b' ≤ c l : c < type r * type s a : α b : β this✝ : type r * typein s b + type r ≤ c this : type r * typein s b + typein r a < c b' : β a' : α e : ¬b = b' h : s b' b ⊢ b' ∈ {b_1 | s b_1 b} ** exact h ** case neg.right α✝ : Type u_1 β✝ : Type u_2 γ : Type u_3 r✝ : α✝ → α✝ → Prop s✝ : β✝ → β✝ → Prop t : γ → γ → Prop α β : Type u_4 r : α → α → Prop s : β → β → Prop inst✝¹ : IsWellOrder α r inst✝ : IsWellOrder β s c : Ordinal.{u_4} h✝ : IsLimit (type s) H : ∀ (b' : Ordinal.{u_4}), b' < type s → type r * b' ≤ c l : c < type r * type s a : α b : β this✝ : type r * typein s b + type r ≤ c this : type r * typein s b + typein r a < c a' : α e : ¬b = b h : r a' a ⊢ b ∈ {b_1 | s b_1 b} ** exact (e rfl).elim ** case refine'_2 α✝ : Type u_1 β✝ : Type u_2 γ : Type u_3 r✝ : α✝ → α✝ → Prop s✝ : β✝ → β✝ → Prop t : γ → γ → Prop α β : Type u_4 r : α → α → Prop s : β → β → Prop inst✝¹ : IsWellOrder α r inst✝ : IsWellOrder β s c : Ordinal.{u_4} h : IsLimit (type s) H : ∀ (b' : Ordinal.{u_4}), b' < type s → type r * b' ≤ c l : c < type r * type s a✝ : α b✝ : β this✝ : type r * typein s b✝ + type r ≤ c this : type r * typein s b✝ + typein r a✝ < c a b : ↑{b | Prod.Lex s r b (b✝, a✝)} ⊢ Subrel (Prod.Lex s r) {b | Prod.Lex s r b (b✝, a✝)} a b → Sum.Lex (Prod.Lex (Subrel s {b | s b b✝}) r) (Subrel r {b | r b a✝}) ((fun a => Subtype.casesOn a fun val h => Prod.casesOn (motive := fun x => x ∈ {b | Prod.Lex s r b (b✝, a✝)} → ↑{b | s b b✝} × α ⊕ ↑{b | r b a✝}) val (fun b' a' h => if e : b✝ = b' then Sum.inr { val := a', property := (_ : a' ∈ {b | r b a✝}) } else Sum.inl ({ val := b', property := (_ : b' ∈ {b | s b b✝}) }, a')) h) a) ((fun a => Subtype.casesOn a fun val h => Prod.casesOn (motive := fun x => x ∈ {b | Prod.Lex s r b (b✝, a✝)} → ↑{b | s b b✝} × α ⊕ ↑{b | r b a✝}) val (fun b' a' h => if e : b✝ = b' then Sum.inr { val := a', property := (_ : a' ∈ {b | r b a✝}) } else Sum.inl ({ val := b', property := (_ : b' ∈ {b | s b b✝}) }, a')) h) b) ** rcases a with ⟨⟨b₁, a₁⟩, h₁⟩ ** case refine'_2.mk.mk α✝ : Type u_1 β✝ : Type u_2 γ : Type u_3 r✝ : α✝ → α✝ → Prop s✝ : β✝ → β✝ → Prop t : γ → γ → Prop α β : Type u_4 r : α → α → Prop s : β → β → Prop inst✝¹ : IsWellOrder α r inst✝ : IsWellOrder β s c : Ordinal.{u_4} h : IsLimit (type s) H : ∀ (b' : Ordinal.{u_4}), b' < type s → type r * b' ≤ c l : c < type r * type s a : α b✝ : β this✝ : type r * typein s b✝ + type r ≤ c this : type r * typein s b✝ + typein r a < c b : ↑{b | Prod.Lex s r b (b✝, a)} b₁ : β a₁ : α h₁ : (b₁, a₁) ∈ {b | Prod.Lex s r b (b✝, a)} ⊢ Subrel (Prod.Lex s r) {b | Prod.Lex s r b (b✝, a)} { val := (b₁, a₁), property := h₁ } b → Sum.Lex (Prod.Lex (Subrel s {b | s b b✝}) r) (Subrel r {b | r b a}) ((fun a_2 => Subtype.casesOn a_2 fun val h => Prod.casesOn (motive := fun x => x ∈ {b | Prod.Lex s r b (b✝, a)} → ↑{b | s b b✝} × α ⊕ ↑{b | r b a}) val (fun b' a' h => if e : b✝ = b' then Sum.inr { val := a', property := (_ : a' ∈ {b | r b a}) } else Sum.inl ({ val := b', property := (_ : b' ∈ {b | s b b✝}) }, a')) h) { val := (b₁, a₁), property := h₁ }) ((fun a_2 => Subtype.casesOn a_2 fun val h => Prod.casesOn (motive := fun x => x ∈ {b | Prod.Lex s r b (b✝, a)} → ↑{b | s b b✝} × α ⊕ ↑{b | r b a}) val (fun b' a' h => if e : b✝ = b' then Sum.inr { val := a', property := (_ : a' ∈ {b | r b a}) } else Sum.inl ({ val := b', property := (_ : b' ∈ {b | s b b✝}) }, a')) h) b) ** rcases b with ⟨⟨b₂, a₂⟩, h₂⟩ ** case refine'_2.mk.mk.mk.mk α✝ : Type u_1 β✝ : Type u_2 γ : Type u_3 r✝ : α✝ → α✝ → Prop s✝ : β✝ → β✝ → Prop t : γ → γ → Prop α β : Type u_4 r : α → α → Prop s : β → β → Prop inst✝¹ : IsWellOrder α r inst✝ : IsWellOrder β s c : Ordinal.{u_4} h : IsLimit (type s) H : ∀ (b' : Ordinal.{u_4}), b' < type s → type r * b' ≤ c l : c < type r * type s a : α b : β this✝ : type r * typein s b + type r ≤ c this : type r * typein s b + typein r a < c b₁ : β a₁ : α h₁ : (b₁, a₁) ∈ {b_1 | Prod.Lex s r b_1 (b, a)} b₂ : β a₂ : α h₂ : (b₂, a₂) ∈ {b_1 | Prod.Lex s r b_1 (b, a)} ⊢ Subrel (Prod.Lex s r) {b_1 | Prod.Lex s r b_1 (b, a)} { val := (b₁, a₁), property := h₁ } { val := (b₂, a₂), property := h₂ } → Sum.Lex (Prod.Lex (Subrel s {b_1 | s b_1 b}) r) (Subrel r {b | r b a}) ((fun a_2 => Subtype.casesOn a_2 fun val h => Prod.casesOn (motive := fun x => x ∈ {b_1 | Prod.Lex s r b_1 (b, a)} → ↑{b_1 | s b_1 b} × α ⊕ ↑{b | r b a}) val (fun b' a' h => if e : b = b' then Sum.inr { val := a', property := (_ : a' ∈ {b | r b a}) } else Sum.inl ({ val := b', property := (_ : b' ∈ {b_1 | s b_1 b}) }, a')) h) { val := (b₁, a₁), property := h₁ }) ((fun a_2 => Subtype.casesOn a_2 fun val h => Prod.casesOn (motive := fun x => x ∈ {b_1 | Prod.Lex s r b_1 (b, a)} → ↑{b_1 | s b_1 b} × α ⊕ ↑{b | r b a}) val (fun b' a' h => if e : b = b' then Sum.inr { val := a', property := (_ : a' ∈ {b | r b a}) } else Sum.inl ({ val := b', property := (_ : b' ∈ {b_1 | s b_1 b}) }, a')) h) { val := (b₂, a₂), property := h₂ }) ** intro h ** case refine'_2.mk.mk.mk.mk α✝ : Type u_1 β✝ : Type u_2 γ : Type u_3 r✝ : α✝ → α✝ → Prop s✝ : β✝ → β✝ → Prop t : γ → γ → Prop α β : Type u_4 r : α → α → Prop s : β → β → Prop inst✝¹ : IsWellOrder α r inst✝ : IsWellOrder β s c : Ordinal.{u_4} h✝ : IsLimit (type s) H : ∀ (b' : Ordinal.{u_4}), b' < type s → type r * b' ≤ c l : c < type r * type s a : α b : β this✝ : type r * typein s b + type r ≤ c this : type r * typein s b + typein r a < c b₁ : β a₁ : α h₁ : (b₁, a₁) ∈ {b_1 | Prod.Lex s r b_1 (b, a)} b₂ : β a₂ : α h₂ : (b₂, a₂) ∈ {b_1 | Prod.Lex s r b_1 (b, a)} h : Subrel (Prod.Lex s r) {b_1 | Prod.Lex s r b_1 (b, a)} { val := (b₁, a₁), property := h₁ } { val := (b₂, a₂), property := h₂ } ⊢ Sum.Lex (Prod.Lex (Subrel s {b_1 | s b_1 b}) r) (Subrel r {b | r b a}) ((fun a_1 => Subtype.casesOn a_1 fun val h => Prod.casesOn (motive := fun x => x ∈ {b_1 | Prod.Lex s r b_1 (b, a)} → ↑{b_1 | s b_1 b} × α ⊕ ↑{b | r b a}) val (fun b' a' h => if e : b = b' then Sum.inr { val := a', property := (_ : a' ∈ {b | r b a}) } else Sum.inl ({ val := b', property := (_ : b' ∈ {b_1 | s b_1 b}) }, a')) h) { val := (b₁, a₁), property := h₁ }) ((fun a_1 => Subtype.casesOn a_1 fun val h => Prod.casesOn (motive := fun x => x ∈ {b_1 | Prod.Lex s r b_1 (b, a)} → ↑{b_1 | s b_1 b} × α ⊕ ↑{b | r b a}) val (fun b' a' h => if e : b = b' then Sum.inr { val := a', property := (_ : a' ∈ {b | r b a}) } else Sum.inl ({ val := b', property := (_ : b' ∈ {b_1 | s b_1 b}) }, a')) h) { val := (b₂, a₂), property := h₂ }) ** by_cases e₁ : b = b₁ <;> by_cases e₂ : b = b₂ ** case pos α✝ : Type u_1 β✝ : Type u_2 γ : Type u_3 r✝ : α✝ → α✝ → Prop s✝ : β✝ → β✝ → Prop t : γ → γ → Prop α β : Type u_4 r : α → α → Prop s : β → β → Prop inst✝¹ : IsWellOrder α r inst✝ : IsWellOrder β s c : Ordinal.{u_4} h✝ : IsLimit (type s) H : ∀ (b' : Ordinal.{u_4}), b' < type s → type r * b' ≤ c l : c < type r * type s a : α b : β this✝ : type r * typein s b + type r ≤ c this : type r * typein s b + typein r a < c b₁ : β a₁ : α h₁ : (b₁, a₁) ∈ {b_1 | Prod.Lex s r b_1 (b, a)} b₂ : β a₂ : α h₂ : (b₂, a₂) ∈ {b_1 | Prod.Lex s r b_1 (b, a)} h : Subrel (Prod.Lex s r) {b_1 | Prod.Lex s r b_1 (b, a)} { val := (b₁, a₁), property := h₁ } { val := (b₂, a₂), property := h₂ } e₁ : b = b₁ e₂ : b = b₂ ⊢ Sum.Lex (Prod.Lex (Subrel s {b_1 | s b_1 b}) r) (Subrel r {b | r b a}) ((fun a_1 => Subtype.casesOn a_1 fun val h => Prod.casesOn (motive := fun x => x ∈ {b_1 | Prod.Lex s r b_1 (b, a)} → ↑{b_1 | s b_1 b} × α ⊕ ↑{b | r b a}) val (fun b' a' h => if e : b = b' then Sum.inr { val := a', property := (_ : a' ∈ {b | r b a}) } else Sum.inl ({ val := b', property := (_ : b' ∈ {b_1 | s b_1 b}) }, a')) h) { val := (b₁, a₁), property := h₁ }) ((fun a_1 => Subtype.casesOn a_1 fun val h => Prod.casesOn (motive := fun x => x ∈ {b_1 | Prod.Lex s r b_1 (b, a)} → ↑{b_1 | s b_1 b} × α ⊕ ↑{b | r b a}) val (fun b' a' h => if e : b = b' then Sum.inr { val := a', property := (_ : a' ∈ {b | r b a}) } else Sum.inl ({ val := b', property := (_ : b' ∈ {b_1 | s b_1 b}) }, a')) h) { val := (b₂, a₂), property := h₂ }) ** substs b₁ b₂ ** case pos α✝ : Type u_1 β✝ : Type u_2 γ : Type u_3 r✝ : α✝ → α✝ → Prop s✝ : β✝ → β✝ → Prop t : γ → γ → Prop α β : Type u_4 r : α → α → Prop s : β → β → Prop inst✝¹ : IsWellOrder α r inst✝ : IsWellOrder β s c : Ordinal.{u_4} h✝ : IsLimit (type s) H : ∀ (b' : Ordinal.{u_4}), b' < type s → type r * b' ≤ c l : c < type r * type s a : α b : β this✝ : type r * typein s b + type r ≤ c this : type r * typein s b + typein r a < c a₁ a₂ : α h₁ : (b, a₁) ∈ {b_1 | Prod.Lex s r b_1 (b, a)} h₂ : (b, a₂) ∈ {b_1 | Prod.Lex s r b_1 (b, a)} h : Subrel (Prod.Lex s r) {b_1 | Prod.Lex s r b_1 (b, a)} { val := (b, a₁), property := h₁ } { val := (b, a₂), property := h₂ } ⊢ Sum.Lex (Prod.Lex (Subrel s {b_1 | s b_1 b}) r) (Subrel r {b | r b a}) ((fun a_1 => Subtype.casesOn a_1 fun val h => Prod.casesOn (motive := fun x => x ∈ {b_1 | Prod.Lex s r b_1 (b, a)} → ↑{b_1 | s b_1 b} × α ⊕ ↑{b | r b a}) val (fun b' a' h => if e : b = b' then Sum.inr { val := a', property := (_ : a' ∈ {b | r b a}) } else Sum.inl ({ val := b', property := (_ : b' ∈ {b_1 | s b_1 b}) }, a')) h) { val := (b, a₁), property := h₁ }) ((fun a_1 => Subtype.casesOn a_1 fun val h => Prod.casesOn (motive := fun x => x ∈ {b_1 | Prod.Lex s r b_1 (b, a)} → ↑{b_1 | s b_1 b} × α ⊕ ↑{b | r b a}) val (fun b' a' h => if e : b = b' then Sum.inr { val := a', property := (_ : a' ∈ {b | r b a}) } else Sum.inl ({ val := b', property := (_ : b' ∈ {b_1 | s b_1 b}) }, a')) h) { val := (b, a₂), property := h₂ }) ** simpa only [subrel_val, Prod.lex_def, @irrefl _ s _ b, true_and_iff, false_or_iff, eq_self_iff_true, dif_pos, Sum.lex_inr_inr] using h ** case neg α✝ : Type u_1 β✝ : Type u_2 γ : Type u_3 r✝ : α✝ → α✝ → Prop s✝ : β✝ → β✝ → Prop t : γ → γ → Prop α β : Type u_4 r : α → α → Prop s : β → β → Prop inst✝¹ : IsWellOrder α r inst✝ : IsWellOrder β s c : Ordinal.{u_4} h✝ : IsLimit (type s) H : ∀ (b' : Ordinal.{u_4}), b' < type s → type r * b' ≤ c l : c < type r * type s a : α b : β this✝ : type r * typein s b + type r ≤ c this : type r * typein s b + typein r a < c b₁ : β a₁ : α h₁ : (b₁, a₁) ∈ {b_1 | Prod.Lex s r b_1 (b, a)} b₂ : β a₂ : α h₂ : (b₂, a₂) ∈ {b_1 | Prod.Lex s r b_1 (b, a)} h : Subrel (Prod.Lex s r) {b_1 | Prod.Lex s r b_1 (b, a)} { val := (b₁, a₁), property := h₁ } { val := (b₂, a₂), property := h₂ } e₁ : b = b₁ e₂ : ¬b = b₂ ⊢ Sum.Lex (Prod.Lex (Subrel s {b_1 | s b_1 b}) r) (Subrel r {b | r b a}) ((fun a_1 => Subtype.casesOn a_1 fun val h => Prod.casesOn (motive := fun x => x ∈ {b_1 | Prod.Lex s r b_1 (b, a)} → ↑{b_1 | s b_1 b} × α ⊕ ↑{b | r b a}) val (fun b' a' h => if e : b = b' then Sum.inr { val := a', property := (_ : a' ∈ {b | r b a}) } else Sum.inl ({ val := b', property := (_ : b' ∈ {b_1 | s b_1 b}) }, a')) h) { val := (b₁, a₁), property := h₁ }) ((fun a_1 => Subtype.casesOn a_1 fun val h => Prod.casesOn (motive := fun x => x ∈ {b_1 | Prod.Lex s r b_1 (b, a)} → ↑{b_1 | s b_1 b} × α ⊕ ↑{b | r b a}) val (fun b' a' h => if e : b = b' then Sum.inr { val := a', property := (_ : a' ∈ {b | r b a}) } else Sum.inl ({ val := b', property := (_ : b' ∈ {b_1 | s b_1 b}) }, a')) h) { val := (b₂, a₂), property := h₂ }) ** subst b₁ ** case neg α✝ : Type u_1 β✝ : Type u_2 γ : Type u_3 r✝ : α✝ → α✝ → Prop s✝ : β✝ → β✝ → Prop t : γ → γ → Prop α β : Type u_4 r : α → α → Prop s : β → β → Prop inst✝¹ : IsWellOrder α r inst✝ : IsWellOrder β s c : Ordinal.{u_4} h✝ : IsLimit (type s) H : ∀ (b' : Ordinal.{u_4}), b' < type s → type r * b' ≤ c l : c < type r * type s a : α b : β this✝ : type r * typein s b + type r ≤ c this : type r * typein s b + typein r a < c a₁ : α b₂ : β a₂ : α h₂ : (b₂, a₂) ∈ {b_1 | Prod.Lex s r b_1 (b, a)} e₂ : ¬b = b₂ h₁ : (b, a₁) ∈ {b_1 | Prod.Lex s r b_1 (b, a)} h : Subrel (Prod.Lex s r) {b_1 | Prod.Lex s r b_1 (b, a)} { val := (b, a₁), property := h₁ } { val := (b₂, a₂), property := h₂ } ⊢ Sum.Lex (Prod.Lex (Subrel s {b_1 | s b_1 b}) r) (Subrel r {b | r b a}) ((fun a_1 => Subtype.casesOn a_1 fun val h => Prod.casesOn (motive := fun x => x ∈ {b_1 | Prod.Lex s r b_1 (b, a)} → ↑{b_1 | s b_1 b} × α ⊕ ↑{b | r b a}) val (fun b' a' h => if e : b = b' then Sum.inr { val := a', property := (_ : a' ∈ {b | r b a}) } else Sum.inl ({ val := b', property := (_ : b' ∈ {b_1 | s b_1 b}) }, a')) h) { val := (b, a₁), property := h₁ }) ((fun a_1 => Subtype.casesOn a_1 fun val h => Prod.casesOn (motive := fun x => x ∈ {b_1 | Prod.Lex s r b_1 (b, a)} → ↑{b_1 | s b_1 b} × α ⊕ ↑{b | r b a}) val (fun b' a' h => if e : b = b' then Sum.inr { val := a', property := (_ : a' ∈ {b | r b a}) } else Sum.inl ({ val := b', property := (_ : b' ∈ {b_1 | s b_1 b}) }, a')) h) { val := (b₂, a₂), property := h₂ }) ** simp only [subrel_val, Prod.lex_def, e₂, Prod.lex_def, dif_pos, subrel_val, eq_self_iff_true, or_false_iff, dif_neg, not_false_iff, Sum.lex_inr_inl, false_and_iff] at h ⊢ ** case neg α✝ : Type u_1 β✝ : Type u_2 γ : Type u_3 r✝ : α✝ → α✝ → Prop s✝ : β✝ → β✝ → Prop t : γ → γ → Prop α β : Type u_4 r : α → α → Prop s : β → β → Prop inst✝¹ : IsWellOrder α r inst✝ : IsWellOrder β s c : Ordinal.{u_4} h✝ : IsLimit (type s) H : ∀ (b' : Ordinal.{u_4}), b' < type s → type r * b' ≤ c l : c < type r * type s a : α b : β this✝ : type r * typein s b + type r ≤ c this : type r * typein s b + typein r a < c a₁ : α b₂ : β a₂ : α h₂ : (b₂, a₂) ∈ {b_1 | Prod.Lex s r b_1 (b, a)} e₂ : ¬b = b₂ h₁ : (b, a₁) ∈ {b_1 | Prod.Lex s r b_1 (b, a)} h : s b b₂ ⊢ False ** cases' h₂ with _ _ _ _ h₂_h h₂_h <;> [exact asymm h h₂_h; exact e₂ rfl] ** case pos α✝ : Type u_1 β✝ : Type u_2 γ : Type u_3 r✝ : α✝ → α✝ → Prop s✝ : β✝ → β✝ → Prop t : γ → γ → Prop α β : Type u_4 r : α → α → Prop s : β → β → Prop inst✝¹ : IsWellOrder α r inst✝ : IsWellOrder β s c : Ordinal.{u_4} h✝ : IsLimit (type s) H : ∀ (b' : Ordinal.{u_4}), b' < type s → type r * b' ≤ c l : c < type r * type s a : α b : β this✝ : type r * typein s b + type r ≤ c this : type r * typein s b + typein r a < c b₁ : β a₁ : α h₁ : (b₁, a₁) ∈ {b_1 | Prod.Lex s r b_1 (b, a)} b₂ : β a₂ : α h₂ : (b₂, a₂) ∈ {b_1 | Prod.Lex s r b_1 (b, a)} h : Subrel (Prod.Lex s r) {b_1 | Prod.Lex s r b_1 (b, a)} { val := (b₁, a₁), property := h₁ } { val := (b₂, a₂), property := h₂ } e₁ : ¬b = b₁ e₂ : b = b₂ ⊢ Sum.Lex (Prod.Lex (Subrel s {b_1 | s b_1 b}) r) (Subrel r {b | r b a}) ((fun a_1 => Subtype.casesOn a_1 fun val h => Prod.casesOn (motive := fun x => x ∈ {b_1 | Prod.Lex s r b_1 (b, a)} → ↑{b_1 | s b_1 b} × α ⊕ ↑{b | r b a}) val (fun b' a' h => if e : b = b' then Sum.inr { val := a', property := (_ : a' ∈ {b | r b a}) } else Sum.inl ({ val := b', property := (_ : b' ∈ {b_1 | s b_1 b}) }, a')) h) { val := (b₁, a₁), property := h₁ }) ((fun a_1 => Subtype.casesOn a_1 fun val h => Prod.casesOn (motive := fun x => x ∈ {b_1 | Prod.Lex s r b_1 (b, a)} → ↑{b_1 | s b_1 b} × α ⊕ ↑{b | r b a}) val (fun b' a' h => if e : b = b' then Sum.inr { val := a', property := (_ : a' ∈ {b | r b a}) } else Sum.inl ({ val := b', property := (_ : b' ∈ {b_1 | s b_1 b}) }, a')) h) { val := (b₂, a₂), property := h₂ }) ** simp [e₂, dif_neg e₁, show b₂ ≠ b₁ from e₂ ▸ e₁] ** case neg α✝ : Type u_1 β✝ : Type u_2 γ : Type u_3 r✝ : α✝ → α✝ → Prop s✝ : β✝ → β✝ → Prop t : γ → γ → Prop α β : Type u_4 r : α → α → Prop s : β → β → Prop inst✝¹ : IsWellOrder α r inst✝ : IsWellOrder β s c : Ordinal.{u_4} h✝ : IsLimit (type s) H : ∀ (b' : Ordinal.{u_4}), b' < type s → type r * b' ≤ c l : c < type r * type s a : α b : β this✝ : type r * typein s b + type r ≤ c this : type r * typein s b + typein r a < c b₁ : β a₁ : α h₁ : (b₁, a₁) ∈ {b_1 | Prod.Lex s r b_1 (b, a)} b₂ : β a₂ : α h₂ : (b₂, a₂) ∈ {b_1 | Prod.Lex s r b_1 (b, a)} h : Subrel (Prod.Lex s r) {b_1 | Prod.Lex s r b_1 (b, a)} { val := (b₁, a₁), property := h₁ } { val := (b₂, a₂), property := h₂ } e₁ : ¬b = b₁ e₂ : ¬b = b₂ ⊢ Sum.Lex (Prod.Lex (Subrel s {b_1 | s b_1 b}) r) (Subrel r {b | r b a}) ((fun a_1 => Subtype.casesOn a_1 fun val h => Prod.casesOn (motive := fun x => x ∈ {b_1 | Prod.Lex s r b_1 (b, a)} → ↑{b_1 | s b_1 b} × α ⊕ ↑{b | r b a}) val (fun b' a' h => if e : b = b' then Sum.inr { val := a', property := (_ : a' ∈ {b | r b a}) } else Sum.inl ({ val := b', property := (_ : b' ∈ {b_1 | s b_1 b}) }, a')) h) { val := (b₁, a₁), property := h₁ }) ((fun a_1 => Subtype.casesOn a_1 fun val h => Prod.casesOn (motive := fun x => x ∈ {b_1 | Prod.Lex s r b_1 (b, a)} → ↑{b_1 | s b_1 b} × α ⊕ ↑{b | r b a}) val (fun b' a' h => if e : b = b' then Sum.inr { val := a', property := (_ : a' ∈ {b | r b a}) } else Sum.inl ({ val := b', property := (_ : b' ∈ {b_1 | s b_1 b}) }, a')) h) { val := (b₂, a₂), property := h₂ }) ** simpa only [dif_neg e₁, dif_neg e₂, Prod.lex_def, subrel_val, Subtype.mk_eq_mk, Sum.lex_inl_inl] using h ** Qed
Ordinal.mul_le_of_limit ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b c : Ordinal.{u_4} h : IsLimit b H : ∀ (b' : Ordinal.{u_4}), b' < b → a * b' ≤ c ⊢ ¬c < a * b ** induction a using inductionOn with | H α r => induction b using inductionOn with | H β s => exact mul_le_of_limit_aux h H ** case H α✝ : Type u_1 β : Type u_2 γ : Type u_3 r✝ : α✝ → α✝ → Prop s : β → β → Prop t : γ → γ → Prop b c : Ordinal.{u_4} h : IsLimit b α : Type u_4 r : α → α → Prop inst✝ : IsWellOrder α r H : ∀ (b' : Ordinal.{u_4}), b' < b → type r * b' ≤ c ⊢ ¬c < type r * b ** induction b using inductionOn with | H β s => exact mul_le_of_limit_aux h H ** case H.H α✝ : Type u_1 β✝ : Type u_2 γ : Type u_3 r✝ : α✝ → α✝ → Prop s✝ : β✝ → β✝ → Prop t : γ → γ → Prop c : Ordinal.{u_4} α : Type u_4 r : α → α → Prop inst✝¹ : IsWellOrder α r β : Type u_4 s : β → β → Prop inst✝ : IsWellOrder β s h : IsLimit (type s) H : ∀ (b' : Ordinal.{u_4}), b' < type s → type r * b' ≤ c ⊢ ¬c < type r * type s ** exact mul_le_of_limit_aux h H ** Qed
Ordinal.mul_isNormal ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a : Ordinal.{u_4} h : 0 < a b : Ordinal.{u_4} ⊢ (fun x x_1 => x * x_1) a b < (fun x x_1 => x * x_1) a (succ b) ** dsimp only ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a : Ordinal.{u_4} h : 0 < a b : Ordinal.{u_4} ⊢ a * b < a * succ b ** rw [mul_succ] ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a : Ordinal.{u_4} h : 0 < a b : Ordinal.{u_4} ⊢ a * b < a * b + a ** simpa only [add_zero] using (add_lt_add_iff_left (a * b)).2 h ** Qed
Ordinal.lt_mul_of_limit ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b c : Ordinal.{u_4} h : IsLimit c ⊢ a < b * c ↔ ∃ c', c' < c ∧ a < b * c' ** simpa only [not_ball, not_le, bex_def] using not_congr (@mul_le_of_limit b c a h) ** Qed
Ordinal.mul_pos ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} h₁ : 0 < a h₂ : 0 < b ⊢ 0 < a * b ** simpa only [mul_zero] using mul_lt_mul_of_pos_left h₂ h₁ ** Qed
Ordinal.mul_ne_zero ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} ⊢ a ≠ 0 → b ≠ 0 → a * b ≠ 0 ** simpa only [Ordinal.pos_iff_ne_zero] using mul_pos ** Qed
Ordinal.mul_isLimit_left ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} l : IsLimit a b0 : 0 < b ⊢ IsLimit (a * b) ** rcases zero_or_succ_or_limit b with (rfl | ⟨b, rfl⟩ | lb) ** case inl α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a : Ordinal.{u_4} l : IsLimit a b0 : 0 < 0 ⊢ IsLimit (a * 0) ** exact b0.false.elim ** case inr.inl.intro α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a : Ordinal.{u_4} l : IsLimit a b : Ordinal.{u_4} b0 : 0 < succ b ⊢ IsLimit (a * succ b) ** rw [mul_succ] ** case inr.inl.intro α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a : Ordinal.{u_4} l : IsLimit a b : Ordinal.{u_4} b0 : 0 < succ b ⊢ IsLimit (a * b + a) ** exact add_isLimit _ l ** case inr.inr α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} l : IsLimit a b0 : 0 < b lb : IsLimit b ⊢ IsLimit (a * b) ** exact mul_isLimit l.pos lb ** Qed
Ordinal.smul_eq_mul ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a : Ordinal.{u_4} ⊢ 0 • a = a * ↑0 ** rw [zero_smul, Nat.cast_zero, mul_zero] ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop n : ℕ a : Ordinal.{u_4} ⊢ (n + 1) • a = a * ↑(n + 1) ** rw [succ_nsmul', Nat.cast_add, mul_add, Nat.cast_one, mul_one, smul_eq_mul n] ** Qed
Ordinal.div_nonempty ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} h : b ≠ 0 ⊢ succ a ≤ b * succ a ** simpa only [succ_zero, one_mul] using mul_le_mul_right' (succ_le_of_lt (Ordinal.pos_iff_ne_zero.2 h)) (succ a) ** Qed
Ordinal.lt_mul_succ_div ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} h : b ≠ 0 ⊢ a < b * succ (a / b) ** rw [div_def a h] ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} h : b ≠ 0 ⊢ a < b * succ (sInf {o | a < b * succ o}) ** exact csInf_mem (div_nonempty h) ** Qed
Ordinal.lt_mul_div_add ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} h : b ≠ 0 ⊢ a < b * (a / b) + b ** simpa only [mul_succ] using lt_mul_succ_div a h ** Qed
Ordinal.div_le ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b c : Ordinal.{u_4} b0 : b ≠ 0 h : a < b * succ c ⊢ a / b ≤ c ** rw [div_def a b0] ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b c : Ordinal.{u_4} b0 : b ≠ 0 h : a < b * succ c ⊢ sInf {o | a < b * succ o} ≤ c ** exact csInf_le' h ** Qed
Ordinal.lt_div ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b c : Ordinal.{u_4} h : c ≠ 0 ⊢ a < b / c ↔ c * succ a ≤ b ** rw [← not_le, div_le h, not_lt] ** Qed
Ordinal.div_pos ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop b c : Ordinal.{u_4} h : c ≠ 0 ⊢ 0 < b / c ↔ c ≤ b ** simp [lt_div h] ** Qed
Ordinal.le_div ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b c : Ordinal.{u_4} c0 : c ≠ 0 ⊢ a ≤ b / c ↔ c * a ≤ b ** induction a using limitRecOn with | H₁ => simp only [mul_zero, Ordinal.zero_le] | H₂ _ _ => rw [succ_le_iff, lt_div c0] | H₃ _ h₁ h₂ => revert h₁ h₂ simp (config := { contextual := true }) only [mul_le_of_limit, limit_le, iff_self_iff, forall_true_iff] ** case H₁ α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop b c : Ordinal.{u_4} c0 : c ≠ 0 ⊢ 0 ≤ b / c ↔ c * 0 ≤ b ** simp only [mul_zero, Ordinal.zero_le] ** case H₂ α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop b c : Ordinal.{u_4} c0 : c ≠ 0 o✝ : Ordinal.{u_4} a✝ : o✝ ≤ b / c ↔ c * o✝ ≤ b ⊢ succ o✝ ≤ b / c ↔ c * succ o✝ ≤ b ** rw [succ_le_iff, lt_div c0] ** case H₃ α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop b c : Ordinal.{u_4} c0 : c ≠ 0 o✝ : Ordinal.{u_4} h₁ : IsLimit o✝ h₂ : ∀ (o' : Ordinal.{u_4}), o' < o✝ → (o' ≤ b / c ↔ c * o' ≤ b) ⊢ o✝ ≤ b / c ↔ c * o✝ ≤ b ** revert h₁ h₂ ** case H₃ α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop b c : Ordinal.{u_4} c0 : c ≠ 0 o✝ : Ordinal.{u_4} ⊢ IsLimit o✝ → (∀ (o' : Ordinal.{u_4}), o' < o✝ → (o' ≤ b / c ↔ c * o' ≤ b)) → (o✝ ≤ b / c ↔ c * o✝ ≤ b) ** simp (config := { contextual := true }) only [mul_le_of_limit, limit_le, iff_self_iff, forall_true_iff] ** Qed
Ordinal.div_le_of_le_mul ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b c : Ordinal.{u_4} h : a ≤ b * c b0 : b = 0 ⊢ a / b ≤ c ** simp only [b0, div_zero, Ordinal.zero_le] ** Qed
Ordinal.mul_div_le ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} b0 : b = 0 ⊢ b * (a / b) ≤ a ** simp only [b0, zero_mul, Ordinal.zero_le] ** Qed
Ordinal.mul_add_div ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} b0 : b ≠ 0 c : Ordinal.{u_4} ⊢ (b * a + c) / b = a + c / b ** apply le_antisymm ** case a α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} b0 : b ≠ 0 c : Ordinal.{u_4} ⊢ (b * a + c) / b ≤ a + c / b ** apply (div_le b0).2 ** case a α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} b0 : b ≠ 0 c : Ordinal.{u_4} ⊢ b * a + c < b * succ (a + c / b) ** rw [mul_succ, mul_add, add_assoc, add_lt_add_iff_left] ** case a α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} b0 : b ≠ 0 c : Ordinal.{u_4} ⊢ c < b * (c / b) + b ** apply lt_mul_div_add _ b0 ** case a α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} b0 : b ≠ 0 c : Ordinal.{u_4} ⊢ a + c / b ≤ (b * a + c) / b ** rw [le_div b0, mul_add, add_le_add_iff_left] ** case a α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} b0 : b ≠ 0 c : Ordinal.{u_4} ⊢ b * (c / b) ≤ c ** apply mul_div_le ** Qed
Ordinal.div_eq_zero_of_lt ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} h : a < b ⊢ a / b = 0 ** rw [← Ordinal.le_zero, div_le <| Ordinal.pos_iff_ne_zero.1 <| (Ordinal.zero_le _).trans_lt h] ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} h : a < b ⊢ a < b * succ 0 ** simpa only [succ_zero, mul_one] using h ** Qed
Ordinal.mul_div_cancel ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} b0 : b ≠ 0 ⊢ b * a / b = a ** simpa only [add_zero, zero_div] using mul_add_div a b0 0 ** Qed
Ordinal.div_one ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a : Ordinal.{u_4} ⊢ a / 1 = a ** simpa only [one_mul] using mul_div_cancel a Ordinal.one_ne_zero ** Qed
Ordinal.div_self ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a : Ordinal.{u_4} h : a ≠ 0 ⊢ a / a = 1 ** simpa only [mul_one] using mul_div_cancel 1 h ** Qed
Ordinal.mul_sub ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b c : Ordinal.{u_4} a0 : a = 0 ⊢ a * (b - c) = a * b - a * c ** simp only [a0, zero_mul, sub_self] ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b c : Ordinal.{u_4} a0 : ¬a = 0 d : Ordinal.{u_4} ⊢ a * (b - c) ≤ d ↔ a * b - a * c ≤ d ** rw [sub_le, ← le_div a0, sub_le, ← le_div a0, mul_add_div _ a0] ** Qed
Ordinal.isLimit_add_iff ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} ⊢ IsLimit (a + b) ↔ IsLimit b ∨ b = 0 ∧ IsLimit a ** constructor <;> intro h ** case mpr α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} h : IsLimit b ∨ b = 0 ∧ IsLimit a ⊢ IsLimit (a + b) ** rcases h with (h | ⟨rfl, h⟩) ** case mpr.inl α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} h : IsLimit b ⊢ IsLimit (a + b) case mpr.inr.intro α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a : Ordinal.{u_4} h : IsLimit a ⊢ IsLimit (a + 0) ** exact add_isLimit a h ** case mpr.inr.intro α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a : Ordinal.{u_4} h : IsLimit a ⊢ IsLimit (a + 0) ** simpa only [add_zero] ** case mp α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} h : IsLimit (a + b) ⊢ IsLimit b ∨ b = 0 ∧ IsLimit a ** by_cases h' : b = 0 ** case neg α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} h : IsLimit (a + b) h' : ¬b = 0 ⊢ IsLimit b ∨ b = 0 ∧ IsLimit a ** left ** case neg.h α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} h : IsLimit (a + b) h' : ¬b = 0 ⊢ IsLimit b ** rw [← add_sub_cancel a b] ** case neg.h α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} h : IsLimit (a + b) h' : ¬b = 0 ⊢ IsLimit (a + b - a) ** apply sub_isLimit h ** case neg.h α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} h : IsLimit (a + b) h' : ¬b = 0 ⊢ a < a + b ** suffices : a + 0 < a + b ** case neg.h α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} h : IsLimit (a + b) h' : ¬b = 0 this : a + 0 < a + b ⊢ a < a + b case this α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} h : IsLimit (a + b) h' : ¬b = 0 ⊢ a + 0 < a + b ** simpa only [add_zero] using this ** case this α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} h : IsLimit (a + b) h' : ¬b = 0 ⊢ a + 0 < a + b ** rwa [add_lt_add_iff_left, Ordinal.pos_iff_ne_zero] ** case pos α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} h : IsLimit (a + b) h' : b = 0 ⊢ IsLimit b ∨ b = 0 ∧ IsLimit a ** rw [h', add_zero] at h ** case pos α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} h : IsLimit a h' : b = 0 ⊢ IsLimit b ∨ b = 0 ∧ IsLimit a ** right ** case pos.h α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} h : IsLimit a h' : b = 0 ⊢ b = 0 ∧ IsLimit a ** exact ⟨h', h⟩ ** Qed
Ordinal.dvd_add_iff ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a c b : Ordinal.{u_4} x✝ : a ∣ a * b + c d : Ordinal.{u_4} e : a * b + c = a * d ⊢ c = a * (d - b) ** rw [mul_sub, ← e, add_sub_cancel] ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a c b : Ordinal.{u_4} x✝ : a ∣ c d : Ordinal.{u_4} e : c = a * d ⊢ a ∣ a * b + c ** rw [e, ← mul_add] ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a c b : Ordinal.{u_4} x✝ : a ∣ c d : Ordinal.{u_4} e : c = a * d ⊢ a ∣ a * (b + d) ** apply dvd_mul_right ** Qed
Ordinal.div_mul_cancel ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a : Ordinal.{u_4} a0 : a ≠ 0 b : Ordinal.{u_4} ⊢ a * (a * b / a) = a * b ** rw [mul_div_cancel _ a0] ** Qed
Ordinal.le_of_dvd ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a x✝ : Ordinal.{u_4} b0 : x✝ ≠ 0 b : Ordinal.{u_4} e : x✝ = a * b ⊢ a ≤ x✝ ** subst e ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} b0 : a * b ≠ 0 ⊢ a ≤ a * b ** simpa only [mul_one] using mul_le_mul_left' (one_le_iff_ne_zero.2 fun h : b = 0 => by simp only [h, mul_zero, Ne] at b0) a ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} b0 : a * b ≠ 0 h : b = 0 ⊢ False ** simp only [h, mul_zero, Ne] at b0 ** Qed
Ordinal.dvd_antisymm ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} h₁ : a ∣ b h₂ : b ∣ a a0 : a = 0 ⊢ a = b ** subst a ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop b : Ordinal.{u_4} h₁ : 0 ∣ b h₂ : b ∣ 0 ⊢ 0 = b ** exact (eq_zero_of_zero_dvd h₁).symm ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} h₁ : a ∣ b h₂ : b ∣ a a0 : ¬a = 0 b0 : b = 0 ⊢ a = b ** subst b ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a : Ordinal.{u_4} a0 : ¬a = 0 h₁ : a ∣ 0 h₂ : 0 ∣ a ⊢ a = 0 ** exact eq_zero_of_zero_dvd h₂ ** Qed
Ordinal.mod_zero ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a : Ordinal.{u_4} ⊢ a % 0 = a ** simp only [mod_def, div_zero, zero_mul, sub_zero] ** Qed
Ordinal.mod_eq_of_lt ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} h : a < b ⊢ a % b = a ** simp only [mod_def, div_eq_zero_of_lt h, mul_zero, sub_zero] ** Qed
Ordinal.zero_mod ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop b : Ordinal.{u_4} ⊢ 0 % b = 0 ** simp only [mod_def, zero_div, mul_zero, sub_self] ** Qed
Ordinal.mod_lt ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} h : b ≠ 0 ⊢ b * (a / b) + a % b < b * (a / b) + b ** rw [div_add_mod] ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} h : b ≠ 0 ⊢ a < b * (a / b) + b ** exact lt_mul_div_add a h ** Qed
Ordinal.mod_self ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a : Ordinal.{u_4} a0 : a = 0 ⊢ a % a = 0 ** simp only [a0, zero_mod] ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a : Ordinal.{u_4} a0 : ¬a = 0 ⊢ a % a = 0 ** simp only [mod_def, div_self a0, mul_one, sub_self] ** Qed
Ordinal.mod_one ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a : Ordinal.{u_4} ⊢ a % 1 = 0 ** simp only [mod_def, div_one, one_mul, sub_self] ** Qed
Ordinal.dvd_of_mod_eq_zero ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} H : a % b = 0 ⊢ a = b * (a / b) ** simpa [H] using (div_add_mod a b).symm ** Qed
Ordinal.mod_eq_zero_of_dvd ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} H : b ∣ a ⊢ a % b = 0 ** rcases H with ⟨c, rfl⟩ ** case intro α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop b c : Ordinal.{u_4} ⊢ b * c % b = 0 ** rcases eq_or_ne b 0 with (rfl | hb) ** case intro.inl α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop c : Ordinal.{u_4} ⊢ 0 * c % 0 = 0 ** simp ** case intro.inr α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop b c : Ordinal.{u_4} hb : b ≠ 0 ⊢ b * c % b = 0 ** simp [mod_def, hb] ** Qed
Ordinal.mul_add_mod_self ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop x y z : Ordinal.{u_4} ⊢ (x * y + z) % x = z % x ** rcases eq_or_ne x 0 with rfl | hx ** case inl α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop y z : Ordinal.{u_4} ⊢ (0 * y + z) % 0 = z % 0 ** simp ** case inr α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop x y z : Ordinal.{u_4} hx : x ≠ 0 ⊢ (x * y + z) % x = z % x ** rwa [mod_def, mul_add_div, mul_add, ← sub_sub, add_sub_cancel, mod_def] ** Qed
Ordinal.mul_mod ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop x y : Ordinal.{u_4} ⊢ x * y % x = 0 ** simpa using mul_add_mod_self x y 0 ** Qed
Ordinal.mod_mod_of_dvd ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b c : Ordinal.{u_4} h : c ∣ b ⊢ a % b % c = a % c ** nth_rw 2 [← div_add_mod a b] ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b c : Ordinal.{u_4} h : c ∣ b ⊢ a % b % c = (b * (a / b) + a % b) % c ** rcases h with ⟨d, rfl⟩ ** case intro α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a c d : Ordinal.{u_4} ⊢ a % (c * d) % c = (c * d * (a / (c * d)) + a % (c * d)) % c ** rw [mul_assoc, mul_add_mod_self] ** Qed
Ordinal.bfamilyOfFamily'_typein ** α : Type u_1 β : Type u_2 γ : Type u_3 r✝ : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u_4 r : ι → ι → Prop inst✝ : IsWellOrder ι r f : ι → α i : ι ⊢ bfamilyOfFamily' r f (typein r i) (_ : typein r i < type r) = f i ** simp only [bfamilyOfFamily', enum_typein] ** Qed
Ordinal.familyOfBFamily'_enum ** α : Type u_1 β : Type u_2 γ : Type u_3 r✝ : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u r : ι → ι → Prop inst✝ : IsWellOrder ι r o : Ordinal.{u} ho : type r = o f : (a : Ordinal.{u}) → a < o → α i : Ordinal.{u} hi : i < o ⊢ i < type r ** rwa [ho] ** α : Type u_1 β : Type u_2 γ : Type u_3 r✝ : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u r : ι → ι → Prop inst✝ : IsWellOrder ι r o : Ordinal.{u} ho : type r = o f : (a : Ordinal.{u}) → a < o → α i : Ordinal.{u} hi : i < o ⊢ familyOfBFamily' r ho f (enum r i (_ : i < type r)) = f i hi ** simp only [familyOfBFamily', typein_enum] ** Qed
Ordinal.familyOfBFamily_enum ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{?u.273825} f : (a : Ordinal.{?u.273825}) → a < o → α i : Ordinal.{?u.273825} hi : i < o ⊢ i < type fun x x_1 => x < x_1 ** convert hi ** case h.e'_4 α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{?u.273825} f : (a : Ordinal.{?u.273825}) → a < o → α i : Ordinal.{?u.273825} hi : i < o ⊢ (type fun x x_1 => x < x_1) = o ** exact type_lt _ ** Qed
Ordinal.range_familyOfBFamily' ** α : Type u_1 β : Type u_2 γ : Type u_3 r✝ : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u r : ι → ι → Prop inst✝ : IsWellOrder ι r o : Ordinal.{u} ho : type r = o f : (a : Ordinal.{u}) → a < o → α ⊢ range (familyOfBFamily' r ho f) = brange o f ** refine' Set.ext fun a => ⟨_, _⟩ ** case refine'_1 α : Type u_1 β : Type u_2 γ : Type u_3 r✝ : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u r : ι → ι → Prop inst✝ : IsWellOrder ι r o : Ordinal.{u} ho : type r = o f : (a : Ordinal.{u}) → a < o → α a : α ⊢ a ∈ range (familyOfBFamily' r ho f) → a ∈ brange o f ** rintro ⟨b, rfl⟩ ** case refine'_1.intro α : Type u_1 β : Type u_2 γ : Type u_3 r✝ : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u r : ι → ι → Prop inst✝ : IsWellOrder ι r o : Ordinal.{u} ho : type r = o f : (a : Ordinal.{u}) → a < o → α b : ι ⊢ familyOfBFamily' r ho f b ∈ brange o f ** apply mem_brange_self ** case refine'_2 α : Type u_1 β : Type u_2 γ : Type u_3 r✝ : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u r : ι → ι → Prop inst✝ : IsWellOrder ι r o : Ordinal.{u} ho : type r = o f : (a : Ordinal.{u}) → a < o → α a : α ⊢ a ∈ brange o f → a ∈ range (familyOfBFamily' r ho f) ** rintro ⟨i, hi, rfl⟩ ** case refine'_2.intro.intro α : Type u_1 β : Type u_2 γ : Type u_3 r✝ : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u r : ι → ι → Prop inst✝ : IsWellOrder ι r o : Ordinal.{u} ho : type r = o f : (a : Ordinal.{u}) → a < o → α i : Ordinal.{u} hi : i < o ⊢ f i hi ∈ range (familyOfBFamily' r ho f) ** exact ⟨_, familyOfBFamily'_enum _ _ _ _ _⟩ ** Qed
Ordinal.brange_bfamilyOfFamily' ** α : Type u_1 β : Type u_2 γ : Type u_3 r✝ : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u r : ι → ι → Prop inst✝ : IsWellOrder ι r f : ι → α ⊢ brange (type r) (bfamilyOfFamily' r f) = range f ** refine' Set.ext fun a => ⟨_, _⟩ ** case refine'_1 α : Type u_1 β : Type u_2 γ : Type u_3 r✝ : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u r : ι → ι → Prop inst✝ : IsWellOrder ι r f : ι → α a : α ⊢ a ∈ brange (type r) (bfamilyOfFamily' r f) → a ∈ range f ** rintro ⟨i, hi, rfl⟩ ** case refine'_1.intro.intro α : Type u_1 β : Type u_2 γ : Type u_3 r✝ : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u r : ι → ι → Prop inst✝ : IsWellOrder ι r f : ι → α i : Ordinal.{u} hi : i < type r ⊢ bfamilyOfFamily' r f i hi ∈ range f ** apply mem_range_self ** case refine'_2 α : Type u_1 β : Type u_2 γ : Type u_3 r✝ : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u r : ι → ι → Prop inst✝ : IsWellOrder ι r f : ι → α a : α ⊢ a ∈ range f → a ∈ brange (type r) (bfamilyOfFamily' r f) ** rintro ⟨b, rfl⟩ ** case refine'_2.intro α : Type u_1 β : Type u_2 γ : Type u_3 r✝ : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u r : ι → ι → Prop inst✝ : IsWellOrder ι r f : ι → α b : ι ⊢ f b ∈ brange (type r) (bfamilyOfFamily' r f) ** exact ⟨_, _, bfamilyOfFamily'_typein _ _ _⟩ ** Qed
Ordinal.brange_const ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u_4} ho : o ≠ 0 c : α ⊢ (brange o fun x x => c) = {c} ** rw [← range_familyOfBFamily] ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u_4} ho : o ≠ 0 c : α ⊢ range (familyOfBFamily o fun x x => c) = {c} ** exact @Set.range_const _ o.out.α (out_nonempty_iff_ne_zero.2 ho) c ** Qed
Ordinal.bddAbove_range ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u f : ι → Ordinal.{max u v} ⊢ ord (iSup (succ ∘ card ∘ f)) ∈ upperBounds (range f) ** rintro a ⟨i, rfl⟩ ** case intro α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u f : ι → Ordinal.{max u v} i : ι ⊢ f i ≤ ord (iSup (succ ∘ card ∘ f)) ** exact le_of_lt (Cardinal.lt_ord.2 ((lt_succ _).trans_le (le_ciSup (Cardinal.bddAbove_range.{_, v} _) _))) ** Qed
Ordinal.sup_le_iff ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u f : ι → Ordinal.{max u v} a : Ordinal.{max u v} ⊢ (∀ (x : Ordinal.{max u v}), x ∈ range f → x ≤ a) ↔ ∀ (i : ι), f i ≤ a ** simp ** Qed
Ordinal.lt_sup ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u f : ι → Ordinal.{max u v} a : Ordinal.{max u v} ⊢ a < sup f ↔ ∃ i, a < f i ** simpa only [not_forall, not_le] using not_congr (@sup_le_iff.{_, v} _ f a) ** Qed
Ordinal.sup_not_succ_of_ne_sup ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u f : ι → Ordinal.{max u v} hf : ∀ (i : ι), f i ≠ sup f a : Ordinal.{max u v} hao : a < sup f ⊢ succ a < sup f ** by_contra' hoa ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u f : ι → Ordinal.{max u v} hf : ∀ (i : ι), f i ≠ sup f a : Ordinal.{max u v} hao : a < sup f hoa : sup f ≤ succ a ⊢ False ** exact hao.not_le (sup_le fun i => le_of_lt_succ <| (lt_of_le_of_ne (le_sup _ _) (hf i)).trans_le hoa) ** Qed
Ordinal.sup_eq_zero_iff ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u f : ι → Ordinal.{max u v} ⊢ sup f = 0 ↔ ∀ (i : ι), f i = 0 ** refine' ⟨fun h i => _, fun h => le_antisymm (sup_le fun i => Ordinal.le_zero.2 (h i)) (Ordinal.zero_le _)⟩ ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u f : ι → Ordinal.{max u v} h : sup f = 0 i : ι ⊢ f i = 0 ** rw [← Ordinal.le_zero, ← h] ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u f : ι → Ordinal.{max u v} h : sup f = 0 i : ι ⊢ f i ≤ sup f ** exact le_sup f i ** Qed
Ordinal.IsNormal.sup ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop f : Ordinal.{max u v} → Ordinal.{max u w} H : IsNormal f ι : Type u g : ι → Ordinal.{max u v} inst✝ : Nonempty ι a : Ordinal.{max u w} ⊢ f (Ordinal.sup g) ≤ a ↔ Ordinal.sup (f ∘ g) ≤ a ** rw [sup_le_iff] ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop f : Ordinal.{max u v} → Ordinal.{max u w} H : IsNormal f ι : Type u g : ι → Ordinal.{max u v} inst✝ : Nonempty ι a : Ordinal.{max u w} ⊢ f (Ordinal.sup g) ≤ a ↔ ∀ (i : ι), (f ∘ g) i ≤ a ** simp only [comp] ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop f : Ordinal.{max u v} → Ordinal.{max u w} H : IsNormal f ι : Type u g : ι → Ordinal.{max u v} inst✝ : Nonempty ι a : Ordinal.{max u w} ⊢ f (Ordinal.sup g) ≤ a ↔ ∀ (i : ι), f (g i) ≤ a ** rw [H.le_set' Set.univ Set.univ_nonempty g] <;> simp [sup_le_iff] ** Qed
Ordinal.sup_sum ** α✝ : Type u_1 β✝ : Type u_2 γ : Type u_3 r : α✝ → α✝ → Prop s : β✝ → β✝ → Prop t : γ → γ → Prop α : Type u β : Type v f : α ⊕ β → Ordinal.{max (max u v) w} ⊢ sup f = max (sup fun a => f (Sum.inl a)) (sup fun b => f (Sum.inr b)) ** apply (sup_le_iff.2 _).antisymm (max_le_iff.2 ⟨_, _⟩) ** α✝ : Type u_1 β✝ : Type u_2 γ : Type u_3 r : α✝ → α✝ → Prop s : β✝ → β✝ → Prop t : γ → γ → Prop α : Type u β : Type v f : α ⊕ β → Ordinal.{max (max u v) w} ⊢ (sup fun a => f (Sum.inl a)) ≤ sup f α✝ : Type u_1 β✝ : Type u_2 γ : Type u_3 r : α✝ → α✝ → Prop s : β✝ → β✝ → Prop t : γ → γ → Prop α : Type u β : Type v f : α ⊕ β → Ordinal.{max (max u v) w} ⊢ (sup fun b => f (Sum.inr b)) ≤ sup f ** all_goals apply sup_le_of_range_subset.{_, max u v, w} rintro i ⟨a, rfl⟩ apply mem_range_self ** α✝ : Type u_1 β✝ : Type u_2 γ : Type u_3 r : α✝ → α✝ → Prop s : β✝ → β✝ → Prop t : γ → γ → Prop α : Type u β : Type v f : α ⊕ β → Ordinal.{max (max u v) w} ⊢ ∀ (i : α ⊕ β), f i ≤ max (sup fun a => f (Sum.inl a)) (sup fun b => f (Sum.inr b)) ** rintro (i | i) ** case inl α✝ : Type u_1 β✝ : Type u_2 γ : Type u_3 r : α✝ → α✝ → Prop s : β✝ → β✝ → Prop t : γ → γ → Prop α : Type u β : Type v f : α ⊕ β → Ordinal.{max (max u v) w} i : α ⊢ f (Sum.inl i) ≤ max (sup fun a => f (Sum.inl a)) (sup fun b => f (Sum.inr b)) ** exact le_max_of_le_left (le_sup _ i) ** case inr α✝ : Type u_1 β✝ : Type u_2 γ : Type u_3 r : α✝ → α✝ → Prop s : β✝ → β✝ → Prop t : γ → γ → Prop α : Type u β : Type v f : α ⊕ β → Ordinal.{max (max u v) w} i : β ⊢ f (Sum.inr i) ≤ max (sup fun a => f (Sum.inl a)) (sup fun b => f (Sum.inr b)) ** exact le_max_of_le_right (le_sup _ i) ** α✝ : Type u_1 β✝ : Type u_2 γ : Type u_3 r : α✝ → α✝ → Prop s : β✝ → β✝ → Prop t : γ → γ → Prop α : Type u β : Type v f : α ⊕ β → Ordinal.{max (max u v) w} ⊢ (sup fun b => f (Sum.inr b)) ≤ sup f ** apply sup_le_of_range_subset.{_, max u v, w} ** α✝ : Type u_1 β✝ : Type u_2 γ : Type u_3 r : α✝ → α✝ → Prop s : β✝ → β✝ → Prop t : γ → γ → Prop α : Type u β : Type v f : α ⊕ β → Ordinal.{max (max u v) w} ⊢ (range fun b => f (Sum.inr b)) ⊆ range f ** rintro i ⟨a, rfl⟩ ** case intro α✝ : Type u_1 β✝ : Type u_2 γ : Type u_3 r : α✝ → α✝ → Prop s : β✝ → β✝ → Prop t : γ → γ → Prop α : Type u β : Type v f : α ⊕ β → Ordinal.{max (max u v) w} a : β ⊢ (fun b => f (Sum.inr b)) a ∈ range f ** apply mem_range_self ** Qed
Ordinal.le_sup_shrink_equiv ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s✝ : β → β → Prop t : γ → γ → Prop s : Set Ordinal.{u} hs : Small.{u, u + 1} ↑s a : Ordinal.{u} ha : a ∈ s ⊢ a ≤ sup fun x => ↑(↑(equivShrink ↑s).symm x) ** convert le_sup.{u, u} (fun x => ((@equivShrink s hs).symm x).val) ((@equivShrink s hs) ⟨a, ha⟩) ** case h.e'_3 α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s✝ : β → β → Prop t : γ → γ → Prop s : Set Ordinal.{u} hs : Small.{u, u + 1} ↑s a : Ordinal.{u} ha : a ∈ s ⊢ a = ↑(↑(equivShrink ↑s).symm (↑(equivShrink ↑s) { val := a, property := ha })) ** rw [symm_apply_apply] ** Qed
Ordinal.sSup_ord ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s✝ : β → β → Prop t : γ → γ → Prop s : Set Cardinal.{u} hs : BddAbove s a : Ordinal.{u} ⊢ ord (sSup s) ≤ a ↔ sSup (ord '' s) ≤ a ** rw [csSup_le_iff' (bddAbove_iff_small.2 (@small_image _ _ _ s (Cardinal.bddAbove_iff_small.1 hs))), ord_le, csSup_le_iff' hs] ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s✝ : β → β → Prop t : γ → γ → Prop s : Set Cardinal.{u} hs : BddAbove s a : Ordinal.{u} ⊢ (∀ (x : Cardinal.{u}), x ∈ s → x ≤ card a) ↔ ∀ (x : Ordinal.{u}), x ∈ ord '' s → x ≤ a ** simp [ord_le] ** Qed
Ordinal.iSup_ord ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Sort u_4 f : ι → Cardinal.{u_5} hf : BddAbove (range f) ⊢ ord (iSup f) = ⨆ i, ord (f i) ** unfold iSup ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Sort u_4 f : ι → Cardinal.{u_5} hf : BddAbove (range f) ⊢ ord (sSup (range f)) = sSup (range fun i => ord (f i)) ** convert sSup_ord hf ** case h.e'_3.h.e'_3 α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Sort u_4 f : ι → Cardinal.{u_5} hf : BddAbove (range f) ⊢ (range fun i => ord (f i)) = ord '' range f ** conv_lhs => change range (ord ∘ f) ** case h.e'_3.h.e'_3 α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Sort u_4 f : ι → Cardinal.{u_5} hf : BddAbove (range f) ⊢ range (ord ∘ f) = ord '' range f ** rw [range_comp] ** Qed
Ordinal.sup_le_sup ** α : Type u_1 β : Type u_2 γ : Type u_3 r✝ : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι ι' : Type u r : ι → ι → Prop r' : ι' → ι' → Prop inst✝¹ : IsWellOrder ι r inst✝ : IsWellOrder ι' r' o : Ordinal.{u} ho : type r = o ho' : type r' = o f : (a : Ordinal.{u}) → a < o → Ordinal.{max u v} i : ι ⊢ familyOfBFamily' r ho f i ≤ sup (familyOfBFamily' r' ho' f) ** cases' typein_surj r' (by rw [ho', ← ho] exact typein_lt_type r i) with j hj ** case intro α : Type u_1 β : Type u_2 γ : Type u_3 r✝ : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι ι' : Type u r : ι → ι → Prop r' : ι' → ι' → Prop inst✝¹ : IsWellOrder ι r inst✝ : IsWellOrder ι' r' o : Ordinal.{u} ho : type r = o ho' : type r' = o f : (a : Ordinal.{u}) → a < o → Ordinal.{max u v} i : ι j : ι' hj : typein r' j = typein r i ⊢ familyOfBFamily' r ho f i ≤ sup (familyOfBFamily' r' ho' f) ** simp_rw [familyOfBFamily', ← hj] ** case intro α : Type u_1 β : Type u_2 γ : Type u_3 r✝ : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι ι' : Type u r : ι → ι → Prop r' : ι' → ι' → Prop inst✝¹ : IsWellOrder ι r inst✝ : IsWellOrder ι' r' o : Ordinal.{u} ho : type r = o ho' : type r' = o f : (a : Ordinal.{u}) → a < o → Ordinal.{max u v} i : ι j : ι' hj : typein r' j = typein r i ⊢ f (typein r' j) (_ : typein r' j < o) ≤ sup fun i => f (typein r' i) (_ : typein r' i < o) ** apply le_sup ** α : Type u_1 β : Type u_2 γ : Type u_3 r✝ : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι ι' : Type u r : ι → ι → Prop r' : ι' → ι' → Prop inst✝¹ : IsWellOrder ι r inst✝ : IsWellOrder ι' r' o : Ordinal.{u} ho : type r = o ho' : type r' = o f : (a : Ordinal.{u}) → a < o → Ordinal.{max u v} i : ι ⊢ ?m.306421 < type r' ** rw [ho', ← ho] ** α : Type u_1 β : Type u_2 γ : Type u_3 r✝ : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι ι' : Type u r : ι → ι → Prop r' : ι' → ι' → Prop inst✝¹ : IsWellOrder ι r inst✝ : IsWellOrder ι' r' o : Ordinal.{u} ho : type r = o ho' : type r' = o f : (a : Ordinal.{u}) → a < o → Ordinal.{max u v} i : ι ⊢ ?m.306421 < type r α : Type u_1 β : Type u_2 γ : Type u_3 r✝ : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι ι' : Type u r : ι → ι → Prop r' : ι' → ι' → Prop inst✝¹ : IsWellOrder ι r inst✝ : IsWellOrder ι' r' o : Ordinal.{u} ho : type r = o ho' : type r' = o f : (a : Ordinal.{u}) → a < o → Ordinal.{max u v} i : ι ⊢ Ordinal.{u} α : Type u_1 β : Type u_2 γ : Type u_3 r✝ : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι ι' : Type u r : ι → ι → Prop r' : ι' → ι' → Prop inst✝¹ : IsWellOrder ι r inst✝ : IsWellOrder ι' r' o : Ordinal.{u} ho : type r = o ho' : type r' = o f : (a : Ordinal.{u}) → a < o → Ordinal.{max u v} i : ι ⊢ Ordinal.{u} ** exact typein_lt_type r i ** Qed
Ordinal.sup_eq_sup ** α : Type u_1 β : Type u_2 γ : Type u_3 r✝ : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι ι' : Type u r : ι → ι → Prop r' : ι' → ι' → Prop inst✝¹ : IsWellOrder ι r inst✝ : IsWellOrder ι' r' o : Ordinal.{u} ho : type r = o ho' : type r' = o f : (a : Ordinal.{u}) → a < o → Ordinal.{max u v} ⊢ range (familyOfBFamily' r ho f) = range (familyOfBFamily' r' ho' f) ** simp ** Qed
Ordinal.sSup_eq_bsup ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u} f : (a : Ordinal.{u}) → a < o → Ordinal.{max u v} ⊢ sSup (brange o f) = bsup o f ** congr ** case e_a α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u} f : (a : Ordinal.{u}) → a < o → Ordinal.{max u v} ⊢ brange o f = range (familyOfBFamily o f) ** rw [range_familyOfBFamily] ** Qed
Ordinal.bsup_eq_sup' ** α : Type u_1 β : Type u_2 γ : Type u_3 r✝ : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u r : ι → ι → Prop inst✝ : IsWellOrder ι r f : ι → Ordinal.{max u v} ⊢ bsup (type r) (bfamilyOfFamily' r f) = sup f ** simp only [← sup_eq_bsup' r, enum_typein, familyOfBFamily', bfamilyOfFamily'] ** Qed
Ordinal.bsup_eq_bsup ** α : Type u_1 β : Type u_2 γ : Type u_3 r✝ : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u r r' : ι → ι → Prop inst✝¹ : IsWellOrder ι r inst✝ : IsWellOrder ι r' f : ι → Ordinal.{max u v} ⊢ bsup (type r) (bfamilyOfFamily' r f) = bsup (type r') (bfamilyOfFamily' r' f) ** rw [bsup_eq_sup', bsup_eq_sup'] ** Qed
Ordinal.bsup_congr ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o₁ o₂ : Ordinal.{u} f : (a : Ordinal.{u}) → a < o₁ → Ordinal.{max u v} ho : o₁ = o₂ ⊢ bsup o₁ f = bsup o₂ fun a h => f a (_ : a < o₁) ** subst ho ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o₁ : Ordinal.{u} f : (a : Ordinal.{u}) → a < o₁ → Ordinal.{max u v} ⊢ bsup o₁ f = bsup o₁ fun a h => f a (_ : a < o₁) ** rfl ** Qed
Ordinal.bsup_le_iff ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u} f : (a : Ordinal.{u}) → a < o → Ordinal.{max u v} a : Ordinal.{max u v} h : ∀ (i : (Quotient.out o).α), familyOfBFamily o f i ≤ a i : Ordinal.{u} hi : i < o ⊢ f i hi ≤ a ** rw [← familyOfBFamily_enum o f] ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u} f : (a : Ordinal.{u}) → a < o → Ordinal.{max u v} a : Ordinal.{max u v} h : ∀ (i : (Quotient.out o).α), familyOfBFamily o f i ≤ a i : Ordinal.{u} hi : i < o ⊢ familyOfBFamily o f (enum (fun x x_1 => x < x_1) i (_ : i < type fun x x_1 => x < x_1)) ≤ a ** exact h _ ** Qed
Ordinal.lt_bsup ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u} f : (a : Ordinal.{u}) → a < o → Ordinal.{max u v} a : Ordinal.{max u v} ⊢ a < bsup o f ↔ ∃ i hi, a < f i hi ** simpa only [not_forall, not_le] using not_congr (@bsup_le_iff.{_, v} _ f a) ** Qed
Ordinal.IsNormal.bsup ** α✝ : Type u_1 β : Type u_2 γ : Type u_3 r✝ : α✝ → α✝ → Prop s : β → β → Prop t : γ → γ → Prop f : Ordinal.{max u v} → Ordinal.{max u w} H : IsNormal f o : Ordinal.{u} α : Type u r : α → α → Prop x✝ : IsWellOrder α r g : (a : Ordinal.{u}) → a < type r → Ordinal.{max u v} h : type r ≠ 0 ⊢ f (Ordinal.bsup (type r) g) = Ordinal.bsup (type r) fun a h => f (g a h) ** haveI := type_ne_zero_iff_nonempty.1 h ** α✝ : Type u_1 β : Type u_2 γ : Type u_3 r✝ : α✝ → α✝ → Prop s : β → β → Prop t : γ → γ → Prop f : Ordinal.{max u v} → Ordinal.{max u w} H : IsNormal f o : Ordinal.{u} α : Type u r : α → α → Prop x✝ : IsWellOrder α r g : (a : Ordinal.{u}) → a < type r → Ordinal.{max u v} h : type r ≠ 0 this : Nonempty α ⊢ f (Ordinal.bsup (type r) g) = Ordinal.bsup (type r) fun a h => f (g a h) ** rw [← sup_eq_bsup' r, IsNormal.sup.{_, v, w} H, ← sup_eq_bsup' r] <;> rfl ** Qed
Ordinal.bsup_not_succ_of_ne_bsup ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u} f : (a : Ordinal.{u}) → a < o → Ordinal.{max u v} hf : ∀ {i : Ordinal.{u}} (h : i < o), f i h ≠ bsup o f a : Ordinal.{max u v} ⊢ a < bsup o f → succ a < bsup o f ** rw [← sup_eq_bsup] at * ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u} f : (a : Ordinal.{u}) → a < o → Ordinal.{max u v} hf : ∀ {i : Ordinal.{u}} (h : i < o), f i h ≠ sup (familyOfBFamily o f) a : Ordinal.{max u v} ⊢ a < sup (familyOfBFamily o f) → succ a < sup (familyOfBFamily o f) ** exact sup_not_succ_of_ne_sup fun i => hf _ ** Qed
Ordinal.bsup_eq_zero_iff ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u_4} f : (a : Ordinal.{u_4}) → a < o → Ordinal.{max u_5 u_4} ⊢ bsup o f = 0 ↔ ∀ (i : Ordinal.{u_4}) (hi : i < o), f i hi = 0 ** refine' ⟨fun h i hi => _, fun h => le_antisymm (bsup_le fun i hi => Ordinal.le_zero.2 (h i hi)) (Ordinal.zero_le _)⟩ ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u_4} f : (a : Ordinal.{u_4}) → a < o → Ordinal.{max u_5 u_4} h : bsup o f = 0 i : Ordinal.{u_4} hi : i < o ⊢ f i hi = 0 ** rw [← Ordinal.le_zero, ← h] ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u_4} f : (a : Ordinal.{u_4}) → a < o → Ordinal.{max u_5 u_4} h : bsup o f = 0 i : Ordinal.{u_4} hi : i < o ⊢ f i hi ≤ bsup o f ** exact le_bsup f i hi ** Qed
Ordinal.bsup_one ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop f : (a : Ordinal.{u_4}) → a < 1 → Ordinal.{max u_4 u_5} ⊢ bsup 1 f = f 0 (_ : 0 < 1) ** simp_rw [← sup_eq_bsup, sup_unique, familyOfBFamily, familyOfBFamily', typein_one_out] ** Qed
Ordinal.bsup_le_of_brange_subset ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u} o' : Ordinal.{v} f : (a : Ordinal.{u}) → a < o → Ordinal.{max (max u v) w} g : (a : Ordinal.{v}) → a < o' → Ordinal.{max (max u v) w} h : brange o f ⊆ brange o' g i : Ordinal.{u} hi : i < o ⊢ f i hi ≤ bsup o' g ** obtain ⟨j, hj, hj'⟩ := h ⟨i, hi, rfl⟩ ** case intro.intro α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u} o' : Ordinal.{v} f : (a : Ordinal.{u}) → a < o → Ordinal.{max (max u v) w} g : (a : Ordinal.{v}) → a < o' → Ordinal.{max (max u v) w} h : brange o f ⊆ brange o' g i : Ordinal.{u} hi : i < o j : Ordinal.{v} hj : j < o' hj' : g j hj = f i hi ⊢ f i hi ≤ bsup o' g ** rw [← hj'] ** case intro.intro α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u} o' : Ordinal.{v} f : (a : Ordinal.{u}) → a < o → Ordinal.{max (max u v) w} g : (a : Ordinal.{v}) → a < o' → Ordinal.{max (max u v) w} h : brange o f ⊆ brange o' g i : Ordinal.{u} hi : i < o j : Ordinal.{v} hj : j < o' hj' : g j hj = f i hi ⊢ g j hj ≤ bsup o' g ** apply le_bsup ** Qed
Ordinal.lsub_le_iff ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u f : ι → Ordinal.{max u v} a : Ordinal.{max v u} ⊢ lsub f ≤ a ↔ ∀ (i : ι), f i < a ** convert sup_le_iff.{_, v} (f := succ ∘ f) (a := a) using 2 ** case h.e'_2.h.a α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u f : ι → Ordinal.{max u v} a : Ordinal.{max v u} a✝ : ι ⊢ f a✝ < a ↔ (succ ∘ f) a✝ ≤ a ** simp only [comp_apply, succ_le_iff] ** Qed
Ordinal.lt_lsub_iff ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u f : ι → Ordinal.{max u v} a : Ordinal.{max v u} ⊢ a < lsub f ↔ ∃ i, a ≤ f i ** simpa only [not_forall, not_lt, not_le] using not_congr (@lsub_le_iff.{_, v} _ f a) ** Qed
Ordinal.sup_eq_lsub_or_sup_succ_eq_lsub ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u f : ι → Ordinal.{max u v} ⊢ sup f = lsub f ∨ succ (sup f) = lsub f ** cases' eq_or_lt_of_le (sup_le_lsub.{_, v} f) with h h ** case inl α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u f : ι → Ordinal.{max u v} h : sup f = lsub f ⊢ sup f = lsub f ∨ succ (sup f) = lsub f ** exact Or.inl h ** case inr α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u f : ι → Ordinal.{max u v} h : sup f < lsub f ⊢ sup f = lsub f ∨ succ (sup f) = lsub f ** exact Or.inr ((succ_le_of_lt h).antisymm (lsub_le_sup_succ f)) ** Qed
Ordinal.sup_succ_le_lsub ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u f : ι → Ordinal.{max u v} ⊢ succ (sup f) ≤ lsub f ↔ ∃ i, f i = sup f ** refine' ⟨fun h => _, _⟩ ** case refine'_2 α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u f : ι → Ordinal.{max u v} ⊢ (∃ i, f i = sup f) → succ (sup f) ≤ lsub f ** rintro ⟨_, hf⟩ ** case refine'_2.intro α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u f : ι → Ordinal.{max u v} w✝ : ι hf : f w✝ = sup f ⊢ succ (sup f) ≤ lsub f ** rw [succ_le_iff, ← hf] ** case refine'_2.intro α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u f : ι → Ordinal.{max u v} w✝ : ι hf : f w✝ = sup f ⊢ f w✝ < lsub f ** exact lt_lsub _ _ ** case refine'_1 α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u f : ι → Ordinal.{max u v} h : succ (sup f) ≤ lsub f ⊢ ∃ i, f i = sup f ** by_contra' hf ** case refine'_1 α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u f : ι → Ordinal.{max u v} h : succ (sup f) ≤ lsub f hf : ∀ (i : ι), f i ≠ sup f ⊢ False ** exact (succ_le_iff.1 h).ne ((sup_le_lsub f).antisymm (lsub_le (ne_sup_iff_lt_sup.1 hf))) ** Qed
Ordinal.sup_eq_lsub_iff_succ ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u f : ι → Ordinal.{max u v} ⊢ sup f = lsub f ↔ ∀ (a : Ordinal.{max v u}), a < lsub f → succ a < lsub f ** refine' ⟨fun h => _, fun hf => le_antisymm (sup_le_lsub f) (lsub_le fun i => _)⟩ ** case refine'_2 α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u f : ι → Ordinal.{max u v} hf : ∀ (a : Ordinal.{max v u}), a < lsub f → succ a < lsub f i : ι ⊢ f i < sup f ** by_contra' hle ** case refine'_2 α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u f : ι → Ordinal.{max u v} hf : ∀ (a : Ordinal.{max v u}), a < lsub f → succ a < lsub f i : ι hle : sup f ≤ f i ⊢ False ** have heq := (sup_succ_eq_lsub f).2 ⟨i, le_antisymm (le_sup _ _) hle⟩ ** case refine'_2 α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u f : ι → Ordinal.{max u v} hf : ∀ (a : Ordinal.{max v u}), a < lsub f → succ a < lsub f i : ι hle : sup f ≤ f i heq : succ (sup f) = lsub f ⊢ False ** have := hf _ (by rw [← heq] exact lt_succ (sup f)) ** case refine'_2 α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u f : ι → Ordinal.{max u v} hf : ∀ (a : Ordinal.{max v u}), a < lsub f → succ a < lsub f i : ι hle : sup f ≤ f i heq : succ (sup f) = lsub f this : succ (sup f) < lsub f ⊢ False ** rw [heq] at this ** case refine'_2 α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u f : ι → Ordinal.{max u v} hf : ∀ (a : Ordinal.{max v u}), a < lsub f → succ a < lsub f i : ι hle : sup f ≤ f i heq : succ (sup f) = lsub f this : lsub f < lsub f ⊢ False ** exact this.false ** case refine'_1 α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u f : ι → Ordinal.{max u v} h : sup f = lsub f ⊢ ∀ (a : Ordinal.{max v u}), a < lsub f → succ a < lsub f ** rw [← h] ** case refine'_1 α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u f : ι → Ordinal.{max u v} h : sup f = lsub f ⊢ ∀ (a : Ordinal.{max v u}), a < sup f → succ a < sup f ** exact fun a => sup_not_succ_of_ne_sup fun i => (lsub_le_iff.1 (le_of_eq h.symm) i).ne ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u f : ι → Ordinal.{max u v} hf : ∀ (a : Ordinal.{max v u}), a < lsub f → succ a < lsub f i : ι hle : sup f ≤ f i heq : succ (sup f) = lsub f ⊢ ?m.326003 < lsub f ** rw [← heq] ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u f : ι → Ordinal.{max u v} hf : ∀ (a : Ordinal.{max v u}), a < lsub f → succ a < lsub f i : ι hle : sup f ≤ f i heq : succ (sup f) = lsub f ⊢ ?m.326003 < succ (sup f) α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u f : ι → Ordinal.{max u v} hf : ∀ (a : Ordinal.{max v u}), a < lsub f → succ a < lsub f i : ι hle : sup f ≤ f i heq : succ (sup f) = lsub f ⊢ Ordinal.{max v u} ** exact lt_succ (sup f) ** Qed
Ordinal.sup_eq_lsub_iff_lt_sup ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u f : ι → Ordinal.{max u v} h : sup f = lsub f i : ι ⊢ f i < sup f ** rw [h] ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u f : ι → Ordinal.{max u v} h : sup f = lsub f i : ι ⊢ f i < lsub f ** apply lt_lsub ** Qed
Ordinal.lsub_empty ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u_4 h : IsEmpty ι f : ι → Ordinal.{max u_5 u_4} ⊢ lsub f = 0 ** rw [← Ordinal.le_zero, lsub_le_iff] ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u_4 h : IsEmpty ι f : ι → Ordinal.{max u_5 u_4} ⊢ ∀ (i : ι), f i < 0 ** exact h.elim ** Qed
Ordinal.lsub_eq_zero_iff ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u f : ι → Ordinal.{max u v} ⊢ lsub f = 0 ↔ IsEmpty ι ** refine' ⟨fun h => ⟨fun i => _⟩, fun h => @lsub_empty _ h _⟩ ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u f : ι → Ordinal.{max u v} h : lsub f = 0 i : ι ⊢ False ** have := @lsub_pos.{_, v} _ ⟨i⟩ f ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u f : ι → Ordinal.{max u v} h : lsub f = 0 i : ι this : 0 < lsub f ⊢ False ** rw [h] at this ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u f : ι → Ordinal.{max u v} h : lsub f = 0 i : ι this : 0 < 0 ⊢ False ** exact this.false ** Qed
Ordinal.lsub_le_of_range_subset ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u ι' : Type v f : ι → Ordinal.{max (max u v) w} g : ι' → Ordinal.{max (max u v) w} h : range f ⊆ range g ⊢ range (succ ∘ f) ⊆ range (succ ∘ g) ** convert Set.image_subset succ h <;> apply Set.range_comp ** Qed
Ordinal.lsub_typein ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u} ⊢ o ≤ lsub fun i => typein (fun x x_1 => x < x_1) i ** by_contra' h ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u} h : (lsub fun i => typein (fun x x_1 => x < x_1) i) < o ⊢ False ** conv_rhs at h => rw [← type_lt o] ** Qed
Ordinal.sup_typein_limit ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u} ho : ∀ (a : Ordinal.{u}), a < o → succ a < o ⊢ ∀ (a : Ordinal.{u}), a < o → succ a < o ** assumption ** Qed
Ordinal.sup_typein_succ ** case inr α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u} h : succ (sup (typein fun x x_1 => x < x_1)) = lsub (typein fun x x_1 => x < x_1) ⊢ sup (typein fun x x_1 => x < x_1) = o ** rw [← succ_eq_succ_iff, h] ** case inr α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u} h : succ (sup (typein fun x x_1 => x < x_1)) = lsub (typein fun x x_1 => x < x_1) ⊢ lsub (typein fun x x_1 => x < x_1) = succ o ** apply lsub_typein ** case inl α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u} h : sup (typein fun x x_1 => x < x_1) = lsub (typein fun x x_1 => x < x_1) ⊢ sup (typein fun x x_1 => x < x_1) = o ** rw [sup_eq_lsub_iff_succ] at h ** case inl α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u} h : ∀ (a : Ordinal.{u}), a < lsub (typein fun x x_1 => x < x_1) → succ a < lsub (typein fun x x_1 => x < x_1) ⊢ sup (typein fun x x_1 => x < x_1) = o ** simp only [lsub_typein] at h ** case inl α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u} h : ∀ (a : Ordinal.{u}), a < succ o → succ a < succ o ⊢ sup (typein fun x x_1 => x < x_1) = o ** exact (h o (lt_succ o)).false.elim ** Qed
Ordinal.lsub_eq_lsub ** α : Type u_1 β : Type u_2 γ : Type u_3 r✝ : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι ι' : Type u r : ι → ι → Prop r' : ι' → ι' → Prop inst✝¹ : IsWellOrder ι r inst✝ : IsWellOrder ι' r' o : Ordinal.{u} ho : type r = o ho' : type r' = o f : (a : Ordinal.{u}) → a < o → Ordinal.{max u v} ⊢ lsub (familyOfBFamily' r ho f) = lsub (familyOfBFamily' r' ho' f) ** rw [lsub_eq_blsub', lsub_eq_blsub'] ** Qed
Ordinal.blsub_eq_blsub ** α : Type u_1 β : Type u_2 γ : Type u_3 r✝ : α → α → Prop s : β → β → Prop t : γ → γ → Prop ι : Type u r r' : ι → ι → Prop inst✝¹ : IsWellOrder ι r inst✝ : IsWellOrder ι r' f : ι → Ordinal.{max u v} ⊢ blsub (type r) (bfamilyOfFamily' r f) = blsub (type r') (bfamilyOfFamily' r' f) ** rw [blsub_eq_lsub', blsub_eq_lsub'] ** Qed
Ordinal.blsub_congr ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o₁ o₂ : Ordinal.{u} f : (a : Ordinal.{u}) → a < o₁ → Ordinal.{max u v} ho : o₁ = o₂ ⊢ blsub o₁ f = blsub o₂ fun a h => f a (_ : a < o₁) ** subst ho ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o₁ : Ordinal.{u} f : (a : Ordinal.{u}) → a < o₁ → Ordinal.{max u v} ⊢ blsub o₁ f = blsub o₁ fun a h => f a (_ : a < o₁) ** rfl ** Qed
Ordinal.blsub_le_iff ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u} f : (a : Ordinal.{u}) → a < o → Ordinal.{max u v} a : Ordinal.{max u v} ⊢ blsub o f ≤ a ↔ ∀ (i : Ordinal.{u}) (h : i < o), f i h < a ** convert bsup_le_iff.{_, v} (f := fun a ha => succ (f a ha)) (a := a) using 2 ** case h.e'_2.h.a α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u} f : (a : Ordinal.{u}) → a < o → Ordinal.{max u v} a : Ordinal.{max u v} a✝ : Ordinal.{u} ⊢ (∀ (h : a✝ < o), f a✝ h < a) ↔ ∀ (h : a✝ < o), succ (f a✝ h) ≤ a ** simp_rw [succ_le_iff] ** Qed
Ordinal.lt_blsub_iff ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u} f : (b : Ordinal.{u}) → b < o → Ordinal.{max u v} a : Ordinal.{max u v} ⊢ a < blsub o f ↔ ∃ i hi, a ≤ f i hi ** simpa only [not_forall, not_lt, not_le] using not_congr (@blsub_le_iff.{_, v} _ f a) ** Qed
Ordinal.bsup_eq_blsub_or_succ_bsup_eq_blsub ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u} f : (a : Ordinal.{u}) → a < o → Ordinal.{max u v} ⊢ bsup o f = blsub o f ∨ succ (bsup o f) = blsub o f ** rw [← sup_eq_bsup, ← lsub_eq_blsub] ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u} f : (a : Ordinal.{u}) → a < o → Ordinal.{max u v} ⊢ sup (familyOfBFamily o f) = lsub (familyOfBFamily o f) ∨ succ (sup (familyOfBFamily o f)) = lsub (familyOfBFamily o f) ** exact sup_eq_lsub_or_sup_succ_eq_lsub _ ** Qed
Ordinal.bsup_succ_le_blsub ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u} f : (a : Ordinal.{u}) → a < o → Ordinal.{max u v} ⊢ succ (bsup o f) ≤ blsub o f ↔ ∃ i hi, f i hi = bsup o f ** refine' ⟨fun h => _, _⟩ ** case refine'_2 α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u} f : (a : Ordinal.{u}) → a < o → Ordinal.{max u v} ⊢ (∃ i hi, f i hi = bsup o f) → succ (bsup o f) ≤ blsub o f ** rintro ⟨_, _, hf⟩ ** case refine'_2.intro.intro α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u} f : (a : Ordinal.{u}) → a < o → Ordinal.{max u v} w✝¹ : Ordinal.{u} w✝ : w✝¹ < o hf : f w✝¹ w✝ = bsup o f ⊢ succ (bsup o f) ≤ blsub o f ** rw [succ_le_iff, ← hf] ** case refine'_2.intro.intro α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u} f : (a : Ordinal.{u}) → a < o → Ordinal.{max u v} w✝¹ : Ordinal.{u} w✝ : w✝¹ < o hf : f w✝¹ w✝ = bsup o f ⊢ f w✝¹ w✝ < blsub o f ** exact lt_blsub _ _ _ ** case refine'_1 α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u} f : (a : Ordinal.{u}) → a < o → Ordinal.{max u v} h : succ (bsup o f) ≤ blsub o f ⊢ ∃ i hi, f i hi = bsup o f ** by_contra' hf ** case refine'_1 α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u} f : (a : Ordinal.{u}) → a < o → Ordinal.{max u v} h : succ (bsup o f) ≤ blsub o f hf : ∀ (i : Ordinal.{u}) (hi : i < o), f i hi ≠ bsup o f ⊢ False ** exact ne_of_lt (succ_le_iff.1 h) (le_antisymm (bsup_le_blsub f) (blsub_le (lt_bsup_of_ne_bsup.1 hf))) ** Qed