src/HOL/Lambda/ListApplication.thy
changeset 16417 9bc16273c2d4
parent 14066 fe45b97b62ea
child 18241 afdba6b3e383
--- a/src/HOL/Lambda/ListApplication.thy	Fri Jun 17 11:35:35 2005 +0200
+++ b/src/HOL/Lambda/ListApplication.thy	Fri Jun 17 16:12:49 2005 +0200
@@ -6,7 +6,7 @@
 
 header {* Application of a term to a list of terms *}
 
-theory ListApplication = Lambda:
+theory ListApplication imports Lambda begin
 
 syntax
   "_list_application" :: "dB => dB list => dB"    (infixl "\<degree>\<degree>" 150)