src/HOL/Rat.thy
changeset 48891 c0eafbd55de3
parent 47952 36a8c477dae8
child 49962 a8cc904a6820
--- a/src/HOL/Rat.thy	Wed Aug 22 22:47:16 2012 +0200
+++ b/src/HOL/Rat.thy	Wed Aug 22 22:55:41 2012 +0200
@@ -6,7 +6,6 @@
 
 theory Rat
 imports GCD Archimedean_Field
-uses ("Tools/float_syntax.ML")
 begin
 
 subsection {* Rational numbers as quotient *}
@@ -1107,7 +1106,7 @@
 
 syntax "_Float" :: "float_const \<Rightarrow> 'a"    ("_")
 
-use "Tools/float_syntax.ML"
+ML_file "Tools/float_syntax.ML"
 setup Float_Syntax.setup
 
 text{* Test: *}