src/HOL/Lambda/ListBeta.thy
changeset 16417 9bc16273c2d4
parent 12011 1a3a7b3cd9bb
child 18241 afdba6b3e383
--- a/src/HOL/Lambda/ListBeta.thy	Fri Jun 17 11:35:35 2005 +0200
+++ b/src/HOL/Lambda/ListBeta.thy	Fri Jun 17 16:12:49 2005 +0200
@@ -6,7 +6,7 @@
 
 header {* Lifting beta-reduction to lists *}
 
-theory ListBeta = ListApplication + ListOrder:
+theory ListBeta imports ListApplication ListOrder begin
 
 text {*
   Lifting beta-reduction to lists of terms, reducing exactly one element.