Main is (Complex_Main) base entry point in library theories
authorhaftmann
Mon, 23 Mar 2009 08:14:58 +0100
changeset 30664 167da873c3b3
parent 30663 0b6aff7451b2
child 30665 4cf38ea4fad2
Main is (Complex_Main) base entry point in library theories
src/HOL/Library/Executable_Set.thy
--- a/src/HOL/Library/Executable_Set.thy	Mon Mar 23 08:14:24 2009 +0100
+++ b/src/HOL/Library/Executable_Set.thy	Mon Mar 23 08:14:58 2009 +0100
@@ -1,12 +1,11 @@
 (*  Title:      HOL/Library/Executable_Set.thy
-    ID:         $Id$
     Author:     Stefan Berghofer, TU Muenchen
 *)
 
 header {* Implementation of finite sets by lists *}
 
 theory Executable_Set
-imports Plain "~~/src/HOL/List"
+imports Main
 begin
 
 subsection {* Definitional rewrites *}