src/HOL/ex/Efficient_Nat_examples.thy
changeset 29938 a0e54cf21fd4
parent 28661 a287d0e8aa9d
child 41413 64cd30d6b0b8
--- a/src/HOL/ex/Efficient_Nat_examples.thy	Mon Feb 16 19:11:16 2009 +0100
+++ b/src/HOL/ex/Efficient_Nat_examples.thy	Mon Feb 16 19:11:16 2009 +0100
@@ -1,12 +1,11 @@
 (*  Title:      HOL/ex/Efficient_Nat_examples.thy
-    ID:         $Id$
     Author:     Florian Haftmann, TU Muenchen
 *)
 
 header {* Simple examples for Efficient\_Nat theory. *}
 
 theory Efficient_Nat_examples
-imports Main "~~/src/HOL/Real/RealDef" Efficient_Nat
+imports Complex_Main Efficient_Nat
 begin
 
 fun to_n :: "nat \<Rightarrow> nat list" where