Zulip Chat Archive
Stream: mathlib4
Topic: BigOperators theorems for Multiset
Martin Dvořák (Nov 02 2023 at 15:31):
Do we want to systematically create Multiset
versions of theorems from this file?
https://github.com/leanprover-community/mathlib4/blob/master/Mathlib/Data/List/BigOperators/Basic.lean
Otherwise, I'll PR only the one I need for my VCSP.
Eric Wieser (Nov 02 2023 at 15:46):
I would expect we already have many of them
Eric Wieser (Nov 02 2023 at 15:46):
There are a lot of weird theorems in that file due to multiplication not being commutative, which isn't allowed for docs#Multiset.prod
Eric Wieser (Nov 02 2023 at 15:47):
(it is for docs#Multiset.nonCommProd though...)
Martin Dvořák (Nov 02 2023 at 16:39):
Eric Wieser said:
I would expect we already have many of them
Which file(s) do you recommend checking?
Eric Wieser (Nov 02 2023 at 16:40):
Loogle?
Martin Dvořák (Nov 02 2023 at 16:41):
Back to my original question: Do we want to systematically add all those that can be proved for Multiset
but are not in mathlib yet? Or should I just add the one I need now?
Eric Wieser (Nov 02 2023 at 16:52):
Adding just the one you need now (and the obvious variants of it) is fine, and shouldn't be held up by doing the whole file
Eric Wieser (Nov 02 2023 at 16:52):
But it might also be a good idea to do the whole file after you're unblocked
Martin Dvořák (Nov 02 2023 at 17:23):
Martin Dvořák (Nov 03 2023 at 18:25):
I think that, before we add the Multiset
versions, we should address the inconsistencies between the List
versions and the Finset
versions. See my comment here:
https://leanprover.zulipchat.com/#narrow/stream/217875-Is-there-code-for-X.3F/topic/Multiset.2Esum_lt_sum/near/400185099
Last updated: Dec 20 2023 at 11:08 UTC