Skip to content

Commit e88d290

Browse files
committed
chore: remove porting note after simp fix (#9974)
1 parent a686ba8 commit e88d290

File tree

1 file changed

+2
-7
lines changed

1 file changed

+2
-7
lines changed

Mathlib/NumberTheory/WellApproximable.lean

Lines changed: 2 additions & 7 deletions
Original file line numberDiff line numberDiff line change
@@ -326,14 +326,9 @@ theorem addWellApproximable_ae_empty_or_univ (δ : ℕ → ℝ) (hδ : Tendsto
326326
rw [hE₁ p]
327327
cases hp
328328
· cases' hA p with _ h; · contradiction
329-
-- Porting note: was `simp only [h, union_ae_eq_univ_of_ae_eq_univ_left]`
330-
have := union_ae_eq_univ_of_ae_eq_univ_left (t := B ↑p) h
331-
exact union_ae_eq_univ_of_ae_eq_univ_left (t := C ↑p) this
329+
simp only [h, union_ae_eq_univ_of_ae_eq_univ_left]
332330
· cases' hB p with _ h; · contradiction
333-
-- Porting note: was
334-
-- `simp only [h, union_ae_eq_univ_of_ae_eq_univ_left, union_ae_eq_univ_of_ae_eq_univ_right]`
335-
have := union_ae_eq_univ_of_ae_eq_univ_right (s := A ↑p) h
336-
exact union_ae_eq_univ_of_ae_eq_univ_left (t := C ↑p) this
331+
simp only [h, union_ae_eq_univ_of_ae_eq_univ_left, union_ae_eq_univ_of_ae_eq_univ_right]
337332
#align add_circle.add_well_approximable_ae_empty_or_univ AddCircle.addWellApproximable_ae_empty_or_univ
338333

339334
/-- A general version of **Dirichlet's approximation theorem**.

0 commit comments

Comments
 (0)