src/HOL/Nat.thy
changeset 48891 c0eafbd55de3
parent 48560 e0875d956a6b
child 49388 1ffd5a055acf
--- a/src/HOL/Nat.thy	Wed Aug 22 22:47:16 2012 +0200
+++ b/src/HOL/Nat.thy	Wed Aug 22 22:55:41 2012 +0200
@@ -9,14 +9,13 @@
 
 theory Nat
 imports Inductive Typedef Fun Fields
-uses
-  "~~/src/Tools/rat.ML"
-  "Tools/arith_data.ML"
-  ("Tools/nat_arith.ML")
-  "~~/src/Provers/Arith/fast_lin_arith.ML"
-  ("Tools/lin_arith.ML")
 begin
 
+ML_file "~~/src/Tools/rat.ML"
+ML_file "Tools/arith_data.ML"
+ML_file "~~/src/Provers/Arith/fast_lin_arith.ML"
+
+
 subsection {* Type @{text ind} *}
 
 typedecl ind
@@ -1492,7 +1491,7 @@
 
 setup Arith_Data.setup
 
-use "Tools/nat_arith.ML"
+ML_file "Tools/nat_arith.ML"
 
 simproc_setup nateq_cancel_sums
   ("(l::nat) + m = n" | "(l::nat) = m + n" | "Suc m = n" | "m = Suc n") =
@@ -1510,7 +1509,7 @@
   ("(l::nat) + m - n" | "(l::nat) - (m + n)" | "Suc m - n" | "m - Suc n") =
   {* fn phi => fn ss => try Nat_Arith.cancel_diff_conv *}
 
-use "Tools/lin_arith.ML"
+ML_file "Tools/lin_arith.ML"
 setup {* Lin_Arith.global_setup *}
 declaration {* K Lin_Arith.setup *}