src/HOL/IMP/AExp.thy
changeset 45212 e87feee00a4c
parent 45015 fdac1e9880eb
child 45216 a51a70687517
--- a/src/HOL/IMP/AExp.thy	Wed Oct 19 23:07:48 2011 +0200
+++ b/src/HOL/IMP/AExp.thy	Thu Oct 20 09:48:00 2011 +0200
@@ -4,11 +4,11 @@
 
 subsection "Arithmetic Expressions"
 
-type_synonym name = string
+type_synonym vname = string
 type_synonym val = int
-type_synonym state = "name \<Rightarrow> val"
+type_synonym state = "vname \<Rightarrow> val"
 
-datatype aexp = N int | V name | Plus aexp aexp
+datatype aexp = N int | V vname | Plus aexp aexp
 
 fun aval :: "aexp \<Rightarrow> state \<Rightarrow> val" where
 "aval (N n) _ = n" |