Documentation

Mathlib.MeasureTheory.Measure.Haar.NormedSpace

Basic properties of Haar measures on real vector spaces #

The integral of f (R • x) with respect to an additive Haar measure is a multiple of the integral of f. The formula we give works even when f is not integrable or R = 0 thanks to the convention that a non-integrable function has integral zero.

The integral of f (R • x) with respect to an additive Haar measure is a multiple of the integral of f. The formula we give works even when f is not integrable or R = 0 thanks to the convention that a non-integrable function has integral zero.

The integral of f (R⁻¹ • x) with respect to an additive Haar measure is a multiple of the integral of f. The formula we give works even when f is not integrable or R = 0 thanks to the convention that a non-integrable function has integral zero.

The integral of f (R⁻¹ • x) with respect to an additive Haar measure is a multiple of the integral of f. The formula we give works even when f is not integrable or R = 0 thanks to the convention that a non-integrable function has integral zero.

theorem MeasureTheory.Measure.setIntegral_comp_smul {E : Type u_1} [NormedAddCommGroup E] [NormedSpace E] [MeasurableSpace E] [BorelSpace E] [FiniteDimensional E] (μ : MeasureTheory.Measure E) [MeasureTheory.Measure.IsAddHaarMeasure μ] {F : Type u_2} [NormedAddCommGroup F] [NormedSpace F] (f : EF) {R : } (s : Set E) (hR : R 0) :
∫ (x : E) in s, f (R x)μ = |(R ^ FiniteDimensional.finrank E)⁻¹| ∫ (x : E) in R s, f xμ
@[deprecated MeasureTheory.Measure.setIntegral_comp_smul]
theorem MeasureTheory.Measure.set_integral_comp_smul {E : Type u_1} [NormedAddCommGroup E] [NormedSpace E] [MeasurableSpace E] [BorelSpace E] [FiniteDimensional E] (μ : MeasureTheory.Measure E) [MeasureTheory.Measure.IsAddHaarMeasure μ] {F : Type u_2} [NormedAddCommGroup F] [NormedSpace F] (f : EF) {R : } (s : Set E) (hR : R 0) :
∫ (x : E) in s, f (R x)μ = |(R ^ FiniteDimensional.finrank E)⁻¹| ∫ (x : E) in R s, f xμ

Alias of MeasureTheory.Measure.setIntegral_comp_smul.

theorem MeasureTheory.Measure.setIntegral_comp_smul_of_pos {E : Type u_1} [NormedAddCommGroup E] [NormedSpace E] [MeasurableSpace E] [BorelSpace E] [FiniteDimensional E] (μ : MeasureTheory.Measure E) [MeasureTheory.Measure.IsAddHaarMeasure μ] {F : Type u_2} [NormedAddCommGroup F] [NormedSpace F] (f : EF) {R : } (s : Set E) (hR : 0 < R) :
∫ (x : E) in s, f (R x)μ = (R ^ FiniteDimensional.finrank E)⁻¹ ∫ (x : E) in R s, f xμ
@[deprecated MeasureTheory.Measure.setIntegral_comp_smul_of_pos]
theorem MeasureTheory.Measure.set_integral_comp_smul_of_pos {E : Type u_1} [NormedAddCommGroup E] [NormedSpace E] [MeasurableSpace E] [BorelSpace E] [FiniteDimensional E] (μ : MeasureTheory.Measure E) [MeasureTheory.Measure.IsAddHaarMeasure μ] {F : Type u_2} [NormedAddCommGroup F] [NormedSpace F] (f : EF) {R : } (s : Set E) (hR : 0 < R) :
∫ (x : E) in s, f (R x)μ = (R ^ FiniteDimensional.finrank E)⁻¹ ∫ (x : E) in R s, f xμ

Alias of MeasureTheory.Measure.setIntegral_comp_smul_of_pos.

theorem MeasureTheory.Measure.integral_comp_mul_left {F : Type u_2} [NormedAddCommGroup F] [NormedSpace F] (g : F) (a : ) :
∫ (x : ), g (a * x) = |a⁻¹| ∫ (y : ), g y
theorem MeasureTheory.Measure.integral_comp_inv_mul_left {F : Type u_2} [NormedAddCommGroup F] [NormedSpace F] (g : F) (a : ) :
∫ (x : ), g (a⁻¹ * x) = |a| ∫ (y : ), g y
theorem MeasureTheory.Measure.integral_comp_mul_right {F : Type u_2} [NormedAddCommGroup F] [NormedSpace F] (g : F) (a : ) :
∫ (x : ), g (x * a) = |a⁻¹| ∫ (y : ), g y
theorem MeasureTheory.Measure.integral_comp_inv_mul_right {F : Type u_2} [NormedAddCommGroup F] [NormedSpace F] (g : F) (a : ) :
∫ (x : ), g (x * a⁻¹) = |a| ∫ (y : ), g y
theorem MeasureTheory.Measure.integral_comp_div {F : Type u_2} [NormedAddCommGroup F] [NormedSpace F] (g : F) (a : ) :
∫ (x : ), g (x / a) = |a| ∫ (y : ), g y
theorem MeasureTheory.integrable_comp_mul_left_iff {F : Type u_1} [NormedAddCommGroup F] (g : F) {R : } (hR : R 0) :
MeasureTheory.Integrable (fun (x : ) => g (R * x)) MeasureTheory.volume MeasureTheory.Integrable g MeasureTheory.volume
theorem MeasureTheory.Integrable.comp_mul_left' {F : Type u_1} [NormedAddCommGroup F] {g : F} (hg : MeasureTheory.Integrable g MeasureTheory.volume) {R : } (hR : R 0) :
MeasureTheory.Integrable (fun (x : ) => g (R * x)) MeasureTheory.volume
theorem MeasureTheory.integrable_comp_mul_right_iff {F : Type u_1} [NormedAddCommGroup F] (g : F) {R : } (hR : R 0) :
MeasureTheory.Integrable (fun (x : ) => g (x * R)) MeasureTheory.volume MeasureTheory.Integrable g MeasureTheory.volume
theorem MeasureTheory.Integrable.comp_mul_right' {F : Type u_1} [NormedAddCommGroup F] {g : F} (hg : MeasureTheory.Integrable g MeasureTheory.volume) {R : } (hR : R 0) :
MeasureTheory.Integrable (fun (x : ) => g (x * R)) MeasureTheory.volume
theorem MeasureTheory.integrable_comp_div_iff {F : Type u_1} [NormedAddCommGroup F] (g : F) {R : } (hR : R 0) :
MeasureTheory.Integrable (fun (x : ) => g (x / R)) MeasureTheory.volume MeasureTheory.Integrable g MeasureTheory.volume
theorem MeasureTheory.Integrable.comp_div {F : Type u_1} [NormedAddCommGroup F] {g : F} (hg : MeasureTheory.Integrable g MeasureTheory.volume) {R : } (hR : R 0) :
MeasureTheory.Integrable (fun (x : ) => g (x / R)) MeasureTheory.volume
theorem MeasureTheory.integral_comp {E' : Type u_2} {F' : Type u_3} {A : Type u_4} [NormedAddCommGroup E'] [InnerProductSpace E'] [FiniteDimensional E'] [MeasurableSpace E'] [BorelSpace E'] [NormedAddCommGroup F'] [InnerProductSpace F'] [FiniteDimensional F'] [MeasurableSpace F'] [BorelSpace F'] (f : E' ≃ₗᵢ[] F') [NormedAddCommGroup A] [NormedSpace A] (g : F'A) :
∫ (x : E'), g (f x) = ∫ (y : F'), g y