src/HOL/Isar_Examples/Expr_Compiler.thy
changeset 58882 6e2010ab8bd9
parent 58614 7338eb25226c
child 61541 846c72206207
equal deleted inserted replaced
58881:b9556a055632 58882:6e2010ab8bd9
     2     Author:     Markus Wenzel, TU Muenchen
     2     Author:     Markus Wenzel, TU Muenchen
     3 
     3 
     4 Correctness of a simple expression/stack-machine compiler.
     4 Correctness of a simple expression/stack-machine compiler.
     5 *)
     5 *)
     6 
     6 
     7 header \<open>Correctness of a simple expression compiler\<close>
     7 section \<open>Correctness of a simple expression compiler\<close>
     8 
     8 
     9 theory Expr_Compiler
     9 theory Expr_Compiler
    10 imports Main
    10 imports Main
    11 begin
    11 begin
    12 
    12