src/HOL/Int.thy
changeset 28952 15a4b2cf8c34
parent 28724 4656aacba2bc
child 28958 74c60b78969c
--- a/src/HOL/Int.thy	Wed Dec 03 09:53:58 2008 +0100
+++ b/src/HOL/Int.thy	Wed Dec 03 15:58:44 2008 +0100
@@ -16,7 +16,7 @@
   ("~~/src/Provers/Arith/assoc_fold.ML")
   "~~/src/Provers/Arith/cancel_numerals.ML"
   "~~/src/Provers/Arith/combine_numerals.ML"
-  ("int_arith1.ML")
+  ("Tools/int_arith.ML")
 begin
 
 subsection {* The equivalence relation underlying the integers *}
@@ -1427,7 +1427,7 @@
 lemmas int_int_eq = of_nat_eq_iff [where 'a=int]
 
 use "~~/src/Provers/Arith/assoc_fold.ML"
-use "int_arith1.ML"
+use "Tools/int_arith.ML"
 declaration {* K int_arith_setup *}