src/HOL/Library/Coinductive_List.thy
changeset 27487 c8a6ce181805
parent 27368 9f90ac19e32b
child 28693 a1294a197d12
--- a/src/HOL/Library/Coinductive_List.thy	Fri Jul 04 16:33:08 2008 +0200
+++ b/src/HOL/Library/Coinductive_List.thy	Mon Jul 07 08:47:17 2008 +0200
@@ -6,7 +6,7 @@
 header {* Potentially infinite lists as greatest fixed-point *}
 
 theory Coinductive_List
-imports Plain List
+imports Plain "~~/src/HOL/List"
 begin
 
 subsection {* List constructors over the datatype universe *}