--- a/src/HOL/IMP/AExp.thy Thu Oct 20 09:48:00 2011 +0200
+++ b/src/HOL/IMP/AExp.thy Thu Oct 20 10:43:47 2011 +0200
@@ -11,7 +11,7 @@
datatype aexp = N int | V vname | Plus aexp aexp
fun aval :: "aexp \<Rightarrow> state \<Rightarrow> val" where
-"aval (N n) _ = n" |
+"aval (N n) s = n" |
"aval (V x) s = s x" |
"aval (Plus a1 a2) s = aval a1 s + aval a2 s"
--- a/src/HOL/IMP/BExp.thy Thu Oct 20 09:48:00 2011 +0200
+++ b/src/HOL/IMP/BExp.thy Thu Oct 20 10:43:47 2011 +0200
@@ -5,7 +5,7 @@
datatype bexp = Bc bool | Not bexp | And bexp bexp | Less aexp aexp
fun bval :: "bexp \<Rightarrow> state \<Rightarrow> bool" where
-"bval (Bc v) _ = v" |
+"bval (Bc v) s = v" |
"bval (Not b) s = (\<not> bval b s)" |
"bval (And b1 b2) s = (if bval b1 s then bval b2 s else False)" |
"bval (Less a1 a2) s = (aval a1 s < aval a2 s)"