src/HOL/Old_Number_Theory/Pocklington.thy
changeset 57418 6ab1c7cb0b8d
parent 57129 7edb7550663e
child 57512 cc97b347b301
--- a/src/HOL/Old_Number_Theory/Pocklington.thy	Fri Jun 27 22:08:55 2014 +0200
+++ b/src/HOL/Old_Number_Theory/Pocklington.thy	Sat Jun 28 09:16:42 2014 +0200
@@ -575,7 +575,7 @@
 lemma nproduct_cmul:
   assumes fS:"finite S"
   shows "setprod (\<lambda>m. (c::'a::{comm_monoid_mult})* a(m)) S = c ^ (card S) * setprod a S"
-unfolding setprod_timesf setprod_constant[OF fS, of c] ..
+unfolding setprod.distrib setprod_constant[OF fS, of c] ..
 
 lemma coprime_nproduct:
   assumes fS: "finite S" and Sn: "\<forall>x\<in>S. coprime n (a x)"