src/HOL/Analysis/Uniform_Limit.thy
changeset 73932 fd21b4a93043
parent 70817 dd675800469d
child 76722 b1d57dd345e1
--- a/src/HOL/Analysis/Uniform_Limit.thy	Fri Jun 18 15:03:12 2021 +0200
+++ b/src/HOL/Analysis/Uniform_Limit.thy	Thu Jul 08 08:42:36 2021 +0200
@@ -603,7 +603,7 @@
   then have "\<forall>\<^sub>F x in F. \<forall>y\<in>S. b/2 \<le> norm (f x y)"
     apply (rule eventually_mono)
     using b apply (simp only: dist_norm)
-    by (metis (no_types, hide_lams) diff_zero dist_commute dist_norm norm_triangle_half_l not_less)
+    by (metis (no_types, opaque_lifting) diff_zero dist_commute dist_norm norm_triangle_half_l not_less)
   then have "\<forall>\<^sub>F x in F. \<forall>y\<in>S. b/2 \<le> norm (f x y) \<and> norm (f x y - l y) < e * b\<^sup>2 / 2"
     apply (simp only: ball_conj_distrib dist_norm [symmetric])
     apply (rule eventually_conj, assumption)