Skip to content

Commit 6e1dcf1

Browse files
committed
chore(Topology/MetricSpace/Ultra): deprecate mem_ball_iff and mem_closedBall_iff (duplicates) (#28524)
1 parent fd4b225 commit 6e1dcf1

File tree

1 file changed

+2
-15
lines changed

1 file changed

+2
-15
lines changed

Mathlib/Topology/MetricSpace/Ultra/Basic.lean

Lines changed: 2 additions & 15 deletions
Original file line numberDiff line numberDiff line change
@@ -71,13 +71,7 @@ lemma ball_eq_of_mem {x y : X} {r : ℝ} (h : y ∈ ball x r) : ball x r = ball
7171
constructor <;> intro h' <;>
7272
exact (dist_triangle_max _ _ _).trans_lt (max_lt h' (dist_comm x _ ▸ h))
7373

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
8175

8276
lemma ball_subset_trichotomy :
8377
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) :
10397
constructor <;> intro h' <;>
10498
exact (dist_triangle_max _ _ _).trans (max_le h' (dist_comm x _ ▸ h))
10599

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
114101

115102
lemma closedBall_subset_trichotomy :
116103
closedBall x r ⊆ closedBall y s ∨ closedBall y s ⊆ closedBall x r ∨

0 commit comments

Comments
 (0)