src/ZF/Induct/Comb.thy
changeset 16417 9bc16273c2d4
parent 15863 78db9506cc78
child 18415 eb68dc98bda2
--- a/src/ZF/Induct/Comb.thy	Fri Jun 17 11:35:35 2005 +0200
+++ b/src/ZF/Induct/Comb.thy	Fri Jun 17 16:12:49 2005 +0200
@@ -6,7 +6,7 @@
 
 header {* Combinatory Logic example: the Church-Rosser Theorem *}
 
-theory Comb = Main:
+theory Comb imports Main begin
 
 text {*
   Curiously, combinators do not include free variables.