Zulip Chat Archive
Stream: mathlib4
Topic: dcomp, Pi.map?
Yury G. Kudryashov (Aug 11 2024 at 12:56):
We have docs#Function.dcomp which is used only a few times across the library. What do you think about replacing it with a bit less generic
@[inline]
def Pi.map {ι : Sort*} {α β : ι → Sort*} (f : ∀ i, α i → β i) (g : ∀ i, α i) : ∀ i, β i :=
fun i ↦ f i (g i)
so that lemmas like docs#Function.surjective_pi_map can be formulated as |- Surjective (F ∘' ·)
(if we keep notation) or |- Surjective (Pi.map F)
(w/o notation)?
Yury G. Kudryashov (Aug 11 2024 at 12:56):
With current definition, (F ∘' ·)
fails to elaborate.
Yury G. Kudryashov (Aug 11 2024 at 13:14):
More details: (F _ ∘' ·)
elaborates if the type is known.
Yury G. Kudryashov (Aug 12 2024 at 16:26):
See #15694 and #15744 for context
Yury G. Kudryashov (Aug 12 2024 at 16:33):
UPD: making dcomp
less dependent doesn't work with usage in docs#MeasureTheory.lmarginal_image
Last updated: May 02 2025 at 03:31 UTC