src/HOL/Integ/Presburger.thy
changeset 20217 25b068a99d2b
parent 20051 859e7129961b
child 20485 3078fd2eec7b
--- a/src/HOL/Integ/Presburger.thy	Wed Jul 26 13:31:07 2006 +0200
+++ b/src/HOL/Integ/Presburger.thy	Wed Jul 26 19:23:04 2006 +0200
@@ -558,17 +558,13 @@
 lemma decr_lemma: "0 < (d::int) \<Longrightarrow> x - (abs(x-z)+1) * d < z"
 apply(induct rule: int_gr_induct)
  apply simp
- apply arith
 apply (simp add:int_distrib)
-apply arith
 done
 
 lemma incr_lemma: "0 < (d::int) \<Longrightarrow> z < x + (abs(x-z)+1) * d"
 apply(induct rule: int_gr_induct)
  apply simp
- apply arith
 apply (simp add:int_distrib)
-apply arith
 done
 
 lemma  minusinfinity: