doc-src/TutorialI/CodeGen/CodeGen.thy
changeset 16417 9bc16273c2d4
parent 11458 09a6c44a48ea
child 17212 6859484b5b2b
--- a/doc-src/TutorialI/CodeGen/CodeGen.thy	Fri Jun 17 11:35:35 2005 +0200
+++ b/doc-src/TutorialI/CodeGen/CodeGen.thy	Fri Jun 17 16:12:49 2005 +0200
@@ -1,5 +1,5 @@
 (*<*)
-theory CodeGen = Main:
+theory CodeGen imports Main begin
 (*>*)
 
 section{*Case Study: Compiling Expressions*}