src/HOL/Library/Efficient_Nat.thy
changeset 27368 9f90ac19e32b
parent 26467 fdd4d78e1e05
child 27496 f56684dd75a5
--- a/src/HOL/Library/Efficient_Nat.thy	Thu Jun 26 10:06:54 2008 +0200
+++ b/src/HOL/Library/Efficient_Nat.thy	Thu Jun 26 10:07:01 2008 +0200
@@ -6,7 +6,7 @@
 header {* Implementation of natural numbers by target-language integers *}
 
 theory Efficient_Nat
-imports Code_Integer Code_Index
+imports Plain Code_Integer Code_Index
 begin
 
 text {*