src/HOL/List.thy
changeset 25591 0792e02973cc
parent 25571 c9e39eafc7a0
child 25885 6fbc3f54f819
--- a/src/HOL/List.thy	Sun Dec 09 21:44:50 2007 +0100
+++ b/src/HOL/List.thy	Mon Dec 10 11:24:03 2007 +0100
@@ -6,7 +6,7 @@
 header {* The datatype of finite lists *}
 
 theory List
-imports PreList
+imports ATP_Linkup
 uses "Tools/string_syntax.ML"
 begin