src/HOL/Induct/LFilter.thy
changeset 16417 9bc16273c2d4
parent 13612 55d32e76ef4e
child 19736 d8d0f8f51d69
--- a/src/HOL/Induct/LFilter.thy	Fri Jun 17 11:35:35 2005 +0200
+++ b/src/HOL/Induct/LFilter.thy	Fri Jun 17 16:12:49 2005 +0200
@@ -7,7 +7,7 @@
 header {*The "filter" functional for coinductive lists
   --defined by a combination of induction and coinduction*}
 
-theory LFilter = LList:
+theory LFilter imports LList begin
 
 consts
   findRel	:: "('a => bool) => ('a llist * 'a llist)set"