src/HOL/Library/Float.thy
changeset 58410 6d46ad54a2ab
parent 58042 ffa9e39763e3
child 58834 773b378d9313
--- a/src/HOL/Library/Float.thy	Sun Sep 21 16:56:06 2014 +0200
+++ b/src/HOL/Library/Float.thy	Sun Sep 21 16:56:11 2014 +0200
@@ -205,7 +205,7 @@
     done
   assume "a < b"
   then show "\<exists>c. a < c \<and> c < b"
-    apply (intro exI[of _ "(a + b) * Float 1 -1"])
+    apply (intro exI[of _ "(a + b) * Float 1 (- 1)"])
     apply transfer
     apply (simp add: powr_minus)
     done
@@ -1085,8 +1085,8 @@
 
 lemma Float_num[simp]: shows
    "real (Float 1 0) = 1" and "real (Float 1 1) = 2" and "real (Float 1 2) = 4" and
-   "real (Float 1 -1) = 1/2" and "real (Float 1 -2) = 1/4" and "real (Float 1 -3) = 1/8" and
-   "real (Float -1 0) = -1" and "real (Float (number_of n) 0) = number_of n"
+   "real (Float 1 (- 1)) = 1/2" and "real (Float 1 (- 2)) = 1/4" and "real (Float 1 (- 3)) = 1/8" and
+   "real (Float (- 1) 0) = -1" and "real (Float (number_of n) 0) = number_of n"
 using two_powr_int_float[of 2] two_powr_int_float[of "-1"] two_powr_int_float[of "-2"] two_powr_int_float[of "-3"]
 using powr_realpow[of 2 2] powr_realpow[of 2 3]
 using powr_minus[of 2 1] powr_minus[of 2 2] powr_minus[of 2 3]