src/HOL/Library/List_Prefix.thy
changeset 30663 0b6aff7451b2
parent 28562 4e74209f113e
child 37474 ce943f9edf5e
--- a/src/HOL/Library/List_Prefix.thy	Mon Mar 23 08:14:23 2009 +0100
+++ b/src/HOL/Library/List_Prefix.thy	Mon Mar 23 08:14:24 2009 +0100
@@ -1,12 +1,11 @@
 (*  Title:      HOL/Library/List_Prefix.thy
-    ID:         $Id$
     Author:     Tobias Nipkow and Markus Wenzel, TU Muenchen
 *)
 
 header {* List prefixes and postfixes *}
 
 theory List_Prefix
-imports Plain "~~/src/HOL/List"
+imports List Main
 begin
 
 subsection {* Prefix order on lists *}