Skip to content

Commit

Permalink
feat(algebra/big_operators/basic): add finset.prod_to_list (#10842)
Browse files Browse the repository at this point in the history


Co-authored-by: jlh <48520973+Jlh18@users.noreply.github.com>
  • Loading branch information
Jlh18 and Jlh18 committed Dec 17, 2021
1 parent 5558fd9 commit 862a68c
Showing 1 changed file with 8 additions and 0 deletions.
8 changes: 8 additions & 0 deletions src/algebra/big_operators/basic.lean
Expand Up @@ -251,6 +251,14 @@ begin
rw [← prod_union (filter_inter_filter_neg_eq p s).le, filter_union_filter_neg_eq]
end

section to_list

@[simp, to_additive]
lemma prod_to_list (s : finset α) (f : α → β) : (s.to_list.map f).prod = s.prod f :=
by rw [finset.prod, ← multiset.coe_prod, ← multiset.coe_map, finset.coe_to_list]

end to_list

end comm_monoid

end finset
Expand Down

0 comments on commit 862a68c

Please sign in to comment.