Zulip Chat Archive
Stream: mathlib4
Topic: distributivity of composition of continuous linear maps
Sébastien Gouëzel (Sep 13 2024 at 12:30):
I can't believe that we don't have distributivity of finset sums over composition of continuous linear maps, i.e.
import Mathlib
lemma foo {E F G 𝕜 : Type*} [NontriviallyNormedField 𝕜] [NormedAddCommGroup E] [NormedSpace 𝕜 E]
[NormedAddCommGroup F] [NormedSpace 𝕜 F] [NormedAddCommGroup G] [NormedSpace 𝕜 G]
(A : ι → (E →L[𝕜] F)) (B : G →L[𝕜] E) : (∑ i, A i) ∘L B = ∑ i, ((A i) ∘L B) := sorry
Am I missing something?
Notification Bot (Sep 13 2024 at 12:30):
A message was moved here from #mathlib4 > Variables not imported by Sébastien Gouëzel.
Sébastien Gouëzel (Sep 13 2024 at 12:31):
@loogle ContinuousLinearMap, Finset.sum
loogle (Sep 13 2024 at 12:31):
:search: ContinuousLinearMap.map_sum, ContinuousLinearMap.coe_sum, and 69 more
Sébastien Gouëzel (Sep 13 2024 at 12:32):
@loogle Finset.sum, ContinuousLinearMap.comp
loogle (Sep 13 2024 at 12:32):
:shrug: nothing found
Bhavik Mehta (Sep 13 2024 at 14:48):
This looks like it should come from the fact that . ∘L B
is a monoid hom, more specifically a monoid hom class. Do we have this instance?
Yaël Dillies (Sep 13 2024 at 14:50):
I don't see where the MonoidHomClass
would be, but a MonoidHom
I certainly believe!
Sébastien Gouëzel (Sep 13 2024 at 15:24):
It's not that the proof is hard (by ext; simp
works fine). I was more surprised that nobody has needed this strongly enough to add it as a lemma in the library.
Eric Wieser (Sep 13 2024 at 18:50):
Do we have the ring structure on continuous endomorphisms?
Last updated: May 02 2025 at 03:31 UTC