src/HOL/Library/Binomial.thy
changeset 37388 793618618f78
parent 36350 bc7982c54e37
child 39198 f967a16dfcdd
--- a/src/HOL/Library/Binomial.thy	Tue Jun 08 16:37:19 2010 +0200
+++ b/src/HOL/Library/Binomial.thy	Tue Jun 08 16:37:22 2010 +0200
@@ -235,7 +235,7 @@
     have eq: "insert 0 {1 .. n} = {0..n}" by auto
     have th1: "(\<Prod>n\<in>{1\<Colon>nat..n}. a + of_nat n) =
       (\<Prod>n\<in>{0\<Colon>nat..n - 1}. a + 1 + of_nat n)"
-      apply (rule setprod_reindex_cong[where f = "Suc"])
+      apply (rule setprod_reindex_cong [where f = Suc])
       using n0 by (auto simp add: expand_fun_eq field_simps)
     have ?thesis apply (simp add: pochhammer_def)
     unfolding setprod_insert[OF th0, unfolded eq]