Zulip Chat Archive
Stream: Is there code for X?
Topic: Fintype.sum of Fintype.sum
David Renshaw (Oct 08 2023 at 15:15):
import Mathlib.Tactic
import Mathlib.Data.Fintype.BigOperators
open BigOperators
lemma sum_of_sum {α β : Type} [Fintype α] [Fintype β]
(f : α → β → ℤ) :
∑ a : α, ∑ b : β, f a b = ∑ ab : α × β, f.uncurry ab := by sorry
David Renshaw (Oct 08 2023 at 15:16):
Anyone have any ideas about how to prove this? Seems like there ought to be some existing lemma.
Yaël Dillies (Oct 08 2023 at 15:17):
This is exactly docs#Finset.sum_product'
David Renshaw (Oct 08 2023 at 15:18):
nice!
David Renshaw (Oct 08 2023 at 15:18):
I should have tried rw?
first
David Renshaw (Oct 08 2023 at 15:19):
(Finset.sum_product'
is among the suggestions given by rw?
, but not among the top 10)
Yaël Dillies (Oct 08 2023 at 15:22):
Sadly, yael?
is only available on Zulip :grinning:
Henrik Böving (Oct 08 2023 at 15:26):
Maybe we can train an LLM on the corpus of Yael Q&A's ...
Last updated: Dec 20 2023 at 11:08 UTC