src/HOL/IMP/Abs_State.thy
changeset 51698 c0af8bbc5825
parent 51389 8a9f0503b1c0
child 51711 df3426139651
--- a/src/HOL/IMP/Abs_State.thy	Thu Apr 11 16:58:54 2013 +0200
+++ b/src/HOL/IMP/Abs_State.thy	Fri Apr 12 08:27:43 2013 +0200
@@ -6,30 +6,6 @@
 
 subsubsection "Set-based lattices"
 
-instantiation com :: vars
-begin
-
-fun vars_com :: "com \<Rightarrow> vname set" where
-"vars com.SKIP = {}" |
-"vars (x::=e) = {x} \<union> vars e" |
-"vars (c1;c2) = vars c1 \<union> vars c2" |
-"vars (IF b THEN c1 ELSE c2) = vars b \<union> vars c1 \<union> vars c2" |
-"vars (WHILE b DO c) = vars b \<union> vars c"
-
-instance ..
-
-end
-
-
-lemma finite_avars: "finite(vars(a::aexp))"
-by(induction a) simp_all
-
-lemma finite_bvars: "finite(vars(b::bexp))"
-by(induction b) (simp_all add: finite_avars)
-
-lemma finite_cvars: "finite(vars(c::com))"
-by(induction c) (simp_all add: finite_avars finite_bvars)
-
 
 class L =
 fixes L :: "vname set \<Rightarrow> 'a set"