File tree Expand file tree Collapse file tree 1 file changed +2
-7
lines changed Expand file tree Collapse file tree 1 file changed +2
-7
lines changed Original file line number Diff line number Diff 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** .
You can’t perform that action at this time.
0 commit comments