src/HOL/Algebra/UnivPoly.thy
changeset 20282 49c312eaaa11
parent 20217 25b068a99d2b
child 20318 0e0ea63fe768
--- a/src/HOL/Algebra/UnivPoly.thy	Wed Aug 02 13:48:21 2006 +0200
+++ b/src/HOL/Algebra/UnivPoly.thy	Wed Aug 02 16:50:41 2006 +0200
@@ -511,7 +511,7 @@
       have f1: "(\<Oplus>i \<in> {..<n}. ?s i) = \<zero>"
         by (simp cong: R.finsum_cong add: Pi_def)
       from neq have f2: "(\<Oplus>i \<in> {n}. ?s i) = \<zero>"
-        by (simp cong: R.finsum_cong add: Pi_def) arith
+        by (simp cong: R.finsum_cong add: Pi_def)
       have f3: "n < k ==> (\<Oplus>i \<in> {n<..k}. ?s i) = \<zero>"
         by (simp cong: R.finsum_cong add: order_less_imp_not_eq Pi_def)
       show ?thesis