src/HOL/Hyperreal/Poly.thy
changeset 20256 5024ba0831a6
parent 20217 25b068a99d2b
child 20432 07ec57376051
--- a/src/HOL/Hyperreal/Poly.thy	Sun Jul 30 02:06:01 2006 +0200
+++ b/src/HOL/Hyperreal/Poly.thy	Sun Jul 30 05:53:10 2006 +0200
@@ -425,7 +425,7 @@
 lemma poly_add_length [rule_format]:
      "\<forall>p2. length (p1 +++ p2) =
              (if (length p1 < length p2) then length p2 else length p1)"
-apply (induct "p1", simp_all, arith)
+apply (induct "p1", simp_all)
 done
 
 lemma poly_root_mult_length: "length([a,b] *** p) = Suc (length p)"