src/HOL/IMP/AExp.thy
changeset 45255 ffc06165d272
parent 45246 4fbeabee6487
child 49191 3601bf546775
--- a/src/HOL/IMP/AExp.thy	Sun Oct 23 17:37:21 2011 +1100
+++ b/src/HOL/IMP/AExp.thy	Sun Oct 23 14:03:37 2011 +0200
@@ -8,12 +8,16 @@
 type_synonym val = int
 type_synonym state = "vname \<Rightarrow> val"
 
+text_raw{*\begin{isaverbatimwrite}\newcommand{\AExpaexpdef}{% *}
 datatype aexp = N int | V vname | Plus aexp aexp
+text_raw{*}\end{isaverbatimwrite}*}
 
+text_raw{*\begin{isaverbatimwrite}\newcommand{\AExpavaldef}{% *}
 fun aval :: "aexp \<Rightarrow> state \<Rightarrow> val" where
 "aval (N n) s = n" |
 "aval (V x) s = s x" |
 "aval (Plus a1 a2) s = aval a1 s + aval a2 s"
+text_raw{*}\end{isaverbatimwrite}*}
 
 
 value "aval (Plus (V ''x'') (N 5)) (\<lambda>x. if x = ''x'' then 7 else 0)"
@@ -48,7 +52,7 @@
 @{text"\<tau>\<^isub>1 \<Rightarrow> \<tau>\<^isub>2"} where @{text "\<tau>\<^isub>2"} has a @{text 0}. *}
 
 
-subsection "Optimization"
+subsection "Constant Folding"
 
 text{* Evaluate constant subsexpressions: *}