Zulip Chat Archive
Stream: maths
Topic: smul invariant measure
Yury G. Kudryashov (Oct 28 2021 at 22:55):
I suggest to generalize left/right-invariant measures to
@[to_additive]
def is_smul_invariant (M : Type*) {α : Type*} [has_scalar M α] [measurable_space α] (μ : set α → ℝ≥0∞) : Prop :=
∀ (g : M) {A : set α} (h : measurable_set A), μ ((λ h, g • h) ⁻¹' A) = μ A
Then is_mul_left_invariant (μ : measure G) = is_smul_invariant G μ
and is_mul_right_invariant (μ : measure G) = is_smul_invariant Gᵒᵖ μ
.
Yury G. Kudryashov (Oct 28 2021 at 22:56):
@Floris van Doorn @Sebastien Gouezel What do you think?
Yury G. Kudryashov (Oct 28 2021 at 22:57):
Also, I think about replacing def
with a class
.
Alex J. Best (Oct 28 2021 at 23:06):
I do this in https://github.com/leanprover-community/mathlib/pull/2819/files but it should probably be an independent PR first, so +1 from me :smile:
Floris van Doorn (Oct 28 2021 at 23:10):
Yeah, that is probably a good idea.
Sebastien Gouezel (Oct 29 2021 at 07:24):
Looks good to me.
Last updated: Dec 20 2023 at 11:08 UTC