src/HOL/IMP/Def_Ass_Exp.thy
changeset 45200 1f1897ac7877
parent 43158 686fa0a0696e
child 45212 e87feee00a4c
--- a/src/HOL/IMP/Def_Ass_Exp.thy	Wed Oct 19 09:11:21 2011 +0200
+++ b/src/HOL/IMP/Def_Ass_Exp.thy	Wed Oct 19 16:32:12 2011 +0200
@@ -18,7 +18,7 @@
 
 
 fun bval :: "bexp \<Rightarrow> state \<Rightarrow> bool option" where
-"bval (B bv) s = Some bv" |
+"bval (Bc v) s = Some v" |
 "bval (Not b) s = (case bval b s of None \<Rightarrow> None | Some bv \<Rightarrow> Some(\<not> bv))" |
 "bval (And b\<^isub>1 b\<^isub>2) s = (case (bval b\<^isub>1 s, bval b\<^isub>2 s) of
   (Some bv\<^isub>1, Some bv\<^isub>2) \<Rightarrow> Some(bv\<^isub>1 & bv\<^isub>2) | _ \<Rightarrow> None)" |