Skip to content

Commit

Permalink
Merge pull request #3 from RemyDegenne/tight
Browse files Browse the repository at this point in the history
Add def of Separating
  • Loading branch information
RemyDegenne authored Dec 29, 2023
2 parents 014bb56 + 6189a5c commit 1b6ecbb
Show file tree
Hide file tree
Showing 3 changed files with 38 additions and 1 deletion.
1 change: 1 addition & 0 deletions Clt.lean
Original file line number Diff line number Diff line change
@@ -1,5 +1,6 @@
-- This module serves as the root of the `Clt` library.
-- Import modules here that should be built as part of the library.
import Clt.Tight
import Clt.Separating
import Clt.CharFun
import Clt.ExpPoly
35 changes: 35 additions & 0 deletions Clt/Separating.lean
Original file line number Diff line number Diff line change
@@ -0,0 +1,35 @@
/-
Copyright (c) 2023 Rémy Degenne. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Rémy Degenne
-/
import Mathlib.Topology.ContinuousFunction.Compact
import Mathlib.MeasureTheory.Measure.ProbabilityMeasure

/-!
# Separating sets of functions
-/

open BoundedContinuousFunction

open scoped ENNReal

namespace MeasureTheory

variable {α E : Type*} [MeasurableSpace α] [TopologicalSpace α] [NormedRing E] [NormedAlgebra ℝ E]

/-- A subalgebra `A` of the bounded continuous function from `α` to `E` is separating in the
probability measures if for all probability measures `μ ≠ ν`, there exists `f ∈ A` such that
`∫ x, f x ∂μ ≠ ∫ x, f x ∂ν`. -/
structure Separating (A : Subalgebra ℝ (α →ᵇ E)) : Prop :=
(exists_ne : ∀ ⦃μ ν : ProbabilityMeasure α⦄, μ ≠ ν → ∃ f ∈ A, ∫ x, f x ∂μ ≠ ∫ x, f x ∂ν)

lemma ProbabilityMeasure.ext_of_Separating {μ ν : ProbabilityMeasure α} {A : Subalgebra ℝ (α →ᵇ E)}
(hA : Separating A) (h : ∀ f ∈ A, ∫ x, f x ∂μ = ∫ x, f x ∂ν) :
μ = ν := by
by_contra h_ne
obtain ⟨f, hfA, hf_ne⟩ := hA.exists_ne h_ne
exact hf_ne (h f hfA)

end MeasureTheory
3 changes: 2 additions & 1 deletion blueprint/src/chapter/separating.tex
Original file line number Diff line number Diff line change
Expand Up @@ -6,6 +6,7 @@ \chapter{Separating subalgebras}
\end{definition}

\begin{definition}\label{def:separating}
\lean{MeasureTheory.Separating} \leanok
A set $\mathcal F$ of functions $E \to F$ is separating in $\mathcal P(E)$ if for all probability measures $\mu, \nu$ on $E$ with $\mu \ne \nu$, there exists $f \in \mathcal F$ with $\mu[f] \ne \nu[f]$.
\end{definition}

Expand Down Expand Up @@ -93,6 +94,7 @@ \chapter{Separating subalgebras}
\end{proof}

\begin{lemma}\label{lem:Cb_eq_of_separating}
\uses{def:separates_points}
Let $\mathcal A$ be a subalgebra of $C_b(E, \mathbb{C})$ that separates points. Let $\mu, \nu$ be two probability measures. If for all $f \in \mathcal A$, $\mu[f] = \nu[f]$, then for all $g \in C_b(E, \mathbb{C})$, $\mu[g] = \nu[g]$.
\end{lemma}

Expand All @@ -115,7 +117,6 @@ \chapter{Separating subalgebras}
\end{proof}

\begin{theorem}[Subalgebras separating points]\label{thm:separating_starSubalgebra}
\uses{def:separates_points}
Let $E$ be a complete separable pseudo-metric space. Let $\mathcal A \subseteq C_b(E, \mathbb{C})$ be a star-subalgebra that separates points. Then $\mathcal A$ is separating in $\mathcal P(E)$.
\end{theorem}

Expand Down

0 comments on commit 1b6ecbb

Please sign in to comment.