src/HOL/Analysis/Arcwise_Connected.thy
changeset 68527 2f4e2aab190a
parent 67968 a5ad4c015d1c
child 68833 fde093888c16
--- a/src/HOL/Analysis/Arcwise_Connected.thy	Thu Jun 28 10:13:54 2018 +0200
+++ b/src/HOL/Analysis/Arcwise_Connected.thy	Thu Jun 28 14:13:57 2018 +0100
@@ -1243,7 +1243,7 @@
         by (metis atLeastAtMost_iff a_ge_0 b_le_1 order.trans)+
       moreover have "y < \<delta> + c (real m / 2 ^ n)" "c (real m / 2 ^ n) < \<delta> + y"
         using y apply simp_all
-        using alec [of m n] cleb [of m n] n real_sum_of_halves close_ab [OF \<open>odd m\<close>, of n]
+        using alec [of m n] cleb [of m n] n field_sum_of_halves close_ab [OF \<open>odd m\<close>, of n]
         by linarith+
       moreover note \<open>0 < m\<close> mless \<open>0 \<le> x\<close> \<open>x \<le> 1\<close>
       ultimately show "\<exists>k. \<exists>m\<in>{0<..<2 ^ k}. dist (h (real m / 2 ^ k)) (f x) < e"