formal
stringlengths
41
427k
informal
stringclasses
1 value
Ordinal.opow_mul_add_lt_opow_mul_succ ** b u w v : Ordinal.{u_1} hw : w < b ^ u ⊢ b ^ u * v + w < b ^ u * succ v ** rwa [mul_succ, add_lt_add_iff_left] ** Qed
Ordinal.opow_mul_add_lt_opow_succ ** b u v w : Ordinal.{u_1} hvb : v < b hw : w < b ^ u ⊢ b ^ u * v + w < b ^ succ u ** convert (opow_mul_add_lt_opow_mul_succ v hw).trans_le (mul_le_mul_left' (succ_le_of_lt hvb) _) using 1 ** case h.e'_4 b u v w : Ordinal.{u_1} hvb : v < b hw : w < b ^ u ⊢ b ^ succ u = b ^ u * b ** exact opow_succ b u ** Qed
Ordinal.log_opow_mul_add ** b u v w : Ordinal.{u_1} hb : 1 < b hv : v ≠ 0 hvb : v < b hw : w < b ^ u ⊢ log b (b ^ u * v + w) = u ** have hne' := (opow_mul_add_pos (zero_lt_one.trans hb).ne' u hv w).ne' ** b u v w : Ordinal.{u_1} hb : 1 < b hv : v ≠ 0 hvb : v < b hw : w < b ^ u hne' : b ^ u * v + w ≠ 0 ⊢ log b (b ^ u * v + w) = u ** by_contra' hne ** b u v w : Ordinal.{u_1} hb : 1 < b hv : v ≠ 0 hvb : v < b hw : w < b ^ u hne' : b ^ u * v + w ≠ 0 hne : log b (b ^ u * v + w) ≠ u ⊢ False ** cases' lt_or_gt_of_ne hne with h h ** case inl b u v w : Ordinal.{u_1} hb : 1 < b hv : v ≠ 0 hvb : v < b hw : w < b ^ u hne' : b ^ u * v + w ≠ 0 hne : log b (b ^ u * v + w) ≠ u h : log b (b ^ u * v + w) < u ⊢ False ** rw [← lt_opow_iff_log_lt hb hne'] at h ** case inl b u v w : Ordinal.{u_1} hb : 1 < b hv : v ≠ 0 hvb : v < b hw : w < b ^ u hne' : b ^ u * v + w ≠ 0 hne : log b (b ^ u * v + w) ≠ u h : b ^ u * v + w < b ^ u ⊢ False ** exact h.not_le ((le_mul_left _ (Ordinal.pos_iff_ne_zero.2 hv)).trans (le_add_right _ _)) ** case inr b u v w : Ordinal.{u_1} hb : 1 < b hv : v ≠ 0 hvb : v < b hw : w < b ^ u hne' : b ^ u * v + w ≠ 0 hne : log b (b ^ u * v + w) ≠ u h : log b (b ^ u * v + w) > u ⊢ False ** conv at h => change u < log b (b ^ u * v + w) ** case inr b u v w : Ordinal.{u_1} hb : 1 < b hv : v ≠ 0 hvb : v < b hw : w < b ^ u hne' : b ^ u * v + w ≠ 0 hne : log b (b ^ u * v + w) ≠ u h : u < log b (b ^ u * v + w) ⊢ False ** rw [← succ_le_iff, ← opow_le_iff_le_log hb hne'] at h ** case inr b u v w : Ordinal.{u_1} hb : 1 < b hv : v ≠ 0 hvb : v < b hw : w < b ^ u hne' : b ^ u * v + w ≠ 0 hne : log b (b ^ u * v + w) ≠ u h✝ : u < log b (b ^ u * v + w) h : b ^ succ u ≤ b ^ u * v + w ⊢ False ** exact (not_lt_of_le h) (opow_mul_add_lt_opow_succ hvb hw) ** Qed
Ordinal.log_opow ** b : Ordinal.{u_1} hb : 1 < b x : Ordinal.{u_1} ⊢ log b (b ^ x) = x ** convert log_opow_mul_add hb zero_ne_one.symm hb (opow_pos x (zero_lt_one.trans hb)) using 1 ** case h.e'_2 b : Ordinal.{u_1} hb : 1 < b x : Ordinal.{u_1} ⊢ log b (b ^ x) = log b (b ^ x * 1 + 0) ** rw [add_zero, mul_one] ** Qed
Ordinal.div_opow_log_pos ** b o : Ordinal.{u_1} ho : o ≠ 0 ⊢ 0 < o / b ^ log b o ** rcases eq_zero_or_pos b with (rfl | hb) ** case inl o : Ordinal.{u_1} ho : o ≠ 0 ⊢ 0 < o / 0 ^ log 0 o ** simpa using Ordinal.pos_iff_ne_zero.2 ho ** case inr b o : Ordinal.{u_1} ho : o ≠ 0 hb : 0 < b ⊢ 0 < o / b ^ log b o ** rw [div_pos (opow_ne_zero _ hb.ne')] ** case inr b o : Ordinal.{u_1} ho : o ≠ 0 hb : 0 < b ⊢ b ^ log b o ≤ o ** exact opow_log_le_self b ho ** Qed
Ordinal.div_opow_log_lt ** b o : Ordinal.{u_1} hb : 1 < b ⊢ o / b ^ log b o < b ** rw [div_lt (opow_pos _ (zero_lt_one.trans hb)).ne', ← opow_succ] ** b o : Ordinal.{u_1} hb : 1 < b ⊢ o < b ^ succ (log b o) ** exact lt_opow_succ_log_self hb o ** Qed
Ordinal.add_log_le_log_mul ** x y b : Ordinal.{u_1} hx : x ≠ 0 hy : y ≠ 0 ⊢ log b x + log b y ≤ log b (x * y) ** by_cases hb : 1 < b ** case neg x y b : Ordinal.{u_1} hx : x ≠ 0 hy : y ≠ 0 hb : ¬1 < b ⊢ log b x + log b y ≤ log b (x * y) ** simp only [log_of_not_one_lt_left hb, zero_add, le_refl] ** case pos x y b : Ordinal.{u_1} hx : x ≠ 0 hy : y ≠ 0 hb : 1 < b ⊢ log b x + log b y ≤ log b (x * y) ** rw [← opow_le_iff_le_log hb (mul_ne_zero hx hy), opow_add] ** case pos x y b : Ordinal.{u_1} hx : x ≠ 0 hy : y ≠ 0 hb : 1 < b ⊢ b ^ log b x * b ^ log b y ≤ x * y ** exact mul_le_mul' (opow_log_le_self b hx) (opow_log_le_self b hy) ** Qed
Ordinal.nat_cast_opow ** m : ℕ ⊢ ↑(m ^ 0) = ↑m ^ ↑0 ** simp ** m n : ℕ ⊢ ↑(m ^ (n + 1)) = ↑m ^ ↑(n + 1) ** rw [pow_succ', nat_cast_mul, nat_cast_opow m n, Nat.cast_succ, add_one_eq_succ, opow_succ] ** Qed
Ordinal.sup_opow_nat ** o : Ordinal.{u_1} ho : 0 < o ⊢ (sup fun n => o ^ ↑n) = o ^ ω ** rcases lt_or_eq_of_le (one_le_iff_pos.2 ho) with (ho₁ | rfl) ** case inl o : Ordinal.{u_1} ho : 0 < o ho₁ : 1 < o ⊢ (sup fun n => o ^ ↑n) = o ^ ω ** exact (opow_isNormal ho₁).apply_omega ** case inr ho : 0 < 1 ⊢ (sup fun n => 1 ^ ↑n) = 1 ^ ω ** rw [one_opow] ** case inr ho : 0 < 1 ⊢ (sup fun n => 1 ^ ↑n) = 1 ** refine' le_antisymm (sup_le fun n => by rw [one_opow]) _ ** case inr ho : 0 < 1 ⊢ 1 ≤ sup fun n => 1 ^ ↑n ** convert le_sup (fun n : ℕ => 1^n) 0 ** case h.e'_3 ho : 0 < 1 ⊢ 1 = 1 ^ ↑0 ** rw [Nat.cast_zero, opow_zero] ** ho : 0 < 1 n : ℕ ⊢ 1 ^ ↑n ≤ 1 ** rw [one_opow] ** Qed
Cardinal.isUnit_iff ** a b : Cardinal.{u} n m : ℕ ⊢ IsUnit a ↔ a = 1 ** refine' ⟨fun h => _, by rintro rfl exact isUnit_one⟩ ** a b : Cardinal.{u} n m : ℕ h : IsUnit a ⊢ a = 1 ** rcases eq_or_ne a 0 with (rfl | ha) ** case inr a b : Cardinal.{u} n m : ℕ h : IsUnit a ha : a ≠ 0 ⊢ a = 1 ** rw [isUnit_iff_forall_dvd] at h ** case inr a b : Cardinal.{u} n m : ℕ h : ∀ (y : Cardinal.{u}), a ∣ y ha : a ≠ 0 ⊢ a = 1 ** cases' h 1 with t ht ** case inr.intro a b : Cardinal.{u} n m : ℕ h : ∀ (y : Cardinal.{u}), a ∣ y ha : a ≠ 0 t : Cardinal.{u} ht : 1 = a * t ⊢ a = 1 ** rw [eq_comm, mul_eq_one_iff'] at ht ** a b : Cardinal.{u} n m : ℕ ⊢ a = 1 → IsUnit a ** rintro rfl ** b : Cardinal.{u} n m : ℕ ⊢ IsUnit 1 ** exact isUnit_one ** case inl b : Cardinal.{u} n m : ℕ h : IsUnit 0 ⊢ 0 = 1 ** exact (not_isUnit_zero h).elim ** case inr.intro a b : Cardinal.{u} n m : ℕ h : ∀ (y : Cardinal.{u}), a ∣ y ha : a ≠ 0 t : Cardinal.{u} ht : a = 1 ∧ t = 1 ⊢ a = 1 ** exact ht.1 ** case inr.intro.ha a b : Cardinal.{u} n m : ℕ h : ∀ (y : Cardinal.{u}), a ∣ y ha : a ≠ 0 t : Cardinal.{u} ht : a * t = 1 ⊢ 1 ≤ a ** exact one_le_iff_ne_zero.mpr ha ** case inr.intro.hb a b : Cardinal.{u} n m : ℕ h : ∀ (y : Cardinal.{u}), a ∣ y ha : a ≠ 0 t : Cardinal.{u} ht : a * t = 1 ⊢ 1 ≤ t ** apply one_le_iff_ne_zero.mpr ** case inr.intro.hb a b : Cardinal.{u} n m : ℕ h : ∀ (y : Cardinal.{u}), a ∣ y ha : a ≠ 0 t : Cardinal.{u} ht : a * t = 1 ⊢ t ≠ 0 ** intro h ** case inr.intro.hb a b : Cardinal.{u} n m : ℕ h✝ : ∀ (y : Cardinal.{u}), a ∣ y ha : a ≠ 0 t : Cardinal.{u} ht : a * t = 1 h : t = 0 ⊢ False ** rw [h, mul_zero] at ht ** case inr.intro.hb a b : Cardinal.{u} n m : ℕ h✝ : ∀ (y : Cardinal.{u}), a ∣ y ha : a ≠ 0 t : Cardinal.{u} ht : 0 = 1 h : t = 0 ⊢ False ** exact zero_ne_one ht ** Qed
Cardinal.le_of_dvd ** a✝ b✝ : Cardinal.{u} n m : ℕ a x : Cardinal.{u_1} b0 : x ≠ 0 b : Cardinal.{u_1} hab : x = a * b ⊢ a ≤ x ** simpa only [hab, mul_one] using mul_le_mul_left' (one_le_iff_ne_zero.2 fun h : b = 0 => b0 (by rwa [h, mul_zero] at hab)) a ** a✝ b✝ : Cardinal.{u} n m : ℕ a x : Cardinal.{u_1} b0 : x ≠ 0 b : Cardinal.{u_1} hab : x = a * b h : b = 0 ⊢ x = 0 ** rwa [h, mul_zero] at hab ** Qed
Cardinal.prime_of_aleph0_le ** a b : Cardinal.{u} n m : ℕ ha : ℵ₀ ≤ a ⊢ Prime a ** refine' ⟨(aleph0_pos.trans_le ha).ne', _, fun b c hbc => _⟩ ** case refine'_2 a b✝ : Cardinal.{u} n m : ℕ ha : ℵ₀ ≤ a b c : Cardinal.{u} hbc : a ∣ b * c ⊢ a ∣ b ∨ a ∣ c ** cases' eq_or_ne (b * c) 0 with hz hz ** case refine'_2.inr a b✝ : Cardinal.{u} n m : ℕ ha : ℵ₀ ≤ a b c : Cardinal.{u} hbc : a ∣ b * c hz : b * c ≠ 0 ⊢ a ∣ b ∨ a ∣ c ** wlog h : c ≤ b ** a✝ a b✝ : Cardinal.{u} n m : ℕ ha : ℵ₀ ≤ a b c : Cardinal.{u} hbc : a ∣ b * c hz : b * c ≠ 0 h : c ≤ b ⊢ a ∣ b ∨ a ∣ c ** left ** case h a✝ a b✝ : Cardinal.{u} n m : ℕ ha : ℵ₀ ≤ a b c : Cardinal.{u} hbc : a ∣ b * c hz : b * c ≠ 0 h : c ≤ b ⊢ a ∣ b ** have habc := le_of_dvd hz hbc ** case h a✝ a b✝ : Cardinal.{u} n m : ℕ ha : ℵ₀ ≤ a b c : Cardinal.{u} hbc : a ∣ b * c hz : b * c ≠ 0 h : c ≤ b habc : a ≤ b * c ⊢ a ∣ b ** rwa [mul_eq_max' <| ha.trans <| habc, max_def', if_pos h] at hbc ** case refine'_1 a b : Cardinal.{u} n m : ℕ ha : ℵ₀ ≤ a ⊢ ¬IsUnit a ** rw [isUnit_iff] ** case refine'_1 a b : Cardinal.{u} n m : ℕ ha : ℵ₀ ≤ a ⊢ ¬a = 1 ** exact (one_lt_aleph0.trans_le ha).ne' ** case refine'_2.inl a b✝ : Cardinal.{u} n m : ℕ ha : ℵ₀ ≤ a b c : Cardinal.{u} hbc : a ∣ b * c hz : b * c = 0 ⊢ a ∣ b ∨ a ∣ c ** rcases mul_eq_zero.mp hz with (rfl | rfl) <;> simp ** case refine'_2.inr.inr a b✝ : Cardinal.{u} n m : ℕ ha : ℵ₀ ≤ a b c : Cardinal.{u} hbc : a ∣ b * c hz : b * c ≠ 0 this : ∀ {a : Cardinal.{u}} {b : Cardinal.{u}} {n m : ℕ}, ℵ₀ ≤ a → ∀ (b c : Cardinal.{u}), a ∣ b * c → b * c ≠ 0 → c ≤ b → a ∣ b ∨ a ∣ c h : ¬c ≤ b ⊢ a ∣ b ∨ a ∣ c ** cases le_total c b <;> [skip; rw [or_comm]] <;> apply_assumption ** case refine'_2.inr.inr.inl.b a b✝ : Cardinal.{u} n m : ℕ ha : ℵ₀ ≤ a b c : Cardinal.{u} hbc : a ∣ b * c hz : b * c ≠ 0 this : ∀ {a : Cardinal.{u}} {b : Cardinal.{u}} {n m : ℕ}, ℵ₀ ≤ a → ∀ (b c : Cardinal.{u}), a ∣ b * c → b * c ≠ 0 → c ≤ b → a ∣ b ∨ a ∣ c h : ¬c ≤ b h✝ : c ≤ b hz_symm : 0 ≠ b * c ⊢ Cardinal.{u} case refine'_2.inr.inr.inl.n a b✝ : Cardinal.{u} n m : ℕ ha : ℵ₀ ≤ a b c : Cardinal.{u} hbc : a ∣ b * c hz : b * c ≠ 0 this : ∀ {a : Cardinal.{u}} {b : Cardinal.{u}} {n m : ℕ}, ℵ₀ ≤ a → ∀ (b c : Cardinal.{u}), a ∣ b * c → b * c ≠ 0 → c ≤ b → a ∣ b ∨ a ∣ c h : ¬c ≤ b h✝ : c ≤ b hz_symm : 0 ≠ b * c ⊢ ℕ case refine'_2.inr.inr.inl.m a b✝ : Cardinal.{u} n m : ℕ ha : ℵ₀ ≤ a b c : Cardinal.{u} hbc : a ∣ b * c hz : b * c ≠ 0 this : ∀ {a : Cardinal.{u}} {b : Cardinal.{u}} {n m : ℕ}, ℵ₀ ≤ a → ∀ (b c : Cardinal.{u}), a ∣ b * c → b * c ≠ 0 → c ≤ b → a ∣ b ∨ a ∣ c h : ¬c ≤ b h✝ : c ≤ b hz_symm : 0 ≠ b * c ⊢ ℕ case refine'_2.inr.inr.inl.ha a b✝ : Cardinal.{u} n m : ℕ ha : ℵ₀ ≤ a b c : Cardinal.{u} hbc : a ∣ b * c hz : b * c ≠ 0 this : ∀ {a : Cardinal.{u}} {b : Cardinal.{u}} {n m : ℕ}, ℵ₀ ≤ a → ∀ (b c : Cardinal.{u}), a ∣ b * c → b * c ≠ 0 → c ≤ b → a ∣ b ∨ a ∣ c h : ¬c ≤ b h✝ : c ≤ b hz_symm : 0 ≠ b * c ⊢ ℵ₀ ≤ a case refine'_2.inr.inr.inl.hbc a b✝ : Cardinal.{u} n m : ℕ ha : ℵ₀ ≤ a b c : Cardinal.{u} hbc : a ∣ b * c hz : b * c ≠ 0 this : ∀ {a : Cardinal.{u}} {b : Cardinal.{u}} {n m : ℕ}, ℵ₀ ≤ a → ∀ (b c : Cardinal.{u}), a ∣ b * c → b * c ≠ 0 → c ≤ b → a ∣ b ∨ a ∣ c h : ¬c ≤ b h✝ : c ≤ b hz_symm : 0 ≠ b * c ⊢ a ∣ b * c case refine'_2.inr.inr.inl.hz a b✝ : Cardinal.{u} n m : ℕ ha : ℵ₀ ≤ a b c : Cardinal.{u} hbc : a ∣ b * c hz : b * c ≠ 0 this : ∀ {a : Cardinal.{u}} {b : Cardinal.{u}} {n m : ℕ}, ℵ₀ ≤ a → ∀ (b c : Cardinal.{u}), a ∣ b * c → b * c ≠ 0 → c ≤ b → a ∣ b ∨ a ∣ c h : ¬c ≤ b h✝ : c ≤ b hz_symm : 0 ≠ b * c ⊢ b * c ≠ 0 case refine'_2.inr.inr.inl.h a b✝ : Cardinal.{u} n m : ℕ ha : ℵ₀ ≤ a b c : Cardinal.{u} hbc : a ∣ b * c hz : b * c ≠ 0 this : ∀ {a : Cardinal.{u}} {b : Cardinal.{u}} {n m : ℕ}, ℵ₀ ≤ a → ∀ (b c : Cardinal.{u}), a ∣ b * c → b * c ≠ 0 → c ≤ b → a ∣ b ∨ a ∣ c h : ¬c ≤ b h✝ : c ≤ b hz_symm : 0 ≠ b * c ⊢ c ≤ b case refine'_2.inr.inr.inr.b a b✝ : Cardinal.{u} n m : ℕ ha : ℵ₀ ≤ a b c : Cardinal.{u} hbc : a ∣ b * c hz : b * c ≠ 0 this : ∀ {a : Cardinal.{u}} {b : Cardinal.{u}} {n m : ℕ}, ℵ₀ ≤ a → ∀ (b c : Cardinal.{u}), a ∣ b * c → b * c ≠ 0 → c ≤ b → a ∣ b ∨ a ∣ c h : ¬c ≤ b h✝ : b ≤ c hz_symm : 0 ≠ b * c ⊢ Cardinal.{u} case refine'_2.inr.inr.inr.n a b✝ : Cardinal.{u} n m : ℕ ha : ℵ₀ ≤ a b c : Cardinal.{u} hbc : a ∣ b * c hz : b * c ≠ 0 this : ∀ {a : Cardinal.{u}} {b : Cardinal.{u}} {n m : ℕ}, ℵ₀ ≤ a → ∀ (b c : Cardinal.{u}), a ∣ b * c → b * c ≠ 0 → c ≤ b → a ∣ b ∨ a ∣ c h : ¬c ≤ b h✝ : b ≤ c hz_symm : 0 ≠ b * c ⊢ ℕ case refine'_2.inr.inr.inr.m a b✝ : Cardinal.{u} n m : ℕ ha : ℵ₀ ≤ a b c : Cardinal.{u} hbc : a ∣ b * c hz : b * c ≠ 0 this : ∀ {a : Cardinal.{u}} {b : Cardinal.{u}} {n m : ℕ}, ℵ₀ ≤ a → ∀ (b c : Cardinal.{u}), a ∣ b * c → b * c ≠ 0 → c ≤ b → a ∣ b ∨ a ∣ c h : ¬c ≤ b h✝ : b ≤ c hz_symm : 0 ≠ b * c ⊢ ℕ case refine'_2.inr.inr.inr.ha a b✝ : Cardinal.{u} n m : ℕ ha : ℵ₀ ≤ a b c : Cardinal.{u} hbc : a ∣ b * c hz : b * c ≠ 0 this : ∀ {a : Cardinal.{u}} {b : Cardinal.{u}} {n m : ℕ}, ℵ₀ ≤ a → ∀ (b c : Cardinal.{u}), a ∣ b * c → b * c ≠ 0 → c ≤ b → a ∣ b ∨ a ∣ c h : ¬c ≤ b h✝ : b ≤ c hz_symm : 0 ≠ b * c ⊢ ℵ₀ ≤ a case refine'_2.inr.inr.inr.hbc a b✝ : Cardinal.{u} n m : ℕ ha : ℵ₀ ≤ a b c : Cardinal.{u} hbc : a ∣ b * c hz : b * c ≠ 0 this : ∀ {a : Cardinal.{u}} {b : Cardinal.{u}} {n m : ℕ}, ℵ₀ ≤ a → ∀ (b c : Cardinal.{u}), a ∣ b * c → b * c ≠ 0 → c ≤ b → a ∣ b ∨ a ∣ c h : ¬c ≤ b h✝ : b ≤ c hz_symm : 0 ≠ b * c ⊢ a ∣ c * b case refine'_2.inr.inr.inr.hz a b✝ : Cardinal.{u} n m : ℕ ha : ℵ₀ ≤ a b c : Cardinal.{u} hbc : a ∣ b * c hz : b * c ≠ 0 this : ∀ {a : Cardinal.{u}} {b : Cardinal.{u}} {n m : ℕ}, ℵ₀ ≤ a → ∀ (b c : Cardinal.{u}), a ∣ b * c → b * c ≠ 0 → c ≤ b → a ∣ b ∨ a ∣ c h : ¬c ≤ b h✝ : b ≤ c hz_symm : 0 ≠ b * c ⊢ c * b ≠ 0 case refine'_2.inr.inr.inr.h a b✝ : Cardinal.{u} n m : ℕ ha : ℵ₀ ≤ a b c : Cardinal.{u} hbc : a ∣ b * c hz : b * c ≠ 0 this : ∀ {a : Cardinal.{u}} {b : Cardinal.{u}} {n m : ℕ}, ℵ₀ ≤ a → ∀ (b c : Cardinal.{u}), a ∣ b * c → b * c ≠ 0 → c ≤ b → a ∣ b ∨ a ∣ c h : ¬c ≤ b h✝ : b ≤ c hz_symm : 0 ≠ b * c ⊢ b ≤ c ** assumption' ** case refine'_2.inr.inr.inr.hbc a b✝ : Cardinal.{u} n m : ℕ ha : ℵ₀ ≤ a b c : Cardinal.{u} hbc : a ∣ b * c hz : b * c ≠ 0 this : ∀ {a : Cardinal.{u}} {b : Cardinal.{u}} {n m : ℕ}, ℵ₀ ≤ a → ∀ (b c : Cardinal.{u}), a ∣ b * c → b * c ≠ 0 → c ≤ b → a ∣ b ∨ a ∣ c h : ¬c ≤ b h✝ : b ≤ c hz_symm : 0 ≠ b * c ⊢ a ∣ c * b case refine'_2.inr.inr.inr.hz a b✝ : Cardinal.{u} n m : ℕ ha : ℵ₀ ≤ a b c : Cardinal.{u} hbc : a ∣ b * c hz : b * c ≠ 0 this : ∀ {a : Cardinal.{u}} {b : Cardinal.{u}} {n m : ℕ}, ℵ₀ ≤ a → ∀ (b c : Cardinal.{u}), a ∣ b * c → b * c ≠ 0 → c ≤ b → a ∣ b ∨ a ∣ c h : ¬c ≤ b h✝ : b ≤ c hz_symm : 0 ≠ b * c ⊢ c * b ≠ 0 ** all_goals rwa [mul_comm] ** case refine'_2.inr.inr.inr.hz a b✝ : Cardinal.{u} n m : ℕ ha : ℵ₀ ≤ a b c : Cardinal.{u} hbc : a ∣ b * c hz : b * c ≠ 0 this : ∀ {a : Cardinal.{u}} {b : Cardinal.{u}} {n m : ℕ}, ℵ₀ ≤ a → ∀ (b c : Cardinal.{u}), a ∣ b * c → b * c ≠ 0 → c ≤ b → a ∣ b ∨ a ∣ c h : ¬c ≤ b h✝ : b ≤ c hz_symm : 0 ≠ b * c ⊢ c * b ≠ 0 ** rwa [mul_comm] ** Qed
Cardinal.not_irreducible_of_aleph0_le ** a b : Cardinal.{u} n m : ℕ ha : ℵ₀ ≤ a ⊢ ¬Irreducible a ** rw [irreducible_iff, not_and_or] ** a b : Cardinal.{u} n m : ℕ ha : ℵ₀ ≤ a ⊢ ¬¬IsUnit a ∨ ¬∀ (a_1 b : Cardinal.{u}), a = a_1 * b → IsUnit a_1 ∨ IsUnit b ** refine' Or.inr fun h => _ ** a b : Cardinal.{u} n m : ℕ ha : ℵ₀ ≤ a h : ∀ (a_1 b : Cardinal.{u}), a = a_1 * b → IsUnit a_1 ∨ IsUnit b ⊢ False ** simpa [mul_aleph0_eq ha, isUnit_iff, (one_lt_aleph0.trans_le ha).ne', one_lt_aleph0.ne'] using h a ℵ₀ ** Qed
Cardinal.nat_coe_dvd_iff ** a b : Cardinal.{u} n m : ℕ ⊢ ↑n ∣ ↑m ↔ n ∣ m ** refine' ⟨_, fun ⟨h, ht⟩ => ⟨h, by exact_mod_cast ht⟩⟩ ** a b : Cardinal.{u} n m : ℕ ⊢ ↑n ∣ ↑m → n ∣ m ** rintro ⟨k, hk⟩ ** case intro a b : Cardinal.{u} n m : ℕ k : Cardinal.{u_1} hk : ↑m = ↑n * k ⊢ n ∣ m ** have : ↑m < ℵ₀ := nat_lt_aleph0 m ** case intro a b : Cardinal.{u} n m : ℕ k : Cardinal.{u_1} hk : ↑m = ↑n * k this : ↑m < ℵ₀ ⊢ n ∣ m ** rw [hk, mul_lt_aleph0_iff] at this ** case intro a b : Cardinal.{u} n m : ℕ k : Cardinal.{u_1} hk : ↑m = ↑n * k this : ↑n = 0 ∨ k = 0 ∨ ↑n < ℵ₀ ∧ k < ℵ₀ ⊢ n ∣ m ** rcases this with (h | h | ⟨-, hk'⟩) ** case intro.inl a b : Cardinal.{u} n m : ℕ k : Cardinal.{u_1} hk : ↑m = ↑n * k h : ↑n = 0 ⊢ n ∣ m case intro.inr.inl a b : Cardinal.{u} n m : ℕ k : Cardinal.{u_1} hk : ↑m = ↑n * k h : k = 0 ⊢ n ∣ m case intro.inr.inr.intro a b : Cardinal.{u} n m : ℕ k : Cardinal.{u_1} hk : ↑m = ↑n * k hk' : k < ℵ₀ ⊢ n ∣ m ** iterate 2 simp only [h, mul_zero, zero_mul, Nat.cast_eq_zero] at hk; simp [hk] ** case intro.inr.inr.intro a b : Cardinal.{u} n m : ℕ k : Cardinal.{u_1} hk : ↑m = ↑n * k hk' : k < ℵ₀ ⊢ n ∣ m ** lift k to ℕ using hk' ** case intro.inr.inr.intro.intro a b : Cardinal.{u} n m k : ℕ hk : ↑m = ↑n * ↑k ⊢ n ∣ m ** exact ⟨k, by exact_mod_cast hk⟩ ** a b : Cardinal.{u} n m : ℕ x✝ : n ∣ m h : ℕ ht : m = n * h ⊢ ↑m = ↑n * ↑h ** exact_mod_cast ht ** case intro.inr.inl a b : Cardinal.{u} n m : ℕ k : Cardinal.{u_1} hk : ↑m = ↑n * k h : k = 0 ⊢ n ∣ m case intro.inr.inr.intro a b : Cardinal.{u} n m : ℕ k : Cardinal.{u_1} hk : ↑m = ↑n * k hk' : k < ℵ₀ ⊢ n ∣ m ** simp only [h, mul_zero, zero_mul, Nat.cast_eq_zero] at hk ** case intro.inr.inl a b : Cardinal.{u} n m : ℕ k : Cardinal.{u_1} h : k = 0 hk : m = 0 ⊢ n ∣ m case intro.inr.inr.intro a b : Cardinal.{u} n m : ℕ k : Cardinal.{u_1} hk : ↑m = ↑n * k hk' : k < ℵ₀ ⊢ n ∣ m ** simp [hk] ** a b : Cardinal.{u} n m k : ℕ hk : ↑m = ↑n * ↑k ⊢ m = n * k ** exact_mod_cast hk ** Qed
Cardinal.nat_is_prime_iff ** a b : Cardinal.{u} n m : ℕ ⊢ Prime ↑n ↔ Nat.Prime n ** simp only [Prime, Nat.prime_iff] ** a b : Cardinal.{u} n m : ℕ ⊢ (↑n ≠ 0 ∧ ¬IsUnit ↑n ∧ ∀ (a b : Cardinal.{u_1}), ↑n ∣ a * b → ↑n ∣ a ∨ ↑n ∣ b) ↔ n ≠ 0 ∧ ¬IsUnit n ∧ ∀ (a b : ℕ), n ∣ a * b → n ∣ a ∨ n ∣ b ** refine' and_congr (by simp) (and_congr _ ⟨fun h b c hbc => _, fun h b c hbc => _⟩) ** case refine'_3 a b✝ : Cardinal.{u} n m : ℕ h : ∀ (a b : ℕ), n ∣ a * b → n ∣ a ∨ n ∣ b b c : Cardinal.{u_1} hbc : ↑n ∣ b * c ⊢ ↑n ∣ b ∨ ↑n ∣ c ** cases' lt_or_le (b * c) ℵ₀ with h' h' ** case refine'_3.inr a b✝ : Cardinal.{u} n m : ℕ h : ∀ (a b : ℕ), n ∣ a * b → n ∣ a ∨ n ∣ b b c : Cardinal.{u_1} hbc : ↑n ∣ b * c h' : ℵ₀ ≤ b * c ⊢ ↑n ∣ b ∨ ↑n ∣ c ** rcases aleph0_le_mul_iff.mp h' with ⟨hb, hc, hℵ₀⟩ ** case refine'_3.inr.intro.intro a b✝ : Cardinal.{u} n m : ℕ h : ∀ (a b : ℕ), n ∣ a * b → n ∣ a ∨ n ∣ b b c : Cardinal.{u_1} hbc : ↑n ∣ b * c h' : ℵ₀ ≤ b * c hb : b ≠ 0 hc : c ≠ 0 hℵ₀ : ℵ₀ ≤ b ∨ ℵ₀ ≤ c ⊢ ↑n ∣ b ∨ ↑n ∣ c ** have hn : (n : Cardinal) ≠ 0 := by intro h rw [h, zero_dvd_iff, mul_eq_zero] at hbc cases hbc <;> contradiction ** case refine'_3.inr.intro.intro a b✝ : Cardinal.{u} n m : ℕ h : ∀ (a b : ℕ), n ∣ a * b → n ∣ a ∨ n ∣ b b c : Cardinal.{u_1} hbc : ↑n ∣ b * c h' : ℵ₀ ≤ b * c hb : b ≠ 0 hc : c ≠ 0 hℵ₀ : ℵ₀ ≤ b ∨ ℵ₀ ≤ c hn : ↑n ≠ 0 ⊢ ↑n ∣ b ∨ ↑n ∣ c ** wlog hℵ₀b : ℵ₀ ≤ b ** case refine'_3.inr.intro.intro.inr a b✝ : Cardinal.{u} n m : ℕ h : ∀ (a b : ℕ), n ∣ a * b → n ∣ a ∨ n ∣ b b c : Cardinal.{u_1} hbc : ↑n ∣ b * c h' : ℵ₀ ≤ b * c hb : b ≠ 0 hc : c ≠ 0 hℵ₀ : ℵ₀ ≤ b ∨ ℵ₀ ≤ c hn : ↑n ≠ 0 this : ∀ {a b : Cardinal.{u}} {n : ℕ} {m : ℕ}, (∀ (a b : ℕ), n ∣ a * b → n ∣ a ∨ n ∣ b) → ∀ (b c : Cardinal.{u_1}), ↑n ∣ b * c → ℵ₀ ≤ b * c → b ≠ 0 → c ≠ 0 → ℵ₀ ≤ b ∨ ℵ₀ ≤ c → ↑n ≠ 0 → ℵ₀ ≤ b → ↑n ∣ b ∨ ↑n ∣ c hℵ₀b : ¬ℵ₀ ≤ b ⊢ ↑n ∣ b ∨ ↑n ∣ c n✝ : ℕ a b✝ : Cardinal.{u} n m : ℕ h : ∀ (a b : ℕ), n ∣ a * b → n ∣ a ∨ n ∣ b b c : Cardinal.{u_1} hbc : ↑n ∣ b * c h' : ℵ₀ ≤ b * c hb : b ≠ 0 hc : c ≠ 0 hℵ₀ : ℵ₀ ≤ b ∨ ℵ₀ ≤ c hn : ↑n ≠ 0 hℵ₀b : ℵ₀ ≤ b ⊢ ↑n ∣ b ∨ ↑n ∣ c ** refine' (this h c b _ _ hc hb hℵ₀.symm hn (hℵ₀.resolve_left hℵ₀b)).symm <;> try assumption ** case refine'_3.inr.intro.intro.inr.refine'_4 a b✝ : Cardinal.{u} n m : ℕ h : ∀ (a b : ℕ), n ∣ a * b → n ∣ a ∨ n ∣ b b c : Cardinal.{u_1} hbc : ↑n ∣ b * c h' : ℵ₀ ≤ b * c hb : b ≠ 0 hc : c ≠ 0 hℵ₀ : ℵ₀ ≤ b ∨ ℵ₀ ≤ c hn : ↑n ≠ 0 this : ∀ {a b : Cardinal.{u}} {n : ℕ} {m : ℕ}, (∀ (a b : ℕ), n ∣ a * b → n ∣ a ∨ n ∣ b) → ∀ (b c : Cardinal.{u_1}), ↑n ∣ b * c → ℵ₀ ≤ b * c → b ≠ 0 → c ≠ 0 → ℵ₀ ≤ b ∨ ℵ₀ ≤ c → ↑n ≠ 0 → ℵ₀ ≤ b → ↑n ∣ b ∨ ↑n ∣ c hℵ₀b : ¬ℵ₀ ≤ b ⊢ ↑n ∣ c * b case refine'_3.inr.intro.intro.inr.refine'_5 a b✝ : Cardinal.{u} n m : ℕ h : ∀ (a b : ℕ), n ∣ a * b → n ∣ a ∨ n ∣ b b c : Cardinal.{u_1} hbc : ↑n ∣ b * c h' : ℵ₀ ≤ b * c hb : b ≠ 0 hc : c ≠ 0 hℵ₀ : ℵ₀ ≤ b ∨ ℵ₀ ≤ c hn : ↑n ≠ 0 this : ∀ {a b : Cardinal.{u}} {n : ℕ} {m : ℕ}, (∀ (a b : ℕ), n ∣ a * b → n ∣ a ∨ n ∣ b) → ∀ (b c : Cardinal.{u_1}), ↑n ∣ b * c → ℵ₀ ≤ b * c → b ≠ 0 → c ≠ 0 → ℵ₀ ≤ b ∨ ℵ₀ ≤ c → ↑n ≠ 0 → ℵ₀ ≤ b → ↑n ∣ b ∨ ↑n ∣ c hℵ₀b : ¬ℵ₀ ≤ b ⊢ ℵ₀ ≤ c * b n✝ : ℕ a b✝ : Cardinal.{u} n m : ℕ h : ∀ (a b : ℕ), n ∣ a * b → n ∣ a ∨ n ∣ b b c : Cardinal.{u_1} hbc : ↑n ∣ b * c h' : ℵ₀ ≤ b * c hb : b ≠ 0 hc : c ≠ 0 hℵ₀ : ℵ₀ ≤ b ∨ ℵ₀ ≤ c hn : ↑n ≠ 0 hℵ₀b : ℵ₀ ≤ b ⊢ ↑n ∣ b ∨ ↑n ∣ c ** rwa [mul_comm] at hbc ** case refine'_3.inr.intro.intro.inr.refine'_5 a b✝ : Cardinal.{u} n m : ℕ h : ∀ (a b : ℕ), n ∣ a * b → n ∣ a ∨ n ∣ b b c : Cardinal.{u_1} hbc : ↑n ∣ b * c h' : ℵ₀ ≤ b * c hb : b ≠ 0 hc : c ≠ 0 hℵ₀ : ℵ₀ ≤ b ∨ ℵ₀ ≤ c hn : ↑n ≠ 0 this : ∀ {a b : Cardinal.{u}} {n : ℕ} {m : ℕ}, (∀ (a b : ℕ), n ∣ a * b → n ∣ a ∨ n ∣ b) → ∀ (b c : Cardinal.{u_1}), ↑n ∣ b * c → ℵ₀ ≤ b * c → b ≠ 0 → c ≠ 0 → ℵ₀ ≤ b ∨ ℵ₀ ≤ c → ↑n ≠ 0 → ℵ₀ ≤ b → ↑n ∣ b ∨ ↑n ∣ c hℵ₀b : ¬ℵ₀ ≤ b ⊢ ℵ₀ ≤ c * b n✝ : ℕ a b✝ : Cardinal.{u} n m : ℕ h : ∀ (a b : ℕ), n ∣ a * b → n ∣ a ∨ n ∣ b b c : Cardinal.{u_1} hbc : ↑n ∣ b * c h' : ℵ₀ ≤ b * c hb : b ≠ 0 hc : c ≠ 0 hℵ₀ : ℵ₀ ≤ b ∨ ℵ₀ ≤ c hn : ↑n ≠ 0 hℵ₀b : ℵ₀ ≤ b ⊢ ↑n ∣ b ∨ ↑n ∣ c ** rwa [mul_comm] at h' ** n✝ : ℕ a b✝ : Cardinal.{u} n m : ℕ h : ∀ (a b : ℕ), n ∣ a * b → n ∣ a ∨ n ∣ b b c : Cardinal.{u_1} hbc : ↑n ∣ b * c h' : ℵ₀ ≤ b * c hb : b ≠ 0 hc : c ≠ 0 hℵ₀ : ℵ₀ ≤ b ∨ ℵ₀ ≤ c hn : ↑n ≠ 0 hℵ₀b : ℵ₀ ≤ b ⊢ ↑n ∣ b ∨ ↑n ∣ c ** exact Or.inl (dvd_of_le_of_aleph0_le hn ((nat_lt_aleph0 n).le.trans hℵ₀b) hℵ₀b) ** a b : Cardinal.{u} n m : ℕ ⊢ ↑n ≠ 0 ↔ n ≠ 0 ** simp ** case refine'_1 a b : Cardinal.{u} n m : ℕ ⊢ ¬IsUnit ↑n ↔ ¬IsUnit n ** simp only [isUnit_iff, Nat.isUnit_iff] ** case refine'_1 a b : Cardinal.{u} n m : ℕ ⊢ ¬↑n = 1 ↔ ¬n = 1 ** exact_mod_cast Iff.rfl ** case refine'_2 a b✝ : Cardinal.{u} n m : ℕ h : ∀ (a b : Cardinal.{u_1}), ↑n ∣ a * b → ↑n ∣ a ∨ ↑n ∣ b b c : ℕ hbc : n ∣ b * c ⊢ n ∣ b ∨ n ∣ c ** exact_mod_cast h b c (by exact_mod_cast hbc) ** a b✝ : Cardinal.{u} n m : ℕ h : ∀ (a b : Cardinal.{u_1}), ↑n ∣ a * b → ↑n ∣ a ∨ ↑n ∣ b b c : ℕ hbc : n ∣ b * c ⊢ ↑n ∣ ↑b * ↑c ** exact_mod_cast hbc ** case refine'_3.inl a b✝ : Cardinal.{u} n m : ℕ h : ∀ (a b : ℕ), n ∣ a * b → n ∣ a ∨ n ∣ b b c : Cardinal.{u_1} hbc : ↑n ∣ b * c h' : b * c < ℵ₀ ⊢ ↑n ∣ b ∨ ↑n ∣ c ** rcases mul_lt_aleph0_iff.mp h' with (rfl | rfl | ⟨hb, hc⟩) ** case refine'_3.inl.inr.inr.intro a b✝ : Cardinal.{u} n m : ℕ h : ∀ (a b : ℕ), n ∣ a * b → n ∣ a ∨ n ∣ b b c : Cardinal.{u_1} hbc : ↑n ∣ b * c h' : b * c < ℵ₀ hb : b < ℵ₀ hc : c < ℵ₀ ⊢ ↑n ∣ b ∨ ↑n ∣ c ** lift b to ℕ using hb ** case refine'_3.inl.inr.inr.intro.intro a b✝ : Cardinal.{u} n m : ℕ h : ∀ (a b : ℕ), n ∣ a * b → n ∣ a ∨ n ∣ b c : Cardinal.{u_1} hc : c < ℵ₀ b : ℕ hbc : ↑n ∣ ↑b * c h' : ↑b * c < ℵ₀ ⊢ ↑n ∣ ↑b ∨ ↑n ∣ c ** lift c to ℕ using hc ** case refine'_3.inl.inr.inr.intro.intro.intro a b✝ : Cardinal.{u} n m : ℕ h : ∀ (a b : ℕ), n ∣ a * b → n ∣ a ∨ n ∣ b b c : ℕ hbc : ↑n ∣ ↑b * ↑c h' : ↑b * ↑c < ℵ₀ ⊢ ↑n ∣ ↑b ∨ ↑n ∣ ↑c ** exact_mod_cast h b c (by exact_mod_cast hbc) ** case refine'_3.inl.inl a b : Cardinal.{u} n m : ℕ h : ∀ (a b : ℕ), n ∣ a * b → n ∣ a ∨ n ∣ b c : Cardinal.{u_1} hbc : ↑n ∣ 0 * c h' : 0 * c < ℵ₀ ⊢ ↑n ∣ 0 ∨ ↑n ∣ c ** simp ** case refine'_3.inl.inr.inl a b✝ : Cardinal.{u} n m : ℕ h : ∀ (a b : ℕ), n ∣ a * b → n ∣ a ∨ n ∣ b b : Cardinal.{u_1} hbc : ↑n ∣ b * 0 h' : b * 0 < ℵ₀ ⊢ ↑n ∣ b ∨ ↑n ∣ 0 ** simp ** a b✝ : Cardinal.{u} n m : ℕ h : ∀ (a b : ℕ), n ∣ a * b → n ∣ a ∨ n ∣ b b c : ℕ hbc : ↑n ∣ ↑b * ↑c h' : ↑b * ↑c < ℵ₀ ⊢ n ∣ b * c ** exact_mod_cast hbc ** a b✝ : Cardinal.{u} n m : ℕ h : ∀ (a b : ℕ), n ∣ a * b → n ∣ a ∨ n ∣ b b c : Cardinal.{u_1} hbc : ↑n ∣ b * c h' : ℵ₀ ≤ b * c hb : b ≠ 0 hc : c ≠ 0 hℵ₀ : ℵ₀ ≤ b ∨ ℵ₀ ≤ c ⊢ ↑n ≠ 0 ** intro h ** a b✝ : Cardinal.{u} n m : ℕ h✝ : ∀ (a b : ℕ), n ∣ a * b → n ∣ a ∨ n ∣ b b c : Cardinal.{u_1} hbc : ↑n ∣ b * c h' : ℵ₀ ≤ b * c hb : b ≠ 0 hc : c ≠ 0 hℵ₀ : ℵ₀ ≤ b ∨ ℵ₀ ≤ c h : ↑n = 0 ⊢ False ** rw [h, zero_dvd_iff, mul_eq_zero] at hbc ** a b✝ : Cardinal.{u} n m : ℕ h✝ : ∀ (a b : ℕ), n ∣ a * b → n ∣ a ∨ n ∣ b b c : Cardinal.{u_1} hbc : b = 0 ∨ c = 0 h' : ℵ₀ ≤ b * c hb : b ≠ 0 hc : c ≠ 0 hℵ₀ : ℵ₀ ≤ b ∨ ℵ₀ ≤ c h : ↑n = 0 ⊢ False ** cases hbc <;> contradiction ** case refine'_3.inr.intro.intro.inr.refine'_3 a b✝ : Cardinal.{u} n m : ℕ h : ∀ (a b : ℕ), n ∣ a * b → n ∣ a ∨ n ∣ b b c : Cardinal.{u_1} hbc : ↑n ∣ b * c h' : ℵ₀ ≤ b * c hb : b ≠ 0 hc : c ≠ 0 hℵ₀ : ℵ₀ ≤ b ∨ ℵ₀ ≤ c hn : ↑n ≠ 0 this : ∀ {a b : Cardinal.{u}} {n : ℕ} {m : ℕ}, (∀ (a b : ℕ), n ∣ a * b → n ∣ a ∨ n ∣ b) → ∀ (b c : Cardinal.{u_1}), ↑n ∣ b * c → ℵ₀ ≤ b * c → b ≠ 0 → c ≠ 0 → ℵ₀ ≤ b ∨ ℵ₀ ≤ c → ↑n ≠ 0 → ℵ₀ ≤ b → ↑n ∣ b ∨ ↑n ∣ c hℵ₀b : ¬ℵ₀ ≤ b ⊢ ℕ ** assumption ** Qed
Cardinal.is_prime_iff ** a✝ b : Cardinal.{u} n m : ℕ a : Cardinal.{u_1} ⊢ Prime a ↔ ℵ₀ ≤ a ∨ ∃ p, a = ↑p ∧ Nat.Prime p ** cases' le_or_lt ℵ₀ a with h h ** case inr a✝ b : Cardinal.{u} n m : ℕ a : Cardinal.{u_1} h : a < ℵ₀ ⊢ Prime a ↔ ℵ₀ ≤ a ∨ ∃ p, a = ↑p ∧ Nat.Prime p ** lift a to ℕ using id h ** case inr.intro a✝ b : Cardinal.{u} n m a : ℕ h : ↑a < ℵ₀ ⊢ Prime ↑a ↔ ℵ₀ ≤ ↑a ∨ ∃ p, ↑a = ↑p ∧ Nat.Prime p ** simp [not_le.mpr h] ** case inl a✝ b : Cardinal.{u} n m : ℕ a : Cardinal.{u_1} h : ℵ₀ ≤ a ⊢ Prime a ↔ ℵ₀ ≤ a ∨ ∃ p, a = ↑p ∧ Nat.Prime p ** simp [h] ** Qed
Cardinal.isPrimePow_iff ** a✝ b : Cardinal.{u} n m : ℕ a : Cardinal.{u_1} ⊢ IsPrimePow a ↔ ℵ₀ ≤ a ∨ ∃ n, a = ↑n ∧ IsPrimePow n ** by_cases h : ℵ₀ ≤ a ** case neg a✝ b : Cardinal.{u} n m : ℕ a : Cardinal.{u_1} h : ¬ℵ₀ ≤ a ⊢ IsPrimePow a ↔ ℵ₀ ≤ a ∨ ∃ n, a = ↑n ∧ IsPrimePow n ** simp only [h, Nat.cast_inj, exists_eq_left', false_or_iff, isPrimePow_nat_iff] ** case neg a✝ b : Cardinal.{u} n m : ℕ a : Cardinal.{u_1} h : ¬ℵ₀ ≤ a ⊢ IsPrimePow a ↔ ∃ n, a = ↑n ∧ ∃ p k, Nat.Prime p ∧ 0 < k ∧ p ^ k = n ** lift a to ℕ using not_le.mp h ** case neg.intro a✝ b : Cardinal.{u} n m a : ℕ h : ¬ℵ₀ ≤ ↑a ⊢ IsPrimePow ↑a ↔ ∃ n, ↑a = ↑n ∧ ∃ p k, Nat.Prime p ∧ 0 < k ∧ p ^ k = n ** rw [isPrimePow_def] ** case neg.intro a✝ b : Cardinal.{u} n m a : ℕ h : ¬ℵ₀ ≤ ↑a ⊢ (∃ p k, Prime p ∧ 0 < k ∧ p ^ k = ↑a) ↔ ∃ n, ↑a = ↑n ∧ ∃ p k, Nat.Prime p ∧ 0 < k ∧ p ^ k = n ** refine' ⟨_, fun ⟨n, han, p, k, hp, hk, h⟩ => ⟨p, k, nat_is_prime_iff.2 hp, hk, by rw [han]; exact_mod_cast h⟩⟩ ** case neg.intro a✝ b : Cardinal.{u} n m a : ℕ h : ¬ℵ₀ ≤ ↑a ⊢ (∃ p k, Prime p ∧ 0 < k ∧ p ^ k = ↑a) → ∃ n, ↑a = ↑n ∧ ∃ p k, Nat.Prime p ∧ 0 < k ∧ p ^ k = n ** rintro ⟨p, k, hp, hk, hpk⟩ ** case neg.intro.intro.intro.intro.intro a✝ b : Cardinal.{u} n m a : ℕ h : ¬ℵ₀ ≤ ↑a p : Cardinal.{u_1} k : ℕ hp : Prime p hk : 0 < k hpk : p ^ k = ↑a ⊢ ∃ n, ↑a = ↑n ∧ ∃ p k, Nat.Prime p ∧ 0 < k ∧ p ^ k = n ** have key : p ^ 1 ≤ ↑a := by rw [←hpk]; apply power_le_power_left hp.ne_zero; exact_mod_cast hk ** case neg.intro.intro.intro.intro.intro a✝ b : Cardinal.{u} n m a : ℕ h : ¬ℵ₀ ≤ ↑a p : Cardinal.{u_1} k : ℕ hp : Prime p hk : 0 < k hpk : p ^ k = ↑a key : p ^ 1 ≤ ↑a ⊢ ∃ n, ↑a = ↑n ∧ ∃ p k, Nat.Prime p ∧ 0 < k ∧ p ^ k = n ** rw [power_one] at key ** case neg.intro.intro.intro.intro.intro a✝ b : Cardinal.{u} n m a : ℕ h : ¬ℵ₀ ≤ ↑a p : Cardinal.{u_1} k : ℕ hp : Prime p hk : 0 < k hpk : p ^ k = ↑a key : p ≤ ↑a ⊢ ∃ n, ↑a = ↑n ∧ ∃ p k, Nat.Prime p ∧ 0 < k ∧ p ^ k = n ** lift p to ℕ using key.trans_lt (nat_lt_aleph0 a) ** case neg.intro.intro.intro.intro.intro.intro a✝ b : Cardinal.{u} n m a : ℕ h : ¬ℵ₀ ≤ ↑a k : ℕ hk : 0 < k p : ℕ hp : Prime ↑p hpk : ↑p ^ k = ↑a key : ↑p ≤ ↑a ⊢ ∃ n, ↑a = ↑n ∧ ∃ p k, Nat.Prime p ∧ 0 < k ∧ p ^ k = n ** exact ⟨a, rfl, p, k, nat_is_prime_iff.mp hp, hk, by exact_mod_cast hpk⟩ ** case pos a✝ b : Cardinal.{u} n m : ℕ a : Cardinal.{u_1} h : ℵ₀ ≤ a ⊢ IsPrimePow a ↔ ℵ₀ ≤ a ∨ ∃ n, a = ↑n ∧ IsPrimePow n ** simp [h, (prime_of_aleph0_le h).isPrimePow] ** a✝ b : Cardinal.{u} n✝ m a : ℕ h✝ : ¬ℵ₀ ≤ ↑a x✝ : ∃ n, ↑a = ↑n ∧ ∃ p k, Nat.Prime p ∧ 0 < k ∧ p ^ k = n n : ℕ han : ↑a = ↑n p k : ℕ hp : Nat.Prime p hk : 0 < k h : p ^ k = n ⊢ ↑p ^ k = ↑a ** rw [han] ** a✝ b : Cardinal.{u} n✝ m a : ℕ h✝ : ¬ℵ₀ ≤ ↑a x✝ : ∃ n, ↑a = ↑n ∧ ∃ p k, Nat.Prime p ∧ 0 < k ∧ p ^ k = n n : ℕ han : ↑a = ↑n p k : ℕ hp : Nat.Prime p hk : 0 < k h : p ^ k = n ⊢ ↑p ^ k = ↑n ** exact_mod_cast h ** a✝ b : Cardinal.{u} n m a : ℕ h : ¬ℵ₀ ≤ ↑a p : Cardinal.{u_1} k : ℕ hp : Prime p hk : 0 < k hpk : p ^ k = ↑a ⊢ p ^ 1 ≤ ↑a ** rw [←hpk] ** a✝ b : Cardinal.{u} n m a : ℕ h : ¬ℵ₀ ≤ ↑a p : Cardinal.{u_1} k : ℕ hp : Prime p hk : 0 < k hpk : p ^ k = ↑a ⊢ p ^ 1 ≤ p ^ k ** apply power_le_power_left hp.ne_zero ** a✝ b : Cardinal.{u} n m a : ℕ h : ¬ℵ₀ ≤ ↑a p : Cardinal.{u_1} k : ℕ hp : Prime p hk : 0 < k hpk : p ^ k = ↑a ⊢ 1 ≤ ↑k ** exact_mod_cast hk ** a✝ b : Cardinal.{u} n m a : ℕ h : ¬ℵ₀ ≤ ↑a k : ℕ hk : 0 < k p : ℕ hp : Prime ↑p hpk : ↑p ^ k = ↑a key : ↑p ≤ ↑a ⊢ p ^ k = a ** exact_mod_cast hpk ** Qed
isOpen_lt ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderClosedTopology α inst✝ : TopologicalSpace β f g : β → α hf : Continuous f hg : Continuous g ⊢ IsOpen {b | f b < g b} ** simpa only [lt_iff_not_le] using (isClosed_le hg hf).isOpen_compl ** Qed
Ioo_subset_closure_interior ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderClosedTopology α a b : α ⊢ Ioo a b ⊆ closure (interior (Ioo a b)) ** simp only [interior_Ioo, subset_closure] ** Qed
Ioo_mem_nhdsWithin_Ioi ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderClosedTopology α a✝ b✝ : α inst✝ : TopologicalSpace γ a b c : α H : b ∈ Ico a c ⊢ Iio c ∩ Ioi b ⊆ Ioo a c ** rw [inter_comm, Ioi_inter_Iio] ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderClosedTopology α a✝ b✝ : α inst✝ : TopologicalSpace γ a b c : α H : b ∈ Ico a c ⊢ Ioo b c ⊆ Ioo a c ** exact Ioo_subset_Ioo_left H.1 ** Qed
continuousWithinAt_Ioc_iff_Ioi ** α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderClosedTopology α a✝ b✝ : α inst✝¹ : TopologicalSpace γ inst✝ : TopologicalSpace β a b : α f : α → β h : a < b ⊢ ContinuousWithinAt f (Ioc a b) a ↔ ContinuousWithinAt f (Ioi a) a ** simp only [ContinuousWithinAt, nhdsWithin_Ioc_eq_nhdsWithin_Ioi h] ** Qed
continuousWithinAt_Ioo_iff_Ioi ** α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderClosedTopology α a✝ b✝ : α inst✝¹ : TopologicalSpace γ inst✝ : TopologicalSpace β a b : α f : α → β h : a < b ⊢ ContinuousWithinAt f (Ioo a b) a ↔ ContinuousWithinAt f (Ioi a) a ** simp only [ContinuousWithinAt, nhdsWithin_Ioo_eq_nhdsWithin_Ioi h] ** Qed
Ioo_mem_nhdsWithin_Iio ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderClosedTopology α a✝ b✝ : α inst✝ : TopologicalSpace γ a b c : α H : b ∈ Ioc a c ⊢ Ioo a c ∈ 𝓝[Iio b] b ** simpa only [dual_Ioo] using Ioo_mem_nhdsWithin_Ioi (show toDual b ∈ Ico (toDual c) (toDual a) from H.symm) ** Qed
nhdsWithin_Ico_eq_nhdsWithin_Iio ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderClosedTopology α a✝ b✝ : α inst✝ : TopologicalSpace γ a b : α h : a < b ⊢ 𝓝[Ico a b] b = 𝓝[Iio b] b ** simpa only [dual_Ioc] using nhdsWithin_Ioc_eq_nhdsWithin_Ioi h.dual ** Qed
nhdsWithin_Ioo_eq_nhdsWithin_Iio ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderClosedTopology α a✝ b✝ : α inst✝ : TopologicalSpace γ a b : α h : a < b ⊢ 𝓝[Ioo a b] b = 𝓝[Iio b] b ** simpa only [dual_Ioo] using nhdsWithin_Ioo_eq_nhdsWithin_Ioi h.dual ** Qed
continuousWithinAt_Ico_iff_Iio ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderClosedTopology α a✝ b✝ : α inst✝ : TopologicalSpace γ a b : α f : α → γ h : a < b ⊢ ContinuousWithinAt f (Ico a b) b ↔ ContinuousWithinAt f (Iio b) b ** simp only [ContinuousWithinAt, nhdsWithin_Ico_eq_nhdsWithin_Iio h] ** Qed
continuousWithinAt_Ioo_iff_Iio ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderClosedTopology α a✝ b✝ : α inst✝ : TopologicalSpace γ a b : α f : α → γ h : a < b ⊢ ContinuousWithinAt f (Ioo a b) b ↔ ContinuousWithinAt f (Iio b) b ** simp only [ContinuousWithinAt, nhdsWithin_Ioo_eq_nhdsWithin_Iio h] ** Qed
Ico_mem_nhdsWithin_Ici ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderClosedTopology α a✝ b✝ : α inst✝ : TopologicalSpace γ a b c : α H : b ∈ Ico a c ⊢ Iio c ∩ Ici b ⊆ Ico a c ** simp only [inter_comm, Ici_inter_Iio, Ico_subset_Ico_left H.1] ** Qed
continuousWithinAt_Icc_iff_Ici ** α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderClosedTopology α a✝ b✝ : α inst✝¹ : TopologicalSpace γ inst✝ : TopologicalSpace β a b : α f : α → β h : a < b ⊢ ContinuousWithinAt f (Icc a b) a ↔ ContinuousWithinAt f (Ici a) a ** simp only [ContinuousWithinAt, nhdsWithin_Icc_eq_nhdsWithin_Ici h] ** Qed
continuousWithinAt_Ico_iff_Ici ** α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderClosedTopology α a✝ b✝ : α inst✝¹ : TopologicalSpace γ inst✝ : TopologicalSpace β a b : α f : α → β h : a < b ⊢ ContinuousWithinAt f (Ico a b) a ↔ ContinuousWithinAt f (Ici a) a ** simp only [ContinuousWithinAt, nhdsWithin_Ico_eq_nhdsWithin_Ici h] ** Qed
Ioc_mem_nhdsWithin_Iic ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderClosedTopology α a✝ b✝ : α inst✝ : TopologicalSpace γ a b c : α H : b ∈ Ioc a c ⊢ Ioc a c ∈ 𝓝[Iic b] b ** simpa only [dual_Ico] using Ico_mem_nhdsWithin_Ici (show toDual b ∈ Ico (toDual c) (toDual a) from H.symm) ** Qed
nhdsWithin_Icc_eq_nhdsWithin_Iic ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderClosedTopology α a✝ b✝ : α inst✝ : TopologicalSpace γ a b : α h : a < b ⊢ 𝓝[Icc a b] b = 𝓝[Iic b] b ** simpa only [dual_Icc] using nhdsWithin_Icc_eq_nhdsWithin_Ici h.dual ** Qed
nhdsWithin_Ioc_eq_nhdsWithin_Iic ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderClosedTopology α a✝ b✝ : α inst✝ : TopologicalSpace γ a b : α h : a < b ⊢ 𝓝[Ioc a b] b = 𝓝[Iic b] b ** simpa only [dual_Ico] using nhdsWithin_Ico_eq_nhdsWithin_Ici h.dual ** Qed
continuousWithinAt_Icc_iff_Iic ** α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderClosedTopology α a✝ b✝ : α inst✝¹ : TopologicalSpace γ inst✝ : TopologicalSpace β a b : α f : α → β h : a < b ⊢ ContinuousWithinAt f (Icc a b) b ↔ ContinuousWithinAt f (Iic b) b ** simp only [ContinuousWithinAt, nhdsWithin_Icc_eq_nhdsWithin_Iic h] ** Qed
continuousWithinAt_Ioc_iff_Iic ** α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderClosedTopology α a✝ b✝ : α inst✝¹ : TopologicalSpace γ inst✝ : TopologicalSpace β a b : α f : α → β h : a < b ⊢ ContinuousWithinAt f (Ioc a b) b ↔ ContinuousWithinAt f (Iic b) b ** simp only [ContinuousWithinAt, nhdsWithin_Ioc_eq_nhdsWithin_Iic h] ** Qed
frontier_le_subset_eq ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderClosedTopology α f g : β → α inst✝ : TopologicalSpace β hf : Continuous f hg : Continuous g ⊢ frontier {b | f b ≤ g b} ⊆ {b | f b = g b} ** rw [frontier_eq_closure_inter_closure, closure_le_eq hf hg] ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderClosedTopology α f g : β → α inst✝ : TopologicalSpace β hf : Continuous f hg : Continuous g ⊢ {b | f b ≤ g b} ∩ closure {b | f b ≤ g b}ᶜ ⊆ {b | f b = g b} ** rintro b ⟨hb₁, hb₂⟩ ** case intro α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderClosedTopology α f g : β → α inst✝ : TopologicalSpace β hf : Continuous f hg : Continuous g b : β hb₁ : b ∈ {b | f b ≤ g b} hb₂ : b ∈ closure {b | f b ≤ g b}ᶜ ⊢ b ∈ {b | f b = g b} ** refine' le_antisymm hb₁ (closure_lt_subset_le hg hf _) ** case intro α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderClosedTopology α f g : β → α inst✝ : TopologicalSpace β hf : Continuous f hg : Continuous g b : β hb₁ : b ∈ {b | f b ≤ g b} hb₂ : b ∈ closure {b | f b ≤ g b}ᶜ ⊢ b ∈ closure {b | g b < f b} ** convert hb₂ using 2 ** case h.e'_5.h.e'_3 α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderClosedTopology α f g : β → α inst✝ : TopologicalSpace β hf : Continuous f hg : Continuous g b : β hb₁ : b ∈ {b | f b ≤ g b} hb₂ : b ∈ closure {b | f b ≤ g b}ᶜ ⊢ {b | g b < f b} = {b | f b ≤ g b}ᶜ ** simp only [not_le.symm] ** case h.e'_5.h.e'_3 α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderClosedTopology α f g : β → α inst✝ : TopologicalSpace β hf : Continuous f hg : Continuous g b : β hb₁ : b ∈ {b | f b ≤ g b} hb₂ : b ∈ closure {b | f b ≤ g b}ᶜ ⊢ {b | ¬f b ≤ g b} = {b | f b ≤ g b}ᶜ ** rfl ** Qed
frontier_lt_subset_eq ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderClosedTopology α f g : β → α inst✝ : TopologicalSpace β hf : Continuous f hg : Continuous g ⊢ frontier {b | f b < g b} ⊆ {b | f b = g b} ** simpa only [← not_lt, ← compl_setOf, frontier_compl, eq_comm] using frontier_le_subset_eq hg hf ** Qed
continuous_if_le ** α : Type u β : Type v γ : Type w inst✝⁵ : TopologicalSpace α inst✝⁴ : LinearOrder α inst✝³ : OrderClosedTopology α f g : β → α inst✝² : TopologicalSpace β inst✝¹ : TopologicalSpace γ inst✝ : (x : β) → Decidable (f x ≤ g x) f' g' : β → γ hf : Continuous f hg : Continuous g hf' : ContinuousOn f' {x | f x ≤ g x} hg' : ContinuousOn g' {x | g x ≤ f x} hfg : ∀ (x : β), f x = g x → f' x = g' x ⊢ Continuous fun x => if f x ≤ g x then f' x else g' x ** refine' continuous_if (fun a ha => hfg _ (frontier_le_subset_eq hf hg ha)) _ (hg'.mono _) ** case refine'_1 α : Type u β : Type v γ : Type w inst✝⁵ : TopologicalSpace α inst✝⁴ : LinearOrder α inst✝³ : OrderClosedTopology α f g : β → α inst✝² : TopologicalSpace β inst✝¹ : TopologicalSpace γ inst✝ : (x : β) → Decidable (f x ≤ g x) f' g' : β → γ hf : Continuous f hg : Continuous g hf' : ContinuousOn f' {x | f x ≤ g x} hg' : ContinuousOn g' {x | g x ≤ f x} hfg : ∀ (x : β), f x = g x → f' x = g' x ⊢ ContinuousOn (fun x => f' x) (closure {x | f x ≤ g x}) ** rwa [(isClosed_le hf hg).closure_eq] ** case refine'_2 α : Type u β : Type v γ : Type w inst✝⁵ : TopologicalSpace α inst✝⁴ : LinearOrder α inst✝³ : OrderClosedTopology α f g : β → α inst✝² : TopologicalSpace β inst✝¹ : TopologicalSpace γ inst✝ : (x : β) → Decidable (f x ≤ g x) f' g' : β → γ hf : Continuous f hg : Continuous g hf' : ContinuousOn f' {x | f x ≤ g x} hg' : ContinuousOn g' {x | g x ≤ f x} hfg : ∀ (x : β), f x = g x → f' x = g' x ⊢ closure {x | ¬f x ≤ g x} ⊆ {x | g x ≤ f x} ** simp only [not_le] ** case refine'_2 α : Type u β : Type v γ : Type w inst✝⁵ : TopologicalSpace α inst✝⁴ : LinearOrder α inst✝³ : OrderClosedTopology α f g : β → α inst✝² : TopologicalSpace β inst✝¹ : TopologicalSpace γ inst✝ : (x : β) → Decidable (f x ≤ g x) f' g' : β → γ hf : Continuous f hg : Continuous g hf' : ContinuousOn f' {x | f x ≤ g x} hg' : ContinuousOn g' {x | g x ≤ f x} hfg : ∀ (x : β), f x = g x → f' x = g' x ⊢ closure {x | g x < f x} ⊆ {x | g x ≤ f x} ** exact closure_lt_subset_le hg hf ** Qed
Continuous.min ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderClosedTopology α f g : β → α inst✝ : TopologicalSpace β hf : Continuous f hg : Continuous g ⊢ Continuous fun b => min (f b) (g b) ** simp only [min_def] ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderClosedTopology α f g : β → α inst✝ : TopologicalSpace β hf : Continuous f hg : Continuous g ⊢ Continuous fun b => if f b ≤ g b then f b else g b ** exact hf.if_le hg hf hg fun x => id ** Qed
Filter.Tendsto.max_right ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderClosedTopology α f g : β → α l : Filter β a : α h : Tendsto f l (𝓝 a) ⊢ Tendsto (fun i => max a (f i)) l (𝓝 a) ** convert ((continuous_max.comp (@Continuous.Prod.mk α α _ _ a)).tendsto a).comp h ** case h.e'_5.h.e'_3 α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderClosedTopology α f g : β → α l : Filter β a : α h : Tendsto f l (𝓝 a) ⊢ a = ((fun p => max p.1 p.2) ∘ fun b => (a, b)) a ** simp ** Qed
Filter.Tendsto.max_left ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderClosedTopology α f g : β → α l : Filter β a : α h : Tendsto f l (𝓝 a) ⊢ Tendsto (fun i => max (f i) a) l (𝓝 a) ** simp_rw [max_comm _ a] ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderClosedTopology α f g : β → α l : Filter β a : α h : Tendsto f l (𝓝 a) ⊢ Tendsto (fun i => max a (f i)) l (𝓝 a) ** exact h.max_right ** Qed
Filter.tendsto_nhds_max_right ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderClosedTopology α f g : β → α l : Filter β a : α h : Tendsto f l (𝓝[Ioi a] a) ⊢ Tendsto (fun i => max a (f i)) l (𝓝[Ioi a] a) ** obtain ⟨h₁ : Tendsto f l (𝓝 a), h₂ : ∀ᶠ i in l, f i ∈ Ioi a⟩ := tendsto_nhdsWithin_iff.mp h ** case intro α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderClosedTopology α f g : β → α l : Filter β a : α h : Tendsto f l (𝓝[Ioi a] a) h₁ : Tendsto f l (𝓝 a) h₂ : ∀ᶠ (i : β) in l, f i ∈ Ioi a ⊢ Tendsto (fun i => max a (f i)) l (𝓝[Ioi a] a) ** exact tendsto_nhdsWithin_iff.mpr ⟨h₁.max_right, h₂.mono fun i hi => lt_max_of_lt_right hi⟩ ** Qed
Filter.tendsto_nhds_max_left ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderClosedTopology α f g : β → α l : Filter β a : α h : Tendsto f l (𝓝[Ioi a] a) ⊢ Tendsto (fun i => max (f i) a) l (𝓝[Ioi a] a) ** simp_rw [max_comm _ a] ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderClosedTopology α f g : β → α l : Filter β a : α h : Tendsto f l (𝓝[Ioi a] a) ⊢ Tendsto (fun i => max a (f i)) l (𝓝[Ioi a] a) ** exact Filter.tendsto_nhds_max_right h ** Qed
Dense.exists_le' ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderClosedTopology α f g : β → α s : Set α hs : Dense s hbot : ∀ (x : α), IsBot x → x ∈ s x : α ⊢ ∃ y, y ∈ s ∧ y ≤ x ** by_cases hx : IsBot x ** case pos α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderClosedTopology α f g : β → α s : Set α hs : Dense s hbot : ∀ (x : α), IsBot x → x ∈ s x : α hx : IsBot x ⊢ ∃ y, y ∈ s ∧ y ≤ x ** exact ⟨x, hbot x hx, le_rfl⟩ ** case neg α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderClosedTopology α f g : β → α s : Set α hs : Dense s hbot : ∀ (x : α), IsBot x → x ∈ s x : α hx : ¬IsBot x ⊢ ∃ y, y ∈ s ∧ y ≤ x ** simp only [IsBot, not_forall, not_le] at hx ** case neg α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderClosedTopology α f g : β → α s : Set α hs : Dense s hbot : ∀ (x : α), IsBot x → x ∈ s x : α hx : ∃ x_1, x_1 < x ⊢ ∃ y, y ∈ s ∧ y ≤ x ** rcases hs.exists_mem_open isOpen_Iio hx with ⟨y, hys, hy : y < x⟩ ** case neg.intro.intro α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderClosedTopology α f g : β → α s : Set α hs : Dense s hbot : ∀ (x : α), IsBot x → x ∈ s x : α hx : ∃ x_1, x_1 < x y : α hys : y ∈ s hy : y < x ⊢ ∃ y, y ∈ s ∧ y ≤ x ** exact ⟨y, hys, hy.le⟩ ** Qed
Dense.Ioi_eq_biUnion ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderClosedTopology α f g : β → α inst✝ : DenselyOrdered α s : Set α hs : Dense s x : α ⊢ Ioi x = ⋃ y ∈ s ∩ Ioi x, Ioi y ** refine Subset.antisymm (fun z hz ↦ ?_) (iUnion₂_subset fun y hy ↦ Ioi_subset_Ioi (le_of_lt hy.2)) ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderClosedTopology α f g : β → α inst✝ : DenselyOrdered α s : Set α hs : Dense s x z : α hz : z ∈ Ioi x ⊢ z ∈ ⋃ y ∈ s ∩ Ioi x, Ioi y ** rcases hs.exists_between hz with ⟨y, hys, hxy, hyz⟩ ** case intro.intro.intro α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderClosedTopology α f g : β → α inst✝ : DenselyOrdered α s : Set α hs : Dense s x z : α hz : z ∈ Ioi x y : α hys : y ∈ s hxy : x < y hyz : y < z ⊢ z ∈ ⋃ y ∈ s ∩ Ioi x, Ioi y ** exact mem_iUnion₂.2 ⟨y, ⟨hys, hxy⟩, hyz⟩ ** Qed
isOpen_iff_generate_intervals ** α : Type u β : Type v γ : Type w inst✝¹ : TopologicalSpace α inst✝ : Preorder α t : OrderTopology α s : Set α ⊢ IsOpen s ↔ GenerateOpen {s | ∃ a, s = Ioi a ∨ s = Iio a} s ** rfl ** Qed
nhds_eq_order ** α : Type u β : Type v γ : Type w inst✝¹ : TopologicalSpace α inst✝ : Preorder α t : OrderTopology α a : α ⊢ 𝓝 a = (⨅ b ∈ Iio a, 𝓟 (Ioi b)) ⊓ ⨅ b ∈ Ioi a, 𝓟 (Iio b) ** rw [t.topology_eq_generate_intervals, nhds_generateFrom] ** α : Type u β : Type v γ : Type w inst✝¹ : TopologicalSpace α inst✝ : Preorder α t : OrderTopology α a : α ⊢ ⨅ s ∈ {s | a ∈ s ∧ s ∈ {s | ∃ a, s = Ioi a ∨ s = Iio a}}, 𝓟 s = (⨅ b ∈ Iio a, 𝓟 (Ioi b)) ⊓ ⨅ b ∈ Ioi a, 𝓟 (Iio b) ** simp_rw [mem_setOf_eq, @and_comm (a ∈ _), exists_or, or_and_right, iInf_or, iInf_and, iInf_exists, iInf_inf_eq, iInf_comm (ι := Set α), iInf_iInf_eq_left, mem_Ioi, mem_Iio] ** Qed
tendsto_order ** α : Type u β : Type v γ : Type w inst✝¹ : TopologicalSpace α inst✝ : Preorder α t : OrderTopology α f : β → α a : α x : Filter β ⊢ Tendsto f x (𝓝 a) ↔ (∀ (a' : α), a' < a → ∀ᶠ (b : β) in x, a' < f b) ∧ ∀ (a' : α), a' > a → ∀ᶠ (b : β) in x, f b < a' ** simp only [nhds_eq_order a, tendsto_inf, tendsto_iInf, tendsto_principal] ** α : Type u β : Type v γ : Type w inst✝¹ : TopologicalSpace α inst✝ : Preorder α t : OrderTopology α f : β → α a : α x : Filter β ⊢ ((∀ (i : α), i ∈ Iio a → ∀ᶠ (a : β) in x, f a ∈ Ioi i) ∧ ∀ (i : α), i ∈ Ioi a → ∀ᶠ (a : β) in x, f a ∈ Iio i) ↔ (∀ (a' : α), a' < a → ∀ᶠ (b : β) in x, a' < f b) ∧ ∀ (a' : α), a' > a → ∀ᶠ (b : β) in x, f b < a' ** rfl ** Qed
nhds_order_unbounded ** α : Type u β : Type v γ : Type w inst✝¹ : TopologicalSpace α inst✝ : Preorder α t : OrderTopology α a : α hu : ∃ u, a < u hl : ∃ l, l < a ⊢ 𝓝 a = ⨅ l, ⨅ (_ : l < a), ⨅ u, ⨅ (_ : a < u), 𝓟 (Ioo l u) ** simp only [nhds_eq_order, ← inf_biInf, ← biInf_inf, *, ← inf_principal, ← Ioi_inter_Iio] ** α : Type u β : Type v γ : Type w inst✝¹ : TopologicalSpace α inst✝ : Preorder α t : OrderTopology α a : α hu : ∃ u, a < u hl : ∃ l, l < a ⊢ (⨅ b ∈ Iio a, 𝓟 (Ioi b)) ⊓ ⨅ b ∈ Ioi a, 𝓟 (Iio b) = (⨅ i, ⨅ (_ : i < a), 𝓟 (Ioi i)) ⊓ ⨅ i, ⨅ (_ : a < i), 𝓟 (Iio i) ** rfl ** Qed
tendsto_order_unbounded ** α : Type u β : Type v γ : Type w inst✝¹ : TopologicalSpace α inst✝ : Preorder α t : OrderTopology α f : β → α a : α x : Filter β hu : ∃ u, a < u hl : ∃ l, l < a h : ∀ (l u : α), l < a → a < u → ∀ᶠ (b : β) in x, l < f b ∧ f b < u ⊢ Tendsto f x (𝓝 a) ** simp only [nhds_order_unbounded hu hl, tendsto_iInf, tendsto_principal] ** α : Type u β : Type v γ : Type w inst✝¹ : TopologicalSpace α inst✝ : Preorder α t : OrderTopology α f : β → α a : α x : Filter β hu : ∃ u, a < u hl : ∃ l, l < a h : ∀ (l u : α), l < a → a < u → ∀ᶠ (b : β) in x, l < f b ∧ f b < u ⊢ ∀ (i : α), i < a → ∀ (i_2 : α), a < i_2 → ∀ᶠ (a : β) in x, f a ∈ Ioo i i_2 ** exact fun l hl u => h l u hl ** Qed
induced_topology_le_preorder ** α : Type u β : Type v γ : Type w inst✝³ : Preorder α inst✝² : Preorder β inst✝¹ : TopologicalSpace β inst✝ : OrderTopology β f : α → β hf : ∀ {x y : α}, f x < f y ↔ x < y ⊢ induced f inst✝¹ ≤ Preorder.topology α ** let _ := Preorder.topology α ** α : Type u β : Type v γ : Type w inst✝³ : Preorder α inst✝² : Preorder β inst✝¹ : TopologicalSpace β inst✝ : OrderTopology β f : α → β hf : ∀ {x y : α}, f x < f y ↔ x < y x✝ : TopologicalSpace α := Preorder.topology α ⊢ induced f inst✝¹ ≤ Preorder.topology α ** have : OrderTopology α := ⟨rfl⟩ ** α : Type u β : Type v γ : Type w inst✝³ : Preorder α inst✝² : Preorder β inst✝¹ : TopologicalSpace β inst✝ : OrderTopology β f : α → β hf : ∀ {x y : α}, f x < f y ↔ x < y x✝ : TopologicalSpace α := Preorder.topology α this : OrderTopology α ⊢ induced f inst✝¹ ≤ Preorder.topology α ** refine le_of_nhds_le_nhds fun x => ?_ ** α : Type u β : Type v γ : Type w inst✝³ : Preorder α inst✝² : Preorder β inst✝¹ : TopologicalSpace β inst✝ : OrderTopology β f : α → β hf : ∀ {x y : α}, f x < f y ↔ x < y x✝ : TopologicalSpace α := Preorder.topology α this : OrderTopology α x : α ⊢ 𝓝 x ≤ 𝓝 x ** simp only [nhds_eq_order, nhds_induced, comap_inf, comap_iInf, comap_principal, Ioi, Iio, ← hf] ** α : Type u β : Type v γ : Type w inst✝³ : Preorder α inst✝² : Preorder β inst✝¹ : TopologicalSpace β inst✝ : OrderTopology β f : α → β hf : ∀ {x y : α}, f x < f y ↔ x < y x✝ : TopologicalSpace α := Preorder.topology α this : OrderTopology α x : α ⊢ (⨅ i ∈ {x_1 | x_1 < f x}, 𝓟 (f ⁻¹' {x | i < x})) ⊓ ⨅ i ∈ {x_1 | f x < x_1}, 𝓟 (f ⁻¹' {x | x < i}) ≤ (⨅ b ∈ {x_1 | f x_1 < f x}, 𝓟 {x | f b < f x}) ⊓ ⨅ b ∈ {x_1 | f x < f x_1}, 𝓟 {x | f x < f b} ** refine inf_le_inf (le_iInf₂ fun a ha => ?_) (le_iInf₂ fun a ha => ?_) ** case refine_1 α : Type u β : Type v γ : Type w inst✝³ : Preorder α inst✝² : Preorder β inst✝¹ : TopologicalSpace β inst✝ : OrderTopology β f : α → β hf : ∀ {x y : α}, f x < f y ↔ x < y x✝ : TopologicalSpace α := Preorder.topology α this : OrderTopology α x a : α ha : a ∈ {x_1 | f x_1 < f x} ⊢ ⨅ i ∈ {x_1 | x_1 < f x}, 𝓟 (f ⁻¹' {x | i < x}) ≤ 𝓟 {x | f a < f x} case refine_2 α : Type u β : Type v γ : Type w inst✝³ : Preorder α inst✝² : Preorder β inst✝¹ : TopologicalSpace β inst✝ : OrderTopology β f : α → β hf : ∀ {x y : α}, f x < f y ↔ x < y x✝ : TopologicalSpace α := Preorder.topology α this : OrderTopology α x a : α ha : a ∈ {x_1 | f x < f x_1} ⊢ ⨅ i ∈ {x_1 | f x < x_1}, 𝓟 (f ⁻¹' {x | x < i}) ≤ 𝓟 {x | f x < f a} ** exacts [iInf₂_le (f a) ha, iInf₂_le (f a) ha] ** Qed
induced_topology_eq_preorder ** α : Type u β : Type v γ : Type w inst✝³ : Preorder α inst✝² : Preorder β inst✝¹ : TopologicalSpace β inst✝ : OrderTopology β f : α → β hf : ∀ {x y : α}, f x < f y ↔ x < y H₁ : ∀ {a : α} {b : β} {x : α}, b < f a → ¬b < f x → ∃ y, y < a ∧ b ≤ f y H₂ : ∀ {a : α} {b : β} {x : α}, f a < b → ¬f x < b → ∃ y, a < y ∧ f y ≤ b ⊢ induced f inst✝¹ = Preorder.topology α ** let _ := Preorder.topology α ** α : Type u β : Type v γ : Type w inst✝³ : Preorder α inst✝² : Preorder β inst✝¹ : TopologicalSpace β inst✝ : OrderTopology β f : α → β hf : ∀ {x y : α}, f x < f y ↔ x < y H₁ : ∀ {a : α} {b : β} {x : α}, b < f a → ¬b < f x → ∃ y, y < a ∧ b ≤ f y H₂ : ∀ {a : α} {b : β} {x : α}, f a < b → ¬f x < b → ∃ y, a < y ∧ f y ≤ b x✝ : TopologicalSpace α := Preorder.topology α ⊢ induced f inst✝¹ = Preorder.topology α ** have : OrderTopology α := ⟨rfl⟩ ** α : Type u β : Type v γ : Type w inst✝³ : Preorder α inst✝² : Preorder β inst✝¹ : TopologicalSpace β inst✝ : OrderTopology β f : α → β hf : ∀ {x y : α}, f x < f y ↔ x < y H₁ : ∀ {a : α} {b : β} {x : α}, b < f a → ¬b < f x → ∃ y, y < a ∧ b ≤ f y H₂ : ∀ {a : α} {b : β} {x : α}, f a < b → ¬f x < b → ∃ y, a < y ∧ f y ≤ b x✝ : TopologicalSpace α := Preorder.topology α this : OrderTopology α ⊢ induced f inst✝¹ = Preorder.topology α ** refine le_antisymm (induced_topology_le_preorder hf) ?_ ** α : Type u β : Type v γ : Type w inst✝³ : Preorder α inst✝² : Preorder β inst✝¹ : TopologicalSpace β inst✝ : OrderTopology β f : α → β hf : ∀ {x y : α}, f x < f y ↔ x < y H₁ : ∀ {a : α} {b : β} {x : α}, b < f a → ¬b < f x → ∃ y, y < a ∧ b ≤ f y H₂ : ∀ {a : α} {b : β} {x : α}, f a < b → ¬f x < b → ∃ y, a < y ∧ f y ≤ b x✝ : TopologicalSpace α := Preorder.topology α this : OrderTopology α ⊢ Preorder.topology α ≤ induced f inst✝¹ ** refine le_of_nhds_le_nhds fun a => ?_ ** α : Type u β : Type v γ : Type w inst✝³ : Preorder α inst✝² : Preorder β inst✝¹ : TopologicalSpace β inst✝ : OrderTopology β f : α → β hf : ∀ {x y : α}, f x < f y ↔ x < y H₁ : ∀ {a : α} {b : β} {x : α}, b < f a → ¬b < f x → ∃ y, y < a ∧ b ≤ f y H₂ : ∀ {a : α} {b : β} {x : α}, f a < b → ¬f x < b → ∃ y, a < y ∧ f y ≤ b x✝ : TopologicalSpace α := Preorder.topology α this : OrderTopology α a : α ⊢ 𝓝 a ≤ 𝓝 a ** simp only [nhds_eq_order, nhds_induced, comap_inf, comap_iInf, comap_principal] ** α : Type u β : Type v γ : Type w inst✝³ : Preorder α inst✝² : Preorder β inst✝¹ : TopologicalSpace β inst✝ : OrderTopology β f : α → β hf : ∀ {x y : α}, f x < f y ↔ x < y H₁ : ∀ {a : α} {b : β} {x : α}, b < f a → ¬b < f x → ∃ y, y < a ∧ b ≤ f y H₂ : ∀ {a : α} {b : β} {x : α}, f a < b → ¬f x < b → ∃ y, a < y ∧ f y ≤ b x✝ : TopologicalSpace α := Preorder.topology α this : OrderTopology α a : α ⊢ (⨅ b ∈ Iio a, 𝓟 (Ioi b)) ⊓ ⨅ b ∈ Ioi a, 𝓟 (Iio b) ≤ (⨅ i ∈ Iio (f a), 𝓟 (f ⁻¹' Ioi i)) ⊓ ⨅ i ∈ Ioi (f a), 𝓟 (f ⁻¹' Iio i) ** refine inf_le_inf (le_iInf₂ fun b hb => ?_) (le_iInf₂ fun b hb => ?_) ** case refine_1 α : Type u β : Type v γ : Type w inst✝³ : Preorder α inst✝² : Preorder β inst✝¹ : TopologicalSpace β inst✝ : OrderTopology β f : α → β hf : ∀ {x y : α}, f x < f y ↔ x < y H₁ : ∀ {a : α} {b : β} {x : α}, b < f a → ¬b < f x → ∃ y, y < a ∧ b ≤ f y H₂ : ∀ {a : α} {b : β} {x : α}, f a < b → ¬f x < b → ∃ y, a < y ∧ f y ≤ b x✝ : TopologicalSpace α := Preorder.topology α this : OrderTopology α a : α b : β hb : b ∈ Iio (f a) ⊢ ⨅ b ∈ Iio a, 𝓟 (Ioi b) ≤ 𝓟 (f ⁻¹' Ioi b) ** rcases em (∃ x, ¬(b < f x)) with (⟨x, hx⟩ | hb) ** case refine_1.inl.intro α : Type u β : Type v γ : Type w inst✝³ : Preorder α inst✝² : Preorder β inst✝¹ : TopologicalSpace β inst✝ : OrderTopology β f : α → β hf : ∀ {x y : α}, f x < f y ↔ x < y H₁ : ∀ {a : α} {b : β} {x : α}, b < f a → ¬b < f x → ∃ y, y < a ∧ b ≤ f y H₂ : ∀ {a : α} {b : β} {x : α}, f a < b → ¬f x < b → ∃ y, a < y ∧ f y ≤ b x✝ : TopologicalSpace α := Preorder.topology α this : OrderTopology α a : α b : β hb : b ∈ Iio (f a) x : α hx : ¬b < f x ⊢ ⨅ b ∈ Iio a, 𝓟 (Ioi b) ≤ 𝓟 (f ⁻¹' Ioi b) ** rcases H₁ hb hx with ⟨y, hya, hyb⟩ ** case refine_1.inl.intro.intro.intro α : Type u β : Type v γ : Type w inst✝³ : Preorder α inst✝² : Preorder β inst✝¹ : TopologicalSpace β inst✝ : OrderTopology β f : α → β hf : ∀ {x y : α}, f x < f y ↔ x < y H₁ : ∀ {a : α} {b : β} {x : α}, b < f a → ¬b < f x → ∃ y, y < a ∧ b ≤ f y H₂ : ∀ {a : α} {b : β} {x : α}, f a < b → ¬f x < b → ∃ y, a < y ∧ f y ≤ b x✝ : TopologicalSpace α := Preorder.topology α this : OrderTopology α a : α b : β hb : b ∈ Iio (f a) x : α hx : ¬b < f x y : α hya : y < a hyb : b ≤ f y ⊢ ⨅ b ∈ Iio a, 𝓟 (Ioi b) ≤ 𝓟 (f ⁻¹' Ioi b) ** exact iInf₂_le_of_le y hya (principal_mono.2 fun z hz => hyb.trans_lt (hf.2 hz)) ** case refine_1.inr α : Type u β : Type v γ : Type w inst✝³ : Preorder α inst✝² : Preorder β inst✝¹ : TopologicalSpace β inst✝ : OrderTopology β f : α → β hf : ∀ {x y : α}, f x < f y ↔ x < y H₁ : ∀ {a : α} {b : β} {x : α}, b < f a → ¬b < f x → ∃ y, y < a ∧ b ≤ f y H₂ : ∀ {a : α} {b : β} {x : α}, f a < b → ¬f x < b → ∃ y, a < y ∧ f y ≤ b x✝ : TopologicalSpace α := Preorder.topology α this : OrderTopology α a : α b : β hb✝ : b ∈ Iio (f a) hb : ¬∃ x, ¬b < f x ⊢ ⨅ b ∈ Iio a, 𝓟 (Ioi b) ≤ 𝓟 (f ⁻¹' Ioi b) ** push_neg at hb ** case refine_1.inr α : Type u β : Type v γ : Type w inst✝³ : Preorder α inst✝² : Preorder β inst✝¹ : TopologicalSpace β inst✝ : OrderTopology β f : α → β hf : ∀ {x y : α}, f x < f y ↔ x < y H₁ : ∀ {a : α} {b : β} {x : α}, b < f a → ¬b < f x → ∃ y, y < a ∧ b ≤ f y H₂ : ∀ {a : α} {b : β} {x : α}, f a < b → ¬f x < b → ∃ y, a < y ∧ f y ≤ b x✝ : TopologicalSpace α := Preorder.topology α this : OrderTopology α a : α b : β hb✝ : b ∈ Iio (f a) hb : ∀ (x : α), b < f x ⊢ ⨅ b ∈ Iio a, 𝓟 (Ioi b) ≤ 𝓟 (f ⁻¹' Ioi b) ** exact le_principal_iff.2 (univ_mem' hb) ** case refine_2 α : Type u β : Type v γ : Type w inst✝³ : Preorder α inst✝² : Preorder β inst✝¹ : TopologicalSpace β inst✝ : OrderTopology β f : α → β hf : ∀ {x y : α}, f x < f y ↔ x < y H₁ : ∀ {a : α} {b : β} {x : α}, b < f a → ¬b < f x → ∃ y, y < a ∧ b ≤ f y H₂ : ∀ {a : α} {b : β} {x : α}, f a < b → ¬f x < b → ∃ y, a < y ∧ f y ≤ b x✝ : TopologicalSpace α := Preorder.topology α this : OrderTopology α a : α b : β hb : b ∈ Ioi (f a) ⊢ ⨅ b ∈ Ioi a, 𝓟 (Iio b) ≤ 𝓟 (f ⁻¹' Iio b) ** rcases em (∃ x, ¬(f x < b)) with (⟨x, hx⟩ | hb) ** case refine_2.inl.intro α : Type u β : Type v γ : Type w inst✝³ : Preorder α inst✝² : Preorder β inst✝¹ : TopologicalSpace β inst✝ : OrderTopology β f : α → β hf : ∀ {x y : α}, f x < f y ↔ x < y H₁ : ∀ {a : α} {b : β} {x : α}, b < f a → ¬b < f x → ∃ y, y < a ∧ b ≤ f y H₂ : ∀ {a : α} {b : β} {x : α}, f a < b → ¬f x < b → ∃ y, a < y ∧ f y ≤ b x✝ : TopologicalSpace α := Preorder.topology α this : OrderTopology α a : α b : β hb : b ∈ Ioi (f a) x : α hx : ¬f x < b ⊢ ⨅ b ∈ Ioi a, 𝓟 (Iio b) ≤ 𝓟 (f ⁻¹' Iio b) ** rcases H₂ hb hx with ⟨y, hya, hyb⟩ ** case refine_2.inl.intro.intro.intro α : Type u β : Type v γ : Type w inst✝³ : Preorder α inst✝² : Preorder β inst✝¹ : TopologicalSpace β inst✝ : OrderTopology β f : α → β hf : ∀ {x y : α}, f x < f y ↔ x < y H₁ : ∀ {a : α} {b : β} {x : α}, b < f a → ¬b < f x → ∃ y, y < a ∧ b ≤ f y H₂ : ∀ {a : α} {b : β} {x : α}, f a < b → ¬f x < b → ∃ y, a < y ∧ f y ≤ b x✝ : TopologicalSpace α := Preorder.topology α this : OrderTopology α a : α b : β hb : b ∈ Ioi (f a) x : α hx : ¬f x < b y : α hya : a < y hyb : f y ≤ b ⊢ ⨅ b ∈ Ioi a, 𝓟 (Iio b) ≤ 𝓟 (f ⁻¹' Iio b) ** exact iInf₂_le_of_le y hya (principal_mono.2 fun z hz => (hf.2 hz).trans_le hyb) ** case refine_2.inr α : Type u β : Type v γ : Type w inst✝³ : Preorder α inst✝² : Preorder β inst✝¹ : TopologicalSpace β inst✝ : OrderTopology β f : α → β hf : ∀ {x y : α}, f x < f y ↔ x < y H₁ : ∀ {a : α} {b : β} {x : α}, b < f a → ¬b < f x → ∃ y, y < a ∧ b ≤ f y H₂ : ∀ {a : α} {b : β} {x : α}, f a < b → ¬f x < b → ∃ y, a < y ∧ f y ≤ b x✝ : TopologicalSpace α := Preorder.topology α this : OrderTopology α a : α b : β hb✝ : b ∈ Ioi (f a) hb : ¬∃ x, ¬f x < b ⊢ ⨅ b ∈ Ioi a, 𝓟 (Iio b) ≤ 𝓟 (f ⁻¹' Iio b) ** push_neg at hb ** case refine_2.inr α : Type u β : Type v γ : Type w inst✝³ : Preorder α inst✝² : Preorder β inst✝¹ : TopologicalSpace β inst✝ : OrderTopology β f : α → β hf : ∀ {x y : α}, f x < f y ↔ x < y H₁ : ∀ {a : α} {b : β} {x : α}, b < f a → ¬b < f x → ∃ y, y < a ∧ b ≤ f y H₂ : ∀ {a : α} {b : β} {x : α}, f a < b → ¬f x < b → ∃ y, a < y ∧ f y ≤ b x✝ : TopologicalSpace α := Preorder.topology α this : OrderTopology α a : α b : β hb✝ : b ∈ Ioi (f a) hb : ∀ (x : α), f x < b ⊢ ⨅ b ∈ Ioi a, 𝓟 (Iio b) ≤ 𝓟 (f ⁻¹' Iio b) ** exact le_principal_iff.2 (univ_mem' hb) ** Qed
StrictMono.induced_topology_eq_preorder ** α✝ : Type u β✝ : Type v γ : Type w α : Type u_1 β : Type u_2 inst✝² : LinearOrder α inst✝¹ : LinearOrder β t : TopologicalSpace β inst✝ : OrderTopology β f : α → β hf : StrictMono f hc : OrdConnected (range f) ⊢ induced f t = Preorder.topology α ** refine induced_topology_eq_preorder hf.lt_iff_lt (fun h₁ h₂ => ?_) fun h₁ h₂ => ?_ ** case refine_1 α✝ : Type u β✝ : Type v γ : Type w α : Type u_1 β : Type u_2 inst✝² : LinearOrder α inst✝¹ : LinearOrder β t : TopologicalSpace β inst✝ : OrderTopology β f : α → β hf : StrictMono f hc : OrdConnected (range f) a✝ : α b✝ : β x✝ : α h₁ : b✝ < f a✝ h₂ : ¬b✝ < f x✝ ⊢ ∃ y, y < a✝ ∧ b✝ ≤ f y ** rcases hc.out (mem_range_self _) (mem_range_self _) ⟨not_lt.1 h₂, h₁.le⟩ with ⟨y, rfl⟩ ** case refine_1.intro α✝ : Type u β✝ : Type v γ : Type w α : Type u_1 β : Type u_2 inst✝² : LinearOrder α inst✝¹ : LinearOrder β t : TopologicalSpace β inst✝ : OrderTopology β f : α → β hf : StrictMono f hc : OrdConnected (range f) a✝ x✝ y : α h₁ : f y < f a✝ h₂ : ¬f y < f x✝ ⊢ ∃ y_1, y_1 < a✝ ∧ f y ≤ f y_1 ** exact ⟨y, hf.lt_iff_lt.1 h₁, le_rfl⟩ ** case refine_2 α✝ : Type u β✝ : Type v γ : Type w α : Type u_1 β : Type u_2 inst✝² : LinearOrder α inst✝¹ : LinearOrder β t : TopologicalSpace β inst✝ : OrderTopology β f : α → β hf : StrictMono f hc : OrdConnected (range f) a✝ : α b✝ : β x✝ : α h₁ : f a✝ < b✝ h₂ : ¬f x✝ < b✝ ⊢ ∃ y, a✝ < y ∧ f y ≤ b✝ ** rcases hc.out (mem_range_self _) (mem_range_self _) ⟨h₁.le, not_lt.1 h₂⟩ with ⟨y, rfl⟩ ** case refine_2.intro α✝ : Type u β✝ : Type v γ : Type w α : Type u_1 β : Type u_2 inst✝² : LinearOrder α inst✝¹ : LinearOrder β t : TopologicalSpace β inst✝ : OrderTopology β f : α → β hf : StrictMono f hc : OrdConnected (range f) a✝ x✝ y : α h₁ : f a✝ < f y h₂ : ¬f x✝ < f y ⊢ ∃ y_1, a✝ < y_1 ∧ f y_1 ≤ f y ** exact ⟨y, hf.lt_iff_lt.1 h₁, le_rfl⟩ ** Qed
nhdsWithin_Ici_eq'' ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : Preorder α inst✝ : OrderTopology α a : α ⊢ 𝓝[Ici a] a = (⨅ u, ⨅ (_ : a < u), 𝓟 (Iio u)) ⊓ 𝓟 (Ici a) ** rw [nhdsWithin, nhds_eq_order] ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : Preorder α inst✝ : OrderTopology α a : α ⊢ ((⨅ b ∈ Iio a, 𝓟 (Ioi b)) ⊓ ⨅ b ∈ Ioi a, 𝓟 (Iio b)) ⊓ 𝓟 (Ici a) = (⨅ u, ⨅ (_ : a < u), 𝓟 (Iio u)) ⊓ 𝓟 (Ici a) ** refine' le_antisymm (inf_le_inf_right _ inf_le_right) (le_inf (le_inf _ inf_le_left) inf_le_right) ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : Preorder α inst✝ : OrderTopology α a : α ⊢ (⨅ u, ⨅ (_ : a < u), 𝓟 (Iio u)) ⊓ 𝓟 (Ici a) ≤ ⨅ b ∈ Iio a, 𝓟 (Ioi b) ** exact inf_le_right.trans (le_iInf₂ fun l hl => principal_mono.2 <| Ici_subset_Ioi.2 hl) ** Qed
nhdsWithin_Ici_eq' ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : Preorder α inst✝ : OrderTopology α a : α ha : ∃ u, a < u ⊢ 𝓝[Ici a] a = ⨅ u, ⨅ (_ : a < u), 𝓟 (Ico a u) ** simp only [nhdsWithin_Ici_eq'', biInf_inf ha, inf_principal, Iio_inter_Ici] ** Qed
nhdsWithin_Iic_eq' ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : Preorder α inst✝ : OrderTopology α a : α ha : ∃ l, l < a ⊢ 𝓝[Iic a] a = ⨅ l, ⨅ (_ : l < a), 𝓟 (Ioc l a) ** simp only [nhdsWithin_Iic_eq'', biInf_inf ha, inf_principal, Ioi_inter_Iic] ** Qed
nhdsWithin_Iic_basis' ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a : α ha : ∃ l, l < a ⊢ HasBasis (𝓝[Iic a] a) (fun l => l < a) fun l => Ioc l a ** convert nhdsWithin_Ici_basis' (α := αᵒᵈ) ha using 2 ** case h.e'_5.h.h α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a : α ha : ∃ l, l < a e_1✝ : α = αᵒᵈ x✝ : α ⊢ Ioc x✝ a = Ico a x✝ ** exact dual_Ico.symm ** Qed
nhds_top_order ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : Preorder α inst✝¹ : OrderTop α inst✝ : OrderTopology α ⊢ 𝓝 ⊤ = ⨅ l, ⨅ (_ : l < ⊤), 𝓟 (Ioi l) ** simp [nhds_eq_order (⊤ : α)] ** Qed
nhds_bot_order ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : Preorder α inst✝¹ : OrderBot α inst✝ : OrderTopology α ⊢ 𝓝 ⊥ = ⨅ l, ⨅ (_ : ⊥ < l), 𝓟 (Iio l) ** simp [nhds_eq_order (⊥ : α)] ** Qed
nhds_top_basis ** α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderTop α inst✝¹ : OrderTopology α inst✝ : Nontrivial α ⊢ HasBasis (𝓝 ⊤) (fun a => a < ⊤) fun a => Ioi a ** have : ∃ x : α, x < ⊤ := (exists_ne ⊤).imp fun x hx => hx.lt_top ** α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderTop α inst✝¹ : OrderTopology α inst✝ : Nontrivial α this : ∃ x, x < ⊤ ⊢ HasBasis (𝓝 ⊤) (fun a => a < ⊤) fun a => Ioi a ** simpa only [Iic_top, nhdsWithin_univ, Ioc_top] using nhdsWithin_Iic_basis' this ** Qed
tendsto_nhds_top_mono ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace β inst✝² : Preorder β inst✝¹ : OrderTop β inst✝ : OrderTopology β l : Filter α f g : α → β hf : Tendsto f l (𝓝 ⊤) hg : f ≤ᶠ[l] g ⊢ Tendsto g l (𝓝 ⊤) ** simp only [nhds_top_order, tendsto_iInf, tendsto_principal] at hf ⊢ ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace β inst✝² : Preorder β inst✝¹ : OrderTop β inst✝ : OrderTopology β l : Filter α f g : α → β hg : f ≤ᶠ[l] g hf : ∀ (i : β), i < ⊤ → ∀ᶠ (a : α) in l, f a ∈ Ioi i ⊢ ∀ (i : β), i < ⊤ → ∀ᶠ (a : α) in l, g a ∈ Ioi i ** intro x hx ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace β inst✝² : Preorder β inst✝¹ : OrderTop β inst✝ : OrderTopology β l : Filter α f g : α → β hg : f ≤ᶠ[l] g hf : ∀ (i : β), i < ⊤ → ∀ᶠ (a : α) in l, f a ∈ Ioi i x : β hx : x < ⊤ ⊢ ∀ᶠ (a : α) in l, g a ∈ Ioi x ** filter_upwards [hf x hx, hg] with _ using lt_of_lt_of_le ** Qed
exists_Ico_subset_of_mem_nhds' ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a : α s : Set α hs : s ∈ 𝓝 a u : α hu : a < u ⊢ ∃ u', u' ∈ Ioc a u ∧ Ico a u' ⊆ s ** simpa only [OrderDual.exists, exists_prop, dual_Ico, dual_Ioc] using exists_Ioc_subset_of_mem_nhds' (show ofDual ⁻¹' s ∈ 𝓝 (toDual a) from hs) hu.dual ** Qed
exists_Icc_mem_subset_of_mem_nhdsWithin_Ici ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a : α s : Set α hs : s ∈ 𝓝[Ici a] a ⊢ ∃ b, a ≤ b ∧ Icc a b ∈ 𝓝[Ici a] a ∧ Icc a b ⊆ s ** rcases (em (IsMax a)).imp_right not_isMax_iff.mp with (ha | ha) ** case inl α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a : α s : Set α hs : s ∈ 𝓝[Ici a] a ha : IsMax a ⊢ ∃ b, a ≤ b ∧ Icc a b ∈ 𝓝[Ici a] a ∧ Icc a b ⊆ s ** use a ** case h α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a : α s : Set α hs : s ∈ 𝓝[Ici a] a ha : IsMax a ⊢ a ≤ a ∧ Icc a a ∈ 𝓝[Ici a] a ∧ Icc a a ⊆ s ** simpa [ha.Ici_eq] using hs ** case inr α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a : α s : Set α hs : s ∈ 𝓝[Ici a] a ha : ∃ b, a < b ⊢ ∃ b, a ≤ b ∧ Icc a b ∈ 𝓝[Ici a] a ∧ Icc a b ⊆ s ** rcases (nhdsWithin_Ici_basis' ha).mem_iff.mp hs with ⟨b, hab, hbs⟩ ** case inr.intro.intro α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a : α s : Set α hs : s ∈ 𝓝[Ici a] a ha : ∃ b, a < b b : α hab : a < b hbs : Ico a b ⊆ s ⊢ ∃ b, a ≤ b ∧ Icc a b ∈ 𝓝[Ici a] a ∧ Icc a b ⊆ s ** rcases eq_empty_or_nonempty (Ioo a b) with (H | ⟨c, hac, hcb⟩) ** case inr.intro.intro.inl α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a : α s : Set α hs : s ∈ 𝓝[Ici a] a ha : ∃ b, a < b b : α hab : a < b hbs : Ico a b ⊆ s H : Ioo a b = ∅ ⊢ ∃ b, a ≤ b ∧ Icc a b ∈ 𝓝[Ici a] a ∧ Icc a b ⊆ s ** have : Ico a b = Icc a a := by rw [← Icc_union_Ioo_eq_Ico le_rfl hab, H, union_empty] ** case inr.intro.intro.inl α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a : α s : Set α hs : s ∈ 𝓝[Ici a] a ha : ∃ b, a < b b : α hab : a < b hbs : Ico a b ⊆ s H : Ioo a b = ∅ this : Ico a b = Icc a a ⊢ ∃ b, a ≤ b ∧ Icc a b ∈ 𝓝[Ici a] a ∧ Icc a b ⊆ s ** exact ⟨a, le_rfl, this ▸ ⟨Ico_mem_nhdsWithin_Ici' hab, hbs⟩⟩ ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a : α s : Set α hs : s ∈ 𝓝[Ici a] a ha : ∃ b, a < b b : α hab : a < b hbs : Ico a b ⊆ s H : Ioo a b = ∅ ⊢ Ico a b = Icc a a ** rw [← Icc_union_Ioo_eq_Ico le_rfl hab, H, union_empty] ** case inr.intro.intro.inr.intro.intro α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a : α s : Set α hs : s ∈ 𝓝[Ici a] a ha : ∃ b, a < b b : α hab : a < b hbs : Ico a b ⊆ s c : α hac : a < c hcb : c < b ⊢ ∃ b, a ≤ b ∧ Icc a b ∈ 𝓝[Ici a] a ∧ Icc a b ⊆ s ** refine' ⟨c, hac.le, Icc_mem_nhdsWithin_Ici' hac, _⟩ ** case inr.intro.intro.inr.intro.intro α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a : α s : Set α hs : s ∈ 𝓝[Ici a] a ha : ∃ b, a < b b : α hab : a < b hbs : Ico a b ⊆ s c : α hac : a < c hcb : c < b ⊢ Icc a c ⊆ s ** exact (Icc_subset_Ico_right hcb).trans hbs ** Qed
exists_Icc_mem_subset_of_mem_nhdsWithin_Iic ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a : α s : Set α hs : s ∈ 𝓝[Iic a] a ⊢ ∃ b, b ≤ a ∧ Icc b a ∈ 𝓝[Iic a] a ∧ Icc b a ⊆ s ** simpa only [dual_Icc, toDual.surjective.exists] using exists_Icc_mem_subset_of_mem_nhdsWithin_Ici (α := αᵒᵈ) (a := toDual a) hs ** Qed
exists_Icc_mem_subset_of_mem_nhds ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a : α s : Set α hs : s ∈ 𝓝 a ⊢ ∃ b c, a ∈ Icc b c ∧ Icc b c ∈ 𝓝 a ∧ Icc b c ⊆ s ** rcases exists_Icc_mem_subset_of_mem_nhdsWithin_Iic (nhdsWithin_le_nhds hs) with ⟨b, hba, hb_nhds, hbs⟩ ** case intro.intro.intro α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a : α s : Set α hs : s ∈ 𝓝 a b : α hba : b ≤ a hb_nhds : Icc b a ∈ 𝓝[Iic a] a hbs : Icc b a ⊆ s ⊢ ∃ b c, a ∈ Icc b c ∧ Icc b c ∈ 𝓝 a ∧ Icc b c ⊆ s ** rcases exists_Icc_mem_subset_of_mem_nhdsWithin_Ici (nhdsWithin_le_nhds hs) with ⟨c, hac, hc_nhds, hcs⟩ ** case intro.intro.intro.intro.intro.intro α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a : α s : Set α hs : s ∈ 𝓝 a b : α hba : b ≤ a hb_nhds : Icc b a ∈ 𝓝[Iic a] a hbs : Icc b a ⊆ s c : α hac : a ≤ c hc_nhds : Icc a c ∈ 𝓝[Ici a] a hcs : Icc a c ⊆ s ⊢ ∃ b c, a ∈ Icc b c ∧ Icc b c ∈ 𝓝 a ∧ Icc b c ⊆ s ** refine' ⟨b, c, ⟨hba, hac⟩, _⟩ ** case intro.intro.intro.intro.intro.intro α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a : α s : Set α hs : s ∈ 𝓝 a b : α hba : b ≤ a hb_nhds : Icc b a ∈ 𝓝[Iic a] a hbs : Icc b a ⊆ s c : α hac : a ≤ c hc_nhds : Icc a c ∈ 𝓝[Ici a] a hcs : Icc a c ⊆ s ⊢ Icc b c ∈ 𝓝 a ∧ Icc b c ⊆ s ** rw [← Icc_union_Icc_eq_Icc hba hac, ← nhds_left_sup_nhds_right] ** case intro.intro.intro.intro.intro.intro α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a : α s : Set α hs : s ∈ 𝓝 a b : α hba : b ≤ a hb_nhds : Icc b a ∈ 𝓝[Iic a] a hbs : Icc b a ⊆ s c : α hac : a ≤ c hc_nhds : Icc a c ∈ 𝓝[Ici a] a hcs : Icc a c ⊆ s ⊢ Icc b a ∪ Icc a c ∈ 𝓝[Iic a] a ⊔ 𝓝[Ici a] a ∧ Icc b a ∪ Icc a c ⊆ s ** exact ⟨union_mem_sup hb_nhds hc_nhds, union_subset hbs hcs⟩ ** Qed
IsOpen.exists_Ioo_subset ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : Nontrivial α s : Set α hs : IsOpen s h : Set.Nonempty s ⊢ ∃ a b, a < b ∧ Ioo a b ⊆ s ** obtain ⟨x, hx⟩ : ∃ x, x ∈ s := h ** case intro α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : Nontrivial α s : Set α hs : IsOpen s x : α hx : x ∈ s ⊢ ∃ a b, a < b ∧ Ioo a b ⊆ s ** obtain ⟨y, hy⟩ : ∃ y, y ≠ x := exists_ne x ** case intro.intro α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : Nontrivial α s : Set α hs : IsOpen s x : α hx : x ∈ s y : α hy : y ≠ x ⊢ ∃ a b, a < b ∧ Ioo a b ⊆ s ** rcases lt_trichotomy x y with (H | rfl | H) ** case intro.intro.inl α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : Nontrivial α s : Set α hs : IsOpen s x : α hx : x ∈ s y : α hy : y ≠ x H : x < y ⊢ ∃ a b, a < b ∧ Ioo a b ⊆ s ** obtain ⟨u, xu, hu⟩ : ∃ u, x < u ∧ Ico x u ⊆ s := exists_Ico_subset_of_mem_nhds (hs.mem_nhds hx) ⟨y, H⟩ ** case intro.intro.inl.intro.intro α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : Nontrivial α s : Set α hs : IsOpen s x : α hx : x ∈ s y : α hy : y ≠ x H : x < y u : α xu : x < u hu : Ico x u ⊆ s ⊢ ∃ a b, a < b ∧ Ioo a b ⊆ s ** exact ⟨x, u, xu, Ioo_subset_Ico_self.trans hu⟩ ** case intro.intro.inr.inl α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : Nontrivial α s : Set α hs : IsOpen s x : α hx : x ∈ s hy : x ≠ x ⊢ ∃ a b, a < b ∧ Ioo a b ⊆ s ** exact (hy rfl).elim ** case intro.intro.inr.inr α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : Nontrivial α s : Set α hs : IsOpen s x : α hx : x ∈ s y : α hy : y ≠ x H : y < x ⊢ ∃ a b, a < b ∧ Ioo a b ⊆ s ** obtain ⟨l, lx, hl⟩ : ∃ l, l < x ∧ Ioc l x ⊆ s := exists_Ioc_subset_of_mem_nhds (hs.mem_nhds hx) ⟨y, H⟩ ** case intro.intro.inr.inr.intro.intro α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : Nontrivial α s : Set α hs : IsOpen s x : α hx : x ∈ s y : α hy : y ≠ x H : y < x l : α lx : l < x hl : Ioc l x ⊆ s ⊢ ∃ a b, a < b ∧ Ioo a b ⊆ s ** exact ⟨l, x, lx, Ioo_subset_Ioc_self.trans hl⟩ ** Qed
dense_of_exists_between ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : Nontrivial α s : Set α h : ∀ ⦃a b : α⦄, a < b → ∃ c, c ∈ s ∧ a < c ∧ c < b ⊢ Dense s ** refine dense_iff_inter_open.2 fun U U_open U_nonempty => ?_ ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : Nontrivial α s : Set α h : ∀ ⦃a b : α⦄, a < b → ∃ c, c ∈ s ∧ a < c ∧ c < b U : Set α U_open : IsOpen U U_nonempty : Set.Nonempty U ⊢ Set.Nonempty (U ∩ s) ** obtain ⟨a, b, hab, H⟩ : ∃ a b : α, a < b ∧ Ioo a b ⊆ U := U_open.exists_Ioo_subset U_nonempty ** case intro.intro.intro α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : Nontrivial α s : Set α h : ∀ ⦃a b : α⦄, a < b → ∃ c, c ∈ s ∧ a < c ∧ c < b U : Set α U_open : IsOpen U U_nonempty : Set.Nonempty U a b : α hab : a < b H : Ioo a b ⊆ U ⊢ Set.Nonempty (U ∩ s) ** obtain ⟨x, xs, hx⟩ : ∃ x ∈ s, a < x ∧ x < b := h hab ** case intro.intro.intro.intro.intro α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : Nontrivial α s : Set α h : ∀ ⦃a b : α⦄, a < b → ∃ c, c ∈ s ∧ a < c ∧ c < b U : Set α U_open : IsOpen U U_nonempty : Set.Nonempty U a b : α hab : a < b H : Ioo a b ⊆ U x : α xs : x ∈ s hx : a < x ∧ x < b ⊢ Set.Nonempty (U ∩ s) ** exact ⟨x, ⟨H hx, xs⟩⟩ ** Qed
mem_nhds_iff_exists_Ioo_subset' ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a : α s : Set α hl : ∃ l, l < a hu : ∃ u, a < u ⊢ s ∈ 𝓝 a ↔ ∃ l u, a ∈ Ioo l u ∧ Ioo l u ⊆ s ** constructor ** case mp α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a : α s : Set α hl : ∃ l, l < a hu : ∃ u, a < u ⊢ s ∈ 𝓝 a → ∃ l u, a ∈ Ioo l u ∧ Ioo l u ⊆ s ** intro h ** case mp α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a : α s : Set α hl : ∃ l, l < a hu : ∃ u, a < u h : s ∈ 𝓝 a ⊢ ∃ l u, a ∈ Ioo l u ∧ Ioo l u ⊆ s ** rcases exists_Ico_subset_of_mem_nhds h hu with ⟨u, au, hu⟩ ** case mp.intro.intro α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a : α s : Set α hl : ∃ l, l < a hu✝ : ∃ u, a < u h : s ∈ 𝓝 a u : α au : a < u hu : Ico a u ⊆ s ⊢ ∃ l u, a ∈ Ioo l u ∧ Ioo l u ⊆ s ** rcases exists_Ioc_subset_of_mem_nhds h hl with ⟨l, la, hl⟩ ** case mp.intro.intro.intro.intro α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a : α s : Set α hl✝ : ∃ l, l < a hu✝ : ∃ u, a < u h : s ∈ 𝓝 a u : α au : a < u hu : Ico a u ⊆ s l : α la : l < a hl : Ioc l a ⊆ s ⊢ ∃ l u, a ∈ Ioo l u ∧ Ioo l u ⊆ s ** exact ⟨l, u, ⟨la, au⟩, Ioc_union_Ico_eq_Ioo la au ▸ union_subset hl hu⟩ ** case mpr α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a : α s : Set α hl : ∃ l, l < a hu : ∃ u, a < u ⊢ (∃ l u, a ∈ Ioo l u ∧ Ioo l u ⊆ s) → s ∈ 𝓝 a ** rintro ⟨l, u, ha, h⟩ ** case mpr.intro.intro.intro α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a : α s : Set α hl : ∃ l, l < a hu : ∃ u, a < u l u : α ha : a ∈ Ioo l u h : Ioo l u ⊆ s ⊢ s ∈ 𝓝 a ** apply mem_of_superset (Ioo_mem_nhds ha.1 ha.2) h ** Qed
nhds_basis_Ioo' ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a : α hl : ∃ l, l < a hu : ∃ u, a < u s : Set α ⊢ (∃ l u, a ∈ Ioo l u ∧ Ioo l u ⊆ s) ↔ ∃ i, (i.1 < a ∧ a < i.2) ∧ Ioo i.1 i.2 ⊆ s ** simp ** Qed
Dense.topology_eq_generateFrom ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : DenselyOrdered α s : Set α hs : Dense s ⊢ inst✝³ = generateFrom (Ioi '' s ∪ Iio '' s) ** refine (OrderTopology.topology_eq_generate_intervals (α := α)).trans ?_ ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : DenselyOrdered α s : Set α hs : Dense s ⊢ generateFrom {s | ∃ a, s = Ioi a ∨ s = Iio a} = generateFrom (Ioi '' s ∪ Iio '' s) ** refine le_antisymm (generateFrom_anti ?_) (le_generateFrom ?_) ** case refine_1 α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : DenselyOrdered α s : Set α hs : Dense s ⊢ Ioi '' s ∪ Iio '' s ⊆ {s | ∃ a, s = Ioi a ∨ s = Iio a} ** simp only [union_subset_iff, image_subset_iff] ** case refine_1 α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : DenselyOrdered α s : Set α hs : Dense s ⊢ s ⊆ Ioi ⁻¹' {s | ∃ a, s = Ioi a ∨ s = Iio a} ∧ s ⊆ Iio ⁻¹' {s | ∃ a, s = Ioi a ∨ s = Iio a} ** exact ⟨fun a _ ↦ ⟨a, .inl rfl⟩, fun a _ ↦ ⟨a, .inr rfl⟩⟩ ** case refine_2 α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : DenselyOrdered α s : Set α hs : Dense s ⊢ ∀ (s_1 : Set α), s_1 ∈ {s | ∃ a, s = Ioi a ∨ s = Iio a} → IsOpen s_1 ** rintro _ ⟨a, rfl | rfl⟩ ** case refine_2.intro.inl α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : DenselyOrdered α s : Set α hs : Dense s a : α ⊢ IsOpen (Ioi a) ** rw [hs.Ioi_eq_biUnion] ** case refine_2.intro.inl α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : DenselyOrdered α s : Set α hs : Dense s a : α ⊢ IsOpen (⋃ y ∈ s ∩ Ioi a, Ioi y) ** let _ := generateFrom (Ioi '' s ∪ Iio '' s) ** case refine_2.intro.inl α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : DenselyOrdered α s : Set α hs : Dense s a : α x✝ : TopologicalSpace α := generateFrom (Ioi '' s ∪ Iio '' s) ⊢ IsOpen (⋃ y ∈ s ∩ Ioi a, Ioi y) ** exact isOpen_iUnion fun x ↦ isOpen_iUnion fun h ↦ .basic _ <| .inl <| mem_image_of_mem _ h.1 ** case refine_2.intro.inr α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : DenselyOrdered α s : Set α hs : Dense s a : α ⊢ IsOpen (Iio a) ** rw [hs.Iio_eq_biUnion] ** case refine_2.intro.inr α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : DenselyOrdered α s : Set α hs : Dense s a : α ⊢ IsOpen (⋃ y ∈ s ∩ Iio a, Iio y) ** let _ := generateFrom (Ioi '' s ∪ Iio '' s) ** case refine_2.intro.inr α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : DenselyOrdered α s : Set α hs : Dense s a : α x✝ : TopologicalSpace α := generateFrom (Ioi '' s ∪ Iio '' s) ⊢ IsOpen (⋃ y ∈ s ∩ Iio a, Iio y) ** exact isOpen_iUnion fun x ↦ isOpen_iUnion fun h ↦ .basic _ <| .inr <| mem_image_of_mem _ h.1 ** Qed
TopologicalSpace.SecondCountableTopology.of_separableSpace_orderTopology ** α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderTopology α inst✝¹ : DenselyOrdered α inst✝ : SeparableSpace α ⊢ SecondCountableTopology α ** rcases exists_countable_dense α with ⟨s, hc, hd⟩ ** case intro.intro α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderTopology α inst✝¹ : DenselyOrdered α inst✝ : SeparableSpace α s : Set α hc : Set.Countable s hd : Dense s ⊢ SecondCountableTopology α ** refine ⟨⟨_, ?_, hd.topology_eq_generateFrom⟩⟩ ** case intro.intro α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderTopology α inst✝¹ : DenselyOrdered α inst✝ : SeparableSpace α s : Set α hc : Set.Countable s hd : Dense s ⊢ Set.Countable (Ioi '' s ∪ Iio '' s) ** exact (hc.image _).union (hc.image _) ** Qed
countable_setOf_covby_right ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : SecondCountableTopology α ⊢ Set.Countable {x | ∃ y, x ⋖ y} ** nontriviality α ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : SecondCountableTopology α ✝ : Nontrivial α ⊢ Set.Countable {x | ∃ y, x ⋖ y} ** let s := { x : α | ∃ y, x ⋖ y } ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : SecondCountableTopology α ✝ : Nontrivial α s : Set α := {x | ∃ y, x ⋖ y} ⊢ Set.Countable {x | ∃ y, x ⋖ y} ** have : ∀ x ∈ s, ∃ y, x ⋖ y := fun x => id ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : SecondCountableTopology α ✝ : Nontrivial α s : Set α := {x | ∃ y, x ⋖ y} this : ∀ (x : α), x ∈ s → ∃ y, x ⋖ y ⊢ Set.Countable {x | ∃ y, x ⋖ y} ** choose! y hy using this ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : SecondCountableTopology α ✝ : Nontrivial α s : Set α := {x | ∃ y, x ⋖ y} y : α → α hy : ∀ (x : α), x ∈ s → x ⋖ y x ⊢ Set.Countable {x | ∃ y, x ⋖ y} ** have Hy : ∀ x z, x ∈ s → z < y x → z ≤ x := fun x z hx => (hy x hx).le_of_lt ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : SecondCountableTopology α ✝ : Nontrivial α s : Set α := {x | ∃ y, x ⋖ y} y : α → α hy : ∀ (x : α), x ∈ s → x ⋖ y x Hy : ∀ (x z : α), x ∈ s → z < y x → z ≤ x ⊢ Set.Countable {x | ∃ y, x ⋖ y} ** suffices H : ∀ a : Set α, IsOpen a → Set.Countable { x | x ∈ s ∧ x ∈ a ∧ y x ∉ a } ** case H α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : SecondCountableTopology α ✝ : Nontrivial α s : Set α := {x | ∃ y, x ⋖ y} y : α → α hy : ∀ (x : α), x ∈ s → x ⋖ y x Hy : ∀ (x z : α), x ∈ s → z < y x → z ≤ x ⊢ ∀ (a : Set α), IsOpen a → Set.Countable {x | x ∈ s ∧ x ∈ a ∧ ¬y x ∈ a} ** intro a ha ** case H α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : SecondCountableTopology α ✝ : Nontrivial α s : Set α := {x | ∃ y, x ⋖ y} y : α → α hy : ∀ (x : α), x ∈ s → x ⋖ y x Hy : ∀ (x z : α), x ∈ s → z < y x → z ≤ x a : Set α ha : IsOpen a ⊢ Set.Countable {x | x ∈ s ∧ x ∈ a ∧ ¬y x ∈ a} ** suffices H : Set.Countable { x | (x ∈ s ∧ x ∈ a ∧ y x ∉ a) ∧ ¬IsBot x } ** case H α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : SecondCountableTopology α ✝ : Nontrivial α s : Set α := {x | ∃ y, x ⋖ y} y : α → α hy : ∀ (x : α), x ∈ s → x ⋖ y x Hy : ∀ (x z : α), x ∈ s → z < y x → z ≤ x a : Set α ha : IsOpen a ⊢ Set.Countable {x | (x ∈ s ∧ x ∈ a ∧ ¬y x ∈ a) ∧ ¬IsBot x} ** simp only [and_assoc] ** case H α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : SecondCountableTopology α ✝ : Nontrivial α s : Set α := {x | ∃ y, x ⋖ y} y : α → α hy : ∀ (x : α), x ∈ s → x ⋖ y x Hy : ∀ (x z : α), x ∈ s → z < y x → z ≤ x a : Set α ha : IsOpen a ⊢ Set.Countable {x | x ∈ {x | ∃ y, x ⋖ y} ∧ x ∈ a ∧ ¬y x ∈ a ∧ ¬IsBot x} ** let t := { x | x ∈ s ∧ x ∈ a ∧ y x ∉ a ∧ ¬IsBot x } ** case H α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : SecondCountableTopology α ✝ : Nontrivial α s : Set α := {x | ∃ y, x ⋖ y} y : α → α hy : ∀ (x : α), x ∈ s → x ⋖ y x Hy : ∀ (x z : α), x ∈ s → z < y x → z ≤ x a : Set α ha : IsOpen a t : Set α := {x | x ∈ s ∧ x ∈ a ∧ ¬y x ∈ a ∧ ¬IsBot x} ⊢ Set.Countable {x | x ∈ {x | ∃ y, x ⋖ y} ∧ x ∈ a ∧ ¬y x ∈ a ∧ ¬IsBot x} ** have : ∀ x ∈ t, ∃ z < x, Ioc z x ⊆ a := by intro x hx apply exists_Ioc_subset_of_mem_nhds (ha.mem_nhds hx.2.1) simpa only [IsBot, not_forall, not_le] using hx.right.right.right ** case H α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : SecondCountableTopology α ✝ : Nontrivial α s : Set α := {x | ∃ y, x ⋖ y} y : α → α hy : ∀ (x : α), x ∈ s → x ⋖ y x Hy : ∀ (x z : α), x ∈ s → z < y x → z ≤ x a : Set α ha : IsOpen a t : Set α := {x | x ∈ s ∧ x ∈ a ∧ ¬y x ∈ a ∧ ¬IsBot x} this : ∀ (x : α), x ∈ t → ∃ z, z < x ∧ Ioc z x ⊆ a ⊢ Set.Countable {x | x ∈ {x | ∃ y, x ⋖ y} ∧ x ∈ a ∧ ¬y x ∈ a ∧ ¬IsBot x} ** choose! z hz h'z using this ** case H α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : SecondCountableTopology α ✝ : Nontrivial α s : Set α := {x | ∃ y, x ⋖ y} y : α → α hy : ∀ (x : α), x ∈ s → x ⋖ y x Hy : ∀ (x z : α), x ∈ s → z < y x → z ≤ x a : Set α ha : IsOpen a t : Set α := {x | x ∈ s ∧ x ∈ a ∧ ¬y x ∈ a ∧ ¬IsBot x} z : α → α hz : ∀ (x : α), x ∈ t → z x < x h'z : ∀ (x : α), x ∈ t → Ioc (z x) x ⊆ a this : PairwiseDisjoint t fun x => Ioc (z x) x ⊢ Set.Countable {x | x ∈ {x | ∃ y, x ⋖ y} ∧ x ∈ a ∧ ¬y x ∈ a ∧ ¬IsBot x} ** refine' this.countable_of_isOpen (fun x hx => _) fun x hx => ⟨x, hz x hx, le_rfl⟩ ** case H α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : SecondCountableTopology α ✝ : Nontrivial α s : Set α := {x | ∃ y, x ⋖ y} y : α → α hy : ∀ (x : α), x ∈ s → x ⋖ y x Hy : ∀ (x z : α), x ∈ s → z < y x → z ≤ x a : Set α ha : IsOpen a t : Set α := {x | x ∈ s ∧ x ∈ a ∧ ¬y x ∈ a ∧ ¬IsBot x} z : α → α hz : ∀ (x : α), x ∈ t → z x < x h'z : ∀ (x : α), x ∈ t → Ioc (z x) x ⊆ a this : PairwiseDisjoint t fun x => Ioc (z x) x x : α hx : x ∈ t ⊢ IsOpen (Ioc (z x) x) ** suffices H : Ioc (z x) x = Ioo (z x) (y x) ** case H α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : SecondCountableTopology α ✝ : Nontrivial α s : Set α := {x | ∃ y, x ⋖ y} y : α → α hy : ∀ (x : α), x ∈ s → x ⋖ y x Hy : ∀ (x z : α), x ∈ s → z < y x → z ≤ x a : Set α ha : IsOpen a t : Set α := {x | x ∈ s ∧ x ∈ a ∧ ¬y x ∈ a ∧ ¬IsBot x} z : α → α hz : ∀ (x : α), x ∈ t → z x < x h'z : ∀ (x : α), x ∈ t → Ioc (z x) x ⊆ a this : PairwiseDisjoint t fun x => Ioc (z x) x x : α hx : x ∈ t ⊢ Ioc (z x) x = Ioo (z x) (y x) ** exact Subset.antisymm (Ioc_subset_Ioo_right (hy x hx.1).lt) fun u hu => ⟨hu.1, Hy _ _ hx.1 hu.2⟩ ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : SecondCountableTopology α ✝ : Nontrivial α s : Set α := {x | ∃ y, x ⋖ y} y : α → α hy : ∀ (x : α), x ∈ s → x ⋖ y x Hy : ∀ (x z : α), x ∈ s → z < y x → z ≤ x H : ∀ (a : Set α), IsOpen a → Set.Countable {x | x ∈ s ∧ x ∈ a ∧ ¬y x ∈ a} ⊢ Set.Countable {x | ∃ y, x ⋖ y} ** have : s ⊆ ⋃ a ∈ countableBasis α, { x | x ∈ s ∧ x ∈ a ∧ y x ∉ a } := fun x hx => by rcases (isBasis_countableBasis α).exists_mem_of_ne (hy x hx).ne with ⟨a, ab, xa, ya⟩ exact mem_iUnion₂.2 ⟨a, ab, hx, xa, ya⟩ ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : SecondCountableTopology α ✝ : Nontrivial α s : Set α := {x | ∃ y, x ⋖ y} y : α → α hy : ∀ (x : α), x ∈ s → x ⋖ y x Hy : ∀ (x z : α), x ∈ s → z < y x → z ≤ x H : ∀ (a : Set α), IsOpen a → Set.Countable {x | x ∈ s ∧ x ∈ a ∧ ¬y x ∈ a} this : s ⊆ ⋃ a ∈ countableBasis α, {x | x ∈ s ∧ x ∈ a ∧ ¬y x ∈ a} ⊢ Set.Countable {x | ∃ y, x ⋖ y} ** refine Set.Countable.mono this ?_ ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : SecondCountableTopology α ✝ : Nontrivial α s : Set α := {x | ∃ y, x ⋖ y} y : α → α hy : ∀ (x : α), x ∈ s → x ⋖ y x Hy : ∀ (x z : α), x ∈ s → z < y x → z ≤ x H : ∀ (a : Set α), IsOpen a → Set.Countable {x | x ∈ s ∧ x ∈ a ∧ ¬y x ∈ a} this : s ⊆ ⋃ a ∈ countableBasis α, {x | x ∈ s ∧ x ∈ a ∧ ¬y x ∈ a} ⊢ Set.Countable (⋃ a ∈ countableBasis α, {x | x ∈ s ∧ x ∈ a ∧ ¬y x ∈ a}) ** refine' Countable.biUnion (countable_countableBasis α) fun a ha => H _ _ ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : SecondCountableTopology α ✝ : Nontrivial α s : Set α := {x | ∃ y, x ⋖ y} y : α → α hy : ∀ (x : α), x ∈ s → x ⋖ y x Hy : ∀ (x z : α), x ∈ s → z < y x → z ≤ x H : ∀ (a : Set α), IsOpen a → Set.Countable {x | x ∈ s ∧ x ∈ a ∧ ¬y x ∈ a} this : s ⊆ ⋃ a ∈ countableBasis α, {x | x ∈ s ∧ x ∈ a ∧ ¬y x ∈ a} a : Set α ha : a ∈ countableBasis α ⊢ IsOpen a ** exact isOpen_of_mem_countableBasis ha ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : SecondCountableTopology α ✝ : Nontrivial α s : Set α := {x | ∃ y, x ⋖ y} y : α → α hy : ∀ (x : α), x ∈ s → x ⋖ y x Hy : ∀ (x z : α), x ∈ s → z < y x → z ≤ x H : ∀ (a : Set α), IsOpen a → Set.Countable {x | x ∈ s ∧ x ∈ a ∧ ¬y x ∈ a} x : α hx : x ∈ s ⊢ x ∈ ⋃ a ∈ countableBasis α, {x | x ∈ s ∧ x ∈ a ∧ ¬y x ∈ a} ** rcases (isBasis_countableBasis α).exists_mem_of_ne (hy x hx).ne with ⟨a, ab, xa, ya⟩ ** case intro.intro.intro α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : SecondCountableTopology α ✝ : Nontrivial α s : Set α := {x | ∃ y, x ⋖ y} y : α → α hy : ∀ (x : α), x ∈ s → x ⋖ y x Hy : ∀ (x z : α), x ∈ s → z < y x → z ≤ x H : ∀ (a : Set α), IsOpen a → Set.Countable {x | x ∈ s ∧ x ∈ a ∧ ¬y x ∈ a} x : α hx : x ∈ s a : Set α ab : a ∈ countableBasis α xa : x ∈ a ya : ¬y x ∈ a ⊢ x ∈ ⋃ a ∈ countableBasis α, {x | x ∈ s ∧ x ∈ a ∧ ¬y x ∈ a} ** exact mem_iUnion₂.2 ⟨a, ab, hx, xa, ya⟩ ** case H α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : SecondCountableTopology α ✝ : Nontrivial α s : Set α := {x | ∃ y, x ⋖ y} y : α → α hy : ∀ (x : α), x ∈ s → x ⋖ y x Hy : ∀ (x z : α), x ∈ s → z < y x → z ≤ x a : Set α ha : IsOpen a H : Set.Countable {x | (x ∈ s ∧ x ∈ a ∧ ¬y x ∈ a) ∧ ¬IsBot x} ⊢ Set.Countable {x | x ∈ s ∧ x ∈ a ∧ ¬y x ∈ a} ** exact H.of_diff (subsingleton_isBot α).countable ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : SecondCountableTopology α ✝ : Nontrivial α s : Set α := {x | ∃ y, x ⋖ y} y : α → α hy : ∀ (x : α), x ∈ s → x ⋖ y x Hy : ∀ (x z : α), x ∈ s → z < y x → z ≤ x a : Set α ha : IsOpen a t : Set α := {x | x ∈ s ∧ x ∈ a ∧ ¬y x ∈ a ∧ ¬IsBot x} ⊢ ∀ (x : α), x ∈ t → ∃ z, z < x ∧ Ioc z x ⊆ a ** intro x hx ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : SecondCountableTopology α ✝ : Nontrivial α s : Set α := {x | ∃ y, x ⋖ y} y : α → α hy : ∀ (x : α), x ∈ s → x ⋖ y x Hy : ∀ (x z : α), x ∈ s → z < y x → z ≤ x a : Set α ha : IsOpen a t : Set α := {x | x ∈ s ∧ x ∈ a ∧ ¬y x ∈ a ∧ ¬IsBot x} x : α hx : x ∈ t ⊢ ∃ z, z < x ∧ Ioc z x ⊆ a ** apply exists_Ioc_subset_of_mem_nhds (ha.mem_nhds hx.2.1) ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : SecondCountableTopology α ✝ : Nontrivial α s : Set α := {x | ∃ y, x ⋖ y} y : α → α hy : ∀ (x : α), x ∈ s → x ⋖ y x Hy : ∀ (x z : α), x ∈ s → z < y x → z ≤ x a : Set α ha : IsOpen a t : Set α := {x | x ∈ s ∧ x ∈ a ∧ ¬y x ∈ a ∧ ¬IsBot x} x : α hx : x ∈ t ⊢ ∃ l, l < x ** simpa only [IsBot, not_forall, not_le] using hx.right.right.right ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : SecondCountableTopology α ✝ : Nontrivial α s : Set α := {x | ∃ y, x ⋖ y} y : α → α hy : ∀ (x : α), x ∈ s → x ⋖ y x Hy : ∀ (x z : α), x ∈ s → z < y x → z ≤ x a : Set α ha : IsOpen a t : Set α := {x | x ∈ s ∧ x ∈ a ∧ ¬y x ∈ a ∧ ¬IsBot x} z : α → α hz : ∀ (x : α), x ∈ t → z x < x h'z : ∀ (x : α), x ∈ t → Ioc (z x) x ⊆ a x : α xt : x ∈ t x' : α x't : x' ∈ t hxx' : x ≠ x' ⊢ (Disjoint on fun x => Ioc (z x) x) x x' ** rcases hxx'.lt_or_lt with (h' | h') ** case inl α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : SecondCountableTopology α ✝ : Nontrivial α s : Set α := {x | ∃ y, x ⋖ y} y : α → α hy : ∀ (x : α), x ∈ s → x ⋖ y x Hy : ∀ (x z : α), x ∈ s → z < y x → z ≤ x a : Set α ha : IsOpen a t : Set α := {x | x ∈ s ∧ x ∈ a ∧ ¬y x ∈ a ∧ ¬IsBot x} z : α → α hz : ∀ (x : α), x ∈ t → z x < x h'z : ∀ (x : α), x ∈ t → Ioc (z x) x ⊆ a x : α xt : x ∈ t x' : α x't : x' ∈ t hxx' : x ≠ x' h' : x < x' ⊢ (Disjoint on fun x => Ioc (z x) x) x x' ** refine' disjoint_left.2 fun u ux ux' => xt.2.2.1 _ ** case inl α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : SecondCountableTopology α ✝ : Nontrivial α s : Set α := {x | ∃ y, x ⋖ y} y : α → α hy : ∀ (x : α), x ∈ s → x ⋖ y x Hy : ∀ (x z : α), x ∈ s → z < y x → z ≤ x a : Set α ha : IsOpen a t : Set α := {x | x ∈ s ∧ x ∈ a ∧ ¬y x ∈ a ∧ ¬IsBot x} z : α → α hz : ∀ (x : α), x ∈ t → z x < x h'z : ∀ (x : α), x ∈ t → Ioc (z x) x ⊆ a x : α xt : x ∈ t x' : α x't : x' ∈ t hxx' : x ≠ x' h' : x < x' u : α ux : u ∈ (fun x => Ioc (z x) x) x ux' : u ∈ (fun x => Ioc (z x) x) x' ⊢ y x ∈ a ** refine' h'z x' x't ⟨ux'.1.trans_le (ux.2.trans (hy x xt.1).le), _⟩ ** case inl α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : SecondCountableTopology α ✝ : Nontrivial α s : Set α := {x | ∃ y, x ⋖ y} y : α → α hy : ∀ (x : α), x ∈ s → x ⋖ y x Hy : ∀ (x z : α), x ∈ s → z < y x → z ≤ x a : Set α ha : IsOpen a t : Set α := {x | x ∈ s ∧ x ∈ a ∧ ¬y x ∈ a ∧ ¬IsBot x} z : α → α hz : ∀ (x : α), x ∈ t → z x < x h'z : ∀ (x : α), x ∈ t → Ioc (z x) x ⊆ a x : α xt : x ∈ t x' : α x't : x' ∈ t hxx' : x ≠ x' h' : x < x' u : α ux : u ∈ (fun x => Ioc (z x) x) x ux' : u ∈ (fun x => Ioc (z x) x) x' ⊢ y x ≤ x' ** by_contra' H ** case inl α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : SecondCountableTopology α ✝ : Nontrivial α s : Set α := {x | ∃ y, x ⋖ y} y : α → α hy : ∀ (x : α), x ∈ s → x ⋖ y x Hy : ∀ (x z : α), x ∈ s → z < y x → z ≤ x a : Set α ha : IsOpen a t : Set α := {x | x ∈ s ∧ x ∈ a ∧ ¬y x ∈ a ∧ ¬IsBot x} z : α → α hz : ∀ (x : α), x ∈ t → z x < x h'z : ∀ (x : α), x ∈ t → Ioc (z x) x ⊆ a x : α xt : x ∈ t x' : α x't : x' ∈ t hxx' : x ≠ x' h' : x < x' u : α ux : u ∈ (fun x => Ioc (z x) x) x ux' : u ∈ (fun x => Ioc (z x) x) x' H : x' < y x ⊢ False ** exact lt_irrefl _ ((Hy _ _ xt.1 H).trans_lt h') ** case inr α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : SecondCountableTopology α ✝ : Nontrivial α s : Set α := {x | ∃ y, x ⋖ y} y : α → α hy : ∀ (x : α), x ∈ s → x ⋖ y x Hy : ∀ (x z : α), x ∈ s → z < y x → z ≤ x a : Set α ha : IsOpen a t : Set α := {x | x ∈ s ∧ x ∈ a ∧ ¬y x ∈ a ∧ ¬IsBot x} z : α → α hz : ∀ (x : α), x ∈ t → z x < x h'z : ∀ (x : α), x ∈ t → Ioc (z x) x ⊆ a x : α xt : x ∈ t x' : α x't : x' ∈ t hxx' : x ≠ x' h' : x' < x ⊢ (Disjoint on fun x => Ioc (z x) x) x x' ** refine' disjoint_left.2 fun u ux ux' => x't.2.2.1 _ ** case inr α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : SecondCountableTopology α ✝ : Nontrivial α s : Set α := {x | ∃ y, x ⋖ y} y : α → α hy : ∀ (x : α), x ∈ s → x ⋖ y x Hy : ∀ (x z : α), x ∈ s → z < y x → z ≤ x a : Set α ha : IsOpen a t : Set α := {x | x ∈ s ∧ x ∈ a ∧ ¬y x ∈ a ∧ ¬IsBot x} z : α → α hz : ∀ (x : α), x ∈ t → z x < x h'z : ∀ (x : α), x ∈ t → Ioc (z x) x ⊆ a x : α xt : x ∈ t x' : α x't : x' ∈ t hxx' : x ≠ x' h' : x' < x u : α ux : u ∈ (fun x => Ioc (z x) x) x ux' : u ∈ (fun x => Ioc (z x) x) x' ⊢ y x' ∈ a ** refine' h'z x xt ⟨ux.1.trans_le (ux'.2.trans (hy x' x't.1).le), _⟩ ** case inr α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : SecondCountableTopology α ✝ : Nontrivial α s : Set α := {x | ∃ y, x ⋖ y} y : α → α hy : ∀ (x : α), x ∈ s → x ⋖ y x Hy : ∀ (x z : α), x ∈ s → z < y x → z ≤ x a : Set α ha : IsOpen a t : Set α := {x | x ∈ s ∧ x ∈ a ∧ ¬y x ∈ a ∧ ¬IsBot x} z : α → α hz : ∀ (x : α), x ∈ t → z x < x h'z : ∀ (x : α), x ∈ t → Ioc (z x) x ⊆ a x : α xt : x ∈ t x' : α x't : x' ∈ t hxx' : x ≠ x' h' : x' < x u : α ux : u ∈ (fun x => Ioc (z x) x) x ux' : u ∈ (fun x => Ioc (z x) x) x' ⊢ y x' ≤ x ** by_contra' H ** case inr α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : SecondCountableTopology α ✝ : Nontrivial α s : Set α := {x | ∃ y, x ⋖ y} y : α → α hy : ∀ (x : α), x ∈ s → x ⋖ y x Hy : ∀ (x z : α), x ∈ s → z < y x → z ≤ x a : Set α ha : IsOpen a t : Set α := {x | x ∈ s ∧ x ∈ a ∧ ¬y x ∈ a ∧ ¬IsBot x} z : α → α hz : ∀ (x : α), x ∈ t → z x < x h'z : ∀ (x : α), x ∈ t → Ioc (z x) x ⊆ a x : α xt : x ∈ t x' : α x't : x' ∈ t hxx' : x ≠ x' h' : x' < x u : α ux : u ∈ (fun x => Ioc (z x) x) x ux' : u ∈ (fun x => Ioc (z x) x) x' H : x < y x' ⊢ False ** exact lt_irrefl _ ((Hy _ _ x't.1 H).trans_lt h') ** case H α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : SecondCountableTopology α ✝ : Nontrivial α s : Set α := {x | ∃ y, x ⋖ y} y : α → α hy : ∀ (x : α), x ∈ s → x ⋖ y x Hy : ∀ (x z : α), x ∈ s → z < y x → z ≤ x a : Set α ha : IsOpen a t : Set α := {x | x ∈ s ∧ x ∈ a ∧ ¬y x ∈ a ∧ ¬IsBot x} z : α → α hz : ∀ (x : α), x ∈ t → z x < x h'z : ∀ (x : α), x ∈ t → Ioc (z x) x ⊆ a this : PairwiseDisjoint t fun x => Ioc (z x) x x : α hx : x ∈ t H : Ioc (z x) x = Ioo (z x) (y x) ⊢ IsOpen (Ioc (z x) x) ** rw [H] ** case H α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : SecondCountableTopology α ✝ : Nontrivial α s : Set α := {x | ∃ y, x ⋖ y} y : α → α hy : ∀ (x : α), x ∈ s → x ⋖ y x Hy : ∀ (x z : α), x ∈ s → z < y x → z ≤ x a : Set α ha : IsOpen a t : Set α := {x | x ∈ s ∧ x ∈ a ∧ ¬y x ∈ a ∧ ¬IsBot x} z : α → α hz : ∀ (x : α), x ∈ t → z x < x h'z : ∀ (x : α), x ∈ t → Ioc (z x) x ⊆ a this : PairwiseDisjoint t fun x => Ioc (z x) x x : α hx : x ∈ t H : Ioc (z x) x = Ioo (z x) (y x) ⊢ IsOpen (Ioo (z x) (y x)) ** exact isOpen_Ioo ** Qed
countable_of_isolated_right' ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : SecondCountableTopology α ⊢ Set.Countable {x | ∃ y, x < y ∧ Ioo x y = ∅} ** simpa only [← covby_iff_Ioo_eq] using countable_setOf_covby_right ** Qed
countable_setOf_covby_left ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : SecondCountableTopology α ⊢ Set.Countable {x | ∃ y, y ⋖ x} ** convert countable_setOf_covby_right (α := αᵒᵈ) using 5 ** case h.e'_2.h.h.e'_2.h.h.h.e'_2.h.h.a α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : SecondCountableTopology α e_1✝ : α = αᵒᵈ x✝¹ x✝ : α ⊢ x✝ ⋖ x✝¹ ↔ x✝¹ ⋖ x✝ ** exact toDual_covby_toDual_iff.symm ** Qed
countable_of_isolated_left' ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : SecondCountableTopology α ⊢ Set.Countable {x | ∃ y, y < x ∧ Ioo y x = ∅} ** simpa only [← covby_iff_Ioo_eq] using countable_setOf_covby_left ** Qed
countable_image_lt_image_Ioi ** α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderTopology α inst✝¹ : LinearOrder β f : β → α inst✝ : SecondCountableTopology α ⊢ Set.Countable {x | ∃ z, f x < z ∧ ∀ (y : β), x < y → z ≤ f y} ** nontriviality β ** α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderTopology α inst✝¹ : LinearOrder β f : β → α inst✝ : SecondCountableTopology α ✝ : Nontrivial β ⊢ Set.Countable {x | ∃ z, f x < z ∧ ∀ (y : β), x < y → z ≤ f y} ** have : Nonempty α := Nonempty.map f (by infer_instance) ** α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderTopology α inst✝¹ : LinearOrder β f : β → α inst✝ : SecondCountableTopology α ✝ : Nontrivial β this : Nonempty α ⊢ Set.Countable {x | ∃ z, f x < z ∧ ∀ (y : β), x < y → z ≤ f y} ** let s := {x | ∃ z, f x < z ∧ ∀ y, x < y → z ≤ f y} ** α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderTopology α inst✝¹ : LinearOrder β f : β → α inst✝ : SecondCountableTopology α ✝ : Nontrivial β this : Nonempty α s : Set β := {x | ∃ z, f x < z ∧ ∀ (y : β), x < y → z ≤ f y} ⊢ Set.Countable {x | ∃ z, f x < z ∧ ∀ (y : β), x < y → z ≤ f y} ** have : ∀ x, x ∈ s → ∃ z, f x < z ∧ ∀ y, x < y → z ≤ f y := fun x hx ↦ hx ** α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderTopology α inst✝¹ : LinearOrder β f : β → α inst✝ : SecondCountableTopology α ✝ : Nontrivial β this✝ : Nonempty α s : Set β := {x | ∃ z, f x < z ∧ ∀ (y : β), x < y → z ≤ f y} this : ∀ (x : β), x ∈ s → ∃ z, f x < z ∧ ∀ (y : β), x < y → z ≤ f y ⊢ Set.Countable {x | ∃ z, f x < z ∧ ∀ (y : β), x < y → z ≤ f y} ** choose! z hz using this ** α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderTopology α inst✝¹ : LinearOrder β f : β → α inst✝ : SecondCountableTopology α ✝ : Nontrivial β this : Nonempty α s : Set β := {x | ∃ z, f x < z ∧ ∀ (y : β), x < y → z ≤ f y} z : β → α hz : ∀ (x : β), x ∈ s → f x < z x ∧ ∀ (y : β), x < y → z x ≤ f y ⊢ Set.Countable {x | ∃ z, f x < z ∧ ∀ (y : β), x < y → z ≤ f y} ** have I : InjOn f s := by apply StrictMonoOn.injOn intro x hx y _ hxy calc f x < z x := (hz x hx).1 _ ≤ f y := (hz x hx).2 y hxy ** α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderTopology α inst✝¹ : LinearOrder β f : β → α inst✝ : SecondCountableTopology α ✝ : Nontrivial β this : Nonempty α s : Set β := {x | ∃ z, f x < z ∧ ∀ (y : β), x < y → z ≤ f y} z : β → α hz : ∀ (x : β), x ∈ s → f x < z x ∧ ∀ (y : β), x < y → z x ≤ f y I : InjOn f s fs_count : Set.Countable (f '' s) ⊢ Set.Countable {x | ∃ z, f x < z ∧ ∀ (y : β), x < y → z ≤ f y} ** exact MapsTo.countable_of_injOn (mapsTo_image f s) I fs_count ** α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderTopology α inst✝¹ : LinearOrder β f : β → α inst✝ : SecondCountableTopology α ✝ : Nontrivial β ⊢ Nonempty β ** infer_instance ** α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderTopology α inst✝¹ : LinearOrder β f : β → α inst✝ : SecondCountableTopology α ✝ : Nontrivial β this : Nonempty α s : Set β := {x | ∃ z, f x < z ∧ ∀ (y : β), x < y → z ≤ f y} z : β → α hz : ∀ (x : β), x ∈ s → f x < z x ∧ ∀ (y : β), x < y → z x ≤ f y ⊢ InjOn f s ** apply StrictMonoOn.injOn ** case H α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderTopology α inst✝¹ : LinearOrder β f : β → α inst✝ : SecondCountableTopology α ✝ : Nontrivial β this : Nonempty α s : Set β := {x | ∃ z, f x < z ∧ ∀ (y : β), x < y → z ≤ f y} z : β → α hz : ∀ (x : β), x ∈ s → f x < z x ∧ ∀ (y : β), x < y → z x ≤ f y ⊢ StrictMonoOn f s ** intro x hx y _ hxy ** case H α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderTopology α inst✝¹ : LinearOrder β f : β → α inst✝ : SecondCountableTopology α ✝ : Nontrivial β this : Nonempty α s : Set β := {x | ∃ z, f x < z ∧ ∀ (y : β), x < y → z ≤ f y} z : β → α hz : ∀ (x : β), x ∈ s → f x < z x ∧ ∀ (y : β), x < y → z x ≤ f y x : β hx : x ∈ s y : β x✝ : y ∈ s hxy : x < y ⊢ f x < f y ** calc f x < z x := (hz x hx).1 _ ≤ f y := (hz x hx).2 y hxy ** α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderTopology α inst✝¹ : LinearOrder β f : β → α inst✝ : SecondCountableTopology α ✝ : Nontrivial β this : Nonempty α s : Set β := {x | ∃ z, f x < z ∧ ∀ (y : β), x < y → z ≤ f y} z : β → α hz : ∀ (x : β), x ∈ s → f x < z x ∧ ∀ (y : β), x < y → z x ≤ f y I : InjOn f s A : PairwiseDisjoint (f '' s) fun x => Ioo x (z (invFunOn f s x)) ⊢ Set.Countable (f '' s) ** apply Set.PairwiseDisjoint.countable_of_Ioo A ** α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderTopology α inst✝¹ : LinearOrder β f : β → α inst✝ : SecondCountableTopology α ✝ : Nontrivial β this : Nonempty α s : Set β := {x | ∃ z, f x < z ∧ ∀ (y : β), x < y → z ≤ f y} z : β → α hz : ∀ (x : β), x ∈ s → f x < z x ∧ ∀ (y : β), x < y → z x ≤ f y I : InjOn f s A : PairwiseDisjoint (f '' s) fun x => Ioo x (z (invFunOn f s x)) ⊢ ∀ (x : α), x ∈ f '' s → x < z (invFunOn f s x) ** rintro _ ⟨y, ys, rfl⟩ ** case intro.intro α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderTopology α inst✝¹ : LinearOrder β f : β → α inst✝ : SecondCountableTopology α ✝ : Nontrivial β this : Nonempty α s : Set β := {x | ∃ z, f x < z ∧ ∀ (y : β), x < y → z ≤ f y} z : β → α hz : ∀ (x : β), x ∈ s → f x < z x ∧ ∀ (y : β), x < y → z x ≤ f y I : InjOn f s A : PairwiseDisjoint (f '' s) fun x => Ioo x (z (invFunOn f s x)) y : β ys : y ∈ s ⊢ f y < z (invFunOn f s (f y)) ** simpa only [I.leftInvOn_invFunOn ys] using (hz y ys).1 ** α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderTopology α inst✝¹ : LinearOrder β f : β → α inst✝ : SecondCountableTopology α ✝ : Nontrivial β this : Nonempty α s : Set β := {x | ∃ z, f x < z ∧ ∀ (y : β), x < y → z ≤ f y} z : β → α hz : ∀ (x : β), x ∈ s → f x < z x ∧ ∀ (y : β), x < y → z x ≤ f y I : InjOn f s ⊢ PairwiseDisjoint (f '' s) fun x => Ioo x (z (invFunOn f s x)) ** rintro _ ⟨u, us, rfl⟩ _ ⟨v, vs, rfl⟩ huv ** case intro.intro.intro.intro α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderTopology α inst✝¹ : LinearOrder β f : β → α inst✝ : SecondCountableTopology α ✝ : Nontrivial β this : Nonempty α s : Set β := {x | ∃ z, f x < z ∧ ∀ (y : β), x < y → z ≤ f y} z : β → α hz : ∀ (x : β), x ∈ s → f x < z x ∧ ∀ (y : β), x < y → z x ≤ f y I : InjOn f s u : β us : u ∈ s v : β vs : v ∈ s huv : f u ≠ f v ⊢ (Disjoint on fun x => Ioo x (z (invFunOn f s x))) (f u) (f v) ** wlog hle : u ≤ v generalizing u v ** α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderTopology α inst✝¹ : LinearOrder β f : β → α inst✝ : SecondCountableTopology α ✝ : Nontrivial β this : Nonempty α s : Set β := {x | ∃ z, f x < z ∧ ∀ (y : β), x < y → z ≤ f y} z : β → α hz : ∀ (x : β), x ∈ s → f x < z x ∧ ∀ (y : β), x < y → z x ≤ f y I : InjOn f s u : β us : u ∈ s v : β vs : v ∈ s huv : f u ≠ f v hle : u ≤ v ⊢ (Disjoint on fun x => Ioo x (z (invFunOn f s x))) (f u) (f v) ** have hlt : u < v := hle.lt_of_ne (ne_of_apply_ne _ huv) ** α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderTopology α inst✝¹ : LinearOrder β f : β → α inst✝ : SecondCountableTopology α ✝ : Nontrivial β this : Nonempty α s : Set β := {x | ∃ z, f x < z ∧ ∀ (y : β), x < y → z ≤ f y} z : β → α hz : ∀ (x : β), x ∈ s → f x < z x ∧ ∀ (y : β), x < y → z x ≤ f y I : InjOn f s u : β us : u ∈ s v : β vs : v ∈ s huv : f u ≠ f v hle : u ≤ v hlt : u < v ⊢ (Disjoint on fun x => Ioo x (z (invFunOn f s x))) (f u) (f v) ** apply disjoint_iff_forall_ne.2 ** α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderTopology α inst✝¹ : LinearOrder β f : β → α inst✝ : SecondCountableTopology α ✝ : Nontrivial β this : Nonempty α s : Set β := {x | ∃ z, f x < z ∧ ∀ (y : β), x < y → z ≤ f y} z : β → α hz : ∀ (x : β), x ∈ s → f x < z x ∧ ∀ (y : β), x < y → z x ≤ f y I : InjOn f s u : β us : u ∈ s v : β vs : v ∈ s huv : f u ≠ f v hle : u ≤ v hlt : u < v ⊢ ∀ ⦃a : α⦄, a ∈ (fun x => Ioo x (z (invFunOn f s x))) (f u) → ∀ ⦃b : α⦄, b ∈ (fun x => Ioo x (z (invFunOn f s x))) (f v) → a ≠ b ** rintro a ha b hb rfl ** α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderTopology α inst✝¹ : LinearOrder β f : β → α inst✝ : SecondCountableTopology α ✝ : Nontrivial β this : Nonempty α s : Set β := {x | ∃ z, f x < z ∧ ∀ (y : β), x < y → z ≤ f y} z : β → α hz : ∀ (x : β), x ∈ s → f x < z x ∧ ∀ (y : β), x < y → z x ≤ f y I : InjOn f s u : β us : u ∈ s v : β vs : v ∈ s huv : f u ≠ f v hle : u ≤ v hlt : u < v a : α ha : a ∈ (fun x => Ioo x (z (invFunOn f s x))) (f u) hb : a ∈ (fun x => Ioo x (z (invFunOn f s x))) (f v) ⊢ False ** simp only [I.leftInvOn_invFunOn us, I.leftInvOn_invFunOn vs] at ha hb ** α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderTopology α inst✝¹ : LinearOrder β f : β → α inst✝ : SecondCountableTopology α ✝ : Nontrivial β this : Nonempty α s : Set β := {x | ∃ z, f x < z ∧ ∀ (y : β), x < y → z ≤ f y} z : β → α hz : ∀ (x : β), x ∈ s → f x < z x ∧ ∀ (y : β), x < y → z x ≤ f y I : InjOn f s u : β us : u ∈ s v : β vs : v ∈ s huv : f u ≠ f v hle : u ≤ v hlt : u < v a : α ha : a ∈ Ioo (f u) (z u) hb : a ∈ Ioo (f v) (z v) ⊢ False ** exact lt_irrefl _ ((ha.2.trans_le ((hz u us).2 v hlt)).trans hb.1) ** case intro.intro.intro.intro.inr α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderTopology α inst✝¹ : LinearOrder β f : β → α inst✝ : SecondCountableTopology α ✝ : Nontrivial β this✝ : Nonempty α s : Set β := {x | ∃ z, f x < z ∧ ∀ (y : β), x < y → z ≤ f y} z : β → α hz : ∀ (x : β), x ∈ s → f x < z x ∧ ∀ (y : β), x < y → z x ≤ f y I : InjOn f s u : β us : u ∈ s v : β vs : v ∈ s huv : f u ≠ f v this : ∀ (u : β), u ∈ s → ∀ (v : β), v ∈ s → f u ≠ f v → u ≤ v → (Disjoint on fun x => Ioo x (z (invFunOn f s x))) (f u) (f v) hle : ¬u ≤ v ⊢ (Disjoint on fun x => Ioo x (z (invFunOn f s x))) (f u) (f v) ** exact (this v vs u us huv.symm (le_of_not_le hle)).symm ** Qed
pi_Iio_mem_nhds ** α : Type u β : Type v γ : Type w inst✝⁷ : TopologicalSpace α inst✝⁶ : LinearOrder α inst✝⁵ : OrderTopology α ι : Type u_1 π : ι → Type u_2 inst✝⁴ : Finite ι inst✝³ : (i : ι) → LinearOrder (π i) inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : ∀ (i : ι), OrderTopology (π i) a b x : (i : ι) → π i a' b' x' : ι → α inst✝ : Nonempty ι ha : ∀ (i : ι), x i < a i ⊢ Iio a ∈ 𝓝 x ** refine' mem_of_superset (set_pi_mem_nhds Set.finite_univ fun i _ => _) (pi_univ_Iio_subset a) ** α : Type u β : Type v γ : Type w inst✝⁷ : TopologicalSpace α inst✝⁶ : LinearOrder α inst✝⁵ : OrderTopology α ι : Type u_1 π : ι → Type u_2 inst✝⁴ : Finite ι inst✝³ : (i : ι) → LinearOrder (π i) inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : ∀ (i : ι), OrderTopology (π i) a b x : (i : ι) → π i a' b' x' : ι → α inst✝ : Nonempty ι ha : ∀ (i : ι), x i < a i i : ι x✝ : i ∈ univ ⊢ Iio (a i) ∈ 𝓝 (x i) ** exact Iio_mem_nhds (ha i) ** Qed
pi_Ioc_mem_nhds ** α : Type u β : Type v γ : Type w inst✝⁷ : TopologicalSpace α inst✝⁶ : LinearOrder α inst✝⁵ : OrderTopology α ι : Type u_1 π : ι → Type u_2 inst✝⁴ : Finite ι inst✝³ : (i : ι) → LinearOrder (π i) inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : ∀ (i : ι), OrderTopology (π i) a b x : (i : ι) → π i a' b' x' : ι → α inst✝ : Nonempty ι ha : ∀ (i : ι), a i < x i hb : ∀ (i : ι), x i < b i ⊢ Ioc a b ∈ 𝓝 x ** refine' mem_of_superset (set_pi_mem_nhds Set.finite_univ fun i _ => _) (pi_univ_Ioc_subset a b) ** α : Type u β : Type v γ : Type w inst✝⁷ : TopologicalSpace α inst✝⁶ : LinearOrder α inst✝⁵ : OrderTopology α ι : Type u_1 π : ι → Type u_2 inst✝⁴ : Finite ι inst✝³ : (i : ι) → LinearOrder (π i) inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : ∀ (i : ι), OrderTopology (π i) a b x : (i : ι) → π i a' b' x' : ι → α inst✝ : Nonempty ι ha : ∀ (i : ι), a i < x i hb : ∀ (i : ι), x i < b i i : ι x✝ : i ∈ univ ⊢ Ioc (a i) (b i) ∈ 𝓝 (x i) ** exact Ioc_mem_nhds (ha i) (hb i) ** Qed
pi_Ico_mem_nhds ** α : Type u β : Type v γ : Type w inst✝⁷ : TopologicalSpace α inst✝⁶ : LinearOrder α inst✝⁵ : OrderTopology α ι : Type u_1 π : ι → Type u_2 inst✝⁴ : Finite ι inst✝³ : (i : ι) → LinearOrder (π i) inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : ∀ (i : ι), OrderTopology (π i) a b x : (i : ι) → π i a' b' x' : ι → α inst✝ : Nonempty ι ha : ∀ (i : ι), a i < x i hb : ∀ (i : ι), x i < b i ⊢ Ico a b ∈ 𝓝 x ** refine' mem_of_superset (set_pi_mem_nhds Set.finite_univ fun i _ => _) (pi_univ_Ico_subset a b) ** α : Type u β : Type v γ : Type w inst✝⁷ : TopologicalSpace α inst✝⁶ : LinearOrder α inst✝⁵ : OrderTopology α ι : Type u_1 π : ι → Type u_2 inst✝⁴ : Finite ι inst✝³ : (i : ι) → LinearOrder (π i) inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : ∀ (i : ι), OrderTopology (π i) a b x : (i : ι) → π i a' b' x' : ι → α inst✝ : Nonempty ι ha : ∀ (i : ι), a i < x i hb : ∀ (i : ι), x i < b i i : ι x✝ : i ∈ univ ⊢ Ico (a i) (b i) ∈ 𝓝 (x i) ** exact Ico_mem_nhds (ha i) (hb i) ** Qed
pi_Ioo_mem_nhds ** α : Type u β : Type v γ : Type w inst✝⁷ : TopologicalSpace α inst✝⁶ : LinearOrder α inst✝⁵ : OrderTopology α ι : Type u_1 π : ι → Type u_2 inst✝⁴ : Finite ι inst✝³ : (i : ι) → LinearOrder (π i) inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : ∀ (i : ι), OrderTopology (π i) a b x : (i : ι) → π i a' b' x' : ι → α inst✝ : Nonempty ι ha : ∀ (i : ι), a i < x i hb : ∀ (i : ι), x i < b i ⊢ Ioo a b ∈ 𝓝 x ** refine' mem_of_superset (set_pi_mem_nhds Set.finite_univ fun i _ => _) (pi_univ_Ioo_subset a b) ** α : Type u β : Type v γ : Type w inst✝⁷ : TopologicalSpace α inst✝⁶ : LinearOrder α inst✝⁵ : OrderTopology α ι : Type u_1 π : ι → Type u_2 inst✝⁴ : Finite ι inst✝³ : (i : ι) → LinearOrder (π i) inst✝² : (i : ι) → TopologicalSpace (π i) inst✝¹ : ∀ (i : ι), OrderTopology (π i) a b x : (i : ι) → π i a' b' x' : ι → α inst✝ : Nonempty ι ha : ∀ (i : ι), a i < x i hb : ∀ (i : ι), x i < b i i : ι x✝ : i ∈ univ ⊢ Ioo (a i) (b i) ∈ 𝓝 (x i) ** exact Ioo_mem_nhds (ha i) (hb i) ** Qed
disjoint_nhds_atTop ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : NoMaxOrder α x : α ⊢ Disjoint (𝓝 x) atTop ** rcases exists_gt x with ⟨y, hy : x < y⟩ ** case intro α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : NoMaxOrder α x y : α hy : x < y ⊢ Disjoint (𝓝 x) atTop ** refine' disjoint_of_disjoint_of_mem _ (Iio_mem_nhds hy) (mem_atTop y) ** case intro α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : NoMaxOrder α x y : α hy : x < y ⊢ Disjoint (Iio y) {b | y ≤ b} ** exact disjoint_left.mpr fun z => not_le.2 ** Qed
TFAE_mem_nhdsWithin_Ioi ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a b : α hab : a < b s : Set α ⊢ TFAE [s ∈ 𝓝[Ioi a] a, s ∈ 𝓝[Ioc a b] a, s ∈ 𝓝[Ioo a b] a, ∃ u, u ∈ Ioc a b ∧ Ioo a u ⊆ s, ∃ u, u ∈ Ioi a ∧ Ioo a u ⊆ s] ** tfae_have 1 ↔ 2 ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a b : α hab : a < b s : Set α tfae_1_iff_2 : s ∈ 𝓝[Ioi a] a ↔ s ∈ 𝓝[Ioc a b] a ⊢ TFAE [s ∈ 𝓝[Ioi a] a, s ∈ 𝓝[Ioc a b] a, s ∈ 𝓝[Ioo a b] a, ∃ u, u ∈ Ioc a b ∧ Ioo a u ⊆ s, ∃ u, u ∈ Ioi a ∧ Ioo a u ⊆ s] ** tfae_have 1 ↔ 3 ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a b : α hab : a < b s : Set α tfae_1_iff_2 : s ∈ 𝓝[Ioi a] a ↔ s ∈ 𝓝[Ioc a b] a tfae_1_iff_3 : s ∈ 𝓝[Ioi a] a ↔ s ∈ 𝓝[Ioo a b] a ⊢ TFAE [s ∈ 𝓝[Ioi a] a, s ∈ 𝓝[Ioc a b] a, s ∈ 𝓝[Ioo a b] a, ∃ u, u ∈ Ioc a b ∧ Ioo a u ⊆ s, ∃ u, u ∈ Ioi a ∧ Ioo a u ⊆ s] ** tfae_have 4 → 5 ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a b : α hab : a < b s : Set α tfae_1_iff_2 : s ∈ 𝓝[Ioi a] a ↔ s ∈ 𝓝[Ioc a b] a tfae_1_iff_3 : s ∈ 𝓝[Ioi a] a ↔ s ∈ 𝓝[Ioo a b] a tfae_4_to_5 : (∃ u, u ∈ Ioc a b ∧ Ioo a u ⊆ s) → ∃ u, u ∈ Ioi a ∧ Ioo a u ⊆ s ⊢ TFAE [s ∈ 𝓝[Ioi a] a, s ∈ 𝓝[Ioc a b] a, s ∈ 𝓝[Ioo a b] a, ∃ u, u ∈ Ioc a b ∧ Ioo a u ⊆ s, ∃ u, u ∈ Ioi a ∧ Ioo a u ⊆ s] ** tfae_have 5 → 1 ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a b : α hab : a < b s : Set α tfae_1_iff_2 : s ∈ 𝓝[Ioi a] a ↔ s ∈ 𝓝[Ioc a b] a tfae_1_iff_3 : s ∈ 𝓝[Ioi a] a ↔ s ∈ 𝓝[Ioo a b] a tfae_4_to_5 : (∃ u, u ∈ Ioc a b ∧ Ioo a u ⊆ s) → ∃ u, u ∈ Ioi a ∧ Ioo a u ⊆ s tfae_5_to_1 : (∃ u, u ∈ Ioi a ∧ Ioo a u ⊆ s) → s ∈ 𝓝[Ioi a] a ⊢ TFAE [s ∈ 𝓝[Ioi a] a, s ∈ 𝓝[Ioc a b] a, s ∈ 𝓝[Ioo a b] a, ∃ u, u ∈ Ioc a b ∧ Ioo a u ⊆ s, ∃ u, u ∈ Ioi a ∧ Ioo a u ⊆ s] ** tfae_have 1 → 4 ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a b : α hab : a < b s : Set α tfae_1_iff_2 : s ∈ 𝓝[Ioi a] a ↔ s ∈ 𝓝[Ioc a b] a tfae_1_iff_3 : s ∈ 𝓝[Ioi a] a ↔ s ∈ 𝓝[Ioo a b] a tfae_4_to_5 : (∃ u, u ∈ Ioc a b ∧ Ioo a u ⊆ s) → ∃ u, u ∈ Ioi a ∧ Ioo a u ⊆ s tfae_5_to_1 : (∃ u, u ∈ Ioi a ∧ Ioo a u ⊆ s) → s ∈ 𝓝[Ioi a] a tfae_1_to_4 : s ∈ 𝓝[Ioi a] a → ∃ u, u ∈ Ioc a b ∧ Ioo a u ⊆ s ⊢ TFAE [s ∈ 𝓝[Ioi a] a, s ∈ 𝓝[Ioc a b] a, s ∈ 𝓝[Ioo a b] a, ∃ u, u ∈ Ioc a b ∧ Ioo a u ⊆ s, ∃ u, u ∈ Ioi a ∧ Ioo a u ⊆ s] ** tfae_finish ** case tfae_1_iff_2 α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a b : α hab : a < b s : Set α ⊢ s ∈ 𝓝[Ioi a] a ↔ s ∈ 𝓝[Ioc a b] a ** rw [nhdsWithin_Ioc_eq_nhdsWithin_Ioi hab] ** case tfae_1_iff_3 α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a b : α hab : a < b s : Set α tfae_1_iff_2 : s ∈ 𝓝[Ioi a] a ↔ s ∈ 𝓝[Ioc a b] a ⊢ s ∈ 𝓝[Ioi a] a ↔ s ∈ 𝓝[Ioo a b] a ** rw [nhdsWithin_Ioo_eq_nhdsWithin_Ioi hab] ** case tfae_4_to_5 α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a b : α hab : a < b s : Set α tfae_1_iff_2 : s ∈ 𝓝[Ioi a] a ↔ s ∈ 𝓝[Ioc a b] a tfae_1_iff_3 : s ∈ 𝓝[Ioi a] a ↔ s ∈ 𝓝[Ioo a b] a ⊢ (∃ u, u ∈ Ioc a b ∧ Ioo a u ⊆ s) → ∃ u, u ∈ Ioi a ∧ Ioo a u ⊆ s ** exact fun ⟨u, umem, hu⟩ => ⟨u, umem.1, hu⟩ ** case tfae_5_to_1 α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a b : α hab : a < b s : Set α tfae_1_iff_2 : s ∈ 𝓝[Ioi a] a ↔ s ∈ 𝓝[Ioc a b] a tfae_1_iff_3 : s ∈ 𝓝[Ioi a] a ↔ s ∈ 𝓝[Ioo a b] a tfae_4_to_5 : (∃ u, u ∈ Ioc a b ∧ Ioo a u ⊆ s) → ∃ u, u ∈ Ioi a ∧ Ioo a u ⊆ s ⊢ (∃ u, u ∈ Ioi a ∧ Ioo a u ⊆ s) → s ∈ 𝓝[Ioi a] a ** rintro ⟨u, hau, hu⟩ ** case tfae_5_to_1.intro.intro α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a b : α hab : a < b s : Set α tfae_1_iff_2 : s ∈ 𝓝[Ioi a] a ↔ s ∈ 𝓝[Ioc a b] a tfae_1_iff_3 : s ∈ 𝓝[Ioi a] a ↔ s ∈ 𝓝[Ioo a b] a tfae_4_to_5 : (∃ u, u ∈ Ioc a b ∧ Ioo a u ⊆ s) → ∃ u, u ∈ Ioi a ∧ Ioo a u ⊆ s u : α hau : u ∈ Ioi a hu : Ioo a u ⊆ s ⊢ s ∈ 𝓝[Ioi a] a ** exact mem_of_superset (Ioo_mem_nhdsWithin_Ioi ⟨le_refl a, hau⟩) hu ** case tfae_1_to_4 α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a b : α hab : a < b s : Set α tfae_1_iff_2 : s ∈ 𝓝[Ioi a] a ↔ s ∈ 𝓝[Ioc a b] a tfae_1_iff_3 : s ∈ 𝓝[Ioi a] a ↔ s ∈ 𝓝[Ioo a b] a tfae_4_to_5 : (∃ u, u ∈ Ioc a b ∧ Ioo a u ⊆ s) → ∃ u, u ∈ Ioi a ∧ Ioo a u ⊆ s tfae_5_to_1 : (∃ u, u ∈ Ioi a ∧ Ioo a u ⊆ s) → s ∈ 𝓝[Ioi a] a ⊢ s ∈ 𝓝[Ioi a] a → ∃ u, u ∈ Ioc a b ∧ Ioo a u ⊆ s ** intro h ** case tfae_1_to_4 α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a b : α hab : a < b s : Set α tfae_1_iff_2 : s ∈ 𝓝[Ioi a] a ↔ s ∈ 𝓝[Ioc a b] a tfae_1_iff_3 : s ∈ 𝓝[Ioi a] a ↔ s ∈ 𝓝[Ioo a b] a tfae_4_to_5 : (∃ u, u ∈ Ioc a b ∧ Ioo a u ⊆ s) → ∃ u, u ∈ Ioi a ∧ Ioo a u ⊆ s tfae_5_to_1 : (∃ u, u ∈ Ioi a ∧ Ioo a u ⊆ s) → s ∈ 𝓝[Ioi a] a h : s ∈ 𝓝[Ioi a] a ⊢ ∃ u, u ∈ Ioc a b ∧ Ioo a u ⊆ s ** rcases mem_nhdsWithin_iff_exists_mem_nhds_inter.1 h with ⟨v, va, hv⟩ ** case tfae_1_to_4.intro.intro α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a b : α hab : a < b s : Set α tfae_1_iff_2 : s ∈ 𝓝[Ioi a] a ↔ s ∈ 𝓝[Ioc a b] a tfae_1_iff_3 : s ∈ 𝓝[Ioi a] a ↔ s ∈ 𝓝[Ioo a b] a tfae_4_to_5 : (∃ u, u ∈ Ioc a b ∧ Ioo a u ⊆ s) → ∃ u, u ∈ Ioi a ∧ Ioo a u ⊆ s tfae_5_to_1 : (∃ u, u ∈ Ioi a ∧ Ioo a u ⊆ s) → s ∈ 𝓝[Ioi a] a h : s ∈ 𝓝[Ioi a] a v : Set α va : v ∈ 𝓝 a hv : v ∩ Ioi a ⊆ s ⊢ ∃ u, u ∈ Ioc a b ∧ Ioo a u ⊆ s ** rcases exists_Ico_subset_of_mem_nhds' va hab with ⟨u, au, hu⟩ ** case tfae_1_to_4.intro.intro.intro.intro α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a b : α hab : a < b s : Set α tfae_1_iff_2 : s ∈ 𝓝[Ioi a] a ↔ s ∈ 𝓝[Ioc a b] a tfae_1_iff_3 : s ∈ 𝓝[Ioi a] a ↔ s ∈ 𝓝[Ioo a b] a tfae_4_to_5 : (∃ u, u ∈ Ioc a b ∧ Ioo a u ⊆ s) → ∃ u, u ∈ Ioi a ∧ Ioo a u ⊆ s tfae_5_to_1 : (∃ u, u ∈ Ioi a ∧ Ioo a u ⊆ s) → s ∈ 𝓝[Ioi a] a h : s ∈ 𝓝[Ioi a] a v : Set α va : v ∈ 𝓝 a hv : v ∩ Ioi a ⊆ s u : α au : u ∈ Ioc a b hu : Ico a u ⊆ v ⊢ ∃ u, u ∈ Ioc a b ∧ Ioo a u ⊆ s ** refine' ⟨u, au, fun x hx => _⟩ ** case tfae_1_to_4.intro.intro.intro.intro α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a b : α hab : a < b s : Set α tfae_1_iff_2 : s ∈ 𝓝[Ioi a] a ↔ s ∈ 𝓝[Ioc a b] a tfae_1_iff_3 : s ∈ 𝓝[Ioi a] a ↔ s ∈ 𝓝[Ioo a b] a tfae_4_to_5 : (∃ u, u ∈ Ioc a b ∧ Ioo a u ⊆ s) → ∃ u, u ∈ Ioi a ∧ Ioo a u ⊆ s tfae_5_to_1 : (∃ u, u ∈ Ioi a ∧ Ioo a u ⊆ s) → s ∈ 𝓝[Ioi a] a h : s ∈ 𝓝[Ioi a] a v : Set α va : v ∈ 𝓝 a hv : v ∩ Ioi a ⊆ s u : α au : u ∈ Ioc a b hu : Ico a u ⊆ v x : α hx : x ∈ Ioo a u ⊢ x ∈ s ** refine' hv ⟨hu ⟨le_of_lt hx.1, hx.2⟩, _⟩ ** case tfae_1_to_4.intro.intro.intro.intro α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a b : α hab : a < b s : Set α tfae_1_iff_2 : s ∈ 𝓝[Ioi a] a ↔ s ∈ 𝓝[Ioc a b] a tfae_1_iff_3 : s ∈ 𝓝[Ioi a] a ↔ s ∈ 𝓝[Ioo a b] a tfae_4_to_5 : (∃ u, u ∈ Ioc a b ∧ Ioo a u ⊆ s) → ∃ u, u ∈ Ioi a ∧ Ioo a u ⊆ s tfae_5_to_1 : (∃ u, u ∈ Ioi a ∧ Ioo a u ⊆ s) → s ∈ 𝓝[Ioi a] a h : s ∈ 𝓝[Ioi a] a v : Set α va : v ∈ 𝓝 a hv : v ∩ Ioi a ⊆ s u : α au : u ∈ Ioc a b hu : Ico a u ⊆ v x : α hx : x ∈ Ioo a u ⊢ x ∈ Ioi a ** exact hx.1 ** Qed
nhdsWithin_Ioi_eq_bot_iff ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a : α ⊢ 𝓝[Ioi a] a = ⊥ ↔ IsTop a ∨ ∃ b, a ⋖ b ** by_cases ha : IsTop a ** case pos α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a : α ha : IsTop a ⊢ 𝓝[Ioi a] a = ⊥ ↔ IsTop a ∨ ∃ b, a ⋖ b ** simp [ha, ha.isMax.Ioi_eq] ** case neg α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a : α ha : ¬IsTop a ⊢ 𝓝[Ioi a] a = ⊥ ↔ IsTop a ∨ ∃ b, a ⋖ b ** simp only [ha, false_or] ** case neg α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a : α ha : ¬IsTop a ⊢ 𝓝[Ioi a] a = ⊥ ↔ ∃ b, a ⋖ b ** rw [isTop_iff_isMax, not_isMax_iff] at ha ** case neg α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a : α ha : ∃ b, a < b ⊢ 𝓝[Ioi a] a = ⊥ ↔ ∃ b, a ⋖ b ** simp only [(nhdsWithin_Ioi_basis' ha).eq_bot_iff, covby_iff_Ioo_eq] ** Qed
countable_setOf_isolated_right ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : SecondCountableTopology α ⊢ Set.Countable {x | 𝓝[Ioi x] x = ⊥} ** simp only [nhdsWithin_Ioi_eq_bot_iff, setOf_or] ** α : Type u β : Type v γ : Type w inst✝³ : TopologicalSpace α inst✝² : LinearOrder α inst✝¹ : OrderTopology α inst✝ : SecondCountableTopology α ⊢ Set.Countable ({a | IsTop a} ∪ {a | ∃ b, a ⋖ b}) ** exact (subsingleton_isTop α).countable.union countable_setOf_covby_right ** Qed
mem_nhdsWithin_Ioi_iff_exists_Ioc_subset ** α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderTopology α inst✝¹ : NoMaxOrder α inst✝ : DenselyOrdered α a : α s : Set α ⊢ s ∈ 𝓝[Ioi a] a ↔ ∃ u, u ∈ Ioi a ∧ Ioc a u ⊆ s ** rw [mem_nhdsWithin_Ioi_iff_exists_Ioo_subset] ** α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderTopology α inst✝¹ : NoMaxOrder α inst✝ : DenselyOrdered α a : α s : Set α ⊢ (∃ u, u ∈ Ioi a ∧ Ioo a u ⊆ s) ↔ ∃ u, u ∈ Ioi a ∧ Ioc a u ⊆ s ** constructor ** case mp α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderTopology α inst✝¹ : NoMaxOrder α inst✝ : DenselyOrdered α a : α s : Set α ⊢ (∃ u, u ∈ Ioi a ∧ Ioo a u ⊆ s) → ∃ u, u ∈ Ioi a ∧ Ioc a u ⊆ s ** rintro ⟨u, au, as⟩ ** case mp.intro.intro α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderTopology α inst✝¹ : NoMaxOrder α inst✝ : DenselyOrdered α a : α s : Set α u : α au : u ∈ Ioi a as : Ioo a u ⊆ s ⊢ ∃ u, u ∈ Ioi a ∧ Ioc a u ⊆ s ** rcases exists_between au with ⟨v, hv⟩ ** case mp.intro.intro.intro α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderTopology α inst✝¹ : NoMaxOrder α inst✝ : DenselyOrdered α a : α s : Set α u : α au : u ∈ Ioi a as : Ioo a u ⊆ s v : α hv : a < v ∧ v < u ⊢ ∃ u, u ∈ Ioi a ∧ Ioc a u ⊆ s ** exact ⟨v, hv.1, fun x hx => as ⟨hx.1, lt_of_le_of_lt hx.2 hv.2⟩⟩ ** case mpr α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderTopology α inst✝¹ : NoMaxOrder α inst✝ : DenselyOrdered α a : α s : Set α ⊢ (∃ u, u ∈ Ioi a ∧ Ioc a u ⊆ s) → ∃ u, u ∈ Ioi a ∧ Ioo a u ⊆ s ** rintro ⟨u, au, as⟩ ** case mpr.intro.intro α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderTopology α inst✝¹ : NoMaxOrder α inst✝ : DenselyOrdered α a : α s : Set α u : α au : u ∈ Ioi a as : Ioc a u ⊆ s ⊢ ∃ u, u ∈ Ioi a ∧ Ioo a u ⊆ s ** exact ⟨u, au, Subset.trans Ioo_subset_Ioc_self as⟩ ** Qed
TFAE_mem_nhdsWithin_Iio ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a b : α h : a < b s : Set α ⊢ TFAE [s ∈ 𝓝[Iio b] b, s ∈ 𝓝[Ico a b] b, s ∈ 𝓝[Ioo a b] b, ∃ l, l ∈ Ico a b ∧ Ioo l b ⊆ s, ∃ l, l ∈ Iio b ∧ Ioo l b ⊆ s] ** simpa only [exists_prop, OrderDual.exists, dual_Ioi, dual_Ioc, dual_Ioo] using TFAE_mem_nhdsWithin_Ioi h.dual (ofDual ⁻¹' s) ** Qed
mem_nhdsWithin_Iio_iff_exists_Ico_subset ** α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderTopology α inst✝¹ : NoMinOrder α inst✝ : DenselyOrdered α a : α s : Set α ⊢ s ∈ 𝓝[Iio a] a ↔ ∃ l, l ∈ Iio a ∧ Ico l a ⊆ s ** have : ofDual ⁻¹' s ∈ 𝓝[>] toDual a ↔ _ := mem_nhdsWithin_Ioi_iff_exists_Ioc_subset ** α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderTopology α inst✝¹ : NoMinOrder α inst✝ : DenselyOrdered α a : α s : Set α this : ↑ofDual ⁻¹' s ∈ 𝓝[Ioi (↑toDual a)] ↑toDual a ↔ ∃ u, u ∈ Ioi (↑toDual a) ∧ Ioc (↑toDual a) u ⊆ ↑ofDual ⁻¹' s ⊢ s ∈ 𝓝[Iio a] a ↔ ∃ l, l ∈ Iio a ∧ Ico l a ⊆ s ** simpa only [OrderDual.exists, exists_prop, dual_Ioc] using this ** Qed
nhdsWithin_Iio_eq_bot_iff ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a : α ⊢ 𝓝[Iio a] a = ⊥ ↔ IsBot a ∨ ∃ b, b ⋖ a ** convert (config := {preTransparency := .default}) nhdsWithin_Ioi_eq_bot_iff (a := OrderDual.toDual a) using 4 ** case h.e'_2.h.e'_2.h.e'_2.h.h.a α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a : α e_1✝ : α = (fun x => αᵒᵈ) a x✝ : α ⊢ x✝ ⋖ a ↔ ↑toDual a ⋖ x✝ ** exact ofDual_covby_ofDual_iff ** Qed
TFAE_mem_nhdsWithin_Ici ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a b : α hab : a < b s : Set α ⊢ TFAE [s ∈ 𝓝[Ici a] a, s ∈ 𝓝[Icc a b] a, s ∈ 𝓝[Ico a b] a, ∃ u, u ∈ Ioc a b ∧ Ico a u ⊆ s, ∃ u, u ∈ Ioi a ∧ Ico a u ⊆ s] ** tfae_have 1 ↔ 2 ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a b : α hab : a < b s : Set α tfae_1_iff_2 : s ∈ 𝓝[Ici a] a ↔ s ∈ 𝓝[Icc a b] a ⊢ TFAE [s ∈ 𝓝[Ici a] a, s ∈ 𝓝[Icc a b] a, s ∈ 𝓝[Ico a b] a, ∃ u, u ∈ Ioc a b ∧ Ico a u ⊆ s, ∃ u, u ∈ Ioi a ∧ Ico a u ⊆ s] ** tfae_have 1 ↔ 3 ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a b : α hab : a < b s : Set α tfae_1_iff_2 : s ∈ 𝓝[Ici a] a ↔ s ∈ 𝓝[Icc a b] a tfae_1_iff_3 : s ∈ 𝓝[Ici a] a ↔ s ∈ 𝓝[Ico a b] a ⊢ TFAE [s ∈ 𝓝[Ici a] a, s ∈ 𝓝[Icc a b] a, s ∈ 𝓝[Ico a b] a, ∃ u, u ∈ Ioc a b ∧ Ico a u ⊆ s, ∃ u, u ∈ Ioi a ∧ Ico a u ⊆ s] ** tfae_have 1 ↔ 5 ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a b : α hab : a < b s : Set α tfae_1_iff_2 : s ∈ 𝓝[Ici a] a ↔ s ∈ 𝓝[Icc a b] a tfae_1_iff_3 : s ∈ 𝓝[Ici a] a ↔ s ∈ 𝓝[Ico a b] a tfae_1_iff_5 : s ∈ 𝓝[Ici a] a ↔ ∃ u, u ∈ Ioi a ∧ Ico a u ⊆ s ⊢ TFAE [s ∈ 𝓝[Ici a] a, s ∈ 𝓝[Icc a b] a, s ∈ 𝓝[Ico a b] a, ∃ u, u ∈ Ioc a b ∧ Ico a u ⊆ s, ∃ u, u ∈ Ioi a ∧ Ico a u ⊆ s] ** tfae_have 4 → 5 ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a b : α hab : a < b s : Set α tfae_1_iff_2 : s ∈ 𝓝[Ici a] a ↔ s ∈ 𝓝[Icc a b] a tfae_1_iff_3 : s ∈ 𝓝[Ici a] a ↔ s ∈ 𝓝[Ico a b] a tfae_1_iff_5 : s ∈ 𝓝[Ici a] a ↔ ∃ u, u ∈ Ioi a ∧ Ico a u ⊆ s tfae_4_to_5 : (∃ u, u ∈ Ioc a b ∧ Ico a u ⊆ s) → ∃ u, u ∈ Ioi a ∧ Ico a u ⊆ s ⊢ TFAE [s ∈ 𝓝[Ici a] a, s ∈ 𝓝[Icc a b] a, s ∈ 𝓝[Ico a b] a, ∃ u, u ∈ Ioc a b ∧ Ico a u ⊆ s, ∃ u, u ∈ Ioi a ∧ Ico a u ⊆ s] ** tfae_have 5 → 4 ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a b : α hab : a < b s : Set α tfae_1_iff_2 : s ∈ 𝓝[Ici a] a ↔ s ∈ 𝓝[Icc a b] a tfae_1_iff_3 : s ∈ 𝓝[Ici a] a ↔ s ∈ 𝓝[Ico a b] a tfae_1_iff_5 : s ∈ 𝓝[Ici a] a ↔ ∃ u, u ∈ Ioi a ∧ Ico a u ⊆ s tfae_4_to_5 : (∃ u, u ∈ Ioc a b ∧ Ico a u ⊆ s) → ∃ u, u ∈ Ioi a ∧ Ico a u ⊆ s tfae_5_to_4 : (∃ u, u ∈ Ioi a ∧ Ico a u ⊆ s) → ∃ u, u ∈ Ioc a b ∧ Ico a u ⊆ s ⊢ TFAE [s ∈ 𝓝[Ici a] a, s ∈ 𝓝[Icc a b] a, s ∈ 𝓝[Ico a b] a, ∃ u, u ∈ Ioc a b ∧ Ico a u ⊆ s, ∃ u, u ∈ Ioi a ∧ Ico a u ⊆ s] ** tfae_finish ** case tfae_1_iff_2 α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a b : α hab : a < b s : Set α ⊢ s ∈ 𝓝[Ici a] a ↔ s ∈ 𝓝[Icc a b] a ** rw [nhdsWithin_Icc_eq_nhdsWithin_Ici hab] ** case tfae_1_iff_3 α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a b : α hab : a < b s : Set α tfae_1_iff_2 : s ∈ 𝓝[Ici a] a ↔ s ∈ 𝓝[Icc a b] a ⊢ s ∈ 𝓝[Ici a] a ↔ s ∈ 𝓝[Ico a b] a ** rw [nhdsWithin_Ico_eq_nhdsWithin_Ici hab] ** case tfae_1_iff_5 α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a b : α hab : a < b s : Set α tfae_1_iff_2 : s ∈ 𝓝[Ici a] a ↔ s ∈ 𝓝[Icc a b] a tfae_1_iff_3 : s ∈ 𝓝[Ici a] a ↔ s ∈ 𝓝[Ico a b] a ⊢ s ∈ 𝓝[Ici a] a ↔ ∃ u, u ∈ Ioi a ∧ Ico a u ⊆ s ** exact (nhdsWithin_Ici_basis' ⟨b, hab⟩).mem_iff ** case tfae_4_to_5 α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a b : α hab : a < b s : Set α tfae_1_iff_2 : s ∈ 𝓝[Ici a] a ↔ s ∈ 𝓝[Icc a b] a tfae_1_iff_3 : s ∈ 𝓝[Ici a] a ↔ s ∈ 𝓝[Ico a b] a tfae_1_iff_5 : s ∈ 𝓝[Ici a] a ↔ ∃ u, u ∈ Ioi a ∧ Ico a u ⊆ s ⊢ (∃ u, u ∈ Ioc a b ∧ Ico a u ⊆ s) → ∃ u, u ∈ Ioi a ∧ Ico a u ⊆ s ** exact fun ⟨u, umem, hu⟩ => ⟨u, umem.1, hu⟩ ** case tfae_5_to_4 α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a b : α hab : a < b s : Set α tfae_1_iff_2 : s ∈ 𝓝[Ici a] a ↔ s ∈ 𝓝[Icc a b] a tfae_1_iff_3 : s ∈ 𝓝[Ici a] a ↔ s ∈ 𝓝[Ico a b] a tfae_1_iff_5 : s ∈ 𝓝[Ici a] a ↔ ∃ u, u ∈ Ioi a ∧ Ico a u ⊆ s tfae_4_to_5 : (∃ u, u ∈ Ioc a b ∧ Ico a u ⊆ s) → ∃ u, u ∈ Ioi a ∧ Ico a u ⊆ s ⊢ (∃ u, u ∈ Ioi a ∧ Ico a u ⊆ s) → ∃ u, u ∈ Ioc a b ∧ Ico a u ⊆ s ** rintro ⟨u, hua, hus⟩ ** case tfae_5_to_4.intro.intro α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a b : α hab : a < b s : Set α tfae_1_iff_2 : s ∈ 𝓝[Ici a] a ↔ s ∈ 𝓝[Icc a b] a tfae_1_iff_3 : s ∈ 𝓝[Ici a] a ↔ s ∈ 𝓝[Ico a b] a tfae_1_iff_5 : s ∈ 𝓝[Ici a] a ↔ ∃ u, u ∈ Ioi a ∧ Ico a u ⊆ s tfae_4_to_5 : (∃ u, u ∈ Ioc a b ∧ Ico a u ⊆ s) → ∃ u, u ∈ Ioi a ∧ Ico a u ⊆ s u : α hua : u ∈ Ioi a hus : Ico a u ⊆ s ⊢ ∃ u, u ∈ Ioc a b ∧ Ico a u ⊆ s ** exact ⟨min u b, ⟨lt_min hua hab, min_le_right _ _⟩, (Ico_subset_Ico_right <| min_le_left _ _).trans hus⟩ ** Qed
mem_nhdsWithin_Ici_iff_exists_mem_Ioc_Ico_subset ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a u' : α s : Set α hu' : a < u' ⊢ List.get? [s ∈ 𝓝[Ici a] a, s ∈ 𝓝[Icc a u'] a, s ∈ 𝓝[Ico a u'] a, ∃ u, u ∈ Ioc a u' ∧ Ico a u ⊆ s, ∃ u, u ∈ Ioi a ∧ Ico a u ⊆ s] 0 = some (s ∈ 𝓝[Ici a] a) ** norm_num ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a u' : α s : Set α hu' : a < u' ⊢ List.get? [s ∈ 𝓝[Ici a] a, s ∈ 𝓝[Icc a u'] a, s ∈ 𝓝[Ico a u'] a, ∃ u, u ∈ Ioc a u' ∧ Ico a u ⊆ s, ∃ u, u ∈ Ioi a ∧ Ico a u ⊆ s] 3 = some (∃ u, u ∈ Ioc a u' ∧ Ico a u ⊆ s) ** norm_num ** Qed
mem_nhdsWithin_Ici_iff_exists_Ico_subset' ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a u' : α s : Set α hu' : a < u' ⊢ List.get? [s ∈ 𝓝[Ici a] a, s ∈ 𝓝[Icc a u'] a, s ∈ 𝓝[Ico a u'] a, ∃ u, u ∈ Ioc a u' ∧ Ico a u ⊆ s, ∃ u, u ∈ Ioi a ∧ Ico a u ⊆ s] 0 = some (s ∈ 𝓝[Ici a] a) ** norm_num ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a u' : α s : Set α hu' : a < u' ⊢ List.get? [s ∈ 𝓝[Ici a] a, s ∈ 𝓝[Icc a u'] a, s ∈ 𝓝[Ico a u'] a, ∃ u, u ∈ Ioc a u' ∧ Ico a u ⊆ s, ∃ u, u ∈ Ioi a ∧ Ico a u ⊆ s] 4 = some (∃ u, u ∈ Ioi a ∧ Ico a u ⊆ s) ** norm_num ** Qed
mem_nhdsWithin_Ici_iff_exists_Icc_subset ** α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderTopology α inst✝¹ : NoMaxOrder α inst✝ : DenselyOrdered α a : α s : Set α ⊢ s ∈ 𝓝[Ici a] a ↔ ∃ u, a < u ∧ Icc a u ⊆ s ** rw [mem_nhdsWithin_Ici_iff_exists_Ico_subset] ** α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderTopology α inst✝¹ : NoMaxOrder α inst✝ : DenselyOrdered α a : α s : Set α ⊢ (∃ u, u ∈ Ioi a ∧ Ico a u ⊆ s) ↔ ∃ u, a < u ∧ Icc a u ⊆ s ** constructor ** case mp α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderTopology α inst✝¹ : NoMaxOrder α inst✝ : DenselyOrdered α a : α s : Set α ⊢ (∃ u, u ∈ Ioi a ∧ Ico a u ⊆ s) → ∃ u, a < u ∧ Icc a u ⊆ s ** rintro ⟨u, au, as⟩ ** case mp.intro.intro α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderTopology α inst✝¹ : NoMaxOrder α inst✝ : DenselyOrdered α a : α s : Set α u : α au : u ∈ Ioi a as : Ico a u ⊆ s ⊢ ∃ u, a < u ∧ Icc a u ⊆ s ** rcases exists_between au with ⟨v, hv⟩ ** case mp.intro.intro.intro α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderTopology α inst✝¹ : NoMaxOrder α inst✝ : DenselyOrdered α a : α s : Set α u : α au : u ∈ Ioi a as : Ico a u ⊆ s v : α hv : a < v ∧ v < u ⊢ ∃ u, a < u ∧ Icc a u ⊆ s ** exact ⟨v, hv.1, fun x hx => as ⟨hx.1, lt_of_le_of_lt hx.2 hv.2⟩⟩ ** case mpr α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderTopology α inst✝¹ : NoMaxOrder α inst✝ : DenselyOrdered α a : α s : Set α ⊢ (∃ u, a < u ∧ Icc a u ⊆ s) → ∃ u, u ∈ Ioi a ∧ Ico a u ⊆ s ** rintro ⟨u, au, as⟩ ** case mpr.intro.intro α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderTopology α inst✝¹ : NoMaxOrder α inst✝ : DenselyOrdered α a : α s : Set α u : α au : a < u as : Icc a u ⊆ s ⊢ ∃ u, u ∈ Ioi a ∧ Ico a u ⊆ s ** exact ⟨u, au, Subset.trans Ico_subset_Icc_self as⟩ ** Qed
TFAE_mem_nhdsWithin_Iic ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a b : α h : a < b s : Set α ⊢ TFAE [s ∈ 𝓝[Iic b] b, s ∈ 𝓝[Icc a b] b, s ∈ 𝓝[Ioc a b] b, ∃ l, l ∈ Ico a b ∧ Ioc l b ⊆ s, ∃ l, l ∈ Iio b ∧ Ioc l b ⊆ s] ** simpa only [exists_prop, OrderDual.exists, dual_Ici, dual_Ioc, dual_Icc, dual_Ico] using TFAE_mem_nhdsWithin_Ici h.dual (ofDual ⁻¹' s) ** Qed
mem_nhdsWithin_Iic_iff_exists_mem_Ico_Ioc_subset ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a l' : α s : Set α hl' : l' < a ⊢ List.get? [s ∈ 𝓝[Iic a] a, s ∈ 𝓝[Icc l' a] a, s ∈ 𝓝[Ioc l' a] a, ∃ l, l ∈ Ico l' a ∧ Ioc l a ⊆ s, ∃ l, l ∈ Iio a ∧ Ioc l a ⊆ s] 0 = some (s ∈ 𝓝[Iic a] a) ** norm_num ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a l' : α s : Set α hl' : l' < a ⊢ List.get? [s ∈ 𝓝[Iic a] a, s ∈ 𝓝[Icc l' a] a, s ∈ 𝓝[Ioc l' a] a, ∃ l, l ∈ Ico l' a ∧ Ioc l a ⊆ s, ∃ l, l ∈ Iio a ∧ Ioc l a ⊆ s] 3 = some (∃ l, l ∈ Ico l' a ∧ Ioc l a ⊆ s) ** norm_num ** Qed
mem_nhdsWithin_Iic_iff_exists_Ioc_subset' ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a l' : α s : Set α hl' : l' < a ⊢ List.get? [s ∈ 𝓝[Iic a] a, s ∈ 𝓝[Icc l' a] a, s ∈ 𝓝[Ioc l' a] a, ∃ l, l ∈ Ico l' a ∧ Ioc l a ⊆ s, ∃ l, l ∈ Iio a ∧ Ioc l a ⊆ s] 0 = some (s ∈ 𝓝[Iic a] a) ** norm_num ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrder α inst✝ : OrderTopology α a l' : α s : Set α hl' : l' < a ⊢ List.get? [s ∈ 𝓝[Iic a] a, s ∈ 𝓝[Icc l' a] a, s ∈ 𝓝[Ioc l' a] a, ∃ l, l ∈ Ico l' a ∧ Ioc l a ⊆ s, ∃ l, l ∈ Iio a ∧ Ioc l a ⊆ s] 4 = some (∃ l, l ∈ Iio a ∧ Ioc l a ⊆ s) ** norm_num ** Qed
mem_nhdsWithin_Iic_iff_exists_Icc_subset ** α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderTopology α inst✝¹ : NoMinOrder α inst✝ : DenselyOrdered α a : α s : Set α ⊢ (∃ u, ↑toDual a < ↑toDual u ∧ Icc (↑toDual a) (↑toDual u) ⊆ ↑ofDual ⁻¹' s) ↔ ∃ l, l < a ∧ Icc l a ⊆ s ** simp only [dual_Icc] ** α : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α inst✝³ : LinearOrder α inst✝² : OrderTopology α inst✝¹ : NoMinOrder α inst✝ : DenselyOrdered α a : α s : Set α ⊢ (∃ u, ↑toDual a < ↑toDual u ∧ ↑ofDual ⁻¹' Icc u a ⊆ ↑ofDual ⁻¹' s) ↔ ∃ l, l < a ∧ Icc l a ⊆ s ** rfl ** Qed
nhds_eq_iInf_abs_sub ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrderedAddCommGroup α inst✝ : OrderTopology α l : Filter β f g : β → α a : α ⊢ 𝓝 a = ⨅ r, ⨅ (_ : r > 0), 𝓟 {b | |a - b| < r} ** simp only [nhds_eq_order, abs_lt, setOf_and, ← inf_principal, iInf_inf_eq] ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrderedAddCommGroup α inst✝ : OrderTopology α l : Filter β f g : β → α a : α ⊢ (⨅ b ∈ Iio a, 𝓟 (Ioi b)) ⊓ ⨅ b ∈ Ioi a, 𝓟 (Iio b) = (⨅ x, ⨅ (_ : x > 0), 𝓟 {a_1 | -x < a - a_1}) ⊓ ⨅ x, ⨅ (_ : x > 0), 𝓟 {a_1 | a - a_1 < x} ** refine (congr_arg₂ _ ?_ ?_).trans inf_comm ** case refine_1 α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrderedAddCommGroup α inst✝ : OrderTopology α l : Filter β f g : β → α a : α ⊢ ⨅ b ∈ Iio a, 𝓟 (Ioi b) = ⨅ x, ⨅ (_ : x > 0), 𝓟 {a_1 | a - a_1 < x} ** refine (Equiv.subLeft a).iInf_congr fun x => ?_ ** case refine_1 α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrderedAddCommGroup α inst✝ : OrderTopology α l : Filter β f g : β → α a x : α ⊢ ⨅ (_ : ↑(Equiv.subLeft a) x > 0), 𝓟 {a_1 | a - a_1 < ↑(Equiv.subLeft a) x} = ⨅ (_ : x ∈ Iio a), 𝓟 (Ioi x) ** simp [Ioi] ** case refine_2 α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrderedAddCommGroup α inst✝ : OrderTopology α l : Filter β f g : β → α a : α ⊢ ⨅ b ∈ Ioi a, 𝓟 (Iio b) = ⨅ x, ⨅ (_ : x > 0), 𝓟 {a_1 | -x < a - a_1} ** refine (Equiv.subRight a).iInf_congr fun x => ?_ ** case refine_2 α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrderedAddCommGroup α inst✝ : OrderTopology α l : Filter β f g : β → α a x : α ⊢ ⨅ (_ : ↑(Equiv.subRight a) x > 0), 𝓟 {a_1 | -↑(Equiv.subRight a) x < a - a_1} = ⨅ (_ : x ∈ Ioi a), 𝓟 (Iio x) ** simp [Iio] ** Qed
orderTopology_of_nhds_abs ** α✝ : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α✝ inst✝³ : LinearOrderedAddCommGroup α✝ inst✝² : OrderTopology α✝ l : Filter β f g : β → α✝ α : Type u_1 inst✝¹ : TopologicalSpace α inst✝ : LinearOrderedAddCommGroup α h_nhds : ∀ (a : α), 𝓝 a = ⨅ r, ⨅ (_ : r > 0), 𝓟 {b | |a - b| < r} ⊢ OrderTopology α ** refine' ⟨eq_of_nhds_eq_nhds fun a => _⟩ ** α✝ : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α✝ inst✝³ : LinearOrderedAddCommGroup α✝ inst✝² : OrderTopology α✝ l : Filter β f g : β → α✝ α : Type u_1 inst✝¹ : TopologicalSpace α inst✝ : LinearOrderedAddCommGroup α h_nhds : ∀ (a : α), 𝓝 a = ⨅ r, ⨅ (_ : r > 0), 𝓟 {b | |a - b| < r} a : α ⊢ 𝓝 a = 𝓝 a ** rw [h_nhds] ** α✝ : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α✝ inst✝³ : LinearOrderedAddCommGroup α✝ inst✝² : OrderTopology α✝ l : Filter β f g : β → α✝ α : Type u_1 inst✝¹ : TopologicalSpace α inst✝ : LinearOrderedAddCommGroup α h_nhds : ∀ (a : α), 𝓝 a = ⨅ r, ⨅ (_ : r > 0), 𝓟 {b | |a - b| < r} a : α ⊢ ⨅ r, ⨅ (_ : r > 0), 𝓟 {b | |a - b| < r} = 𝓝 a ** letI := Preorder.topology α ** α✝ : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α✝ inst✝³ : LinearOrderedAddCommGroup α✝ inst✝² : OrderTopology α✝ l : Filter β f g : β → α✝ α : Type u_1 inst✝¹ : TopologicalSpace α inst✝ : LinearOrderedAddCommGroup α h_nhds : ∀ (a : α), 𝓝 a = ⨅ r, ⨅ (_ : r > 0), 𝓟 {b | |a - b| < r} a : α this : TopologicalSpace α := Preorder.topology α ⊢ ⨅ r, ⨅ (_ : r > 0), 𝓟 {b | |a - b| < r} = 𝓝 a ** letI : OrderTopology α := ⟨rfl⟩ ** α✝ : Type u β : Type v γ : Type w inst✝⁴ : TopologicalSpace α✝ inst✝³ : LinearOrderedAddCommGroup α✝ inst✝² : OrderTopology α✝ l : Filter β f g : β → α✝ α : Type u_1 inst✝¹ : TopologicalSpace α inst✝ : LinearOrderedAddCommGroup α h_nhds : ∀ (a : α), 𝓝 a = ⨅ r, ⨅ (_ : r > 0), 𝓟 {b | |a - b| < r} a : α this✝ : TopologicalSpace α := Preorder.topology α this : OrderTopology α := { topology_eq_generate_intervals := rfl } ⊢ ⨅ r, ⨅ (_ : r > 0), 𝓟 {b | |a - b| < r} = 𝓝 a ** exact (nhds_eq_iInf_abs_sub a).symm ** Qed
LinearOrderedAddCommGroup.tendsto_nhds ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrderedAddCommGroup α inst✝ : OrderTopology α l : Filter β f g : β → α x : Filter β a : α ⊢ Tendsto f x (𝓝 a) ↔ ∀ (ε : α), ε > 0 → ∀ᶠ (b : β) in x, |f b - a| < ε ** simp [nhds_eq_iInf_abs_sub, abs_sub_comm a] ** Qed
eventually_abs_sub_lt ** α : Type u β : Type v γ : Type w inst✝² : TopologicalSpace α inst✝¹ : LinearOrderedAddCommGroup α inst✝ : OrderTopology α l : Filter β f g : β → α a ε : α hε : 0 < ε ⊢ {x | (fun x => |x - a| < ε) x} ∈ 𝓟 {b | |a - b| < ε} ** simp only [abs_sub_comm, mem_principal_self] ** Qed