src/HOL/Library/Efficient_Nat.thy
changeset 30663 0b6aff7451b2
parent 29937 ffed4bd4bfad
child 31090 3be41b271023
--- a/src/HOL/Library/Efficient_Nat.thy	Mon Mar 23 08:14:23 2009 +0100
+++ b/src/HOL/Library/Efficient_Nat.thy	Mon Mar 23 08:14:24 2009 +0100
@@ -5,7 +5,7 @@
 header {* Implementation of natural numbers by target-language integers *}
 
 theory Efficient_Nat
-imports Code_Index Code_Integer
+imports Code_Index Code_Integer Main
 begin
 
 text {*