src/HOL/IMP/Abs_Int1.thy
changeset 45200 1f1897ac7877
parent 45127 d2eb07a1e01b
child 45623 f682f3f7b726
--- a/src/HOL/IMP/Abs_Int1.thy	Wed Oct 19 09:11:21 2011 +0200
+++ b/src/HOL/IMP/Abs_Int1.thy	Wed Oct 19 16:32:12 2011 +0200
@@ -101,7 +101,7 @@
 
 
 fun bfilter :: "bexp \<Rightarrow> bool \<Rightarrow> 'a st up \<Rightarrow> 'a st up" where
-"bfilter (B bv) res S = (if bv=res then S else Bot)" |
+"bfilter (Bc v) res S = (if v=res then S else Bot)" |
 "bfilter (Not b) res S = bfilter b (\<not> res) S" |
 "bfilter (And b1 b2) res S =
   (if res then bfilter b1 True (bfilter b2 True S)
@@ -130,7 +130,7 @@
 
 lemma bfilter_sound: "s <:up S \<Longrightarrow> bv = bval b s \<Longrightarrow> s <:up bfilter b bv S"
 proof(induction b arbitrary: S bv)
-  case B thus ?case by simp
+  case Bc thus ?case by simp
 next
   case (Not b) thus ?case by simp
 next