File tree Expand file tree Collapse file tree 1 file changed +2
-15
lines changed
Mathlib/Topology/MetricSpace/Ultra Expand file tree Collapse file tree 1 file changed +2
-15
lines changed Original file line number Diff line number Diff line change @@ -71,13 +71,7 @@ lemma ball_eq_of_mem {x y : X} {r : ℝ} (h : y ∈ ball x r) : ball x r = ball
71
71
constructor <;> intro h' <;>
72
72
exact (dist_triangle_max _ _ _).trans_lt (max_lt h' (dist_comm x _ ▸ h))
73
73
74
- lemma mem_ball_iff {x y : X} {r : ℝ} : y ∈ ball x r ↔ x ∈ ball y r := by
75
- cases lt_or_ge 0 r with
76
- | inl hr =>
77
- constructor <;> intro h <;>
78
- rw [← ball_eq_of_mem h] <;>
79
- simp [hr]
80
- | inr hr => simp [ball_eq_empty.mpr hr]
74
+ @[deprecated (since := "2025-08-16")] alias mem_ball_iff := mem_ball_comm
81
75
82
76
lemma ball_subset_trichotomy :
83
77
ball x r ⊆ ball y s ∨ ball y s ⊆ ball x r ∨ Disjoint (ball x r) (ball y s) := by
@@ -103,14 +97,7 @@ lemma closedBall_eq_of_mem {x y : X} {r : ℝ} (h : y ∈ closedBall x r) :
103
97
constructor <;> intro h' <;>
104
98
exact (dist_triangle_max _ _ _).trans (max_le h' (dist_comm x _ ▸ h))
105
99
106
- lemma mem_closedBall_iff {x y : X} {r : ℝ} :
107
- y ∈ closedBall x r ↔ x ∈ closedBall y r := by
108
- cases le_or_gt 0 r with
109
- | inl hr =>
110
- constructor <;> intro h <;>
111
- rw [← closedBall_eq_of_mem h] <;>
112
- simp [hr]
113
- | inr hr => simp [closedBall_eq_empty.mpr hr]
100
+ @[deprecated (since := "2025-08-16")] alias mem_closedBall_iff := mem_closedBall_comm
114
101
115
102
lemma closedBall_subset_trichotomy :
116
103
closedBall x r ⊆ closedBall y s ∨ closedBall y s ⊆ closedBall x r ∨
You can’t perform that action at this time.
0 commit comments