src/HOL/Analysis/Uniform_Limit.thy
changeset 70817 dd675800469d
parent 70136 f03a01a18c6e
child 73932 fd21b4a93043
--- a/src/HOL/Analysis/Uniform_Limit.thy	Wed Oct 09 23:00:52 2019 +0200
+++ b/src/HOL/Analysis/Uniform_Limit.thy	Wed Oct 09 14:51:54 2019 +0000
@@ -596,7 +596,7 @@
       using \<open>e > 0\<close> that b [OF \<open>y \<in> S\<close>] apply (simp add: power2_eq_square)
       by (metis \<open>b > 0\<close> less_eq_real_def mult.left_commute mult_mono')
     finally show ?thesis
-      by (auto simp: dist_norm divide_simps norm_mult norm_divide)
+      by (auto simp: dist_norm field_split_simps norm_mult norm_divide)
   qed
   have "\<forall>\<^sub>F n in F. \<forall>x\<in>S. dist (f n x) (l x) < b/2"
     using uniform_limitD [OF f, of "b/2"] by (simp add: \<open>b > 0\<close>)