--- a/src/HOL/IMP/Procs_Stat_Vars_Stat.thy Wed Oct 19 23:07:48 2011 +0200
+++ b/src/HOL/IMP/Procs_Stat_Vars_Stat.thy Thu Oct 20 09:48:00 2011 +0200
@@ -4,9 +4,9 @@
subsubsection "Static Scoping of Procedures and Variables"
type_synonym addr = nat
-type_synonym venv = "name \<Rightarrow> addr"
+type_synonym venv = "vname \<Rightarrow> addr"
type_synonym store = "addr \<Rightarrow> val"
-type_synonym penv = "(name \<times> com \<times> venv) list"
+type_synonym penv = "(pname \<times> com \<times> venv) list"
fun venv :: "penv \<times> venv \<times> nat \<Rightarrow> venv" where
"venv(_,ve,_) = ve"