src/HOL/IMP/Vars.thy
changeset 45212 e87feee00a4c
parent 45200 1f1897ac7877
child 45716 ccf2cbe86d70
--- a/src/HOL/IMP/Vars.thy	Wed Oct 19 23:07:48 2011 +0200
+++ b/src/HOL/IMP/Vars.thy	Thu Oct 20 09:48:00 2011 +0200
@@ -13,7 +13,7 @@
 via a \emph{type class}, a device that originated with Haskell: *}
  
 class vars =
-fixes vars :: "'a \<Rightarrow> name set"
+fixes vars :: "'a \<Rightarrow> vname set"
 
 text{* This defines a type class ``vars'' with a single
 function of (coincidentally) the same name. Then we define two separated
@@ -22,7 +22,7 @@
 instantiation aexp :: vars
 begin
 
-fun vars_aexp :: "aexp \<Rightarrow> name set" where
+fun vars_aexp :: "aexp \<Rightarrow> vname set" where
 "vars_aexp (N n) = {}" |
 "vars_aexp (V x) = {x}" |
 "vars_aexp (Plus a\<^isub>1 a\<^isub>2) = vars_aexp a\<^isub>1 \<union> vars_aexp a\<^isub>2"
@@ -40,7 +40,7 @@
 instantiation bexp :: vars
 begin
 
-fun vars_bexp :: "bexp \<Rightarrow> name set" where
+fun vars_bexp :: "bexp \<Rightarrow> vname set" where
 "vars_bexp (Bc v) = {}" |
 "vars_bexp (Not b) = vars_bexp b" |
 "vars_bexp (And b\<^isub>1 b\<^isub>2) = vars_bexp b\<^isub>1 \<union> vars_bexp b\<^isub>2" |