src/HOL/Limits.thy
changeset 62390 842917225d56
parent 62379 340738057c8c
child 62393 a620a8756b7c
--- a/src/HOL/Limits.thy	Tue Feb 23 15:37:18 2016 +0100
+++ b/src/HOL/Limits.thy	Tue Feb 23 16:25:08 2016 +0100
@@ -1354,7 +1354,7 @@
   fix Z :: real assume "0 < Z"
   from f \<open>0 < c\<close> have "eventually (\<lambda>x. c / 2 < f x) F"
     by (auto dest!: tendstoD[where e="c / 2"] elim!: eventually_mono
-             simp: dist_real_def abs_real_def split: split_if_asm)
+             simp: dist_real_def abs_real_def split: if_split_asm)
   moreover from g have "eventually (\<lambda>x. (Z / c * 2) \<le> g x) F"
     unfolding filterlim_at_top by auto
   ultimately show "eventually (\<lambda>x. Z \<le> f x * g x) F"