src/HOL/Int.thy
changeset 48891 c0eafbd55de3
parent 48066 c6783c9b87bf
child 49962 a8cc904a6820
--- a/src/HOL/Int.thy	Wed Aug 22 22:47:16 2012 +0200
+++ b/src/HOL/Int.thy	Wed Aug 22 22:55:41 2012 +0200
@@ -7,8 +7,6 @@
 
 theory Int
 imports Equiv_Relations Wellfounded Quotient
-uses
-  ("Tools/int_arith.ML")
 begin
 
 subsection {* Definition of integers as a quotient type *}
@@ -719,7 +717,7 @@
   of_nat_0 of_nat_1 of_nat_Suc of_nat_add of_nat_mult
   of_int_0 of_int_1 of_int_add of_int_mult
 
-use "Tools/int_arith.ML"
+ML_file "Tools/int_arith.ML"
 declaration {* K Int_Arith.setup *}
 
 simproc_setup fast_arith ("(m::'a::linordered_idom) < n" |