formal
stringlengths
41
427k
informal
stringclasses
1 value
Cardinal.le_aleph0_iff_set_countable ** α β : Type u s : Set α ⊢ #↑s ≤ ℵ₀ ↔ Set.Countable s ** rw [mk_le_aleph0_iff, countable_coe_iff] ** Qed
Cardinal.add_lt_aleph0 ** α β : Type u a b : Cardinal.{u_1} m n : ℕ ha : ↑m < ℵ₀ hb : ↑n < ℵ₀ ⊢ ↑m + ↑n < ℵ₀ ** rw [← Nat.cast_add] ** α β : Type u a b : Cardinal.{u_1} m n : ℕ ha : ↑m < ℵ₀ hb : ↑n < ℵ₀ ⊢ ↑(m + n) < ℵ₀ ** apply nat_lt_aleph0 ** Qed
Cardinal.aleph0_le_add_iff ** α β : Type u a b : Cardinal.{u_1} ⊢ ℵ₀ ≤ a + b ↔ ℵ₀ ≤ a ∨ ℵ₀ ≤ b ** simp only [← not_lt, add_lt_aleph0_iff, not_and_or] ** Qed
Cardinal.nsmul_lt_aleph0_iff ** case zero α β : Type u a : Cardinal.{u_1} ⊢ Nat.zero • a < ℵ₀ ↔ Nat.zero = 0 ∨ a < ℵ₀ ** simpa using nat_lt_aleph0 0 ** case succ α β : Type u a : Cardinal.{u_1} n : ℕ ⊢ Nat.succ n • a < ℵ₀ ↔ Nat.succ n = 0 ∨ a < ℵ₀ ** simp only [Nat.succ_ne_zero, false_or_iff] ** case succ α β : Type u a : Cardinal.{u_1} n : ℕ ⊢ Nat.succ n • a < ℵ₀ ↔ a < ℵ₀ ** induction' n with n ih ** case succ.succ α β : Type u a : Cardinal.{u_1} n : ℕ ih : Nat.succ n • a < ℵ₀ ↔ a < ℵ₀ ⊢ Nat.succ (Nat.succ n) • a < ℵ₀ ↔ a < ℵ₀ ** rw [succ_nsmul, add_lt_aleph0_iff, ih, and_self_iff] ** case succ.zero α β : Type u a : Cardinal.{u_1} ⊢ Nat.succ Nat.zero • a < ℵ₀ ↔ a < ℵ₀ ** simp ** Qed
Cardinal.mul_lt_aleph0 ** α β : Type u a b : Cardinal.{u_1} m n : ℕ ha : ↑m < ℵ₀ hb : ↑n < ℵ₀ ⊢ ↑m * ↑n < ℵ₀ ** rw [← Nat.cast_mul] ** α β : Type u a b : Cardinal.{u_1} m n : ℕ ha : ↑m < ℵ₀ hb : ↑n < ℵ₀ ⊢ ↑(m * n) < ℵ₀ ** apply nat_lt_aleph0 ** Qed
Cardinal.mul_lt_aleph0_iff ** α β : Type u a b : Cardinal.{u_1} ⊢ a * b < ℵ₀ ↔ a = 0 ∨ b = 0 ∨ a < ℵ₀ ∧ b < ℵ₀ ** refine' ⟨fun h => _, _⟩ ** case refine'_2 α β : Type u a b : Cardinal.{u_1} ⊢ a = 0 ∨ b = 0 ∨ a < ℵ₀ ∧ b < ℵ₀ → a * b < ℵ₀ ** rintro (rfl | rfl | ⟨ha, hb⟩) <;> simp only [*, mul_lt_aleph0, aleph0_pos, zero_mul, mul_zero] ** case refine'_1 α β : Type u a b : Cardinal.{u_1} h : a * b < ℵ₀ ⊢ a = 0 ∨ b = 0 ∨ a < ℵ₀ ∧ b < ℵ₀ ** by_cases ha : a = 0 ** case neg α β : Type u a b : Cardinal.{u_1} h : a * b < ℵ₀ ha : ¬a = 0 ⊢ a = 0 ∨ b = 0 ∨ a < ℵ₀ ∧ b < ℵ₀ ** right ** case neg.h α β : Type u a b : Cardinal.{u_1} h : a * b < ℵ₀ ha : ¬a = 0 ⊢ b = 0 ∨ a < ℵ₀ ∧ b < ℵ₀ ** by_cases hb : b = 0 ** case neg α β : Type u a b : Cardinal.{u_1} h : a * b < ℵ₀ ha : ¬a = 0 hb : ¬b = 0 ⊢ b = 0 ∨ a < ℵ₀ ∧ b < ℵ₀ ** right ** case neg.h α β : Type u a b : Cardinal.{u_1} h : a * b < ℵ₀ ha : ¬a = 0 hb : ¬b = 0 ⊢ a < ℵ₀ ∧ b < ℵ₀ ** rw [← Ne, ← one_le_iff_ne_zero] at ha hb ** case neg.h α β : Type u a b : Cardinal.{u_1} h : a * b < ℵ₀ ha : 1 ≤ a hb : 1 ≤ b ⊢ a < ℵ₀ ∧ b < ℵ₀ ** constructor ** case pos α β : Type u a b : Cardinal.{u_1} h : a * b < ℵ₀ ha : a = 0 ⊢ a = 0 ∨ b = 0 ∨ a < ℵ₀ ∧ b < ℵ₀ ** exact Or.inl ha ** case pos α β : Type u a b : Cardinal.{u_1} h : a * b < ℵ₀ ha : ¬a = 0 hb : b = 0 ⊢ b = 0 ∨ a < ℵ₀ ∧ b < ℵ₀ ** exact Or.inl hb ** case neg.h.left α β : Type u a b : Cardinal.{u_1} h : a * b < ℵ₀ ha : 1 ≤ a hb : 1 ≤ b ⊢ a < ℵ₀ ** rw [← mul_one a] ** case neg.h.left α β : Type u a b : Cardinal.{u_1} h : a * b < ℵ₀ ha : 1 ≤ a hb : 1 ≤ b ⊢ a * 1 < ℵ₀ ** refine' (mul_le_mul' le_rfl hb).trans_lt h ** case neg.h.right α β : Type u a b : Cardinal.{u_1} h : a * b < ℵ₀ ha : 1 ≤ a hb : 1 ≤ b ⊢ b < ℵ₀ ** rw [← one_mul b] ** case neg.h.right α β : Type u a b : Cardinal.{u_1} h : a * b < ℵ₀ ha : 1 ≤ a hb : 1 ≤ b ⊢ 1 * b < ℵ₀ ** refine' (mul_le_mul' ha le_rfl).trans_lt h ** Qed
Cardinal.aleph0_le_mul_iff ** α β : Type u a b : Cardinal.{u_1} ⊢ ℵ₀ ≤ a * b ↔ a ≠ 0 ∧ b ≠ 0 ∧ (ℵ₀ ≤ a ∨ ℵ₀ ≤ b) ** let h := (@mul_lt_aleph0_iff a b).not ** α β : Type u a b : Cardinal.{u_1} h : ¬a * b < ℵ₀ ↔ ¬(a = 0 ∨ b = 0 ∨ a < ℵ₀ ∧ b < ℵ₀) := Iff.not mul_lt_aleph0_iff ⊢ ℵ₀ ≤ a * b ↔ a ≠ 0 ∧ b ≠ 0 ∧ (ℵ₀ ≤ a ∨ ℵ₀ ≤ b) ** rwa [not_lt, not_or, not_or, not_and_or, not_lt, not_lt] at h ** Qed
Cardinal.aleph0_le_mul_iff' ** α β : Type u a b : Cardinal.{u} ⊢ ℵ₀ ≤ a * b ↔ a ≠ 0 ∧ ℵ₀ ≤ b ∨ ℵ₀ ≤ a ∧ b ≠ 0 ** have : ∀ {a : Cardinal.{u}}, ℵ₀ ≤ a → a ≠ 0 := fun a => ne_bot_of_le_ne_bot aleph0_ne_zero a ** α β : Type u a b : Cardinal.{u} this : ∀ {a : Cardinal.{u}}, ℵ₀ ≤ a → a ≠ 0 ⊢ ℵ₀ ≤ a * b ↔ a ≠ 0 ∧ ℵ₀ ≤ b ∨ ℵ₀ ≤ a ∧ b ≠ 0 ** simp only [aleph0_le_mul_iff, and_or_left, and_iff_right_of_imp this, @and_left_comm (a ≠ 0)] ** α β : Type u a b : Cardinal.{u} this : ∀ {a : Cardinal.{u}}, ℵ₀ ≤ a → a ≠ 0 ⊢ b ≠ 0 ∧ ℵ₀ ≤ a ∨ a ≠ 0 ∧ ℵ₀ ≤ b ↔ a ≠ 0 ∧ ℵ₀ ≤ b ∨ ℵ₀ ≤ a ∧ b ≠ 0 ** simp only [and_comm, or_comm] ** Qed
Cardinal.mul_lt_aleph0_iff_of_ne_zero ** α β : Type u a b : Cardinal.{u_1} ha : a ≠ 0 hb : b ≠ 0 ⊢ a * b < ℵ₀ ↔ a < ℵ₀ ∧ b < ℵ₀ ** simp [mul_lt_aleph0_iff, ha, hb] ** Qed
Cardinal.power_lt_aleph0 ** α β : Type u a b : Cardinal.{u_1} m n : ℕ ha : ↑m < ℵ₀ hb : ↑n < ℵ₀ ⊢ ↑m ^ ↑n < ℵ₀ ** rw [← natCast_pow] ** α β : Type u a b : Cardinal.{u_1} m n : ℕ ha : ↑m < ℵ₀ hb : ↑n < ℵ₀ ⊢ ↑(m ^ n) < ℵ₀ ** apply nat_lt_aleph0 ** Qed
Cardinal.infinite_iff ** α✝ β α : Type u ⊢ Infinite α ↔ ℵ₀ ≤ #α ** rw [← not_lt, lt_aleph0_iff_finite, not_finite_iff_infinite] ** Qed
Cardinal.denumerable_iff ** α✝ β α : Type u h : #α = ℵ₀ ⊢ Nonempty (Denumerable α) ** cases' Quotient.exact h with f ** case intro α✝ β α : Type u h : #α = ℵ₀ f : α ≃ ULift.{u, 0} ℕ ⊢ Nonempty (Denumerable α) ** exact ⟨Denumerable.mk' <| f.trans Equiv.ulift⟩ ** Qed
Cardinal.nat_mul_aleph0 ** α β : Type u n : ℕ hn : n ≠ 0 ⊢ 1 ≤ ↑n ** rwa [← Nat.cast_one, natCast_le, Nat.one_le_iff_ne_zero] ** Qed
Cardinal.aleph0_mul_nat ** α β : Type u n : ℕ hn : n ≠ 0 ⊢ ℵ₀ * ↑n = ℵ₀ ** rw [mul_comm, nat_mul_aleph0 hn] ** Qed
Cardinal.nat_add_aleph0 ** α β : Type u n : ℕ ⊢ ↑n + ℵ₀ = ℵ₀ ** rw [add_comm, aleph0_add_nat] ** Qed
Cardinal.cast_toNat_of_lt_aleph0 ** α β : Type u c : Cardinal.{u_1} h : c < ℵ₀ ⊢ ↑(↑toNat c) = c ** rw [toNat_apply_of_lt_aleph0 h, ← Classical.choose_spec (lt_aleph0.1 h)] ** Qed
Cardinal.cast_toNat_of_aleph0_le ** α β : Type u c : Cardinal.{u_1} h : ℵ₀ ≤ c ⊢ ↑(↑toNat c) = 0 ** rw [toNat_apply_of_aleph0_le h, Nat.cast_zero] ** Qed
Cardinal.toNat_eq_iff_eq_of_lt_aleph0 ** α β : Type u c d : Cardinal.{u_1} hc : c < ℵ₀ hd : d < ℵ₀ ⊢ ↑toNat c = ↑toNat d ↔ c = d ** rw [← natCast_inj, cast_toNat_of_lt_aleph0 hc, cast_toNat_of_lt_aleph0 hd] ** Qed
Cardinal.toNat_le_iff_le_of_lt_aleph0 ** α β : Type u c d : Cardinal.{u_1} hc : c < ℵ₀ hd : d < ℵ₀ ⊢ ↑toNat c ≤ ↑toNat d ↔ c ≤ d ** rw [← natCast_le, cast_toNat_of_lt_aleph0 hc, cast_toNat_of_lt_aleph0 hd] ** Qed
Cardinal.toNat_lt_iff_lt_of_lt_aleph0 ** α β : Type u c d : Cardinal.{u_1} hc : c < ℵ₀ hd : d < ℵ₀ ⊢ ↑toNat c < ↑toNat d ↔ c < d ** rw [← natCast_lt, cast_toNat_of_lt_aleph0 hc, cast_toNat_of_lt_aleph0 hd] ** Qed
Cardinal.toNat_cast ** α β : Type u n : ℕ ⊢ ↑toNat ↑n = n ** rw [toNat_apply_of_lt_aleph0 (nat_lt_aleph0 n), ← natCast_inj] ** α β : Type u n : ℕ ⊢ ↑(choose (_ : ∃ n_1, ↑n = ↑n_1)) = ↑n ** exact (Classical.choose_spec (lt_aleph0.1 (nat_lt_aleph0 n))).symm ** Qed
Cardinal.mk_toNat_eq_card ** α β : Type u inst✝ : Fintype α ⊢ ↑toNat #α = Fintype.card α ** simp ** Qed
Cardinal.zero_toNat ** α β : Type u ⊢ ↑toNat 0 = 0 ** rw [← toNat_cast 0, Nat.cast_zero] ** Qed
Cardinal.one_toNat ** α β : Type u ⊢ ↑toNat 1 = 1 ** rw [← toNat_cast 1, Nat.cast_one] ** Qed
Cardinal.toNat_eq_one ** α β : Type u c : Cardinal.{u_1} ⊢ ↑toNat c = 1 ↔ c = 1 ** rw [toNat_eq_iff one_ne_zero, Nat.cast_one] ** Qed
Cardinal.toNat_lift ** α β : Type u c : Cardinal.{v} ⊢ ↑toNat (lift.{u, v} c) = ↑toNat c ** apply natCast_injective ** case a α β : Type u c : Cardinal.{v} ⊢ ↑(↑toNat (lift.{u, v} c)) = ↑(↑toNat c) ** cases' lt_or_ge c ℵ₀ with hc hc ** case a.inl α β : Type u c : Cardinal.{v} hc : c < ℵ₀ ⊢ ↑(↑toNat (lift.{u, v} c)) = ↑(↑toNat c) ** rw [cast_toNat_of_lt_aleph0, ← lift_natCast.{u,v}, cast_toNat_of_lt_aleph0 hc] ** case a.inl α β : Type u c : Cardinal.{v} hc : c < ℵ₀ ⊢ lift.{u, v} c < ℵ₀ ** rwa [lift_lt_aleph0] ** case a.inr α β : Type u c : Cardinal.{v} hc : c ≥ ℵ₀ ⊢ ↑(↑toNat (lift.{u, v} c)) = ↑(↑toNat c) ** rw [cast_toNat_of_aleph0_le, ← lift_natCast.{u,v}, cast_toNat_of_aleph0_le hc, lift_zero] ** case a.inr α β : Type u c : Cardinal.{v} hc : c ≥ ℵ₀ ⊢ ℵ₀ ≤ lift.{u, v} c ** rwa [aleph0_le_lift] ** Qed
Cardinal.toNat_congr ** α β✝ : Type u β : Type v e : α ≃ β ⊢ ↑toNat #α = ↑toNat #β ** rw [← toNat_lift, (lift_mk_eq.{_,_,v}).mpr ⟨e⟩, toNat_lift] ** Qed
Cardinal.toNat_mul ** α β : Type u x y : Cardinal.{u_1} ⊢ ↑toNat (x * y) = ↑toNat x * ↑toNat y ** rcases eq_or_ne x 0 with (rfl | hx1) ** case inr α β : Type u x y : Cardinal.{u_1} hx1 : x ≠ 0 ⊢ ↑toNat (x * y) = ↑toNat x * ↑toNat y ** rcases eq_or_ne y 0 with (rfl | hy1) ** case inr.inr α β : Type u x y : Cardinal.{u_1} hx1 : x ≠ 0 hy1 : y ≠ 0 ⊢ ↑toNat (x * y) = ↑toNat x * ↑toNat y ** cases' lt_or_le x ℵ₀ with hx2 hx2 ** case inl α β : Type u y : Cardinal.{u_1} ⊢ ↑toNat (0 * y) = ↑toNat 0 * ↑toNat y ** rw [zero_mul, zero_toNat, zero_mul] ** case inr.inl α β : Type u x : Cardinal.{u_1} hx1 : x ≠ 0 ⊢ ↑toNat (x * 0) = ↑toNat x * ↑toNat 0 ** rw [mul_zero, zero_toNat, mul_zero] ** case inr.inr.inl α β : Type u x y : Cardinal.{u_1} hx1 : x ≠ 0 hy1 : y ≠ 0 hx2 : x < ℵ₀ ⊢ ↑toNat (x * y) = ↑toNat x * ↑toNat y ** cases' lt_or_le y ℵ₀ with hy2 hy2 ** case inr.inr.inl.inl α β : Type u x y : Cardinal.{u_1} hx1 : x ≠ 0 hy1 : y ≠ 0 hx2 : x < ℵ₀ hy2 : y < ℵ₀ ⊢ ↑toNat (x * y) = ↑toNat x * ↑toNat y ** lift x to ℕ using hx2 ** case inr.inr.inl.inl.intro α β : Type u y : Cardinal.{u_1} hy1 : y ≠ 0 hy2 : y < ℵ₀ x : ℕ hx1 : ↑x ≠ 0 ⊢ ↑toNat (↑x * y) = ↑toNat ↑x * ↑toNat y ** lift y to ℕ using hy2 ** case inr.inr.inl.inl.intro.intro α β : Type u x : ℕ hx1 : ↑x ≠ 0 y : ℕ hy1 : ↑y ≠ 0 ⊢ ↑toNat (↑x * ↑y) = ↑toNat ↑x * ↑toNat ↑y ** rw [← Nat.cast_mul, toNat_cast, toNat_cast, toNat_cast] ** case inr.inr.inl.inr α β : Type u x y : Cardinal.{u_1} hx1 : x ≠ 0 hy1 : y ≠ 0 hx2 : x < ℵ₀ hy2 : ℵ₀ ≤ y ⊢ ↑toNat (x * y) = ↑toNat x * ↑toNat y ** rw [toNat_apply_of_aleph0_le hy2, mul_zero, toNat_apply_of_aleph0_le] ** case inr.inr.inl.inr α β : Type u x y : Cardinal.{u_1} hx1 : x ≠ 0 hy1 : y ≠ 0 hx2 : x < ℵ₀ hy2 : ℵ₀ ≤ y ⊢ ℵ₀ ≤ x * y ** exact aleph0_le_mul_iff'.2 (Or.inl ⟨hx1, hy2⟩) ** case inr.inr.inr α β : Type u x y : Cardinal.{u_1} hx1 : x ≠ 0 hy1 : y ≠ 0 hx2 : ℵ₀ ≤ x ⊢ ↑toNat (x * y) = ↑toNat x * ↑toNat y ** rw [toNat_apply_of_aleph0_le hx2, zero_mul, toNat_apply_of_aleph0_le] ** case inr.inr.inr α β : Type u x y : Cardinal.{u_1} hx1 : x ≠ 0 hy1 : y ≠ 0 hx2 : ℵ₀ ≤ x ⊢ ℵ₀ ≤ x * y ** exact aleph0_le_mul_iff'.2 (Or.inr ⟨hx2, hy1⟩) ** Qed
Cardinal.toNat_add_of_lt_aleph0 ** α β : Type u a : Cardinal.{u} b : Cardinal.{v} ha : a < ℵ₀ hb : b < ℵ₀ ⊢ ↑toNat (lift.{v, u} a + lift.{u, v} b) = ↑toNat a + ↑toNat b ** apply Cardinal.natCast_injective ** case a α β : Type u a : Cardinal.{u} b : Cardinal.{v} ha : a < ℵ₀ hb : b < ℵ₀ ⊢ ↑(↑toNat (lift.{v, u} a + lift.{u, v} b)) = ↑(↑toNat a + ↑toNat b) ** replace ha : lift.{v, u} a < ℵ₀ := by rwa [lift_lt_aleph0] ** case a α β : Type u a : Cardinal.{u} b : Cardinal.{v} hb : b < ℵ₀ ha : lift.{v, u} a < ℵ₀ ⊢ ↑(↑toNat (lift.{v, u} a + lift.{u, v} b)) = ↑(↑toNat a + ↑toNat b) ** replace hb : lift.{u, v} b < ℵ₀ := by rwa [lift_lt_aleph0] ** case a α β : Type u a : Cardinal.{u} b : Cardinal.{v} ha : lift.{v, u} a < ℵ₀ hb : lift.{u, v} b < ℵ₀ ⊢ ↑(↑toNat (lift.{v, u} a + lift.{u, v} b)) = ↑(↑toNat a + ↑toNat b) ** rw [Nat.cast_add, ← toNat_lift.{v, u} a, ← toNat_lift.{u, v} b, cast_toNat_of_lt_aleph0 ha, cast_toNat_of_lt_aleph0 hb, cast_toNat_of_lt_aleph0 (add_lt_aleph0 ha hb)] ** α β : Type u a : Cardinal.{u} b : Cardinal.{v} ha : a < ℵ₀ hb : b < ℵ₀ ⊢ lift.{v, u} a < ℵ₀ ** rwa [lift_lt_aleph0] ** α β : Type u a : Cardinal.{u} b : Cardinal.{v} hb : b < ℵ₀ ha : lift.{v, u} a < ℵ₀ ⊢ lift.{u, v} b < ℵ₀ ** rwa [lift_lt_aleph0] ** Qed
Cardinal.toPartENat_cast ** α β : Type u n : ℕ ⊢ ↑toPartENat ↑n = ↑n ** rw [toPartENat_apply_of_lt_aleph0 (nat_lt_aleph0 n), toNat_cast] ** Qed
Cardinal.toPartENat_eq_top_iff_le_aleph0 ** α β : Type u c : Cardinal.{u_1} ⊢ ↑toPartENat c = ⊤ ↔ ℵ₀ ≤ c ** cases lt_or_ge c ℵ₀ with | inl hc => simp only [toPartENat_apply_of_lt_aleph0 hc, PartENat.natCast_ne_top, false_iff, not_le, hc] | inr hc => simp only [toPartENat_apply_of_aleph0_le hc, eq_self_iff_true, true_iff]; exact hc ** case inl α β : Type u c : Cardinal.{u_1} hc : c < ℵ₀ ⊢ ↑toPartENat c = ⊤ ↔ ℵ₀ ≤ c ** simp only [toPartENat_apply_of_lt_aleph0 hc, PartENat.natCast_ne_top, false_iff, not_le, hc] ** case inr α β : Type u c : Cardinal.{u_1} hc : c ≥ ℵ₀ ⊢ ↑toPartENat c = ⊤ ↔ ℵ₀ ≤ c ** simp only [toPartENat_apply_of_aleph0_le hc, eq_self_iff_true, true_iff] ** case inr α β : Type u c : Cardinal.{u_1} hc : c ≥ ℵ₀ ⊢ ℵ₀ ≤ c ** exact hc ** Qed
Cardinal.toPartENat_mono ** α β : Type u c c' : Cardinal.{u_1} h : c ≤ c' ⊢ ↑toPartENat c ≤ ↑toPartENat c' ** cases lt_or_ge c ℵ₀ with | inl hc => rw [toPartENat_apply_of_lt_aleph0 hc] cases lt_or_ge c' ℵ₀ with | inl hc' => rw [toPartENat_apply_of_lt_aleph0 hc', PartENat.coe_le_coe] exact toNat_le_of_le_of_lt_aleph0 hc' h | inr hc' => rw [toPartENat_apply_of_aleph0_le hc'] exact le_top | inr hc => rw [toPartENat_apply_of_aleph0_le hc, toPartENat_apply_of_aleph0_le (le_trans hc h)] ** case inl α β : Type u c c' : Cardinal.{u_1} h : c ≤ c' hc : c < ℵ₀ ⊢ ↑toPartENat c ≤ ↑toPartENat c' ** rw [toPartENat_apply_of_lt_aleph0 hc] ** case inl α β : Type u c c' : Cardinal.{u_1} h : c ≤ c' hc : c < ℵ₀ ⊢ ↑(↑toNat c) ≤ ↑toPartENat c' ** cases lt_or_ge c' ℵ₀ with | inl hc' => rw [toPartENat_apply_of_lt_aleph0 hc', PartENat.coe_le_coe] exact toNat_le_of_le_of_lt_aleph0 hc' h | inr hc' => rw [toPartENat_apply_of_aleph0_le hc'] exact le_top ** case inl.inl α β : Type u c c' : Cardinal.{u_1} h : c ≤ c' hc : c < ℵ₀ hc' : c' < ℵ₀ ⊢ ↑(↑toNat c) ≤ ↑toPartENat c' ** rw [toPartENat_apply_of_lt_aleph0 hc', PartENat.coe_le_coe] ** case inl.inl α β : Type u c c' : Cardinal.{u_1} h : c ≤ c' hc : c < ℵ₀ hc' : c' < ℵ₀ ⊢ ↑toNat c ≤ ↑toNat c' ** exact toNat_le_of_le_of_lt_aleph0 hc' h ** case inl.inr α β : Type u c c' : Cardinal.{u_1} h : c ≤ c' hc : c < ℵ₀ hc' : c' ≥ ℵ₀ ⊢ ↑(↑toNat c) ≤ ↑toPartENat c' ** rw [toPartENat_apply_of_aleph0_le hc'] ** case inl.inr α β : Type u c c' : Cardinal.{u_1} h : c ≤ c' hc : c < ℵ₀ hc' : c' ≥ ℵ₀ ⊢ ↑(↑toNat c) ≤ ⊤ ** exact le_top ** case inr α β : Type u c c' : Cardinal.{u_1} h : c ≤ c' hc : c ≥ ℵ₀ ⊢ ↑toPartENat c ≤ ↑toPartENat c' ** rw [toPartENat_apply_of_aleph0_le hc, toPartENat_apply_of_aleph0_le (le_trans hc h)] ** Qed
Cardinal.toPartENat_lift ** α β : Type u c : Cardinal.{v} ⊢ ↑toPartENat (lift.{u, v} c) = ↑toPartENat c ** cases' lt_or_ge c ℵ₀ with hc hc ** case inl α β : Type u c : Cardinal.{v} hc : c < ℵ₀ ⊢ ↑toPartENat (lift.{u, v} c) = ↑toPartENat c ** rw [toPartENat_apply_of_lt_aleph0 hc, Cardinal.toPartENat_apply_of_lt_aleph0 _] ** case inl α β : Type u c : Cardinal.{v} hc : c < ℵ₀ ⊢ ↑(↑toNat (lift.{u, v} c)) = ↑(↑toNat c) α β : Type u c : Cardinal.{v} hc : c < ℵ₀ ⊢ lift.{u, v} c < ℵ₀ ** simp only [toNat_lift] ** α β : Type u c : Cardinal.{v} hc : c < ℵ₀ ⊢ lift.{u, v} c < ℵ₀ ** rw [lift_lt_aleph0] ** α β : Type u c : Cardinal.{v} hc : c < ℵ₀ ⊢ c < ℵ₀ ** exact hc ** case inr α β : Type u c : Cardinal.{v} hc : c ≥ ℵ₀ ⊢ ↑toPartENat (lift.{u, v} c) = ↑toPartENat c ** rw [toPartENat_apply_of_aleph0_le hc, toPartENat_apply_of_aleph0_le _] ** α β : Type u c : Cardinal.{v} hc : c ≥ ℵ₀ ⊢ ℵ₀ ≤ lift.{u, v} c ** rw [aleph0_le_lift] ** α β : Type u c : Cardinal.{v} hc : c ≥ ℵ₀ ⊢ ℵ₀ ≤ c ** exact hc ** Qed
Cardinal.toPartENat_congr ** α β✝ : Type u β : Type v e : α ≃ β ⊢ ↑toPartENat #α = ↑toPartENat #β ** rw [← toPartENat_lift, lift_mk_eq.{_, _,v}.mpr ⟨e⟩, toPartENat_lift] ** Qed
Cardinal.mk_toPartENat_eq_coe_card ** α β : Type u inst✝ : Fintype α ⊢ ↑toPartENat #α = ↑(Fintype.card α) ** simp ** Qed
Cardinal.sum_lt_prod ** α β : Type u ι : Type u_1 f g : ι → Cardinal.{u_2} H : ∀ (i : ι), f i < g i x✝ : sum f ≥ prod g F : ((i : ι) → Quotient.out (g i)) ↪ (i : ι) × Quotient.out (f i) ⊢ False ** have : Inhabited (∀ i : ι, (g i).out) := by refine' ⟨fun i => Classical.choice <| mk_ne_zero_iff.1 _⟩ rw [mk_out] exact (H i).ne_bot ** α β : Type u ι : Type u_1 f g : ι → Cardinal.{u_2} H : ∀ (i : ι), f i < g i x✝ : sum f ≥ prod g F : ((i : ι) → Quotient.out (g i)) ↪ (i : ι) × Quotient.out (f i) this : Inhabited ((i : ι) → Quotient.out (g i)) ⊢ False ** let G := invFun F ** α β : Type u ι : Type u_1 f g : ι → Cardinal.{u_2} H : ∀ (i : ι), f i < g i x✝ : sum f ≥ prod g F : ((i : ι) → Quotient.out (g i)) ↪ (i : ι) × Quotient.out (f i) this : Inhabited ((i : ι) → Quotient.out (g i)) G : (i : ι) × Quotient.out (f i) → (i : ι) → Quotient.out (g i) := invFun ↑F ⊢ False ** have sG : Surjective G := invFun_surjective F.2 ** α β : Type u ι : Type u_1 f g : ι → Cardinal.{u_2} H : ∀ (i : ι), f i < g i x✝ : sum f ≥ prod g F : ((i : ι) → Quotient.out (g i)) ↪ (i : ι) × Quotient.out (f i) this : Inhabited ((i : ι) → Quotient.out (g i)) G : (i : ι) × Quotient.out (f i) → (i : ι) → Quotient.out (g i) := invFun ↑F sG : Surjective G ⊢ False ** choose C hc using show ∀ i, ∃ b, ∀ a, G ⟨i, a⟩ i ≠ b by intro i simp only [not_exists.symm, not_forall.symm] refine' fun h => (H i).not_le _ rw [← mk_out (f i), ← mk_out (g i)] exact ⟨Embedding.ofSurjective _ h⟩ ** α β : Type u ι : Type u_1 f g : ι → Cardinal.{u_2} H : ∀ (i : ι), f i < g i x✝ : sum f ≥ prod g F : ((i : ι) → Quotient.out (g i)) ↪ (i : ι) × Quotient.out (f i) this : Inhabited ((i : ι) → Quotient.out (g i)) G : (i : ι) × Quotient.out (f i) → (i : ι) → Quotient.out (g i) := invFun ↑F sG : Surjective G C : (i : ι) → Quotient.out (g i) hc : ∀ (i : ι) (a : Quotient.out (f i)), G { fst := i, snd := a } i ≠ C i ⊢ False ** let ⟨⟨i, a⟩, h⟩ := sG C ** α β : Type u ι : Type u_1 f g : ι → Cardinal.{u_2} H : ∀ (i : ι), f i < g i x✝ : sum f ≥ prod g F : ((i : ι) → Quotient.out (g i)) ↪ (i : ι) × Quotient.out (f i) this : Inhabited ((i : ι) → Quotient.out (g i)) G : (i : ι) × Quotient.out (f i) → (i : ι) → Quotient.out (g i) := invFun ↑F sG : Surjective G C : (i : ι) → Quotient.out (g i) hc : ∀ (i : ι) (a : Quotient.out (f i)), G { fst := i, snd := a } i ≠ C i i : ι a : Quotient.out (f i) h : G { fst := i, snd := a } = C ⊢ False ** exact hc i a (congr_fun h _) ** α β : Type u ι : Type u_1 f g : ι → Cardinal.{u_2} H : ∀ (i : ι), f i < g i x✝ : sum f ≥ prod g F : ((i : ι) → Quotient.out (g i)) ↪ (i : ι) × Quotient.out (f i) ⊢ Inhabited ((i : ι) → Quotient.out (g i)) ** refine' ⟨fun i => Classical.choice <| mk_ne_zero_iff.1 _⟩ ** α β : Type u ι : Type u_1 f g : ι → Cardinal.{u_2} H : ∀ (i : ι), f i < g i x✝ : sum f ≥ prod g F : ((i : ι) → Quotient.out (g i)) ↪ (i : ι) × Quotient.out (f i) i : ι ⊢ #(Quotient.out (g i)) ≠ 0 ** rw [mk_out] ** α β : Type u ι : Type u_1 f g : ι → Cardinal.{u_2} H : ∀ (i : ι), f i < g i x✝ : sum f ≥ prod g F : ((i : ι) → Quotient.out (g i)) ↪ (i : ι) × Quotient.out (f i) i : ι ⊢ g i ≠ 0 ** exact (H i).ne_bot ** α β : Type u ι : Type u_1 f g : ι → Cardinal.{u_2} H : ∀ (i : ι), f i < g i x✝ : sum f ≥ prod g F : ((i : ι) → Quotient.out (g i)) ↪ (i : ι) × Quotient.out (f i) this : Inhabited ((i : ι) → Quotient.out (g i)) G : (i : ι) × Quotient.out (f i) → (i : ι) → Quotient.out (g i) := invFun ↑F sG : Surjective G ⊢ ∀ (i : ι), ∃ b, ∀ (a : Quotient.out (f i)), G { fst := i, snd := a } i ≠ b ** intro i ** α β : Type u ι : Type u_1 f g : ι → Cardinal.{u_2} H : ∀ (i : ι), f i < g i x✝ : sum f ≥ prod g F : ((i : ι) → Quotient.out (g i)) ↪ (i : ι) × Quotient.out (f i) this : Inhabited ((i : ι) → Quotient.out (g i)) G : (i : ι) × Quotient.out (f i) → (i : ι) → Quotient.out (g i) := invFun ↑F sG : Surjective G i : ι ⊢ ∃ b, ∀ (a : Quotient.out (f i)), G { fst := i, snd := a } i ≠ b ** simp only [not_exists.symm, not_forall.symm] ** α β : Type u ι : Type u_1 f g : ι → Cardinal.{u_2} H : ∀ (i : ι), f i < g i x✝ : sum f ≥ prod g F : ((i : ι) → Quotient.out (g i)) ↪ (i : ι) × Quotient.out (f i) this : Inhabited ((i : ι) → Quotient.out (g i)) G : (i : ι) × Quotient.out (f i) → (i : ι) → Quotient.out (g i) := invFun ↑F sG : Surjective G i : ι ⊢ ¬∀ (x : Quotient.out (g i)), ∃ x_1, invFun ↑F { fst := i, snd := x_1 } i = x ** refine' fun h => (H i).not_le _ ** α β : Type u ι : Type u_1 f g : ι → Cardinal.{u_2} H : ∀ (i : ι), f i < g i x✝ : sum f ≥ prod g F : ((i : ι) → Quotient.out (g i)) ↪ (i : ι) × Quotient.out (f i) this : Inhabited ((i : ι) → Quotient.out (g i)) G : (i : ι) × Quotient.out (f i) → (i : ι) → Quotient.out (g i) := invFun ↑F sG : Surjective G i : ι h : ∀ (x : Quotient.out (g i)), ∃ x_1, invFun ↑F { fst := i, snd := x_1 } i = x ⊢ g i ≤ f i ** rw [← mk_out (f i), ← mk_out (g i)] ** α β : Type u ι : Type u_1 f g : ι → Cardinal.{u_2} H : ∀ (i : ι), f i < g i x✝ : sum f ≥ prod g F : ((i : ι) → Quotient.out (g i)) ↪ (i : ι) × Quotient.out (f i) this : Inhabited ((i : ι) → Quotient.out (g i)) G : (i : ι) × Quotient.out (f i) → (i : ι) → Quotient.out (g i) := invFun ↑F sG : Surjective G i : ι h : ∀ (x : Quotient.out (g i)), ∃ x_1, invFun ↑F { fst := i, snd := x_1 } i = x ⊢ #(Quotient.out (g i)) ≤ #(Quotient.out (f i)) ** exact ⟨Embedding.ofSurjective _ h⟩ ** Qed
Cardinal.mk_vector ** α✝ β α : Type u n : ℕ ⊢ #(Fin n → α) = #α ^ n ** simp ** Qed
Cardinal.mk_list_eq_sum_pow ** α✝ β α : Type u ⊢ #((n : ℕ) × Vector α n) = sum fun n => #α ^ n ** simp ** Qed
Cardinal.mk_emptyCollection_iff ** α✝ β α : Type u s : Set α ⊢ #↑s = 0 ↔ s = ∅ ** constructor ** case mp α✝ β α : Type u s : Set α ⊢ #↑s = 0 → s = ∅ ** intro h ** case mp α✝ β α : Type u s : Set α h : #↑s = 0 ⊢ s = ∅ ** rw [mk_eq_zero_iff] at h ** case mp α✝ β α : Type u s : Set α h : IsEmpty ↑s ⊢ s = ∅ ** exact eq_empty_iff_forall_not_mem.2 fun x hx => h.elim' ⟨x, hx⟩ ** case mpr α✝ β α : Type u s : Set α ⊢ s = ∅ → #↑s = 0 ** rintro rfl ** case mpr α✝ β α : Type u ⊢ #↑∅ = 0 ** exact mk_emptyCollection _ ** Qed
Cardinal.mk_sUnion_le ** α✝ β α : Type u A : Set (Set α) ⊢ #↑(⋃₀ A) ≤ #↑A * ⨆ s, #↑↑s ** rw [sUnion_eq_iUnion] ** α✝ β α : Type u A : Set (Set α) ⊢ #↑(⋃ i, ↑i) ≤ #↑A * ⨆ s, #↑↑s ** apply mk_iUnion_le ** Qed
Cardinal.mk_biUnion_le ** α✝ β ι α : Type u A : ι → Set α s : Set ι ⊢ #↑(⋃ x ∈ s, A x) ≤ #↑s * ⨆ x, #↑(A ↑x) ** rw [biUnion_eq_iUnion] ** α✝ β ι α : Type u A : ι → Set α s : Set ι ⊢ #↑(⋃ x, A ↑x) ≤ #↑s * ⨆ x, #↑(A ↑x) ** apply mk_iUnion_le ** Qed
Cardinal.mk_set_eq_nat_iff_finset ** α✝ β : Type u α : Type u_1 s : Set α n : ℕ ⊢ #↑s = ↑n ↔ ∃ t, ↑t = s ∧ Finset.card t = n ** constructor ** case mp α✝ β : Type u α : Type u_1 s : Set α n : ℕ ⊢ #↑s = ↑n → ∃ t, ↑t = s ∧ Finset.card t = n ** intro h ** case mp α✝ β : Type u α : Type u_1 s : Set α n : ℕ h : #↑s = ↑n ⊢ ∃ t, ↑t = s ∧ Finset.card t = n ** lift s to Finset α using lt_aleph0_iff_set_finite.1 (h.symm ▸ nat_lt_aleph0 n) ** case mp.intro α✝ β : Type u α : Type u_1 n : ℕ s : Finset α h : #↑↑s = ↑n ⊢ ∃ t, ↑t = ↑s ∧ Finset.card t = n ** simpa using h ** case mpr α✝ β : Type u α : Type u_1 s : Set α n : ℕ ⊢ (∃ t, ↑t = s ∧ Finset.card t = n) → #↑s = ↑n ** rintro ⟨t, rfl, rfl⟩ ** case mpr.intro.intro α✝ β : Type u α : Type u_1 t : Finset α ⊢ #↑↑t = ↑(Finset.card t) ** exact mk_coe_finset ** Qed
Cardinal.mk_eq_nat_iff_finset ** α β : Type u n : ℕ ⊢ #α = ↑n ↔ ∃ t, ↑t = univ ∧ Finset.card t = n ** rw [← mk_univ, mk_set_eq_nat_iff_finset] ** Qed
Cardinal.mk_eq_nat_iff_fintype ** α β : Type u n : ℕ ⊢ #α = ↑n ↔ ∃ h, Fintype.card α = n ** rw [mk_eq_nat_iff_finset] ** α β : Type u n : ℕ ⊢ (∃ t, ↑t = univ ∧ Finset.card t = n) ↔ ∃ h, Fintype.card α = n ** constructor ** case mp α β : Type u n : ℕ ⊢ (∃ t, ↑t = univ ∧ Finset.card t = n) → ∃ h, Fintype.card α = n ** rintro ⟨t, ht, hn⟩ ** case mp.intro.intro α β : Type u n : ℕ t : Finset α ht : ↑t = univ hn : Finset.card t = n ⊢ ∃ h, Fintype.card α = n ** exact ⟨⟨t, eq_univ_iff_forall.1 ht⟩, hn⟩ ** case mpr α β : Type u n : ℕ ⊢ (∃ h, Fintype.card α = n) → ∃ t, ↑t = univ ∧ Finset.card t = n ** rintro ⟨⟨t, ht⟩, hn⟩ ** case mpr.intro.mk α β : Type u n : ℕ t : Finset α ht : ∀ (x : α), x ∈ t hn : Fintype.card α = n ⊢ ∃ t, ↑t = univ ∧ Finset.card t = n ** exact ⟨t, eq_univ_iff_forall.2 ht, hn⟩ ** Qed
Cardinal.mk_insert ** α✝ β α : Type u s : Set α a : α h : ¬a ∈ s ⊢ #↑(insert a s) = #↑s + 1 ** rw [← union_singleton, mk_union_of_disjoint, mk_singleton] ** α✝ β α : Type u s : Set α a : α h : ¬a ∈ s ⊢ Disjoint s {a} ** simpa ** Qed
Cardinal.mk_le_iff_forall_finset_subset_card_le ** α✝ β α : Type u n : ℕ t : Set α ⊢ #↑t ≤ ↑n ↔ ∀ (s : Finset α), ↑s ⊆ t → Finset.card s ≤ n ** refine ⟨fun H s hs ↦ by simpa using (mk_le_mk_of_subset hs).trans H, fun H ↦ ?_⟩ ** α✝ β α : Type u n : ℕ t : Set α H : ∀ (s : Finset α), ↑s ⊆ t → Finset.card s ≤ n ⊢ #↑t ≤ ↑n ** apply card_le_of (fun s ↦ ?_) ** α✝ β α : Type u n : ℕ t : Set α H : ∀ (s : Finset α), ↑s ⊆ t → Finset.card s ≤ n s : Finset ↑t ⊢ Finset.card s ≤ n ** let u : Finset α := s.image Subtype.val ** α✝ β α : Type u n : ℕ t : Set α H : ∀ (s : Finset α), ↑s ⊆ t → Finset.card s ≤ n s : Finset ↑t u : Finset α := Finset.image Subtype.val s ⊢ Finset.card s ≤ n ** have : u.card = s.card := Finset.card_image_of_injOn (injOn_of_injective Subtype.coe_injective _) ** α✝ β α : Type u n : ℕ t : Set α H : ∀ (s : Finset α), ↑s ⊆ t → Finset.card s ≤ n s : Finset ↑t u : Finset α := Finset.image Subtype.val s this : Finset.card u = Finset.card s ⊢ Finset.card s ≤ n ** rw [← this] ** α✝ β α : Type u n : ℕ t : Set α H : ∀ (s : Finset α), ↑s ⊆ t → Finset.card s ≤ n s : Finset ↑t u : Finset α := Finset.image Subtype.val s this : Finset.card u = Finset.card s ⊢ Finset.card u ≤ n ** apply H ** case a α✝ β α : Type u n : ℕ t : Set α H : ∀ (s : Finset α), ↑s ⊆ t → Finset.card s ≤ n s : Finset ↑t u : Finset α := Finset.image Subtype.val s this : Finset.card u = Finset.card s ⊢ ↑u ⊆ t ** simp only [Finset.coe_image, image_subset_iff, Subtype.coe_preimage_self, subset_univ] ** α✝ β α : Type u n : ℕ t : Set α H : #↑t ≤ ↑n s : Finset α hs : ↑s ⊆ t ⊢ Finset.card s ≤ n ** simpa using (mk_le_mk_of_subset hs).trans H ** Qed
Cardinal.mk_diff_add_mk ** α β : Type u S T : Set α h : T ⊆ S ⊢ #↑(S \ T) + #↑T = #↑S ** refine (mk_union_of_disjoint <| ?_).symm.trans <| by rw [diff_union_of_subset h] ** α β : Type u S T : Set α h : T ⊆ S ⊢ Disjoint (S \ T) T ** exact disjoint_sdiff_self_left ** α β : Type u S T : Set α h : T ⊆ S ⊢ #↑(S \ T ∪ T) = #↑S ** rw [diff_union_of_subset h] ** Qed
Cardinal.mk_union_le_aleph0 ** α✝ β : Type u α : Type u_1 P Q : Set α ⊢ #↑(P ∪ Q) ≤ ℵ₀ ↔ #↑P ≤ ℵ₀ ∧ #↑Q ≤ ℵ₀ ** simp only [le_aleph0_iff_subtype_countable, mem_union, setOf_mem_eq, Set.union_def, ← countable_union] ** Qed
Cardinal.mk_preimage_of_injective_lift ** α✝ β✝ α : Type u β : Type v f : α → β s : Set β h : Injective f ⊢ lift.{v, u} #↑(f ⁻¹' s) ≤ lift.{u, v} #↑s ** rw [lift_mk_le.{0}] ** α✝ β✝ α : Type u β : Type v f : α → β s : Set β h : Injective f ⊢ Nonempty (↑(f ⁻¹' s) ↪ ↑s) ** use Subtype.coind (fun x => f x.1) fun x => mem_preimage.mp x.2 ** case inj' α✝ β✝ α : Type u β : Type v f : α → β s : Set β h : Injective f ⊢ Injective (Subtype.coind (fun x => f ↑x) (_ : ∀ (x : ↑(f ⁻¹' s)), f ↑x ∈ s)) ** apply Subtype.coind_injective ** case inj'.hf α✝ β✝ α : Type u β : Type v f : α → β s : Set β h : Injective f ⊢ Injective fun x => f ↑x ** exact h.comp Subtype.val_injective ** Qed
Cardinal.mk_preimage_of_subset_range_lift ** α✝ β✝ α : Type u β : Type v f : α → β s : Set β h : s ⊆ range f ⊢ lift.{u, v} #↑s ≤ lift.{v, u} #↑(f ⁻¹' s) ** rw [lift_mk_le.{0}] ** α✝ β✝ α : Type u β : Type v f : α → β s : Set β h : s ⊆ range f ⊢ Nonempty (↑s ↪ ↑(f ⁻¹' s)) ** refine' ⟨⟨_, _⟩⟩ ** case refine'_2 α✝ β✝ α : Type u β : Type v f : α → β s : Set β h : s ⊆ range f ⊢ Injective fun a => Subtype.casesOn a fun y hy => Subtype.casesOn (subtype_of_exists (_ : y ∈ range f)) fun x property => Eq.ndrec (motive := fun y => y ∈ s → ↑(f ⁻¹' s)) (fun hy => { val := x, property := hy }) property hy ** rintro ⟨y, hy⟩ ⟨y', hy'⟩ ** case refine'_2.mk.mk α✝ β✝ α : Type u β : Type v f : α → β s : Set β h : s ⊆ range f y : β hy : y ∈ s y' : β hy' : y' ∈ s ⊢ (fun a => Subtype.casesOn a fun y hy => Subtype.casesOn (subtype_of_exists (_ : y ∈ range f)) fun x property => Eq.ndrec (motive := fun y => y ∈ s → ↑(f ⁻¹' s)) (fun hy => { val := x, property := hy }) property hy) { val := y, property := hy } = (fun a => Subtype.casesOn a fun y hy => Subtype.casesOn (subtype_of_exists (_ : y ∈ range f)) fun x property => Eq.ndrec (motive := fun y => y ∈ s → ↑(f ⁻¹' s)) (fun hy => { val := x, property := hy }) property hy) { val := y', property := hy' } → { val := y, property := hy } = { val := y', property := hy' } ** dsimp ** case refine'_2.mk.mk α✝ β✝ α : Type u β : Type v f : α → β s : Set β h : s ⊆ range f y : β hy : y ∈ s y' : β hy' : y' ∈ s ⊢ Eq.rec (motive := fun x x_1 => x ∈ s → ↑(f ⁻¹' s)) (fun hy_1 => { val := ↑(subtype_of_exists (_ : y ∈ range f)), property := hy_1 }) (_ : f ↑(subtype_of_exists (_ : y ∈ range f)) = y) hy = Eq.rec (motive := fun x x_1 => x ∈ s → ↑(f ⁻¹' s)) (fun hy => { val := ↑(subtype_of_exists (_ : y' ∈ range f)), property := hy }) (_ : f ↑(subtype_of_exists (_ : y' ∈ range f)) = y') hy' → { val := y, property := hy } = { val := y', property := hy' } ** rcases Classical.subtype_of_exists (h hy) with ⟨x, rfl⟩ ** case refine'_2.mk.mk.mk α✝ β✝ α : Type u β : Type v f : α → β s : Set β h : s ⊆ range f y' : β hy' : y' ∈ s x : α hy : f x ∈ s ⊢ Eq.rec (motive := fun x_1 x => x_1 ∈ s → ↑(f ⁻¹' s)) (fun hy => { val := ↑{ val := x, property := (_ : f x = f x) }, property := hy }) (_ : f ↑{ val := x, property := (_ : f x = f x) } = f x) hy = Eq.rec (motive := fun x x_1 => x ∈ s → ↑(f ⁻¹' s)) (fun hy => { val := ↑(subtype_of_exists (_ : y' ∈ range f)), property := hy }) (_ : f ↑(subtype_of_exists (_ : y' ∈ range f)) = y') hy' → { val := f x, property := hy } = { val := y', property := hy' } ** rcases Classical.subtype_of_exists (h hy') with ⟨x', rfl⟩ ** case refine'_2.mk.mk.mk.mk α✝ β✝ α : Type u β : Type v f : α → β s : Set β h : s ⊆ range f x : α hy : f x ∈ s x' : α hy' : f x' ∈ s ⊢ Eq.rec (motive := fun x_1 x => x_1 ∈ s → ↑(f ⁻¹' s)) (fun hy => { val := ↑{ val := x, property := (_ : f x = f x) }, property := hy }) (_ : f ↑{ val := x, property := (_ : f x = f x) } = f x) hy = Eq.rec (motive := fun x x_1 => x ∈ s → ↑(f ⁻¹' s)) (fun hy => { val := ↑{ val := x', property := (_ : f x' = f x') }, property := hy }) (_ : f ↑{ val := x', property := (_ : f x' = f x') } = f x') hy' → { val := f x, property := hy } = { val := f x', property := hy' } ** simp ** case refine'_2.mk.mk.mk.mk α✝ β✝ α : Type u β : Type v f : α → β s : Set β h : s ⊆ range f x : α hy : f x ∈ s x' : α hy' : f x' ∈ s ⊢ x = x' → f x = f x' ** intro hxx' ** case refine'_2.mk.mk.mk.mk α✝ β✝ α : Type u β : Type v f : α → β s : Set β h : s ⊆ range f x : α hy : f x ∈ s x' : α hy' : f x' ∈ s hxx' : x = x' ⊢ f x = f x' ** rw [hxx'] ** case refine'_1 α✝ β✝ α : Type u β : Type v f : α → β s : Set β h : s ⊆ range f ⊢ ↑s → ↑(f ⁻¹' s) ** rintro ⟨y, hy⟩ ** case refine'_1.mk α✝ β✝ α : Type u β : Type v f : α → β s : Set β h : s ⊆ range f y : β hy : y ∈ s ⊢ ↑(f ⁻¹' s) ** rcases Classical.subtype_of_exists (h hy) with ⟨x, rfl⟩ ** case refine'_1.mk.mk α✝ β✝ α : Type u β : Type v f : α → β s : Set β h : s ⊆ range f x : α hy : f x ∈ s ⊢ ↑(f ⁻¹' s) ** exact ⟨x, hy⟩ ** Qed
Cardinal.mk_preimage_of_injective ** α β : Type u f : α → β s : Set β h : Injective f ⊢ #↑(f ⁻¹' s) ≤ #↑s ** rw [← lift_id #(↑(f ⁻¹' s)), ← lift_id #(↑s)] ** α β : Type u f : α → β s : Set β h : Injective f ⊢ lift.{u, u} #↑(f ⁻¹' s) ≤ lift.{u, u} #↑s ** exact mk_preimage_of_injective_lift f s h ** Qed
Cardinal.mk_preimage_of_subset_range ** α β : Type u f : α → β s : Set β h : s ⊆ range f ⊢ #↑s ≤ #↑(f ⁻¹' s) ** rw [← lift_id #(↑(f ⁻¹' s)), ← lift_id #(↑s)] ** α β : Type u f : α → β s : Set β h : s ⊆ range f ⊢ lift.{u, u} #↑s ≤ lift.{u, u} #↑(f ⁻¹' s) ** exact mk_preimage_of_subset_range_lift f s h ** Qed
Cardinal.mk_preimage_of_injective_of_subset_range ** α β : Type u f : α → β s : Set β h : Injective f h2 : s ⊆ range f ⊢ #↑(f ⁻¹' s) = #↑s ** convert mk_preimage_of_injective_of_subset_range_lift.{u, u} f s h h2 using 1 <;> rw [lift_id] ** Qed
Cardinal.mk_subset_ge_of_subset_image_lift ** α✝ β✝ α : Type u β : Type v f : α → β s : Set α t : Set β h : t ⊆ f '' s ⊢ lift.{u, v} #↑t ≤ lift.{v, u} #↑{x | x ∈ s ∧ f x ∈ t} ** rw [image_eq_range] at h ** α✝ β✝ α : Type u β : Type v f : α → β s : Set α t : Set β h : t ⊆ range fun x => f ↑x ⊢ lift.{u, v} #↑t ≤ lift.{v, u} #↑{x | x ∈ s ∧ f x ∈ t} ** convert mk_preimage_of_subset_range_lift _ _ h using 1 ** case h.e'_4 α✝ β✝ α : Type u β : Type v f : α → β s : Set α t : Set β h : t ⊆ range fun x => f ↑x ⊢ lift.{v, u} #↑{x | x ∈ s ∧ f x ∈ t} = lift.{v, u} #↑((fun x => f ↑x) ⁻¹' t) ** rw [mk_sep] ** case h.e'_4 α✝ β✝ α : Type u β : Type v f : α → β s : Set α t : Set β h : t ⊆ range fun x => f ↑x ⊢ lift.{v, u} #↑{x | f ↑x ∈ t} = lift.{v, u} #↑((fun x => f ↑x) ⁻¹' t) ** rfl ** Qed
Cardinal.mk_subset_ge_of_subset_image ** α β : Type u f : α → β s : Set α t : Set β h : t ⊆ f '' s ⊢ #↑t ≤ #↑{x | x ∈ s ∧ f x ∈ t} ** rw [image_eq_range] at h ** α β : Type u f : α → β s : Set α t : Set β h : t ⊆ range fun x => f ↑x ⊢ #↑t ≤ #↑{x | x ∈ s ∧ f x ∈ t} ** convert mk_preimage_of_subset_range _ _ h using 1 ** case h.e'_4 α β : Type u f : α → β s : Set α t : Set β h : t ⊆ range fun x => f ↑x ⊢ #↑{x | x ∈ s ∧ f x ∈ t} = #↑((fun x => f ↑x) ⁻¹' t) ** rw [mk_sep] ** case h.e'_4 α β : Type u f : α → β s : Set α t : Set β h : t ⊆ range fun x => f ↑x ⊢ #↑{x | f ↑x ∈ t} = #↑((fun x => f ↑x) ⁻¹' t) ** rfl ** Qed
Cardinal.le_mk_iff_exists_subset ** α✝ β : Type u c : Cardinal.{u} α : Type u s : Set α ⊢ c ≤ #↑s ↔ ∃ p, p ⊆ s ∧ #↑p = c ** rw [le_mk_iff_exists_set, ← Subtype.exists_set_subtype] ** α✝ β : Type u c : Cardinal.{u} α : Type u s : Set α ⊢ (∃ p, #↑p = c) ↔ ∃ s_1, #↑(Subtype.val '' s_1) = c ** apply exists_congr ** case h α✝ β : Type u c : Cardinal.{u} α : Type u s : Set α ⊢ ∀ (a : Set ↑s), #↑a = c ↔ #↑(Subtype.val '' a) = c ** intro t ** case h α✝ β : Type u c : Cardinal.{u} α : Type u s : Set α t : Set ↑s ⊢ #↑t = c ↔ #↑(Subtype.val '' t) = c ** rw [mk_image_eq] ** case h α✝ β : Type u c : Cardinal.{u} α : Type u s : Set α t : Set ↑s ⊢ Injective Subtype.val ** apply Subtype.val_injective ** Qed
Cardinal.two_le_iff ** α β : Type u ⊢ 2 ≤ #α ↔ ∃ x y, x ≠ y ** rw [← Nat.cast_two, nat_succ, succ_le_iff, Nat.cast_one, one_lt_iff_nontrivial, nontrivial_iff] ** Qed
Cardinal.two_le_iff' ** α β : Type u x : α ⊢ 2 ≤ #α ↔ ∃ y, y ≠ x ** rw [two_le_iff, ← nontrivial_iff, nontrivial_iff_exists_ne x] ** Qed
Cardinal.mk_eq_two_iff ** α β : Type u ⊢ #α = 2 ↔ ∃ x y, x ≠ y ∧ {x, y} = univ ** simp only [← @Nat.cast_two Cardinal, mk_eq_nat_iff_finset, Finset.card_eq_two] ** α β : Type u ⊢ (∃ t, ↑t = univ ∧ ∃ x y, x ≠ y ∧ t = {x, y}) ↔ ∃ x y, x ≠ y ∧ {x, y} = univ ** constructor ** case mp α β : Type u ⊢ (∃ t, ↑t = univ ∧ ∃ x y, x ≠ y ∧ t = {x, y}) → ∃ x y, x ≠ y ∧ {x, y} = univ ** rintro ⟨t, ht, x, y, hne, rfl⟩ ** case mp.intro.intro.intro.intro.intro α β : Type u x y : α hne : x ≠ y ht : ↑{x, y} = univ ⊢ ∃ x y, x ≠ y ∧ {x, y} = univ ** exact ⟨x, y, hne, by simpa using ht⟩ ** α β : Type u x y : α hne : x ≠ y ht : ↑{x, y} = univ ⊢ {x, y} = univ ** simpa using ht ** case mpr α β : Type u ⊢ (∃ x y, x ≠ y ∧ {x, y} = univ) → ∃ t, ↑t = univ ∧ ∃ x y, x ≠ y ∧ t = {x, y} ** rintro ⟨x, y, hne, h⟩ ** case mpr.intro.intro.intro α β : Type u x y : α hne : x ≠ y h : {x, y} = univ ⊢ ∃ t, ↑t = univ ∧ ∃ x y, x ≠ y ∧ t = {x, y} ** exact ⟨{x, y}, by simpa using h, x, y, hne, rfl⟩ ** α β : Type u x y : α hne : x ≠ y h : {x, y} = univ ⊢ ↑{x, y} = univ ** simpa using h ** Qed
Cardinal.mk_eq_two_iff' ** α β : Type u x : α ⊢ #α = 2 ↔ ∃! y, y ≠ x ** rw [mk_eq_two_iff] ** α β : Type u x : α ⊢ (∃ x y, x ≠ y ∧ {x, y} = univ) ↔ ∃! y, y ≠ x ** constructor ** case mp α β : Type u x : α ⊢ (∃ x y, x ≠ y ∧ {x, y} = univ) → ∃! y, y ≠ x ** rintro ⟨a, b, hne, h⟩ ** case mp.intro.intro.intro α β : Type u x a b : α hne : a ≠ b h : {a, b} = univ ⊢ ∃! y, y ≠ x ** simp only [eq_univ_iff_forall, mem_insert_iff, mem_singleton_iff] at h ** case mp.intro.intro.intro α β : Type u x a b : α hne : a ≠ b h : ∀ (x : α), x = a ∨ x = b ⊢ ∃! y, y ≠ x ** rcases h x with (rfl | rfl) ** case mp.intro.intro.intro.inl α β : Type u x b : α hne : x ≠ b h : ∀ (x_1 : α), x_1 = x ∨ x_1 = b ⊢ ∃! y, y ≠ x case mp.intro.intro.intro.inr α β : Type u x a : α hne : a ≠ x h : ∀ (x_1 : α), x_1 = a ∨ x_1 = x ⊢ ∃! y, y ≠ x ** exacts [⟨b, hne.symm, fun z => (h z).resolve_left⟩, ⟨a, hne, fun z => (h z).resolve_right⟩] ** case mpr α β : Type u x : α ⊢ (∃! y, y ≠ x) → ∃ x y, x ≠ y ∧ {x, y} = univ ** rintro ⟨y, hne, hy⟩ ** case mpr.intro.intro α β : Type u x y : α hne : y ≠ x hy : ∀ (y_1 : α), (fun y => y ≠ x) y_1 → y_1 = y ⊢ ∃ x y, x ≠ y ∧ {x, y} = univ ** exact ⟨x, y, hne.symm, eq_univ_of_forall fun z => or_iff_not_imp_left.2 (hy z)⟩ ** Qed
Cardinal.exists_not_mem_of_length_lt ** α✝ β : Type u α : Type u_1 l : List α h : ↑(List.length l) < #α ⊢ ∃ z, ¬z ∈ l ** contrapose! h ** α✝ β : Type u α : Type u_1 l : List α h : ∀ (z : α), z ∈ l ⊢ #α ≤ ↑(List.length l) ** calc #α = #(Set.univ : Set α) := mk_univ.symm _ ≤ #l.toFinset := mk_le_mk_of_subset fun x _ => List.mem_toFinset.mpr (h x) _ = l.toFinset.card := Cardinal.mk_coe_finset _ ≤ l.length := Cardinal.natCast_le.mpr (List.toFinset_card_le l) ** Qed
Cardinal.three_le ** α✝ β : Type u α : Type u_1 h : 3 ≤ #α x y : α ⊢ ∃ z, z ≠ x ∧ z ≠ y ** have : ↑(3 : ℕ) ≤ #α ** case this α✝ β : Type u α : Type u_1 h : 3 ≤ #α x y : α ⊢ ↑3 ≤ #α α✝ β : Type u α : Type u_1 h : 3 ≤ #α x y : α this : ↑3 ≤ #α ⊢ ∃ z, z ≠ x ∧ z ≠ y ** simpa using h ** α✝ β : Type u α : Type u_1 h : 3 ≤ #α x y : α this : ↑3 ≤ #α ⊢ ∃ z, z ≠ x ∧ z ≠ y ** have : ↑(2 : ℕ) < #α ** case this α✝ β : Type u α : Type u_1 h : 3 ≤ #α x y : α this : ↑3 ≤ #α ⊢ ↑2 < #α α✝ β : Type u α : Type u_1 h : 3 ≤ #α x y : α this✝ : ↑3 ≤ #α this : ↑2 < #α ⊢ ∃ z, z ≠ x ∧ z ≠ y ** rwa [← succ_le_iff, ← Cardinal.nat_succ] ** α✝ β : Type u α : Type u_1 h : 3 ≤ #α x y : α this✝ : ↑3 ≤ #α this : ↑2 < #α ⊢ ∃ z, z ≠ x ∧ z ≠ y ** have := exists_not_mem_of_length_lt [x, y] this ** α✝ β : Type u α : Type u_1 h : 3 ≤ #α x y : α this✝¹ : ↑3 ≤ #α this✝ : ↑2 < #α this : ∃ z, ¬z ∈ [x, y] ⊢ ∃ z, z ≠ x ∧ z ≠ y ** simpa [not_or] using this ** Qed
Cardinal.le_powerlt ** α β : Type u b c a : Cardinal.{u} h : c < b ⊢ a ^ c ≤ a ^< b ** refine le_ciSup (f := fun y : Iio b => a^y) ?_ ⟨c, h⟩ ** α β : Type u b c a : Cardinal.{u} h : c < b ⊢ BddAbove (range fun y => a ^ ↑y) ** rw [← image_eq_range] ** α β : Type u b c a : Cardinal.{u} h : c < b ⊢ BddAbove (HPow.hPow a '' Iio b) ** exact bddAbove_image.{u, u} _ bddAbove_Iio ** Qed
Cardinal.powerlt_le ** α β : Type u a b c : Cardinal.{u} ⊢ a ^< b ≤ c ↔ ∀ (x : Cardinal.{u}), x < b → a ^ x ≤ c ** rw [powerlt, ciSup_le_iff'] ** α β : Type u a b c : Cardinal.{u} ⊢ (∀ (i : ↑(Iio b)), a ^ ↑i ≤ c) ↔ ∀ (x : Cardinal.{u}), x < b → a ^ x ≤ c ** simp ** case h α β : Type u a b c : Cardinal.{u} ⊢ BddAbove (range fun c => a ^ ↑c) ** rw [← image_eq_range] ** case h α β : Type u a b c : Cardinal.{u} ⊢ BddAbove (HPow.hPow a '' Iio b) ** exact bddAbove_image.{u, u} _ bddAbove_Iio ** Qed
Cardinal.zero_powerlt ** α β : Type u a : Cardinal.{u_1} h : a ≠ 0 ⊢ 0 ^< a = 1 ** apply (powerlt_le.2 fun c _ => zero_power_le _).antisymm ** α β : Type u a : Cardinal.{u_1} h : a ≠ 0 ⊢ 1 ≤ 0 ^< a ** rw [← power_zero] ** α β : Type u a : Cardinal.{u_1} h : a ≠ 0 ⊢ ?m.858249 ^ 0 ≤ 0 ^< a α β : Type u a : Cardinal.{u_1} h : a ≠ 0 ⊢ Cardinal.{u_1} ** exact le_powerlt 0 (pos_iff_ne_zero.2 h) ** Qed
Cardinal.powerlt_zero ** α β : Type u a : Cardinal.{u_1} ⊢ a ^< 0 = 0 ** convert Cardinal.iSup_of_empty _ ** case convert_3 α β : Type u a : Cardinal.{u_1} ⊢ IsEmpty ↑(Iio 0) ** exact Subtype.isEmpty_of_false fun x => mem_Iio.not.mpr (Cardinal.zero_le x).not_lt ** Qed
Cardinal.mk_le_of_module ** α β R : Type u E : Type v inst✝⁴ : AddCommGroup E inst✝³ : Ring R inst✝² : Module R E inst✝¹ : Nontrivial E inst✝ : NoZeroSMulDivisors R E ⊢ lift.{v, u} #R ≤ lift.{u, v} #E ** obtain ⟨x, hx⟩ : ∃ (x : E), x ≠ 0 := exists_ne 0 ** case intro α β R : Type u E : Type v inst✝⁴ : AddCommGroup E inst✝³ : Ring R inst✝² : Module R E inst✝¹ : Nontrivial E inst✝ : NoZeroSMulDivisors R E x : E hx : x ≠ 0 ⊢ lift.{v, u} #R ≤ lift.{u, v} #E ** have : Injective (fun k ↦ k • x) := smul_left_injective R hx ** case intro α β R : Type u E : Type v inst✝⁴ : AddCommGroup E inst✝³ : Ring R inst✝² : Module R E inst✝¹ : Nontrivial E inst✝ : NoZeroSMulDivisors R E x : E hx : x ≠ 0 this : Injective fun k => k • x ⊢ lift.{v, u} #R ≤ lift.{u, v} #E ** exact lift_mk_le_lift_mk_of_injective this ** Qed
Ordinal.lift_succ ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a : Ordinal.{v} ⊢ lift.{u, v} (succ a) = succ (lift.{u, v} a) ** rw [← add_one_eq_succ, lift_add, lift_one] ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a : Ordinal.{v} ⊢ lift.{u, v} a + 1 = succ (lift.{u, v} a) ** rfl ** Qed
Ordinal.add_left_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 ** simp only [le_antisymm_iff, add_le_add_iff_left] ** Qed
Ordinal.add_lt_add_iff_left' ** α : 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 [← not_le, ← not_le, add_le_add_iff_left] ** Qed
Ordinal.add_le_add_iff_right ** α : 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 ** simp ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} n : ℕ ⊢ a + ↑(n + 1) ≤ b + ↑(n + 1) ↔ a ≤ b ** simp only [nat_cast_succ, add_succ, add_succ, succ_le_succ_iff, add_le_add_iff_right] ** Qed
Ordinal.add_right_cancel ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} n : ℕ ⊢ a + ↑n = b + ↑n ↔ a = b ** simp only [le_antisymm_iff, add_le_add_iff_right] ** Qed
Ordinal.add_eq_zero_iff ** α✝ : Type u_1 β✝ : Type u_2 γ : Type u_3 r✝ : α✝ → α✝ → Prop s✝ : β✝ → β✝ → Prop t : γ → γ → Prop a b : Ordinal.{u_4} α : Type u_4 r : α → α → Prop x✝¹ : IsWellOrder α r β : Type u_4 s : β → β → Prop x✝ : IsWellOrder β s ⊢ type r + type s = 0 ↔ type r = 0 ∧ type s = 0 ** simp_rw [← type_sum_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 r : α → α → Prop x✝¹ : IsWellOrder α r β : Type u_4 s : β → β → Prop x✝ : IsWellOrder β s ⊢ IsEmpty (α ⊕ β) ↔ IsEmpty α ∧ IsEmpty β ** exact isEmpty_sum ** Qed
Ordinal.pred_succ ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u_4} ⊢ pred (succ o) = o ** have h : ∃ a, succ o = succ a := ⟨_, rfl⟩ ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u_4} h : ∃ a, succ o = succ a ⊢ pred (succ o) = o ** simpa only [pred, dif_pos h] using (succ_injective <| Classical.choose_spec h).symm ** Qed
Ordinal.pred_le_self ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u_4} h : ∃ a, o = succ a ⊢ pred o ≤ o ** let ⟨a, e⟩ := h ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u_4} h : ∃ a, o = succ a a : Ordinal.{u_4} e : o = succ a ⊢ pred o ≤ o ** rw [e, pred_succ] ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u_4} h : ∃ a, o = succ a a : Ordinal.{u_4} e : o = succ a ⊢ a ≤ succ a ** exact le_succ a ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u_4} h : ¬∃ a, o = succ a ⊢ pred o ≤ o ** rw [pred, dif_neg h] ** Qed
Ordinal.pred_eq_iff_not_succ ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u_4} e : pred o = o x✝ : ∃ a, o = succ a a : Ordinal.{u_4} e' : o = succ a ⊢ False ** rw [e', pred_succ] at e ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u_4} x✝ : ∃ a, o = succ a a : Ordinal.{u_4} e : a = succ a e' : o = succ a ⊢ False ** exact (lt_succ a).ne e ** Qed
Ordinal.pred_eq_iff_not_succ' ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u_4} ⊢ pred o = o ↔ ∀ (a : Ordinal.{u_4}), o ≠ succ a ** simpa using pred_eq_iff_not_succ ** Qed
Ordinal.pred_lt_iff_is_succ ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u_4} ⊢ pred o < o ↔ ¬pred o = o ** simp only [le_antisymm_iff, pred_le_self, true_and_iff, not_le] ** Qed
Ordinal.succ_pred_iff_is_succ ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u_4} x✝ : ∃ a, o = succ a a : Ordinal.{u_4} e : o = succ a ⊢ succ (pred o) = o ** simp only [e, pred_succ] ** Qed
Ordinal.lt_pred ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} h : ∃ a, b = succ a ⊢ a < pred b ↔ succ a < b ** let ⟨c, e⟩ := h ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} h : ∃ a, b = succ a c : Ordinal.{u_4} e : b = succ c ⊢ a < pred b ↔ succ a < b ** rw [e, pred_succ, succ_lt_succ_iff] ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} h : ¬∃ a, b = succ a ⊢ a < pred b ↔ succ a < b ** simp only [pred, dif_neg h, succ_lt_of_not_succ h] ** Qed
Ordinal.lift_is_succ ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{v} x✝ : ∃ a, lift.{u, v} o = succ a a : Ordinal.{max v u} h : lift.{u, v} o = succ a b : Ordinal.{v} e : lift.{u, v} b = a ⊢ lift.{?u.92282, v} o = lift.{?u.92282, v} (succ b) ** rw [h, ← e, lift_succ] ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{v} x✝ : ∃ a, o = succ a a : Ordinal.{v} h : o = succ a ⊢ lift.{u, v} o = succ (lift.{u, v} a) ** simp only [h, lift_succ] ** Qed
Ordinal.lift_pred ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{v} h : ∃ a, o = succ a ⊢ lift.{u, v} (pred o) = pred (lift.{u, v} o) ** cases' h with a e ** case intro α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o a : Ordinal.{v} e : o = succ a ⊢ lift.{u, v} (pred o) = pred (lift.{u, v} o) ** simp only [e, pred_succ, lift_succ] ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{v} h : ¬∃ a, o = succ a ⊢ lift.{u, v} (pred o) = pred (lift.{u, v} o) ** rw [pred_eq_iff_not_succ.2 h, pred_eq_iff_not_succ.2 (mt lift_is_succ.1 h)] ** Qed
Ordinal.lt_limit ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u_4} h : IsLimit o a : Ordinal.{u_4} ⊢ a < o ↔ ∃ x, x < o ∧ a < x ** simpa only [not_ball, not_le, bex_def] using not_congr (@limit_le _ h a) ** Qed
Ordinal.lift_isLimit ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u_4} ⊢ lift.{u_5, u_4} o = 0 ↔ o = 0 ** simpa only [lift_zero] using @lift_inj o 0 ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u_4} H : ∀ (a : Ordinal.{max u_4 u_5}), a < lift.{u_5, u_4} o → succ a < lift.{u_5, u_4} o a : Ordinal.{u_4} h : a < o ⊢ lift.{?u.96114, u_4} (succ a) < lift.{?u.96114, u_4} o ** simpa only [lift_succ] using H _ (lift_lt.2 h) ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u_4} H : ∀ (a : Ordinal.{u_4}), a < o → succ a < o a : Ordinal.{max u_4 u_5} h : a < lift.{u_5, u_4} o ⊢ succ a < lift.{u_5, u_4} o ** obtain ⟨a', rfl⟩ := lift_down h.le ** case intro α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u_4} H : ∀ (a : Ordinal.{u_4}), a < o → succ a < o a' : Ordinal.{u_4} h : lift.{u_5, u_4} a' < lift.{u_5, u_4} o ⊢ succ (lift.{u_5, u_4} a') < lift.{u_5, u_4} o ** rw [← lift_succ, lift_lt] ** case intro α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u_4} H : ∀ (a : Ordinal.{u_4}), a < o → succ a < o a' : Ordinal.{u_4} h : lift.{u_5, u_4} a' < lift.{u_5, u_4} o ⊢ succ a' < o ** exact H a' (lift_lt.1 h) ** Qed
Ordinal.IsLimit.one_lt ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u_4} h : IsLimit o ⊢ 1 < o ** simpa only [succ_zero] using h.2 _ h.pos ** Qed
Ordinal.limitRecOn_zero ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop C : Ordinal.{u_4} → Sort u_5 H₁ : C 0 H₂ : (o : Ordinal.{u_4}) → C o → C (succ o) H₃ : (o : Ordinal.{u_4}) → IsLimit o → ((o' : Ordinal.{u_4}) → o' < o → C o') → C o ⊢ limitRecOn 0 H₁ H₂ H₃ = H₁ ** rw [limitRecOn, lt_wf.fix_eq, dif_pos rfl] ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop C : Ordinal.{u_4} → Sort u_5 H₁ : C 0 H₂ : (o : Ordinal.{u_4}) → C o → C (succ o) H₃ : (o : Ordinal.{u_4}) → IsLimit o → ((o' : Ordinal.{u_4}) → o' < o → C o') → C o ⊢ Eq.mpr (_ : C 0 = C 0) H₁ = H₁ ** rfl ** Qed
Ordinal.limitRecOn_succ ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop C : Ordinal.{u_4} → Sort u_5 o : Ordinal.{u_4} H₁ : C 0 H₂ : (o : Ordinal.{u_4}) → C o → C (succ o) H₃ : (o : Ordinal.{u_4}) → IsLimit o → ((o' : Ordinal.{u_4}) → o' < o → C o') → C o ⊢ limitRecOn (succ o) H₁ H₂ H₃ = H₂ o (limitRecOn o H₁ H₂ H₃) ** have h : ∃ a, succ o = succ a := ⟨_, rfl⟩ ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop C : Ordinal.{u_4} → Sort u_5 o : Ordinal.{u_4} H₁ : C 0 H₂ : (o : Ordinal.{u_4}) → C o → C (succ o) H₃ : (o : Ordinal.{u_4}) → IsLimit o → ((o' : Ordinal.{u_4}) → o' < o → C o') → C o h : ∃ a, succ o = succ a ⊢ limitRecOn (succ o) H₁ H₂ H₃ = H₂ o (limitRecOn o H₁ H₂ H₃) ** rw [limitRecOn, lt_wf.fix_eq, dif_neg (succ_ne_zero o), dif_pos h] ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop C : Ordinal.{u_4} → Sort u_5 o : Ordinal.{u_4} H₁ : C 0 H₂ : (o : Ordinal.{u_4}) → C o → C (succ o) H₃ : (o : Ordinal.{u_4}) → IsLimit o → ((o' : Ordinal.{u_4}) → o' < o → C o') → C o h : ∃ a, succ o = succ a ⊢ Eq.mpr (_ : C (succ o) = C (succ (pred (succ o)))) (H₂ (pred (succ o)) ((fun y x => WellFounded.fix lt_wf (fun o IH => if o0 : o = 0 then Eq.mpr (_ : C o = C 0) H₁ else if h : ∃ a, o = succ a then Eq.mpr (_ : C o = C (succ (pred o))) (H₂ (pred o) (IH (pred o) (_ : pred o < o))) else H₃ o (_ : o ≠ 0 ∧ ∀ (a : Ordinal.{u_4}), a < o → succ a < o) IH) y) (pred (succ o)) (_ : pred (succ o) < succ o))) = H₂ o (limitRecOn o H₁ H₂ H₃) ** generalize limitRecOn.proof_2 (succ o) h = h₂ ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop C : Ordinal.{u_4} → Sort u_5 o : Ordinal.{u_4} H₁ : C 0 H₂ : (o : Ordinal.{u_4}) → C o → C (succ o) H₃ : (o : Ordinal.{u_4}) → IsLimit o → ((o' : Ordinal.{u_4}) → o' < o → C o') → C o h : ∃ a, succ o = succ a h₂ : C (succ o) = C (succ (pred (succ o))) ⊢ Eq.mpr h₂ (H₂ (pred (succ o)) ((fun y x => WellFounded.fix lt_wf (fun o IH => if o0 : o = 0 then Eq.mpr (_ : C o = C 0) H₁ else if h : ∃ a, o = succ a then Eq.mpr (_ : C o = C (succ (pred o))) (H₂ (pred o) (IH (pred o) (_ : pred o < o))) else H₃ o (_ : o ≠ 0 ∧ ∀ (a : Ordinal.{u_4}), a < o → succ a < o) IH) y) (pred (succ o)) (_ : pred (succ o) < succ o))) = H₂ o (limitRecOn o H₁ H₂ H₃) ** generalize limitRecOn.proof_3 (succ o) h = h₃ ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop C : Ordinal.{u_4} → Sort u_5 o : Ordinal.{u_4} H₁ : C 0 H₂ : (o : Ordinal.{u_4}) → C o → C (succ o) H₃ : (o : Ordinal.{u_4}) → IsLimit o → ((o' : Ordinal.{u_4}) → o' < o → C o') → C o h : ∃ a, succ o = succ a h₂ : C (succ o) = C (succ (pred (succ o))) h₃ : pred (succ o) < succ o ⊢ Eq.mpr h₂ (H₂ (pred (succ o)) ((fun y x => WellFounded.fix lt_wf (fun o IH => if o0 : o = 0 then Eq.mpr (_ : C o = C 0) H₁ else if h : ∃ a, o = succ a then Eq.mpr (_ : C o = C (succ (pred o))) (H₂ (pred o) (IH (pred o) (_ : pred o < o))) else H₃ o (_ : o ≠ 0 ∧ ∀ (a : Ordinal.{u_4}), a < o → succ a < o) IH) y) (pred (succ o)) h₃)) = H₂ o (limitRecOn o H₁ H₂ H₃) ** revert h₂ h₃ ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop C : Ordinal.{u_4} → Sort u_5 o : Ordinal.{u_4} H₁ : C 0 H₂ : (o : Ordinal.{u_4}) → C o → C (succ o) H₃ : (o : Ordinal.{u_4}) → IsLimit o → ((o' : Ordinal.{u_4}) → o' < o → C o') → C o h : ∃ a, succ o = succ a ⊢ ∀ (h₂ : C (succ o) = C (succ (pred (succ o)))) (h₃ : pred (succ o) < succ o), Eq.mpr h₂ (H₂ (pred (succ o)) ((fun y x => WellFounded.fix lt_wf (fun o IH => if o0 : o = 0 then Eq.mpr (_ : C o = C 0) H₁ else if h : ∃ a, o = succ a then Eq.mpr (_ : C o = C (succ (pred o))) (H₂ (pred o) (IH (pred o) (_ : pred o < o))) else H₃ o (_ : o ≠ 0 ∧ ∀ (a : Ordinal.{u_4}), a < o → succ a < o) IH) y) (pred (succ o)) h₃)) = H₂ o (limitRecOn o H₁ H₂ H₃) ** generalize e : pred (succ o) = o' ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop C : Ordinal.{u_4} → Sort u_5 o : Ordinal.{u_4} H₁ : C 0 H₂ : (o : Ordinal.{u_4}) → C o → C (succ o) H₃ : (o : Ordinal.{u_4}) → IsLimit o → ((o' : Ordinal.{u_4}) → o' < o → C o') → C o h : ∃ a, succ o = succ a o' : Ordinal.{u_4} e : pred (succ o) = o' ⊢ ∀ (h₂ : C (succ o) = C (succ o')) (h₃ : o' < succ o), Eq.mpr h₂ (H₂ o' ((fun y x => WellFounded.fix lt_wf (fun o IH => if o0 : o = 0 then Eq.mpr (_ : C o = C 0) H₁ else if h : ∃ a, o = succ a then Eq.mpr (_ : C o = C (succ (pred o))) (H₂ (pred o) (IH (pred o) (_ : pred o < o))) else H₃ o (_ : o ≠ 0 ∧ ∀ (a : Ordinal.{u_4}), a < o → succ a < o) IH) y) o' h₃)) = H₂ o (limitRecOn o H₁ H₂ H₃) ** intros ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop C : Ordinal.{u_4} → Sort u_5 o : Ordinal.{u_4} H₁ : C 0 H₂ : (o : Ordinal.{u_4}) → C o → C (succ o) H₃ : (o : Ordinal.{u_4}) → IsLimit o → ((o' : Ordinal.{u_4}) → o' < o → C o') → C o h : ∃ a, succ o = succ a o' : Ordinal.{u_4} e : pred (succ o) = o' h₂✝ : C (succ o) = C (succ o') h₃✝ : o' < succ o ⊢ Eq.mpr h₂✝ (H₂ o' ((fun y x => WellFounded.fix lt_wf (fun o IH => if o0 : o = 0 then Eq.mpr (_ : C o = C 0) H₁ else if h : ∃ a, o = succ a then Eq.mpr (_ : C o = C (succ (pred o))) (H₂ (pred o) (IH (pred o) (_ : pred o < o))) else H₃ o (_ : o ≠ 0 ∧ ∀ (a : Ordinal.{u_4}), a < o → succ a < o) IH) y) o' h₃✝)) = H₂ o (limitRecOn o H₁ H₂ H₃) ** rw [pred_succ] at e ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop C : Ordinal.{u_4} → Sort u_5 o : Ordinal.{u_4} H₁ : C 0 H₂ : (o : Ordinal.{u_4}) → C o → C (succ o) H₃ : (o : Ordinal.{u_4}) → IsLimit o → ((o' : Ordinal.{u_4}) → o' < o → C o') → C o h : ∃ a, succ o = succ a o' : Ordinal.{u_4} e : o = o' h₂✝ : C (succ o) = C (succ o') h₃✝ : o' < succ o ⊢ Eq.mpr h₂✝ (H₂ o' ((fun y x => WellFounded.fix lt_wf (fun o IH => if o0 : o = 0 then Eq.mpr (_ : C o = C 0) H₁ else if h : ∃ a, o = succ a then Eq.mpr (_ : C o = C (succ (pred o))) (H₂ (pred o) (IH (pred o) (_ : pred o < o))) else H₃ o (_ : o ≠ 0 ∧ ∀ (a : Ordinal.{u_4}), a < o → succ a < o) IH) y) o' h₃✝)) = H₂ o (limitRecOn o H₁ H₂ H₃) ** subst o' ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop C : Ordinal.{u_4} → Sort u_5 o : Ordinal.{u_4} H₁ : C 0 H₂ : (o : Ordinal.{u_4}) → C o → C (succ o) H₃ : (o : Ordinal.{u_4}) → IsLimit o → ((o' : Ordinal.{u_4}) → o' < o → C o') → C o h : ∃ a, succ o = succ a h₂✝ : C (succ o) = C (succ o) h₃✝ : o < succ o ⊢ Eq.mpr h₂✝ (H₂ o ((fun y x => WellFounded.fix lt_wf (fun o IH => if o0 : o = 0 then Eq.mpr (_ : C o = C 0) H₁ else if h : ∃ a, o = succ a then Eq.mpr (_ : C o = C (succ (pred o))) (H₂ (pred o) (IH (pred o) (_ : pred o < o))) else H₃ o (_ : o ≠ 0 ∧ ∀ (a : Ordinal.{u_4}), a < o → succ a < o) IH) y) o h₃✝)) = H₂ o (limitRecOn o H₁ H₂ H₃) ** rfl ** Qed
Ordinal.limitRecOn_limit ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop C : Ordinal.{u_4} → Sort u_5 o : Ordinal.{u_4} H₁ : C 0 H₂ : (o : Ordinal.{u_4}) → C o → C (succ o) H₃ : (o : Ordinal.{u_4}) → IsLimit o → ((o' : Ordinal.{u_4}) → o' < o → C o') → C o h : IsLimit o ⊢ limitRecOn o H₁ H₂ H₃ = H₃ o h fun x _h => limitRecOn x H₁ H₂ H₃ ** rw [limitRecOn, lt_wf.fix_eq, dif_neg h.1, dif_neg (not_succ_of_isLimit h)] ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop C : Ordinal.{u_4} → Sort u_5 o : Ordinal.{u_4} H₁ : C 0 H₂ : (o : Ordinal.{u_4}) → C o → C (succ o) H₃ : (o : Ordinal.{u_4}) → IsLimit o → ((o' : Ordinal.{u_4}) → o' < o → C o') → C o h : IsLimit o ⊢ (H₃ o (_ : o ≠ 0 ∧ ∀ (a : Ordinal.{u_4}), a < o → succ a < o) fun y x => WellFounded.fix lt_wf (fun o IH => if o0 : o = 0 then Eq.mpr (_ : C o = C 0) H₁ else if h : ∃ a, o = succ a then Eq.mpr (_ : C o = C (succ (pred o))) (H₂ (pred o) (IH (pred o) (_ : pred o < o))) else H₃ o (_ : o ≠ 0 ∧ ∀ (a : Ordinal.{u_4}), a < o → succ a < o) IH) y) = H₃ o h fun x _h => limitRecOn x H₁ H₂ H₃ ** rfl ** Qed
Ordinal.enum_succ_eq_top ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{?u.103680} ⊢ o < type fun x x_1 => x < x_1 ** rw [type_lt] ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{?u.103680} ⊢ o < succ o ** exact lt_succ o ** Qed
Ordinal.has_succ_of_type_succ_lt ** α✝ : Type u_1 β : Type u_2 γ : Type u_3 r✝ : α✝ → α✝ → Prop s : β → β → Prop t : γ → γ → Prop α : Type u_4 r : α → α → Prop wo : IsWellOrder α r h : ∀ (a : Ordinal.{u_4}), a < type r → succ a < type r x : α ⊢ ∃ y, r x y ** use enum r (succ (typein r x)) (h _ (typein_lt_type r x)) ** case h α✝ : Type u_1 β : Type u_2 γ : Type u_3 r✝ : α✝ → α✝ → Prop s : β → β → Prop t : γ → γ → Prop α : Type u_4 r : α → α → Prop wo : IsWellOrder α r h : ∀ (a : Ordinal.{u_4}), a < type r → succ a < type r x : α ⊢ r x (enum r (succ (typein r x)) (_ : succ (typein r x) < type r)) ** convert (enum_lt_enum (typein_lt_type r x) (h _ (typein_lt_type r x))).mpr (lt_succ _) ** case h.e'_1 α✝ : Type u_1 β : Type u_2 γ : Type u_3 r✝ : α✝ → α✝ → Prop s : β → β → Prop t : γ → γ → Prop α : Type u_4 r : α → α → Prop wo : IsWellOrder α r h : ∀ (a : Ordinal.{u_4}), a < type r → succ a < type r x : α ⊢ x = enum r (typein r x) (_ : typein r x < type r) ** rw [enum_typein] ** Qed
Ordinal.out_no_max_of_succ_lt ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u_4} ho : ∀ (a : Ordinal.{u_4}), a < o → succ a < o ⊢ ∀ (a : Ordinal.{u_4}), (a < type fun a b => a < b) → succ a < type fun a b => a < b ** rwa [type_lt] ** Qed
Ordinal.bounded_singleton ** α : Type u_1 β : Type u_2 γ : Type u_3 r✝ : α → α → Prop s : β → β → Prop t : γ → γ → Prop r : α → α → Prop inst✝ : IsWellOrder α r hr : IsLimit (type r) x : α ⊢ Bounded r {x} ** refine' ⟨enum r (succ (typein r x)) (hr.2 _ (typein_lt_type r x)), _⟩ ** α : Type u_1 β : Type u_2 γ : Type u_3 r✝ : α → α → Prop s : β → β → Prop t : γ → γ → Prop r : α → α → Prop inst✝ : IsWellOrder α r hr : IsLimit (type r) x : α ⊢ ∀ (b : α), b ∈ {x} → r b (enum r (succ (typein r x)) (_ : succ (typein r x) < type r)) ** intro b hb ** α : Type u_1 β : Type u_2 γ : Type u_3 r✝ : α → α → Prop s : β → β → Prop t : γ → γ → Prop r : α → α → Prop inst✝ : IsWellOrder α r hr : IsLimit (type r) x b : α hb : b ∈ {x} ⊢ r b (enum r (succ (typein r x)) (_ : succ (typein r x) < type r)) ** rw [mem_singleton_iff.1 hb] ** α : Type u_1 β : Type u_2 γ : Type u_3 r✝ : α → α → Prop s : β → β → Prop t : γ → γ → Prop r : α → α → Prop inst✝ : IsWellOrder α r hr : IsLimit (type r) x b : α hb : b ∈ {x} ⊢ r x (enum r (succ (typein r x)) (_ : succ (typein r x) < type r)) ** nth_rw 1 [← enum_typein r x] ** α : Type u_1 β : Type u_2 γ : Type u_3 r✝ : α → α → Prop s : β → β → Prop t : γ → γ → Prop r : α → α → Prop inst✝ : IsWellOrder α r hr : IsLimit (type r) x b : α hb : b ∈ {x} ⊢ r (enum r (typein r x) (_ : typein r x < type r)) (enum r (succ (typein r x)) (_ : succ (typein r x) < type r)) ** rw [@enum_lt_enum _ r] ** α : Type u_1 β : Type u_2 γ : Type u_3 r✝ : α → α → Prop s : β → β → Prop t : γ → γ → Prop r : α → α → Prop inst✝ : IsWellOrder α r hr : IsLimit (type r) x b : α hb : b ∈ {x} ⊢ typein r x < succ (typein r x) ** apply lt_succ ** Qed
Ordinal.type_subrel_lt ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u} ⊢ type (Subrel (fun x x_1 => x < x_1) {o' | o' < o}) = lift.{u + 1, u} o ** refine' Quotient.inductionOn o _ ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u} ⊢ ∀ (a : WellOrder), type (Subrel (fun x x_1 => x < x_1) {o' | o' < Quotient.mk isEquivalent a}) = lift.{u + 1, u} (Quotient.mk isEquivalent a) ** rintro ⟨α, r, wo⟩ ** case mk α✝ : Type u_1 β : Type u_2 γ : Type u_3 r✝ : α✝ → α✝ → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u} α : Type u r : α → α → Prop wo : IsWellOrder α r ⊢ type (Subrel (fun x x_1 => x < x_1) {o' | o' < Quotient.mk isEquivalent { α := α, r := r, wo := wo }}) = lift.{u + 1, u} (Quotient.mk isEquivalent { α := α, r := r, wo := wo }) ** apply Quotient.sound ** case mk.a α✝ : Type u_1 β : Type u_2 γ : Type u_3 r✝ : α✝ → α✝ → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u} α : Type u r : α → α → Prop wo : IsWellOrder α r ⊢ { α := ↑{o' | o' < Quotient.mk isEquivalent { α := α, r := r, wo := wo }}, r := Subrel (fun x x_1 => x < x_1) {o' | o' < Quotient.mk isEquivalent { α := α, r := r, wo := wo }}, wo := (_ : IsWellOrder (↑{o' | o' < Quotient.mk isEquivalent { α := α, r := r, wo := wo }}) (Subrel (fun x x_1 => x < x_1) {o' | o' < Quotient.mk isEquivalent { α := α, r := r, wo := wo }})) } ≈ { α := ULift.{u + 1, u} { α := α, r := r, wo := wo }.α, r := ULift.down ⁻¹'o { α := α, r := r, wo := wo }.r, wo := (_ : IsWellOrder (ULift.{u + 1, u} { α := α, r := r, wo := wo }.α) (ULift.down ⁻¹'o { α := α, r := r, wo := wo }.r)) } ** constructor ** case mk.a.val α✝ : Type u_1 β : Type u_2 γ : Type u_3 r✝ : α✝ → α✝ → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u} α : Type u r : α → α → Prop wo : IsWellOrder α r ⊢ Subrel (fun x x_1 => x < x_1) {o' | o' < Quotient.mk isEquivalent { α := α, r := r, wo := wo }} ≃r ULift.down ⁻¹'o { α := α, r := r, wo := wo }.r ** refine' ((RelIso.preimage Equiv.ulift r).trans (enumIso r).symm).symm ** Qed
Ordinal.mk_initialSeg ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop o : Ordinal.{u} ⊢ #↑{o' | o' < o} = Cardinal.lift.{u + 1, u} (card o) ** rw [lift_card, ← type_subrel_lt, card_type] ** Qed
Ordinal.IsNormal.limit_lt ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop f : Ordinal.{u_4} → Ordinal.{u_5} H : IsNormal f o : Ordinal.{u_4} h : IsLimit o a : Ordinal.{u_5} ⊢ ¬a < f o ↔ ¬∃ b, b < o ∧ a < f b ** simpa only [exists_prop, not_exists, not_and, not_lt] using H.2 _ h a ** Qed
Ordinal.IsNormal.inj ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop f : Ordinal.{u_4} → Ordinal.{u_5} H : IsNormal f a b : Ordinal.{u_4} ⊢ f a = f b ↔ a = b ** simp only [le_antisymm_iff, H.le_iff] ** Qed
Ordinal.IsNormal.le_set ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop f : Ordinal.{u_4} → Ordinal.{u_5} o : Ordinal.{u_5} H : IsNormal f p : Set Ordinal.{u_4} p0 : Set.Nonempty p b : Ordinal.{u_4} H₂ : ∀ (o : Ordinal.{u_4}), b ≤ o ↔ ∀ (a : Ordinal.{u_4}), a ∈ p → a ≤ o h : ∀ (a : Ordinal.{u_4}), a ∈ p → f a ≤ o ⊢ f b ≤ o ** induction b using limitRecOn with | H₁ => cases' p0 with x px have := Ordinal.le_zero.1 ((H₂ _).1 (Ordinal.zero_le _) _ px) rw [this] at px exact h _ px | H₂ S _ => rcases not_ball.1 (mt (H₂ S).2 <| (lt_succ S).not_le) with ⟨a, h₁, h₂⟩ exact (H.le_iff.2 <| succ_le_of_lt <| not_le.1 h₂).trans (h _ h₁) | H₃ S L _ => refine' (H.2 _ L _).2 fun a h' => _ rcases not_ball.1 (mt (H₂ a).2 h'.not_le) with ⟨b, h₁, h₂⟩ exact (H.le_iff.2 <| (not_le.1 h₂).le).trans (h _ h₁) ** case H₁ α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop f : Ordinal.{u_4} → Ordinal.{u_5} o : Ordinal.{u_5} H : IsNormal f p : Set Ordinal.{u_4} p0 : Set.Nonempty p h : ∀ (a : Ordinal.{u_4}), a ∈ p → f a ≤ o H₂ : ∀ (o : Ordinal.{u_4}), 0 ≤ o ↔ ∀ (a : Ordinal.{u_4}), a ∈ p → a ≤ o ⊢ f 0 ≤ o ** cases' p0 with x px ** case H₁.intro α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop f : Ordinal.{u_4} → Ordinal.{u_5} o : Ordinal.{u_5} H : IsNormal f p : Set Ordinal.{u_4} h : ∀ (a : Ordinal.{u_4}), a ∈ p → f a ≤ o H₂ : ∀ (o : Ordinal.{u_4}), 0 ≤ o ↔ ∀ (a : Ordinal.{u_4}), a ∈ p → a ≤ o x : Ordinal.{u_4} px : x ∈ p ⊢ f 0 ≤ o ** have := Ordinal.le_zero.1 ((H₂ _).1 (Ordinal.zero_le _) _ px) ** case H₁.intro α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop f : Ordinal.{u_4} → Ordinal.{u_5} o : Ordinal.{u_5} H : IsNormal f p : Set Ordinal.{u_4} h : ∀ (a : Ordinal.{u_4}), a ∈ p → f a ≤ o H₂ : ∀ (o : Ordinal.{u_4}), 0 ≤ o ↔ ∀ (a : Ordinal.{u_4}), a ∈ p → a ≤ o x : Ordinal.{u_4} px : x ∈ p this : x = 0 ⊢ f 0 ≤ o ** rw [this] at px ** case H₁.intro α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop f : Ordinal.{u_4} → Ordinal.{u_5} o : Ordinal.{u_5} H : IsNormal f p : Set Ordinal.{u_4} h : ∀ (a : Ordinal.{u_4}), a ∈ p → f a ≤ o H₂ : ∀ (o : Ordinal.{u_4}), 0 ≤ o ↔ ∀ (a : Ordinal.{u_4}), a ∈ p → a ≤ o x : Ordinal.{u_4} px : 0 ∈ p this : x = 0 ⊢ f 0 ≤ o ** exact h _ px ** case H₂ α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop f : Ordinal.{u_4} → Ordinal.{u_5} o : Ordinal.{u_5} H : IsNormal f p : Set Ordinal.{u_4} p0 : Set.Nonempty p h : ∀ (a : Ordinal.{u_4}), a ∈ p → f a ≤ o S : Ordinal.{u_4} a✝ : (∀ (o : Ordinal.{u_4}), S ≤ o ↔ ∀ (a : Ordinal.{u_4}), a ∈ p → a ≤ o) → f S ≤ o H₂ : ∀ (o : Ordinal.{u_4}), succ S ≤ o ↔ ∀ (a : Ordinal.{u_4}), a ∈ p → a ≤ o ⊢ f (succ S) ≤ o ** rcases not_ball.1 (mt (H₂ S).2 <| (lt_succ S).not_le) with ⟨a, h₁, h₂⟩ ** case H₂.intro.intro α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop f : Ordinal.{u_4} → Ordinal.{u_5} o : Ordinal.{u_5} H : IsNormal f p : Set Ordinal.{u_4} p0 : Set.Nonempty p h : ∀ (a : Ordinal.{u_4}), a ∈ p → f a ≤ o S : Ordinal.{u_4} a✝ : (∀ (o : Ordinal.{u_4}), S ≤ o ↔ ∀ (a : Ordinal.{u_4}), a ∈ p → a ≤ o) → f S ≤ o H₂ : ∀ (o : Ordinal.{u_4}), succ S ≤ o ↔ ∀ (a : Ordinal.{u_4}), a ∈ p → a ≤ o a : Ordinal.{u_4} h₁ : a ∈ p h₂ : ¬a ≤ S ⊢ f (succ S) ≤ o ** exact (H.le_iff.2 <| succ_le_of_lt <| not_le.1 h₂).trans (h _ h₁) ** case H₃ α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop f : Ordinal.{u_4} → Ordinal.{u_5} o : Ordinal.{u_5} H : IsNormal f p : Set Ordinal.{u_4} p0 : Set.Nonempty p h : ∀ (a : Ordinal.{u_4}), a ∈ p → f a ≤ o S : Ordinal.{u_4} L : IsLimit S a✝ : ∀ (o' : Ordinal.{u_4}), o' < S → (∀ (o : Ordinal.{u_4}), o' ≤ o ↔ ∀ (a : Ordinal.{u_4}), a ∈ p → a ≤ o) → f o' ≤ o H₂ : ∀ (o : Ordinal.{u_4}), S ≤ o ↔ ∀ (a : Ordinal.{u_4}), a ∈ p → a ≤ o ⊢ f S ≤ o ** refine' (H.2 _ L _).2 fun a h' => _ ** case H₃ α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop f : Ordinal.{u_4} → Ordinal.{u_5} o : Ordinal.{u_5} H : IsNormal f p : Set Ordinal.{u_4} p0 : Set.Nonempty p h : ∀ (a : Ordinal.{u_4}), a ∈ p → f a ≤ o S : Ordinal.{u_4} L : IsLimit S a✝ : ∀ (o' : Ordinal.{u_4}), o' < S → (∀ (o : Ordinal.{u_4}), o' ≤ o ↔ ∀ (a : Ordinal.{u_4}), a ∈ p → a ≤ o) → f o' ≤ o H₂ : ∀ (o : Ordinal.{u_4}), S ≤ o ↔ ∀ (a : Ordinal.{u_4}), a ∈ p → a ≤ o a : Ordinal.{u_4} h' : a < S ⊢ f a ≤ o ** rcases not_ball.1 (mt (H₂ a).2 h'.not_le) with ⟨b, h₁, h₂⟩ ** case H₃.intro.intro α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop f : Ordinal.{u_4} → Ordinal.{u_5} o : Ordinal.{u_5} H : IsNormal f p : Set Ordinal.{u_4} p0 : Set.Nonempty p h : ∀ (a : Ordinal.{u_4}), a ∈ p → f a ≤ o S : Ordinal.{u_4} L : IsLimit S a✝ : ∀ (o' : Ordinal.{u_4}), o' < S → (∀ (o : Ordinal.{u_4}), o' ≤ o ↔ ∀ (a : Ordinal.{u_4}), a ∈ p → a ≤ o) → f o' ≤ o H₂ : ∀ (o : Ordinal.{u_4}), S ≤ o ↔ ∀ (a : Ordinal.{u_4}), a ∈ p → a ≤ o a : Ordinal.{u_4} h' : a < S b : Ordinal.{u_4} h₁ : b ∈ p h₂ : ¬b ≤ a ⊢ f a ≤ o ** exact (H.le_iff.2 <| (not_le.1 h₂).le).trans (h _ h₁) ** Qed
Ordinal.IsNormal.le_set' ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop f : Ordinal.{u_4} → Ordinal.{u_5} o : Ordinal.{u_5} H : IsNormal f p : Set α p0 : Set.Nonempty p g : α → Ordinal.{u_4} b : Ordinal.{u_4} H₂ : ∀ (o : Ordinal.{u_4}), b ≤ o ↔ ∀ (a : α), a ∈ p → g a ≤ o ⊢ f b ≤ o ↔ ∀ (a : α), a ∈ p → f (g a) ≤ o ** simpa [H₂] using H.le_set (g '' p) (p0.image g) b ** Qed
Ordinal.add_le_of_limit ** 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 ** intro l ** 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 l : c < type r + type s ⊢ ∀ (x : β), Sum.Lex r s (Sum.inr x) (enum (Sum.Lex r s) c l) ** intro x ** 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 l : c < type r + type s x : β ⊢ Sum.Lex r s (Sum.inr x) (enum (Sum.Lex r s) c l) ** rw [← typein_lt_typein (Sum.Lex r s), typein_enum] ** 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 l : c < type r + type s x : β ⊢ typein (Sum.Lex r s) (Sum.inr x) < c ** have := H _ (h.2 _ (typein_lt_type s x)) ** 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 l : c < type r + type s x : β this : type r + succ (typein s x) ≤ c ⊢ typein (Sum.Lex r s) (Sum.inr x) < c ** rw [add_succ, succ_le_iff] at this ** 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 l : c < type r + type s x : β this : type r + typein s x < c ⊢ typein (Sum.Lex r s) (Sum.inr x) < 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 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 l : c < type r + type s this : ∀ (x : β), Sum.Lex r s (Sum.inr x) (enum (Sum.Lex r s) c l) ⊢ False ** revert this ** α✝ : 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 l : c < type r + type s ⊢ (∀ (x : β), Sum.Lex r s (Sum.inr x) (enum (Sum.Lex r s) c l)) → False ** cases' enum _ _ l with x x <;> intro this ** case inl α✝ : 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 l : c < type r + type s x : α this : ∀ (x_1 : β), Sum.Lex r s (Sum.inr x_1) (Sum.inl x) ⊢ False ** cases this (enum s 0 h.pos) ** case inr α✝ : 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 l : c < type r + type s x : β this : ∀ (x_1 : β), Sum.Lex r s (Sum.inr x_1) (Sum.inr x) ⊢ False ** exact irrefl _ (this _) ** case H.H.refine'_1 α✝ : 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 l : c < type r + type s x : β this : type r + typein s x < c a : ↑{b | Sum.Lex r s b (Sum.inr x)} ⊢ α ⊕ ↑{b | s b x} ** rcases a with ⟨a | b, h⟩ ** case H.H.refine'_1.mk.inl α✝ : 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 l : c < type r + type s x : β this : type r + typein s x < c a : α h : Sum.inl a ∈ {b | Sum.Lex r s b (Sum.inr x)} ⊢ α ⊕ ↑{b | s b x} ** exact Sum.inl a ** case H.H.refine'_1.mk.inr α✝ : 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 l : c < type r + type s x : β this : type r + typein s x < c b : β h : Sum.inr b ∈ {b | Sum.Lex r s b (Sum.inr x)} ⊢ α ⊕ ↑{b | s b x} ** exact Sum.inr ⟨b, by cases h; assumption⟩ ** α✝ : 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 l : c < type r + type s x : β this : type r + typein s x < c b : β h : Sum.inr b ∈ {b | Sum.Lex r s b (Sum.inr x)} ⊢ b ∈ {b | s b x} ** cases h ** case inr α✝ : 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 l : c < type r + type s x : β this : type r + typein s x < c b : β h✝ : s b x ⊢ b ∈ {b | s b x} ** assumption ** case H.H.refine'_2 α✝ : 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 l : c < type r + type s x : β this : type r + typein s x < c a b : ↑{b | Sum.Lex r s b (Sum.inr x)} ⊢ Subrel (Sum.Lex r s) {b | Sum.Lex r s b (Sum.inr x)} a b → Sum.Lex r (Subrel s {b | s b x}) ((fun a => Subtype.casesOn a fun val h => Sum.casesOn (motive := fun x_1 => x_1 ∈ {b | Sum.Lex r s b (Sum.inr x)} → α ⊕ ↑{b | s b x}) val (fun a h => Sum.inl a) (fun b h => Sum.inr { val := b, property := (_ : b ∈ {b | s b x}) }) h) a) ((fun a => Subtype.casesOn a fun val h => Sum.casesOn (motive := fun x_1 => x_1 ∈ {b | Sum.Lex r s b (Sum.inr x)} → α ⊕ ↑{b | s b x}) val (fun a h => Sum.inl a) (fun b h => Sum.inr { val := b, property := (_ : b ∈ {b | s b x}) }) h) b) ** rcases a with ⟨a | a, h₁⟩ <;> rcases b with ⟨b | b, h₂⟩ <;> cases h₁ <;> cases h₂ <;> rintro ⟨⟩ <;> constructor <;> assumption ** Qed
Ordinal.add_sub_cancel_of_le ** α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} h : b ≤ a ⊢ b + (a - b) ≤ a ** rcases zero_or_succ_or_limit (a - b) with (e | ⟨c, e⟩ | l) ** case inl α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} h : b ≤ a e : a - b = 0 ⊢ b + (a - b) ≤ a ** simp only [e, add_zero, h] ** case inr.inl.intro α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} h : b ≤ a c : Ordinal.{u_4} e : a - b = succ c ⊢ b + (a - b) ≤ a ** rw [e, add_succ, succ_le_iff, ← lt_sub, e] ** case inr.inl.intro α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} h : b ≤ a c : Ordinal.{u_4} e : a - b = succ c ⊢ c < succ c ** exact lt_succ c ** case inr.inr α : Type u_1 β : Type u_2 γ : Type u_3 r : α → α → Prop s : β → β → Prop t : γ → γ → Prop a b : Ordinal.{u_4} h : b ≤ a l : IsLimit (a - b) ⊢ b + (a - b) ≤ a ** exact (add_le_of_limit l).2 fun c l => (lt_sub.1 l).le ** Qed