fix latex in Transcendental
authorhoelzl
Sun, 12 Apr 2015 16:04:53 +0200
changeset 60035 4b77fc0b3514
parent 60025 d84b355f341f
child 60036 218fcc645d22
fix latex in Transcendental
src/HOL/Transcendental.thy
--- a/src/HOL/Transcendental.thy	Sun Apr 12 00:26:24 2015 +0200
+++ b/src/HOL/Transcendental.thy	Sun Apr 12 16:04:53 2015 +0200
@@ -5201,7 +5201,7 @@
   then have wnz: "\<And>w. w \<noteq> 0 \<Longrightarrow> (\<Sum>i\<le>n. c (Suc i) * w^i) = 0"
     using Suc  by auto
   then have "(\<lambda>h. \<Sum>i\<le>n. c (Suc i) * h^i) -- 0 --> 0"
-    by (simp cong: LIM_cong)                   --{*the case @{term"w=0"} by continuity}*}
+    by (simp cong: LIM_cong)                   --{*the case @{term"w=0"} by continuity*}
   then have "(\<Sum>i\<le>n. c (Suc i) * 0^i) = 0"
     using isCont_polynom [of 0 "\<lambda>i. c (Suc i)" n] LIM_unique
     by (force simp add: Limits.isCont_iff)