src/HOL/Library/Fundamental_Theorem_Algebra.thy
changeset 41529 ba60efa2fd08
parent 37887 2ae085b07f2f
child 46240 933f35c4e126
--- a/src/HOL/Library/Fundamental_Theorem_Algebra.thy	Wed Jan 12 17:14:27 2011 +0100
+++ b/src/HOL/Library/Fundamental_Theorem_Algebra.thy	Wed Jan 12 17:19:50 2011 +0100
@@ -793,7 +793,7 @@
   assumes "\<forall>x. poly p x = 0 \<longrightarrow> poly q x = 0"
   and "degree p = n" and "n \<noteq> 0"
   shows "p dvd (q ^ n)"
-using prems
+using assms
 proof(induct n arbitrary: p q rule: nat_less_induct)
   fix n::nat fix p q :: "complex poly"
   assume IH: "\<forall>m<n. \<forall>p q.