src/HOL/Isar_examples/ExprCompiler.thy
changeset 16417 9bc16273c2d4
parent 13537 f506eb568121
child 18153 a084aa91f701
--- a/src/HOL/Isar_examples/ExprCompiler.thy	Fri Jun 17 11:35:35 2005 +0200
+++ b/src/HOL/Isar_examples/ExprCompiler.thy	Fri Jun 17 16:12:49 2005 +0200
@@ -7,7 +7,7 @@
 
 header {* Correctness of a simple expression compiler *}
 
-theory ExprCompiler = Main:
+theory ExprCompiler imports Main begin
 
 text {*
  This is a (rather trivial) example of program verification.  We model