src/HOL/Library/Fundamental_Theorem_Algebra.thy
changeset 60449 229bad93377e
parent 60424 c96fff9dcdbc
child 60457 f31f7599ef55
--- a/src/HOL/Library/Fundamental_Theorem_Algebra.thy	Thu Jun 11 22:47:53 2015 +0200
+++ b/src/HOL/Library/Fundamental_Theorem_Algebra.thy	Sat Jun 13 13:09:05 2015 +0200
@@ -1191,7 +1191,7 @@
   shows "\<exists>x. poly (pCons a (pCons b p)) x = (0::complex)"
 proof -
   have False if "h \<noteq> 0" "t = 0" and "pCons a (pCons b p) = pCons h t" for h t
-    using l prems by simp
+    using l that by simp
   then have th: "\<not> (\<exists> h t. h \<noteq> 0 \<and> t = 0 \<and> pCons a (pCons b p) = pCons h t)"
     by blast
   from fundamental_theorem_of_algebra_alt[OF th] show ?thesis