src/HOL/Library/Fundamental_Theorem_Algebra.thy
changeset 32456 341c83339aeb
parent 31337 a9ed5fcc5e39
child 32960 69916a850301
--- a/src/HOL/Library/Fundamental_Theorem_Algebra.thy	Sat Aug 29 14:31:39 2009 +0200
+++ b/src/HOL/Library/Fundamental_Theorem_Algebra.thy	Mon Aug 31 14:09:42 2009 +0200
@@ -577,11 +577,12 @@
 next
   case (pCons c cs)
   {assume c0: "c = 0"
-    from pCons.hyps pCons.prems c0 have ?case apply auto
+    from pCons.hyps pCons.prems c0 have ?case
+      apply (auto)
       apply (rule_tac x="k+1" in exI)
       apply (rule_tac x="a" in exI, clarsimp)
       apply (rule_tac x="q" in exI)
-      by (auto simp add: power_Suc)}
+      by (auto)}
   moreover
   {assume c0: "c\<noteq>0"
     hence ?case apply-