tuned
authornipkow
Fri, 21 Oct 2011 17:39:00 +0200
changeset 45238 ed2bb3b58cc4
parent 45223 62ca94616539
child 45239 ccea94064585
tuned
src/HOL/IMP/AExp.thy
--- a/src/HOL/IMP/AExp.thy	Fri Oct 21 08:25:04 2011 +0200
+++ b/src/HOL/IMP/AExp.thy	Fri Oct 21 17:39:00 2011 +0200
@@ -60,7 +60,7 @@
     (N n1, N n2) \<Rightarrow> N(n1+n2) |
     (a1',a2') \<Rightarrow> Plus a1' a2')"
 
-theorem aval_asimp_const[simp]:
+theorem aval_asimp_const:
   "aval (asimp_const a) s = aval a s"
 apply(induction a)
 apply (auto split: aexp.split)