Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit 608faf0

Browse files
RemyDegennesgouezel
andcommitted
feat(measure_theory/function/conditional_expectation): uniqueness of the conditional expectation (#8802)
The main part of the PR is the new file `ae_eq_of_integral`, in which many different lemmas prove variants of the statement "if two functions have same integral on all sets, then they are equal almost everywhere". In the file `conditional_expectation`, a similar lemma is written for functions which have same integral on all sets in a sub-sigma-algebra and are measurable with respect to that sigma-algebra. This proves the uniqueness of the conditional expectation. Co-authored-by: sgouezel <sebastien.gouezel@univ-rennes1.fr>
1 parent 9a7d9a8 commit 608faf0

File tree

6 files changed

+770
-6
lines changed

6 files changed

+770
-6
lines changed

src/analysis/normed_space/hahn_banach.lean

Lines changed: 14 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -157,4 +157,18 @@ begin
157157
{ exact exists_dual_vector 𝕜 x hx }
158158
end
159159

160+
/-- Variant of Hahn-Banach, eliminating the hypothesis that `x` be nonzero, but only ensuring that
161+
the dual element has norm at most `1` (this can not be improved for the trivial
162+
vector space). -/
163+
theorem exists_dual_vector'' (x : E) :
164+
∃ g : E →L[𝕜] 𝕜, ∥g∥ ≤ 1 ∧ g x = norm' 𝕜 x :=
165+
begin
166+
by_cases hx : x = 0,
167+
{ refine ⟨0, by simp, _⟩,
168+
symmetry,
169+
simp [hx], },
170+
{ rcases exists_dual_vector 𝕜 x hx with ⟨g, g_norm, g_eq⟩,
171+
exact ⟨g, g_norm.le, g_eq⟩ }
172+
end
173+
160174
end dual_vector

0 commit comments

Comments
 (0)