src/HOL/Matrix_LP/ComputeFloat.thy
changeset 65583 8d53b3bebab4
parent 63901 4ce989e962e0
child 66453 cc19f7ca2ed6
--- a/src/HOL/Matrix_LP/ComputeFloat.thy	Tue Apr 25 21:31:28 2017 +0200
+++ b/src/HOL/Matrix_LP/ComputeFloat.thy	Wed Apr 26 15:53:35 2017 +0100
@@ -170,7 +170,7 @@
 lemma float_add:
   "float (a1, e1) + float (a2, e2) =
   (if e1<=e2 then float (a1+a2*2^(nat(e2-e1)), e1) else float (a1*2^(nat (e1-e2))+a2, e2))"
-  by (simp add: float_def algebra_simps powr_realpow[symmetric] powr_divide2[symmetric])
+  by (simp add: float_def algebra_simps powr_realpow[symmetric] powr_diff)
 
 lemma float_mult_l0: "float (0, e) * x = float (0, 0)"
   by (simp add: float_def)