src/HOL/Library/Formal_Power_Series.thy
changeset 37388 793618618f78
parent 36811 4ab4aa5bee1c
child 39198 f967a16dfcdd
--- a/src/HOL/Library/Formal_Power_Series.thy	Tue Jun 08 16:37:19 2010 +0200
+++ b/src/HOL/Library/Formal_Power_Series.thy	Tue Jun 08 16:37:22 2010 +0200
@@ -2031,7 +2031,7 @@
     done
   also have "\<dots> = setsum (\<lambda>i. of_nat (i + 1) * a$(i+1) * (setsum (\<lambda>j. (b^ i)$j * of_nat (n - j + 1) * b$(n - j + 1)) {0..n})) {0.. n}"
     unfolding fps_deriv_nth
-    apply (rule setsum_reindex_cong[where f="Suc"])
+    apply (rule setsum_reindex_cong [where f = Suc])
     by (auto simp add: mult_assoc)
   finally have th0: "(fps_deriv (a oo b))$n = setsum (\<lambda>i. of_nat (i + 1) * a$(i+1) * (setsum (\<lambda>j. (b^ i)$j * of_nat (n - j + 1) * b$(n - j + 1)) {0..n})) {0.. n}" .