PreList imports RecDef
authorhaftmann
Sun, 06 May 2007 21:49:44 +0200
changeset 22844 91c05f4b509e
parent 22843 189e214845dd
child 22845 5f9138bcb3d7
PreList imports RecDef
src/HOL/List.thy
src/HOL/PreList.thy
--- a/src/HOL/List.thy	Sun May 06 21:49:32 2007 +0200
+++ b/src/HOL/List.thy	Sun May 06 21:49:44 2007 +0200
@@ -6,7 +6,7 @@
 header {* The datatype of finite lists *}
 
 theory List
-imports PreList Recdef
+imports PreList
 uses "Tools/string_syntax.ML"
 begin
 
--- a/src/HOL/PreList.thy	Sun May 06 21:49:32 2007 +0200
+++ b/src/HOL/PreList.thy	Sun May 06 21:49:44 2007 +0200
@@ -8,7 +8,7 @@
 
 theory PreList
 imports Wellfounded_Relations Presburger Relation_Power SAT
-  FunDef Extraction
+  FunDef Recdef Extraction
 begin
 
 text {*