src/HOL/Nat.thy
changeset 23263 0c227412b285
parent 23001 3608f0362a91
child 23276 a70934b63910
--- a/src/HOL/Nat.thy	Tue Jun 05 19:22:01 2007 +0200
+++ b/src/HOL/Nat.thy	Tue Jun 05 19:23:09 2007 +0200
@@ -10,7 +10,11 @@
 
 theory Nat
 imports Wellfounded_Recursion Ring_and_Field
-uses ("arith_data.ML")
+uses
+  "~~/src/Tools/rat.ML"
+  "~~/src/Provers/Arith/fast_lin_arith.ML"
+  "~~/src/Provers/Arith/cancel_sums.ML"
+  ("arith_data.ML")
 begin
 
 subsection {* Type @{text ind} *}