fixed spurious proof failure
authorhaftmann
Fri, 20 Feb 2009 14:49:23 +0100
changeset 30012 a717c3dffe4f
parent 30011 cc264a9a033d
child 30013 1e0b8e561cc2
fixed spurious proof failure
src/HOL/Algebra/poly/UnivPoly2.thy
--- a/src/HOL/Algebra/poly/UnivPoly2.thy	Fri Feb 20 14:49:23 2009 +0100
+++ b/src/HOL/Algebra/poly/UnivPoly2.thy	Fri Feb 20 14:49:23 2009 +0100
@@ -1,6 +1,5 @@
 (*
   Title:     Univariate Polynomials
-  Id:        $Id$
   Author:    Clemens Ballarin, started 9 December 1996
   Copyright: Clemens Ballarin
 *)
@@ -388,7 +387,7 @@
   proof (cases k)
     case 0 then show ?thesis by simp ring
   next
-    case Suc then show ?thesis by (simp add: algebra_simps) ring
+    case Suc then show ?thesis by simp (ring, simp)
   qed
   then show "coeff (monom a 0 * p) k = coeff (a *s p) k" by ring
 qed