Skip to content

Commit

Permalink
feat: the volume in a MeasureSpace over an empty index is the Dirac m…
Browse files Browse the repository at this point in the history
…ass (#8799)
  • Loading branch information
sgouezel committed Dec 24, 2023
1 parent 86393c8 commit 640097f
Show file tree
Hide file tree
Showing 2 changed files with 13 additions and 0 deletions.
5 changes: 5 additions & 0 deletions Mathlib/MeasureTheory/Constructions/Pi.lean
Expand Up @@ -421,6 +421,11 @@ theorem pi_of_empty {α : Type*} [Fintype α] [IsEmpty α] {β : α → Type*}
exact isEmptyElim (α := α)
#align measure_theory.measure.pi_of_empty MeasureTheory.Measure.pi_of_empty

lemma volume_pi_eq_dirac {ι : Type*} [Fintype ι] [IsEmpty ι]
{α : ι → Type*} [∀ i, MeasureSpace (α i)] (x : ∀ a, α a := isEmptyElim) :
(volume : Measure (∀ i, α i)) = Measure.dirac x :=
Measure.pi_of_empty _ _

@[simp]
theorem pi_empty_univ {α : Type*} [Fintype α] [IsEmpty α] {β : α → Type*}
{m : ∀ α, MeasurableSpace (β α)} (μ : ∀ a : α, Measure (β a)) :
Expand Down
8 changes: 8 additions & 0 deletions Mathlib/MeasureTheory/Measure/Haar/InnerProductSpace.lean
Expand Up @@ -120,4 +120,12 @@ theorem PiLp.volume_preserving_equiv : MeasurePreserving (WithLp.equiv 2 (ι →
theorem PiLp.volume_preserving_equiv_symm : MeasurePreserving (WithLp.equiv 2 (ι → ℝ)).symm :=
(EuclideanSpace.volume_preserving_measurableEquiv ι).symm

lemma volume_euclideanSpace_eq_dirac [IsEmpty ι] :
(volume : Measure (EuclideanSpace ℝ ι)) = Measure.dirac 0 := by
ext s hs
simp only [← ((EuclideanSpace.volume_preserving_measurableEquiv ι).symm).measure_preimage hs,
volume_pi_eq_dirac 0, MeasurableEquiv.measurableSet_preimage, hs, dirac_apply', indicator,
mem_preimage, Pi.one_apply]
rfl

end PiLp

0 comments on commit 640097f

Please sign in to comment.