src/HOL/Transcendental.thy
changeset 68614 3cb44b0abc5c
parent 68611 4bc4b5c0ccfc
child 68634 db0980691ef4
--- a/src/HOL/Transcendental.thy	Wed Jul 11 09:47:09 2018 +0100
+++ b/src/HOL/Transcendental.thy	Wed Jul 11 15:36:12 2018 +0100
@@ -5697,16 +5697,9 @@
       if x'_bounds: "x' \<in> {- 1 <..< 1}" for x' :: real
     proof -
       from that have "\<bar>x'\<bar> < 1" by auto
-      then have *: "summable (\<lambda>n. (- 1) ^ n * x' ^ (2 * n))"
-        by (rule summable_Integral)
-      show ?thesis
-        unfolding if_eq
-        apply (rule sums_summable [where l="0 + (\<Sum>n. (-1)^n * x'^(2 * n))"])
-        apply (rule sums_if)
-         apply (rule sums_zero)
-        apply (rule summable_sums)
-        apply (rule *)
-        done
+      then show ?thesis
+        using that sums_summable sums_if [OF sums_0 [of "\<lambda>x. 0"] summable_sums [OF summable_Integral]]   
+        by (auto simp add: if_distrib [of "\<lambda>x. x * y" for y] cong: if_cong)
     qed
   qed auto
   then show ?thesis