src/HOL/Nat_Transfer.thy
changeset 47255 30a1692557b0
parent 42870 36abaf4cce1f
child 47324 ed2bad9b7c6a
--- a/src/HOL/Nat_Transfer.thy	Sun Apr 01 09:12:03 2012 +0200
+++ b/src/HOL/Nat_Transfer.thy	Sun Apr 01 16:09:58 2012 +0200
@@ -4,7 +4,7 @@
 header {* Generic transfer machinery;  specific transfer from nats to ints and back. *}
 
 theory Nat_Transfer
-imports Nat_Numeral
+imports Int
 uses ("Tools/transfer.ML")
 begin