src/HOL/Induct/Comb.thy
changeset 16417 9bc16273c2d4
parent 15816 4575c87dd25b
child 16563 a92f96951355
--- a/src/HOL/Induct/Comb.thy	Fri Jun 17 11:35:35 2005 +0200
+++ b/src/HOL/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.