Zulip Chat Archive

Stream: new members

Topic: Gaussian measures


jsodd (Aug 17 2024 at 20:50):

In this topic, I've asked how do we formalise measures on R^n. Here's a more specific question which I'm trying to solve.

I am trying to formalise Gaussian measures, and decided to start from the case of R^n. A Borel measure gamma on R^n is said to be Gaussian if for every linear functional R^n -> R the induced measure gamma o l^{-1} is a Gaussian measure on R. Here's my attempt at formalising this definition:

def isGaussianReal (γ : ProbabilityMeasure ) : Prop := sorry

def isGaussianFinDim (γ : ProbabilityMeasure (n  )) [BorelSpace (n  )]:=
   (l : (n  ) L[] ) (h : AEMeasurable l γ), isGaussianReal (ProbabilityMeasure.map γ h)

However, assuming h : AEMeasurable l γ seems unnecessary, which brings me to the following two quesions:

  1. Where did I specify that n → ℝ is endowed with the Borel sigma-algebra? Is it somehow inferred? If yes, how should I find the definition?
  2. Is there a way to avoid this assumption? It's not really needed.

jsodd (Aug 17 2024 at 21:06):

P.S. If I remove [BorelSpace n → ℝ], nothing changes, this was just my attempt to put this assumption somewhere

Etienne Marion (Aug 17 2024 at 21:15):

Yes, n \to \R is automatically endowed with borel sigma algebra (see docs#Real.borelSpace and docs#Pi.borelSpace)

Etienne Marion (Aug 17 2024 at 21:16):

And you can use docs#Continuous.aemeasurable

Etienne Marion (Aug 17 2024 at 21:20):

If you want to know how an instance is synthesized, you can do

import Mathlib
variable (n : Type) [Finite n]

#synth BorelSpace (n  )

Last updated: May 02 2025 at 03:31 UTC