# HG changeset patch # User blanchet # Date 1396615491 -7200 # Node ID ae4f904c98b03cd78f62c57a956f21bd5ee0a8ee # Parent 6d9a24f8746073f7e15c7a1420e6345bc26b4d55 tuned spaces diff -r 6d9a24f87460 -r ae4f904c98b0 src/HOL/Library/Fundamental_Theorem_Algebra.thy --- a/src/HOL/Library/Fundamental_Theorem_Algebra.thy Fri Apr 04 13:22:26 2014 +0200 +++ b/src/HOL/Library/Fundamental_Theorem_Algebra.thy Fri Apr 04 14:44:51 2014 +0200 @@ -516,10 +516,10 @@ {fix z::'a assume h: "(\d\ + norm a) / norm c \ norm z" from c0 have "norm c > 0" by simp - from h c0 have th0: "\d\ + norm a \ norm (z*c)" + from h c0 have th0: "\d\ + norm a \ norm (z * c)" by (simp add: field_simps norm_mult) have ath: "\mzh mazh ma. mzh <= mazh + ma ==> abs(d) + ma <= mzh ==> d <= mazh" by arith - from norm_diff_ineq[of "z*c" a ] + from norm_diff_ineq[of "z * c" a ] have th1: "norm (z * c) \ norm (a + z * c) + norm a" by (simp add: algebra_simps) from ath[OF th1 th0] have "d \ norm (poly (pCons a (pCons c cs)) z)" @@ -720,7 +720,7 @@ with norm_triangle_ineq[of "complex_of_real (1 - t^k)" "?w^k * ?w * poly s ?w"] have th11: "cmod (1 + ?w^k * (a + ?w * poly s ?w)) \ \1 - t^k\ + cmod (?w^k * ?w * poly s ?w)" unfolding norm_of_real by simp have ath: "\x (t::real). 0\ x \ x < t \ t\1 \ \1 - t\ + x < 1" by arith - have "t *cmod w \ 1 * cmod w" apply (rule mult_mono) using t(1,2) by auto + have "t * cmod w \ 1 * cmod w" apply (rule mult_mono) using t(1,2) by auto then have tw: "cmod ?w \ cmod w" using t(1) by (simp add: norm_mult) from t inv0 have "t* (cmod w ^ (k + 1) * m) < 1" by (simp add: inverse_eq_divide field_simps) @@ -1074,4 +1074,3 @@ shows "poly [:c:] x = y \ c = y" by simp end -