Zulip Chat Archive
Stream: Is there code for X?
Topic: power of product in comm_monoid
Xavier Xarles (Apr 14 2022 at 15:39):
I need this:
lemma pow_prod {G : Type}comm_monoid G(n:nat): (ab)^n=(a^n)*(b^n):=
sorry
I guess one should be able to prove using big_operators.findprod.finprod_pow
Johan Commelin (Apr 14 2022 at 15:40):
Should be mul_pow
.
Xavier Xarles (Apr 14 2022 at 15:42):
ups, thanks, you are right.
Eric Wieser (Apr 14 2022 at 15:56):
For future reference, #backticks
Last updated: Dec 20 2023 at 11:08 UTC