doc-src/TutorialI/CodeGen/CodeGen.thy
changeset 9844 8016321c7de1
parent 9792 bbefb6ce5cb2
child 9933 9feb1e0c4cb3
--- a/doc-src/TutorialI/CodeGen/CodeGen.thy	Tue Sep 05 13:12:00 2000 +0200
+++ b/doc-src/TutorialI/CodeGen/CodeGen.thy	Tue Sep 05 13:53:39 2000 +0200
@@ -2,7 +2,9 @@
 theory CodeGen = Main:
 (*>*)
 
-text{*\noindent
+section{*Case study: compiling expressions*}
+
+text{*\label{sec:ExprCompiler}
 The task is to develop a compiler from a generic type of expressions (built
 up from variables, constants and binary operations) to a stack machine.  This
 generic type of expressions is a generalization of the boolean expressions in