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