Zulip Chat Archive
Stream: new members
Topic: Sum over product set
Pim Otte (Aug 09 2022 at 19:19):
I'm trying to state the equality from exercise 1 here. This involves a sum over all vectors {-1,1}^d. How do I formulate this? I think finset.pi is the thing I should be using, but it seems a little overkill at some points, but I have some trouble grasping the definition in general. It also seems to not be used anywhere else in the library, so I might be on the wrong track. Any pointers?
import data.mv_polynomial.basic
import data.complex.basic
import ring_theory.polynomial.homogeneous
noncomputable theory
open_locale big_operators
open mv_polynomial
def polynomial_identity {R : Type*} [comm_semiring R] (d : ℕ) : (∏ i, (X i): mv_polynomial (fin d) R) = ∑ α in (finset.pi (fin d) ((λ _, (fin 2)))), (X 0) :=
begin
end
Eric Wieser (Aug 09 2022 at 19:27):
finset.pi
is used behind the scenes when you write ∑ f : fin d → ℤˣ, ...
Eric Wieser (Aug 09 2022 at 19:27):
(by docs#pi.fintype)
Eric Wieser (Aug 09 2022 at 19:28):
(also, ℤˣ
is likely a better translation of {1,-1}
than fin 2
)
Pim Otte (Aug 09 2022 at 19:33):
@Eric Wieser Thanks! That's very helpful:)
Last updated: Dec 20 2023 at 11:08 UTC