src/HOL/List.thy
changeset 51738 9e4220605179
parent 51717 9e7d1c139569
child 51875 dafd097dd1f4
--- a/src/HOL/List.thy	Tue Apr 23 11:14:50 2013 +0200
+++ b/src/HOL/List.thy	Tue Apr 23 11:14:51 2013 +0200
@@ -3376,7 +3376,7 @@
   shows "listsum (map f (filter P xs)) = listsum (map f xs)"
   using assms by (induct xs) auto
 
-lemma (in monoid_add) distinct_listsum_conv_Setsum:
+lemma (in comm_monoid_add) distinct_listsum_conv_Setsum:
   "distinct xs \<Longrightarrow> listsum xs = Setsum (set xs)"
   by (induct xs) simp_all