src/HOL/List.thy
changeset 33593 ef54e2108b74
parent 33318 ddd97d9dfbfb
child 33639 603320b93668
--- a/src/HOL/List.thy	Mon Nov 09 21:56:55 2009 +0100
+++ b/src/HOL/List.thy	Tue Nov 10 16:11:37 2009 +0100
@@ -5,7 +5,7 @@
 header {* The datatype of finite lists *}
 
 theory List
-imports Plain Presburger Recdef ATP_Linkup
+imports Plain Presburger ATP_Linkup Recdef
 uses ("Tools/list_code.ML")
 begin