src/HOL/IMP/AExp.thy
changeset 45216 a51a70687517
parent 45212 e87feee00a4c
child 45238 ed2bb3b58cc4
--- 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"