src/HOL/Library/Float.thy
changeset 47230 6584098d5378
parent 47165 9344891b504b
child 47599 400b158f1589
--- a/src/HOL/Library/Float.thy	Fri Mar 30 15:25:47 2012 +0200
+++ b/src/HOL/Library/Float.thy	Fri Mar 30 17:22:17 2012 +0200
@@ -165,9 +165,8 @@
 
   {
     assume bcmp: "b > b'"
-    then have "\<exists>c::nat. b - b' = int c + 1"
-      by arith
-    then guess c ..
+    then obtain c :: nat where "b - b' = int c + 1"
+      by atomize_elim arith
     with a' have "real a' = real (a * 2^c * 2)"
       by (simp add: pow2_def nat_add_distrib)
     with odd have False