src/HOL/Real.thy
changeset 62390 842917225d56
parent 62348 9a5f43dac883
child 62398 a4b68bf18f8d
--- a/src/HOL/Real.thy	Tue Feb 23 15:37:18 2016 +0100
+++ b/src/HOL/Real.thy	Tue Feb 23 16:25:08 2016 +0100
@@ -476,7 +476,7 @@
   shows "inverse (Real X) =
     (if vanishes X then 0 else Real (\<lambda>n. inverse (X n)))"
   using assms inverse_real.transfer zero_real.transfer
-  unfolding cr_real_eq rel_fun_def by (simp split: split_if_asm, metis)
+  unfolding cr_real_eq rel_fun_def by (simp split: if_split_asm, metis)
 
 instance proof
   fix a b c :: real