proper use of float.ML;
authorwenzelm
Thu, 28 Sep 2006 23:42:45 +0200
changeset 20771 89bec28a03c8
parent 20770 2c583720436e
child 20772 7a51ed817ec7
proper use of float.ML;
src/HOL/Real/Float.thy
--- a/src/HOL/Real/Float.thy	Thu Sep 28 23:42:43 2006 +0200
+++ b/src/HOL/Real/Float.thy	Thu Sep 28 23:42:45 2006 +0200
@@ -7,6 +7,7 @@
 
 theory Float
 imports Real
+uses ("float.ML")
 begin
 
 definition
@@ -521,4 +522,6 @@
 (* for use with the compute oracle *)
 lemmas arith = binarith intarith intarithrel natarith powerarith floatarith not_false_eq_true not_true_eq_false
 
+use "float.ML";
+
 end