Zulip Chat Archive
Stream: Is there code for X?
Topic: non finsupp finsupp.dom_congr
Kevin Buzzard (Dec 14 2021 at 03:35):
import algebra.monoid_algebra.basic
variables {S T A : Type*} [add_comm_group A]
/-
finsupp.dom_congr :
Π {α : Type u_4} {β : Type u_5} {M : Type u_6} [_inst_1 : add_comm_monoid M],
α ≃ β → (α →₀ M) ≃+ (β →₀ M)
-/
-- what is the non-finsupp version of finsupp.dom_congr
#find ((S ≃ T) → ((S → A) ≃+ (T → A)))
What's the regular function version called? I don't know how to find out without asking.
Eric Wieser (Dec 14 2021 at 08:14):
Kevin Buzzard (Dec 14 2021 at 11:12):
Oh nice! Thanks! I didn't know →
was called arrow
.
Eric Wieser (Dec 14 2021 at 11:19):
It's a bit annoying that we sometimes have one definition (M ≃ N) → (P ≃+ Q) → ((M → P) ≃+ (N → Q))
(like arrow_congr
) and other times (like finsupp.dom_congr
) have two, (M ≃ N) → ((M → P) ≃+ (N → P))
and (P ≃+ Q) → ((M → P) ≃+ (M → Q))
. IMO the separate definitions make slightly more sense as they're simpler operations.
Last updated: Dec 20 2023 at 11:08 UTC