author | wenzelm |
Fri, 13 May 2011 23:58:40 +0200 | |
changeset 42795 | 66fcc9882784 |
parent 42067 | 66c8281349ec |
child 42866 | b0746bd57a41 |
permissions | -rw-r--r-- |
42067 | 1 |
(* Title: HOL/Probability/Radon_Nikodym.thy |
2 |
Author: Johannes Hölzl, TU München |
|
3 |
*) |
|
4 |
||
5 |
header {*Radon-Nikod{\'y}m derivative*} |
|
6 |
||
38656 | 7 |
theory Radon_Nikodym |
8 |
imports Lebesgue_Integration |
|
9 |
begin |
|
10 |
||
11 |
lemma (in sigma_finite_measure) Ex_finite_integrable_function: |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
12 |
shows "\<exists>h\<in>borel_measurable M. integral\<^isup>P M h \<noteq> \<infinity> \<and> (\<forall>x\<in>space M. 0 < h x \<and> h x < \<infinity>) \<and> (\<forall>x. 0 \<le> h x)" |
38656 | 13 |
proof - |
14 |
obtain A :: "nat \<Rightarrow> 'a set" where |
|
15 |
range: "range A \<subseteq> sets M" and |
|
16 |
space: "(\<Union>i. A i) = space M" and |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
17 |
measure: "\<And>i. \<mu> (A i) \<noteq> \<infinity>" and |
38656 | 18 |
disjoint: "disjoint_family A" |
19 |
using disjoint_sigma_finite by auto |
|
20 |
let "?B i" = "2^Suc i * \<mu> (A i)" |
|
21 |
have "\<forall>i. \<exists>x. 0 < x \<and> x < inverse (?B i)" |
|
22 |
proof |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
23 |
fix i have Ai: "A i \<in> sets M" using range by auto |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
24 |
from measure positive_measure[OF this] |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
25 |
show "\<exists>x. 0 < x \<and> x < inverse (?B i)" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
26 |
by (auto intro!: extreal_dense simp: extreal_0_gt_inverse) |
38656 | 27 |
qed |
28 |
from choice[OF this] obtain n where n: "\<And>i. 0 < n i" |
|
29 |
"\<And>i. n i < inverse (2^Suc i * \<mu> (A i))" by auto |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
30 |
{ fix i have "0 \<le> n i" using n(1)[of i] by auto } note pos = this |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
31 |
let "?h x" = "\<Sum>i. n i * indicator (A i) x" |
38656 | 32 |
show ?thesis |
33 |
proof (safe intro!: bexI[of _ ?h] del: notI) |
|
39092 | 34 |
have "\<And>i. A i \<in> sets M" |
35 |
using range by fastsimp+ |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
36 |
then have "integral\<^isup>P M ?h = (\<Sum>i. n i * \<mu> (A i))" using pos |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
37 |
by (simp add: positive_integral_suminf positive_integral_cmult_indicator) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
38 |
also have "\<dots> \<le> (\<Sum>i. (1 / 2)^Suc i)" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
39 |
proof (rule suminf_le_pos) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
40 |
fix N |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
41 |
have "n N * \<mu> (A N) \<le> inverse (2^Suc N * \<mu> (A N)) * \<mu> (A N)" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
42 |
using positive_measure[OF `A N \<in> sets M`] n[of N] |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
43 |
by (intro extreal_mult_right_mono) auto |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
44 |
also have "\<dots> \<le> (1 / 2) ^ Suc N" |
38656 | 45 |
using measure[of N] n[of N] |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
46 |
by (cases rule: extreal2_cases[of "n N" "\<mu> (A N)"]) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
47 |
(simp_all add: inverse_eq_divide power_divide one_extreal_def extreal_power_divide) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
48 |
finally show "n N * \<mu> (A N) \<le> (1 / 2) ^ Suc N" . |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
49 |
show "0 \<le> n N * \<mu> (A N)" using n[of N] `A N \<in> sets M` by simp |
38656 | 50 |
qed |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
51 |
finally show "integral\<^isup>P M ?h \<noteq> \<infinity>" unfolding suminf_half_series_extreal by auto |
38656 | 52 |
next |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
53 |
{ fix x assume "x \<in> space M" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
54 |
then obtain i where "x \<in> A i" using space[symmetric] by auto |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
55 |
with disjoint n have "?h x = n i" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
56 |
by (auto intro!: suminf_cmult_indicator intro: less_imp_le) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
57 |
then show "0 < ?h x" and "?h x < \<infinity>" using n[of i] by auto } |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
58 |
note pos = this |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
59 |
fix x show "0 \<le> ?h x" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
60 |
proof cases |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
61 |
assume "x \<in> space M" then show "0 \<le> ?h x" using pos by (auto intro: less_imp_le) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
62 |
next |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
63 |
assume "x \<notin> space M" then have "\<And>i. x \<notin> A i" using space by auto |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
64 |
then show "0 \<le> ?h x" by auto |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
65 |
qed |
38656 | 66 |
next |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
67 |
show "?h \<in> borel_measurable M" using range n |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
68 |
by (auto intro!: borel_measurable_psuminf borel_measurable_extreal_times extreal_0_le_mult intro: less_imp_le) |
38656 | 69 |
qed |
70 |
qed |
|
71 |
||
40871 | 72 |
subsection "Absolutely continuous" |
73 |
||
38656 | 74 |
definition (in measure_space) |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
75 |
"absolutely_continuous \<nu> = (\<forall>N\<in>null_sets. \<nu> N = (0 :: extreal))" |
38656 | 76 |
|
41832 | 77 |
lemma (in measure_space) absolutely_continuous_AE: |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
78 |
assumes "measure_space M'" and [simp]: "sets M' = sets M" "space M' = space M" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
79 |
and "absolutely_continuous (measure M')" "AE x. P x" |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
80 |
shows "AE x in M'. P x" |
40859 | 81 |
proof - |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
82 |
interpret \<nu>: measure_space M' by fact |
40859 | 83 |
from `AE x. P x` obtain N where N: "N \<in> null_sets" and "{x\<in>space M. \<not> P x} \<subseteq> N" |
84 |
unfolding almost_everywhere_def by auto |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
85 |
show "AE x in M'. P x" |
40859 | 86 |
proof (rule \<nu>.AE_I') |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
87 |
show "{x\<in>space M'. \<not> P x} \<subseteq> N" by simp fact |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
88 |
from `absolutely_continuous (measure M')` show "N \<in> \<nu>.null_sets" |
40859 | 89 |
using N unfolding absolutely_continuous_def by auto |
90 |
qed |
|
91 |
qed |
|
92 |
||
39097 | 93 |
lemma (in finite_measure_space) absolutely_continuousI: |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
94 |
assumes "finite_measure_space (M\<lparr> measure := \<nu>\<rparr>)" (is "finite_measure_space ?\<nu>") |
39097 | 95 |
assumes v: "\<And>x. \<lbrakk> x \<in> space M ; \<mu> {x} = 0 \<rbrakk> \<Longrightarrow> \<nu> {x} = 0" |
96 |
shows "absolutely_continuous \<nu>" |
|
97 |
proof (unfold absolutely_continuous_def sets_eq_Pow, safe) |
|
98 |
fix N assume "\<mu> N = 0" "N \<subseteq> space M" |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
99 |
interpret v: finite_measure_space ?\<nu> by fact |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
100 |
have "\<nu> N = measure ?\<nu> (\<Union>x\<in>N. {x})" by simp |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
101 |
also have "\<dots> = (\<Sum>x\<in>N. measure ?\<nu> {x})" |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
102 |
proof (rule v.measure_setsum[symmetric]) |
39097 | 103 |
show "finite N" using `N \<subseteq> space M` finite_space by (auto intro: finite_subset) |
104 |
show "disjoint_family_on (\<lambda>i. {i}) N" unfolding disjoint_family_on_def by auto |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
105 |
fix x assume "x \<in> N" thus "{x} \<in> sets ?\<nu>" using `N \<subseteq> space M` sets_eq_Pow by auto |
39097 | 106 |
qed |
107 |
also have "\<dots> = 0" |
|
108 |
proof (safe intro!: setsum_0') |
|
109 |
fix x assume "x \<in> N" |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
110 |
hence "\<mu> {x} \<le> \<mu> N" "0 \<le> \<mu> {x}" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
111 |
using sets_eq_Pow `N \<subseteq> space M` positive_measure[of "{x}"] |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
112 |
by (auto intro!: measure_mono) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
113 |
then have "\<mu> {x} = 0" using `\<mu> N = 0` by simp |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
114 |
thus "measure ?\<nu> {x} = 0" using v[of x] `x \<in> N` `N \<subseteq> space M` by auto |
39097 | 115 |
qed |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
116 |
finally show "\<nu> N = 0" by simp |
39097 | 117 |
qed |
118 |
||
40871 | 119 |
lemma (in measure_space) density_is_absolutely_continuous: |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
120 |
assumes "\<And>A. A \<in> sets M \<Longrightarrow> \<nu> A = (\<integral>\<^isup>+x. f x * indicator A x \<partial>M)" |
40871 | 121 |
shows "absolutely_continuous \<nu>" |
122 |
using assms unfolding absolutely_continuous_def |
|
123 |
by (simp add: positive_integral_null_set) |
|
124 |
||
125 |
subsection "Existence of the Radon-Nikodym derivative" |
|
126 |
||
38656 | 127 |
lemma (in finite_measure) Radon_Nikodym_aux_epsilon: |
128 |
fixes e :: real assumes "0 < e" |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
129 |
assumes "finite_measure (M\<lparr>measure := \<nu>\<rparr>)" |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
130 |
shows "\<exists>A\<in>sets M. \<mu>' (space M) - finite_measure.\<mu>' (M\<lparr>measure := \<nu>\<rparr>) (space M) \<le> |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
131 |
\<mu>' A - finite_measure.\<mu>' (M\<lparr>measure := \<nu>\<rparr>) A \<and> |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
132 |
(\<forall>B\<in>sets M. B \<subseteq> A \<longrightarrow> - e < \<mu>' B - finite_measure.\<mu>' (M\<lparr>measure := \<nu>\<rparr>) B)" |
38656 | 133 |
proof - |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
134 |
interpret M': finite_measure "M\<lparr>measure := \<nu>\<rparr>" by fact |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
135 |
let "?d A" = "\<mu>' A - M'.\<mu>' A" |
38656 | 136 |
let "?A A" = "if (\<forall>B\<in>sets M. B \<subseteq> space M - A \<longrightarrow> -e < ?d B) |
137 |
then {} |
|
138 |
else (SOME B. B \<in> sets M \<and> B \<subseteq> space M - A \<and> ?d B \<le> -e)" |
|
139 |
def A \<equiv> "\<lambda>n. ((\<lambda>B. B \<union> ?A B) ^^ n) {}" |
|
140 |
have A_simps[simp]: |
|
141 |
"A 0 = {}" |
|
142 |
"\<And>n. A (Suc n) = (A n \<union> ?A (A n))" unfolding A_def by simp_all |
|
143 |
{ fix A assume "A \<in> sets M" |
|
144 |
have "?A A \<in> sets M" |
|
145 |
by (auto intro!: someI2[of _ _ "\<lambda>A. A \<in> sets M"] simp: not_less) } |
|
146 |
note A'_in_sets = this |
|
147 |
{ fix n have "A n \<in> sets M" |
|
148 |
proof (induct n) |
|
149 |
case (Suc n) thus "A (Suc n) \<in> sets M" |
|
150 |
using A'_in_sets[of "A n"] by (auto split: split_if_asm) |
|
151 |
qed (simp add: A_def) } |
|
152 |
note A_in_sets = this |
|
153 |
hence "range A \<subseteq> sets M" by auto |
|
154 |
{ fix n B |
|
155 |
assume Ex: "\<exists>B. B \<in> sets M \<and> B \<subseteq> space M - A n \<and> ?d B \<le> -e" |
|
156 |
hence False: "\<not> (\<forall>B\<in>sets M. B \<subseteq> space M - A n \<longrightarrow> -e < ?d B)" by (auto simp: not_less) |
|
157 |
have "?d (A (Suc n)) \<le> ?d (A n) - e" unfolding A_simps if_not_P[OF False] |
|
158 |
proof (rule someI2_ex[OF Ex]) |
|
159 |
fix B assume "B \<in> sets M \<and> B \<subseteq> space M - A n \<and> ?d B \<le> - e" |
|
160 |
hence "A n \<inter> B = {}" "B \<in> sets M" and dB: "?d B \<le> -e" by auto |
|
161 |
hence "?d (A n \<union> B) = ?d (A n) + ?d B" |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
162 |
using `A n \<in> sets M` finite_measure_Union M'.finite_measure_Union by simp |
38656 | 163 |
also have "\<dots> \<le> ?d (A n) - e" using dB by simp |
164 |
finally show "?d (A n \<union> B) \<le> ?d (A n) - e" . |
|
165 |
qed } |
|
166 |
note dA_epsilon = this |
|
167 |
{ fix n have "?d (A (Suc n)) \<le> ?d (A n)" |
|
168 |
proof (cases "\<exists>B. B\<in>sets M \<and> B \<subseteq> space M - A n \<and> ?d B \<le> - e") |
|
169 |
case True from dA_epsilon[OF this] show ?thesis using `0 < e` by simp |
|
170 |
next |
|
171 |
case False |
|
172 |
hence "\<forall>B\<in>sets M. B \<subseteq> space M - A n \<longrightarrow> -e < ?d B" by (auto simp: not_le) |
|
173 |
thus ?thesis by simp |
|
174 |
qed } |
|
175 |
note dA_mono = this |
|
176 |
show ?thesis |
|
177 |
proof (cases "\<exists>n. \<forall>B\<in>sets M. B \<subseteq> space M - A n \<longrightarrow> -e < ?d B") |
|
178 |
case True then obtain n where B: "\<And>B. \<lbrakk> B \<in> sets M; B \<subseteq> space M - A n\<rbrakk> \<Longrightarrow> -e < ?d B" by blast |
|
179 |
show ?thesis |
|
180 |
proof (safe intro!: bexI[of _ "space M - A n"]) |
|
181 |
fix B assume "B \<in> sets M" "B \<subseteq> space M - A n" |
|
182 |
from B[OF this] show "-e < ?d B" . |
|
183 |
next |
|
184 |
show "space M - A n \<in> sets M" by (rule compl_sets) fact |
|
185 |
next |
|
186 |
show "?d (space M) \<le> ?d (space M - A n)" |
|
187 |
proof (induct n) |
|
188 |
fix n assume "?d (space M) \<le> ?d (space M - A n)" |
|
189 |
also have "\<dots> \<le> ?d (space M - A (Suc n))" |
|
190 |
using A_in_sets sets_into_space dA_mono[of n] |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
191 |
by (simp del: A_simps add: finite_measure_Diff M'.finite_measure_Diff) |
38656 | 192 |
finally show "?d (space M) \<le> ?d (space M - A (Suc n))" . |
193 |
qed simp |
|
194 |
qed |
|
195 |
next |
|
196 |
case False hence B: "\<And>n. \<exists>B. B\<in>sets M \<and> B \<subseteq> space M - A n \<and> ?d B \<le> - e" |
|
197 |
by (auto simp add: not_less) |
|
198 |
{ fix n have "?d (A n) \<le> - real n * e" |
|
199 |
proof (induct n) |
|
200 |
case (Suc n) with dA_epsilon[of n, OF B] show ?case by (simp del: A_simps add: real_of_nat_Suc field_simps) |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
201 |
next |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
202 |
case 0 with M'.empty_measure show ?case by (simp add: zero_extreal_def) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
203 |
qed } note dA_less = this |
38656 | 204 |
have decseq: "decseq (\<lambda>n. ?d (A n))" unfolding decseq_eq_incseq |
205 |
proof (rule incseq_SucI) |
|
206 |
fix n show "- ?d (A n) \<le> - ?d (A (Suc n))" using dA_mono[of n] by auto |
|
207 |
qed |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
208 |
have A: "incseq A" by (auto intro!: incseq_SucI) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
209 |
from finite_continuity_from_below[OF _ A] `range A \<subseteq> sets M` |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
210 |
M'.finite_continuity_from_below[OF _ A] |
38656 | 211 |
have convergent: "(\<lambda>i. ?d (A i)) ----> ?d (\<Union>i. A i)" |
212 |
by (auto intro!: LIMSEQ_diff) |
|
213 |
obtain n :: nat where "- ?d (\<Union>i. A i) / e < real n" using reals_Archimedean2 by auto |
|
214 |
moreover from order_trans[OF decseq_le[OF decseq convergent] dA_less] |
|
215 |
have "real n \<le> - ?d (\<Union>i. A i) / e" using `0<e` by (simp add: field_simps) |
|
216 |
ultimately show ?thesis by auto |
|
217 |
qed |
|
218 |
qed |
|
219 |
||
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
220 |
lemma (in finite_measure) restricted_measure_subset: |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
221 |
assumes S: "S \<in> sets M" and X: "X \<subseteq> S" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
222 |
shows "finite_measure.\<mu>' (restricted_space S) X = \<mu>' X" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
223 |
proof cases |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
224 |
note r = restricted_finite_measure[OF S] |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
225 |
{ assume "X \<in> sets M" with S X show ?thesis |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
226 |
unfolding finite_measure.\<mu>'_def[OF r] \<mu>'_def by auto } |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
227 |
{ assume "X \<notin> sets M" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
228 |
moreover then have "S \<inter> X \<notin> sets M" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
229 |
using X by (simp add: Int_absorb1) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
230 |
ultimately show ?thesis |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
231 |
unfolding finite_measure.\<mu>'_def[OF r] \<mu>'_def using S by auto } |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
232 |
qed |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
233 |
|
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
234 |
lemma (in finite_measure) restricted_measure: |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
235 |
assumes X: "S \<in> sets M" "X \<in> sets (restricted_space S)" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
236 |
shows "finite_measure.\<mu>' (restricted_space S) X = \<mu>' X" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
237 |
proof - |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
238 |
from X have "S \<in> sets M" "X \<subseteq> S" by auto |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
239 |
from restricted_measure_subset[OF this] show ?thesis . |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
240 |
qed |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
241 |
|
38656 | 242 |
lemma (in finite_measure) Radon_Nikodym_aux: |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
243 |
assumes "finite_measure (M\<lparr>measure := \<nu>\<rparr>)" (is "finite_measure ?M'") |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
244 |
shows "\<exists>A\<in>sets M. \<mu>' (space M) - finite_measure.\<mu>' (M\<lparr>measure := \<nu>\<rparr>) (space M) \<le> |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
245 |
\<mu>' A - finite_measure.\<mu>' (M\<lparr>measure := \<nu>\<rparr>) A \<and> |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
246 |
(\<forall>B\<in>sets M. B \<subseteq> A \<longrightarrow> 0 \<le> \<mu>' B - finite_measure.\<mu>' (M\<lparr>measure := \<nu>\<rparr>) B)" |
38656 | 247 |
proof - |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
248 |
interpret M': finite_measure ?M' where |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
249 |
"space ?M' = space M" and "sets ?M' = sets M" and "measure ?M' = \<nu>" by fact auto |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
250 |
let "?d A" = "\<mu>' A - M'.\<mu>' A" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
251 |
let "?P A B n" = "A \<in> sets M \<and> A \<subseteq> B \<and> ?d B \<le> ?d A \<and> (\<forall>C\<in>sets M. C \<subseteq> A \<longrightarrow> - 1 / real (Suc n) < ?d C)" |
39092 | 252 |
let "?r S" = "restricted_space S" |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
253 |
{ fix S n assume S: "S \<in> sets M" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
254 |
note r = M'.restricted_finite_measure[of S] restricted_finite_measure[OF S] S |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
255 |
then have "finite_measure (?r S)" "0 < 1 / real (Suc n)" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
256 |
"finite_measure (?r S\<lparr>measure := \<nu>\<rparr>)" by auto |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
257 |
from finite_measure.Radon_Nikodym_aux_epsilon[OF this] guess X .. note X = this |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
258 |
have "?P X S n" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
259 |
proof (intro conjI ballI impI) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
260 |
show "X \<in> sets M" "X \<subseteq> S" using X(1) `S \<in> sets M` by auto |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
261 |
have "S \<in> op \<inter> S ` sets M" using `S \<in> sets M` by auto |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
262 |
then show "?d S \<le> ?d X" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
263 |
using S X restricted_measure[OF S] M'.restricted_measure[OF S] by simp |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
264 |
fix C assume "C \<in> sets M" "C \<subseteq> X" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
265 |
then have "C \<in> sets (restricted_space S)" "C \<subseteq> X" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
266 |
using `S \<in> sets M` `X \<subseteq> S` by auto |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
267 |
with X(2) show "- 1 / real (Suc n) < ?d C" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
268 |
using S X restricted_measure[OF S] M'.restricted_measure[OF S] by auto |
38656 | 269 |
qed |
270 |
hence "\<exists>A. ?P A S n" by auto } |
|
271 |
note Ex_P = this |
|
272 |
def A \<equiv> "nat_rec (space M) (\<lambda>n A. SOME B. ?P B A n)" |
|
273 |
have A_Suc: "\<And>n. A (Suc n) = (SOME B. ?P B (A n) n)" by (simp add: A_def) |
|
274 |
have A_0[simp]: "A 0 = space M" unfolding A_def by simp |
|
275 |
{ fix i have "A i \<in> sets M" unfolding A_def |
|
276 |
proof (induct i) |
|
277 |
case (Suc i) |
|
278 |
from Ex_P[OF this, of i] show ?case unfolding nat_rec_Suc |
|
279 |
by (rule someI2_ex) simp |
|
280 |
qed simp } |
|
281 |
note A_in_sets = this |
|
282 |
{ fix n have "?P (A (Suc n)) (A n) n" |
|
283 |
using Ex_P[OF A_in_sets] unfolding A_Suc |
|
284 |
by (rule someI2_ex) simp } |
|
285 |
note P_A = this |
|
286 |
have "range A \<subseteq> sets M" using A_in_sets by auto |
|
287 |
have A_mono: "\<And>i. A (Suc i) \<subseteq> A i" using P_A by simp |
|
288 |
have mono_dA: "mono (\<lambda>i. ?d (A i))" using P_A by (simp add: mono_iff_le_Suc) |
|
289 |
have epsilon: "\<And>C i. \<lbrakk> C \<in> sets M; C \<subseteq> A (Suc i) \<rbrakk> \<Longrightarrow> - 1 / real (Suc i) < ?d C" |
|
290 |
using P_A by auto |
|
291 |
show ?thesis |
|
292 |
proof (safe intro!: bexI[of _ "\<Inter>i. A i"]) |
|
293 |
show "(\<Inter>i. A i) \<in> sets M" using A_in_sets by auto |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
294 |
have A: "decseq A" using A_mono by (auto intro!: decseq_SucI) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
295 |
from |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
296 |
finite_continuity_from_above[OF `range A \<subseteq> sets M` A] |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
297 |
M'.finite_continuity_from_above[OF `range A \<subseteq> sets M` A] |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
298 |
have "(\<lambda>i. ?d (A i)) ----> ?d (\<Inter>i. A i)" by (intro LIMSEQ_diff) |
38656 | 299 |
thus "?d (space M) \<le> ?d (\<Inter>i. A i)" using mono_dA[THEN monoD, of 0 _] |
300 |
by (rule_tac LIMSEQ_le_const) (auto intro!: exI) |
|
301 |
next |
|
302 |
fix B assume B: "B \<in> sets M" "B \<subseteq> (\<Inter>i. A i)" |
|
303 |
show "0 \<le> ?d B" |
|
304 |
proof (rule ccontr) |
|
305 |
assume "\<not> 0 \<le> ?d B" |
|
306 |
hence "0 < - ?d B" by auto |
|
307 |
from ex_inverse_of_nat_Suc_less[OF this] |
|
308 |
obtain n where *: "?d B < - 1 / real (Suc n)" |
|
309 |
by (auto simp: real_eq_of_nat inverse_eq_divide field_simps) |
|
310 |
have "B \<subseteq> A (Suc n)" using B by (auto simp del: nat_rec_Suc) |
|
311 |
from epsilon[OF B(1) this] * |
|
312 |
show False by auto |
|
313 |
qed |
|
314 |
qed |
|
315 |
qed |
|
316 |
||
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
317 |
lemma (in finite_measure) real_measure: |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
318 |
assumes A: "A \<in> sets M" shows "\<exists>r. 0 \<le> r \<and> \<mu> A = extreal r" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
319 |
using finite_measure[OF A] positive_measure[OF A] by (cases "\<mu> A") auto |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
320 |
|
38656 | 321 |
lemma (in finite_measure) Radon_Nikodym_finite_measure: |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
322 |
assumes "finite_measure (M\<lparr> measure := \<nu>\<rparr>)" (is "finite_measure ?M'") |
38656 | 323 |
assumes "absolutely_continuous \<nu>" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
324 |
shows "\<exists>f \<in> borel_measurable M. \<forall>A\<in>sets M. \<nu> A = (\<integral>\<^isup>+x. f x * indicator A x \<partial>M)" |
38656 | 325 |
proof - |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
326 |
interpret M': finite_measure ?M' |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
327 |
where "space ?M' = space M" and "sets ?M' = sets M" and "measure ?M' = \<nu>" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
328 |
using assms(1) by auto |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
329 |
def G \<equiv> "{g \<in> borel_measurable M. (\<forall>x. 0 \<le> g x) \<and> (\<forall>A\<in>sets M. (\<integral>\<^isup>+x. g x * indicator A x \<partial>M) \<le> \<nu> A)}" |
38656 | 330 |
have "(\<lambda>x. 0) \<in> G" unfolding G_def by auto |
331 |
hence "G \<noteq> {}" by auto |
|
332 |
{ fix f g assume f: "f \<in> G" and g: "g \<in> G" |
|
333 |
have "(\<lambda>x. max (g x) (f x)) \<in> G" (is "?max \<in> G") unfolding G_def |
|
334 |
proof safe |
|
335 |
show "?max \<in> borel_measurable M" using f g unfolding G_def by auto |
|
336 |
let ?A = "{x \<in> space M. f x \<le> g x}" |
|
337 |
have "?A \<in> sets M" using f g unfolding G_def by auto |
|
338 |
fix A assume "A \<in> sets M" |
|
339 |
hence sets: "?A \<inter> A \<in> sets M" "(space M - ?A) \<inter> A \<in> sets M" using `?A \<in> sets M` by auto |
|
340 |
have union: "((?A \<inter> A) \<union> ((space M - ?A) \<inter> A)) = A" |
|
341 |
using sets_into_space[OF `A \<in> sets M`] by auto |
|
342 |
have "\<And>x. x \<in> space M \<Longrightarrow> max (g x) (f x) * indicator A x = |
|
343 |
g x * indicator (?A \<inter> A) x + f x * indicator ((space M - ?A) \<inter> A) x" |
|
344 |
by (auto simp: indicator_def max_def) |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
345 |
hence "(\<integral>\<^isup>+x. max (g x) (f x) * indicator A x \<partial>M) = |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
346 |
(\<integral>\<^isup>+x. g x * indicator (?A \<inter> A) x \<partial>M) + |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
347 |
(\<integral>\<^isup>+x. f x * indicator ((space M - ?A) \<inter> A) x \<partial>M)" |
38656 | 348 |
using f g sets unfolding G_def |
349 |
by (auto cong: positive_integral_cong intro!: positive_integral_add borel_measurable_indicator) |
|
350 |
also have "\<dots> \<le> \<nu> (?A \<inter> A) + \<nu> ((space M - ?A) \<inter> A)" |
|
351 |
using f g sets unfolding G_def by (auto intro!: add_mono) |
|
352 |
also have "\<dots> = \<nu> A" |
|
353 |
using M'.measure_additive[OF sets] union by auto |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
354 |
finally show "(\<integral>\<^isup>+x. max (g x) (f x) * indicator A x \<partial>M) \<le> \<nu> A" . |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
355 |
next |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
356 |
fix x show "0 \<le> max (g x) (f x)" using f g by (auto simp: G_def split: split_max) |
38656 | 357 |
qed } |
358 |
note max_in_G = this |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
359 |
{ fix f assume "incseq f" and f: "\<And>i. f i \<in> G" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
360 |
have "(\<lambda>x. SUP i. f i x) \<in> G" unfolding G_def |
38656 | 361 |
proof safe |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
362 |
show "(\<lambda>x. SUP i. f i x) \<in> borel_measurable M" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
363 |
using f by (auto simp: G_def) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
364 |
{ fix x show "0 \<le> (SUP i. f i x)" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
365 |
using f by (auto simp: G_def intro: le_SUPI2) } |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
366 |
next |
38656 | 367 |
fix A assume "A \<in> sets M" |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
368 |
have "(\<integral>\<^isup>+x. (SUP i. f i x) * indicator A x \<partial>M) = |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
369 |
(\<integral>\<^isup>+x. (SUP i. f i x * indicator A x) \<partial>M)" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
370 |
by (intro positive_integral_cong) (simp split: split_indicator) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
371 |
also have "\<dots> = (SUP i. (\<integral>\<^isup>+x. f i x * indicator A x \<partial>M))" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
372 |
using `incseq f` f `A \<in> sets M` |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
373 |
by (intro positive_integral_monotone_convergence_SUP) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
374 |
(auto simp: G_def incseq_Suc_iff le_fun_def split: split_indicator) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
375 |
finally show "(\<integral>\<^isup>+x. (SUP i. f i x) * indicator A x \<partial>M) \<le> \<nu> A" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
376 |
using f `A \<in> sets M` by (auto intro!: SUP_leI simp: G_def) |
38656 | 377 |
qed } |
378 |
note SUP_in_G = this |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
379 |
let ?y = "SUP g : G. integral\<^isup>P M g" |
38656 | 380 |
have "?y \<le> \<nu> (space M)" unfolding G_def |
381 |
proof (safe intro!: SUP_leI) |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
382 |
fix g assume "\<forall>A\<in>sets M. (\<integral>\<^isup>+x. g x * indicator A x \<partial>M) \<le> \<nu> A" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
383 |
from this[THEN bspec, OF top] show "integral\<^isup>P M g \<le> \<nu> (space M)" |
38656 | 384 |
by (simp cong: positive_integral_cong) |
385 |
qed |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
386 |
from SUPR_countable_SUPR[OF `G \<noteq> {}`, of "integral\<^isup>P M"] guess ys .. note ys = this |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
387 |
then have "\<forall>n. \<exists>g. g\<in>G \<and> integral\<^isup>P M g = ys n" |
38656 | 388 |
proof safe |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
389 |
fix n assume "range ys \<subseteq> integral\<^isup>P M ` G" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
390 |
hence "ys n \<in> integral\<^isup>P M ` G" by auto |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
391 |
thus "\<exists>g. g\<in>G \<and> integral\<^isup>P M g = ys n" by auto |
38656 | 392 |
qed |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
393 |
from choice[OF this] obtain gs where "\<And>i. gs i \<in> G" "\<And>n. integral\<^isup>P M (gs n) = ys n" by auto |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
394 |
hence y_eq: "?y = (SUP i. integral\<^isup>P M (gs i))" using ys by auto |
38656 | 395 |
let "?g i x" = "Max ((\<lambda>n. gs n x) ` {..i})" |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
396 |
def f \<equiv> "\<lambda>x. SUP i. ?g i x" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
397 |
let "?F A x" = "f x * indicator A x" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
398 |
have gs_not_empty: "\<And>i x. (\<lambda>n. gs n x) ` {..i} \<noteq> {}" by auto |
38656 | 399 |
{ fix i have "?g i \<in> G" |
400 |
proof (induct i) |
|
401 |
case 0 thus ?case by simp fact |
|
402 |
next |
|
403 |
case (Suc i) |
|
404 |
with Suc gs_not_empty `gs (Suc i) \<in> G` show ?case |
|
405 |
by (auto simp add: atMost_Suc intro!: max_in_G) |
|
406 |
qed } |
|
407 |
note g_in_G = this |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
408 |
have "incseq ?g" using gs_not_empty |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
409 |
by (auto intro!: incseq_SucI le_funI simp add: atMost_Suc) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
410 |
from SUP_in_G[OF this g_in_G] have "f \<in> G" unfolding f_def . |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
411 |
then have [simp, intro]: "f \<in> borel_measurable M" unfolding G_def by auto |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
412 |
have "integral\<^isup>P M f = (SUP i. integral\<^isup>P M (?g i))" unfolding f_def |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
413 |
using g_in_G `incseq ?g` |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
414 |
by (auto intro!: positive_integral_monotone_convergence_SUP simp: G_def) |
38656 | 415 |
also have "\<dots> = ?y" |
416 |
proof (rule antisym) |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
417 |
show "(SUP i. integral\<^isup>P M (?g i)) \<le> ?y" |
38656 | 418 |
using g_in_G by (auto intro!: exI Sup_mono simp: SUPR_def) |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
419 |
show "?y \<le> (SUP i. integral\<^isup>P M (?g i))" unfolding y_eq |
38656 | 420 |
by (auto intro!: SUP_mono positive_integral_mono Max_ge) |
421 |
qed |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
422 |
finally have int_f_eq_y: "integral\<^isup>P M f = ?y" . |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
423 |
have "\<And>x. 0 \<le> f x" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
424 |
unfolding f_def using `\<And>i. gs i \<in> G` |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
425 |
by (auto intro!: le_SUPI2 Max_ge_iff[THEN iffD2] simp: G_def) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
426 |
let "?t A" = "\<nu> A - (\<integral>\<^isup>+x. ?F A x \<partial>M)" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
427 |
let ?M = "M\<lparr> measure := ?t\<rparr>" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
428 |
interpret M: sigma_algebra ?M |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
429 |
by (intro sigma_algebra_cong) auto |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
430 |
have f_le_\<nu>: "\<And>A. A \<in> sets M \<Longrightarrow> (\<integral>\<^isup>+x. ?F A x \<partial>M) \<le> \<nu> A" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
431 |
using `f \<in> G` unfolding G_def by auto |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
432 |
have fmM: "finite_measure ?M" |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
433 |
proof (default, simp_all add: countably_additive_def positive_def, safe del: notI) |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
434 |
fix A :: "nat \<Rightarrow> 'a set" assume A: "range A \<subseteq> sets M" "disjoint_family A" |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
435 |
have "(\<Sum>n. (\<integral>\<^isup>+x. ?F (A n) x \<partial>M)) = (\<integral>\<^isup>+x. (\<Sum>n. ?F (A n) x) \<partial>M)" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
436 |
using `range A \<subseteq> sets M` `\<And>x. 0 \<le> f x` |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
437 |
by (intro positive_integral_suminf[symmetric]) auto |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
438 |
also have "\<dots> = (\<integral>\<^isup>+x. ?F (\<Union>n. A n) x \<partial>M)" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
439 |
using `\<And>x. 0 \<le> f x` |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
440 |
by (intro positive_integral_cong) (simp add: suminf_cmult_extreal suminf_indicator[OF `disjoint_family A`]) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
441 |
finally have "(\<Sum>n. (\<integral>\<^isup>+x. ?F (A n) x \<partial>M)) = (\<integral>\<^isup>+x. ?F (\<Union>n. A n) x \<partial>M)" . |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
442 |
moreover have "(\<Sum>n. \<nu> (A n)) = \<nu> (\<Union>n. A n)" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
443 |
using M'.measure_countably_additive A by (simp add: comp_def) |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
444 |
moreover have v_fin: "\<nu> (\<Union>i. A i) \<noteq> \<infinity>" using M'.finite_measure A by (simp add: countable_UN) |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
445 |
moreover { |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
446 |
have "(\<integral>\<^isup>+x. ?F (\<Union>i. A i) x \<partial>M) \<le> \<nu> (\<Union>i. A i)" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
447 |
using A `f \<in> G` unfolding G_def by (auto simp: countable_UN) |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
448 |
also have "\<nu> (\<Union>i. A i) < \<infinity>" using v_fin by simp |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
449 |
finally have "(\<integral>\<^isup>+x. ?F (\<Union>i. A i) x \<partial>M) \<noteq> \<infinity>" by simp } |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
450 |
moreover have "\<And>i. (\<integral>\<^isup>+x. ?F (A i) x \<partial>M) \<le> \<nu> (A i)" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
451 |
using A by (intro f_le_\<nu>) auto |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
452 |
ultimately |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
453 |
show "(\<Sum>n. ?t (A n)) = ?t (\<Union>i. A i)" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
454 |
by (subst suminf_extreal_minus) (simp_all add: positive_integral_positive) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
455 |
next |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
456 |
fix A assume A: "A \<in> sets M" show "0 \<le> \<nu> A - \<integral>\<^isup>+ x. ?F A x \<partial>M" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
457 |
using f_le_\<nu>[OF A] `f \<in> G` M'.finite_measure[OF A] by (auto simp: G_def extreal_le_minus_iff) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
458 |
next |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
459 |
show "\<nu> (space M) - (\<integral>\<^isup>+ x. ?F (space M) x \<partial>M) \<noteq> \<infinity>" (is "?a - ?b \<noteq> _") |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
460 |
using positive_integral_positive[of "?F (space M)"] |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
461 |
by (cases rule: extreal2_cases[of ?a ?b]) auto |
38656 | 462 |
qed |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
463 |
then interpret M: finite_measure ?M |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
464 |
where "space ?M = space M" and "sets ?M = sets M" and "measure ?M = ?t" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
465 |
by (simp_all add: fmM) |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
466 |
have ac: "absolutely_continuous ?t" unfolding absolutely_continuous_def |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
467 |
proof |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
468 |
fix N assume N: "N \<in> null_sets" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
469 |
with `absolutely_continuous \<nu>` have "\<nu> N = 0" unfolding absolutely_continuous_def by auto |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
470 |
moreover with N have "(\<integral>\<^isup>+ x. ?F N x \<partial>M) \<le> \<nu> N" using `f \<in> G` by (auto simp: G_def) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
471 |
ultimately show "\<nu> N - (\<integral>\<^isup>+ x. ?F N x \<partial>M) = 0" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
472 |
using positive_integral_positive by (auto intro!: antisym) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
473 |
qed |
38656 | 474 |
have upper_bound: "\<forall>A\<in>sets M. ?t A \<le> 0" |
475 |
proof (rule ccontr) |
|
476 |
assume "\<not> ?thesis" |
|
477 |
then obtain A where A: "A \<in> sets M" and pos: "0 < ?t A" |
|
478 |
by (auto simp: not_le) |
|
479 |
note pos |
|
480 |
also have "?t A \<le> ?t (space M)" |
|
481 |
using M.measure_mono[of A "space M"] A sets_into_space by simp |
|
482 |
finally have pos_t: "0 < ?t (space M)" by simp |
|
483 |
moreover |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
484 |
then have "\<mu> (space M) \<noteq> 0" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
485 |
using ac unfolding absolutely_continuous_def by auto |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
486 |
then have pos_M: "0 < \<mu> (space M)" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
487 |
using positive_measure[OF top] by (simp add: le_less) |
38656 | 488 |
moreover |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
489 |
have "(\<integral>\<^isup>+x. f x * indicator (space M) x \<partial>M) \<le> \<nu> (space M)" |
38656 | 490 |
using `f \<in> G` unfolding G_def by auto |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
491 |
hence "(\<integral>\<^isup>+x. f x * indicator (space M) x \<partial>M) \<noteq> \<infinity>" |
38656 | 492 |
using M'.finite_measure_of_space by auto |
493 |
moreover |
|
494 |
def b \<equiv> "?t (space M) / \<mu> (space M) / 2" |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
495 |
ultimately have b: "b \<noteq> 0 \<and> 0 \<le> b \<and> b \<noteq> \<infinity>" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
496 |
using M'.finite_measure_of_space positive_integral_positive[of "?F (space M)"] |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
497 |
by (cases rule: extreal3_cases[of "integral\<^isup>P M (?F (space M))" "\<nu> (space M)" "\<mu> (space M)"]) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
498 |
(simp_all add: field_simps) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
499 |
then have b: "b \<noteq> 0" "0 \<le> b" "0 < b" "b \<noteq> \<infinity>" by auto |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
500 |
let ?Mb = "?M\<lparr>measure := \<lambda>A. b * \<mu> A\<rparr>" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
501 |
interpret b: sigma_algebra ?Mb by (intro sigma_algebra_cong) auto |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
502 |
have Mb: "finite_measure ?Mb" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
503 |
proof |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
504 |
show "positive ?Mb (measure ?Mb)" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
505 |
using `0 \<le> b` by (auto simp: positive_def) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
506 |
show "countably_additive ?Mb (measure ?Mb)" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
507 |
using `0 \<le> b` measure_countably_additive |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
508 |
by (auto simp: countably_additive_def suminf_cmult_extreal subset_eq) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
509 |
show "measure ?Mb (space ?Mb) \<noteq> \<infinity>" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
510 |
using b by auto |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
511 |
qed |
38656 | 512 |
from M.Radon_Nikodym_aux[OF this] |
513 |
obtain A0 where "A0 \<in> sets M" and |
|
514 |
space_less_A0: "real (?t (space M)) - real (b * \<mu> (space M)) \<le> real (?t A0) - real (b * \<mu> A0)" and |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
515 |
*: "\<And>B. \<lbrakk> B \<in> sets M ; B \<subseteq> A0 \<rbrakk> \<Longrightarrow> 0 \<le> real (?t B) - real (b * \<mu> B)" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
516 |
unfolding M.\<mu>'_def finite_measure.\<mu>'_def[OF Mb] by auto |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
517 |
{ fix B assume B: "B \<in> sets M" "B \<subseteq> A0" |
38656 | 518 |
with *[OF this] have "b * \<mu> B \<le> ?t B" |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
519 |
using M'.finite_measure b finite_measure M.positive_measure[OF B(1)] |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
520 |
by (cases rule: extreal2_cases[of "?t B" "b * \<mu> B"]) auto } |
38656 | 521 |
note bM_le_t = this |
522 |
let "?f0 x" = "f x + b * indicator A0 x" |
|
523 |
{ fix A assume A: "A \<in> sets M" |
|
524 |
hence "A \<inter> A0 \<in> sets M" using `A0 \<in> sets M` by auto |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
525 |
have "(\<integral>\<^isup>+x. ?f0 x * indicator A x \<partial>M) = |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
526 |
(\<integral>\<^isup>+x. f x * indicator A x + b * indicator (A \<inter> A0) x \<partial>M)" |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
527 |
by (auto intro!: positive_integral_cong split: split_indicator) |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
528 |
hence "(\<integral>\<^isup>+x. ?f0 x * indicator A x \<partial>M) = |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
529 |
(\<integral>\<^isup>+x. f x * indicator A x \<partial>M) + b * \<mu> (A \<inter> A0)" |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
530 |
using `A0 \<in> sets M` `A \<inter> A0 \<in> sets M` A b `f \<in> G` |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
531 |
by (simp add: G_def positive_integral_add positive_integral_cmult_indicator) } |
38656 | 532 |
note f0_eq = this |
533 |
{ fix A assume A: "A \<in> sets M" |
|
534 |
hence "A \<inter> A0 \<in> sets M" using `A0 \<in> sets M` by auto |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
535 |
have f_le_v: "(\<integral>\<^isup>+x. f x * indicator A x \<partial>M) \<le> \<nu> A" |
38656 | 536 |
using `f \<in> G` A unfolding G_def by auto |
537 |
note f0_eq[OF A] |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
538 |
also have "(\<integral>\<^isup>+x. f x * indicator A x \<partial>M) + b * \<mu> (A \<inter> A0) \<le> |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
539 |
(\<integral>\<^isup>+x. f x * indicator A x \<partial>M) + ?t (A \<inter> A0)" |
38656 | 540 |
using bM_le_t[OF `A \<inter> A0 \<in> sets M`] `A \<in> sets M` `A0 \<in> sets M` |
541 |
by (auto intro!: add_left_mono) |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
542 |
also have "\<dots> \<le> (\<integral>\<^isup>+x. f x * indicator A x \<partial>M) + ?t A" |
38656 | 543 |
using M.measure_mono[simplified, OF _ `A \<inter> A0 \<in> sets M` `A \<in> sets M`] |
544 |
by (auto intro!: add_left_mono) |
|
545 |
also have "\<dots> \<le> \<nu> A" |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
546 |
using f_le_v M'.finite_measure[simplified, OF `A \<in> sets M`] positive_integral_positive[of "?F A"] |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
547 |
by (cases "\<integral>\<^isup>+x. ?F A x \<partial>M", cases "\<nu> A") auto |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
548 |
finally have "(\<integral>\<^isup>+x. ?f0 x * indicator A x \<partial>M) \<le> \<nu> A" . } |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
549 |
hence "?f0 \<in> G" using `A0 \<in> sets M` b `f \<in> G` unfolding G_def |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
550 |
by (auto intro!: borel_measurable_indicator borel_measurable_extreal_add |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
551 |
borel_measurable_extreal_times extreal_add_nonneg_nonneg) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
552 |
have real: "?t (space M) \<noteq> \<infinity>" "?t A0 \<noteq> \<infinity>" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
553 |
"b * \<mu> (space M) \<noteq> \<infinity>" "b * \<mu> A0 \<noteq> \<infinity>" |
38656 | 554 |
using `A0 \<in> sets M` b |
555 |
finite_measure[of A0] M.finite_measure[of A0] |
|
556 |
finite_measure_of_space M.finite_measure_of_space |
|
557 |
by auto |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
558 |
have int_f_finite: "integral\<^isup>P M f \<noteq> \<infinity>" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
559 |
using M'.finite_measure_of_space pos_t unfolding extreal_less_minus_iff |
38656 | 560 |
by (auto cong: positive_integral_cong) |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
561 |
have "0 < ?t (space M) - b * \<mu> (space M)" unfolding b_def |
38656 | 562 |
using finite_measure_of_space M'.finite_measure_of_space pos_t pos_M |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
563 |
using positive_integral_positive[of "?F (space M)"] |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
564 |
by (cases rule: extreal3_cases[of "\<mu> (space M)" "\<nu> (space M)" "integral\<^isup>P M (?F (space M))"]) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
565 |
(auto simp: field_simps mult_less_cancel_left) |
38656 | 566 |
also have "\<dots> \<le> ?t A0 - b * \<mu> A0" |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
567 |
using space_less_A0 b |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
568 |
using |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
569 |
`A0 \<in> sets M`[THEN M.real_measure] |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
570 |
top[THEN M.real_measure] |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
571 |
apply safe |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
572 |
apply simp |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
573 |
using |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
574 |
`A0 \<in> sets M`[THEN real_measure] |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
575 |
`A0 \<in> sets M`[THEN M'.real_measure] |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
576 |
top[THEN real_measure] |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
577 |
top[THEN M'.real_measure] |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
578 |
by (cases b) auto |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
579 |
finally have 1: "b * \<mu> A0 < ?t A0" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
580 |
using |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
581 |
`A0 \<in> sets M`[THEN M.real_measure] |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
582 |
apply safe |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
583 |
apply simp |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
584 |
using |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
585 |
`A0 \<in> sets M`[THEN real_measure] |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
586 |
`A0 \<in> sets M`[THEN M'.real_measure] |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
587 |
by (cases b) auto |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
588 |
have "0 < ?t A0" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
589 |
using b `A0 \<in> sets M` by (auto intro!: le_less_trans[OF _ 1]) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
590 |
then have "\<mu> A0 \<noteq> 0" using ac unfolding absolutely_continuous_def |
38656 | 591 |
using `A0 \<in> sets M` by auto |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
592 |
then have "0 < \<mu> A0" using positive_measure[OF `A0 \<in> sets M`] by auto |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
593 |
hence "0 < b * \<mu> A0" using b by (auto simp: extreal_zero_less_0_iff) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
594 |
with int_f_finite have "?y + 0 < integral\<^isup>P M f + b * \<mu> A0" unfolding int_f_eq_y |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
595 |
using `f \<in> G` |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
596 |
by (intro extreal_add_strict_mono) (auto intro!: le_SUPI2 positive_integral_positive) |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
597 |
also have "\<dots> = integral\<^isup>P M ?f0" using f0_eq[OF top] `A0 \<in> sets M` sets_into_space |
38656 | 598 |
by (simp cong: positive_integral_cong) |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
599 |
finally have "?y < integral\<^isup>P M ?f0" by simp |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
600 |
moreover from `?f0 \<in> G` have "integral\<^isup>P M ?f0 \<le> ?y" by (auto intro!: le_SUPI) |
38656 | 601 |
ultimately show False by auto |
602 |
qed |
|
603 |
show ?thesis |
|
604 |
proof (safe intro!: bexI[of _ f]) |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
605 |
fix A assume A: "A\<in>sets M" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
606 |
show "\<nu> A = (\<integral>\<^isup>+x. f x * indicator A x \<partial>M)" |
38656 | 607 |
proof (rule antisym) |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
608 |
show "(\<integral>\<^isup>+x. f x * indicator A x \<partial>M) \<le> \<nu> A" |
38656 | 609 |
using `f \<in> G` `A \<in> sets M` unfolding G_def by auto |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
610 |
show "\<nu> A \<le> (\<integral>\<^isup>+x. f x * indicator A x \<partial>M)" |
38656 | 611 |
using upper_bound[THEN bspec, OF `A \<in> sets M`] |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
612 |
using M'.real_measure[OF A] |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
613 |
by (cases "integral\<^isup>P M (?F A)") auto |
38656 | 614 |
qed |
615 |
qed simp |
|
616 |
qed |
|
617 |
||
40859 | 618 |
lemma (in finite_measure) split_space_into_finite_sets_and_rest: |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
619 |
assumes "measure_space (M\<lparr>measure := \<nu>\<rparr>)" (is "measure_space ?N") |
40859 | 620 |
assumes ac: "absolutely_continuous \<nu>" |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
621 |
shows "\<exists>A0\<in>sets M. \<exists>B::nat\<Rightarrow>'a set. disjoint_family B \<and> range B \<subseteq> sets M \<and> A0 = space M - (\<Union>i. B i) \<and> |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
622 |
(\<forall>A\<in>sets M. A \<subseteq> A0 \<longrightarrow> (\<mu> A = 0 \<and> \<nu> A = 0) \<or> (\<mu> A > 0 \<and> \<nu> A = \<infinity>)) \<and> |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
623 |
(\<forall>i. \<nu> (B i) \<noteq> \<infinity>)" |
38656 | 624 |
proof - |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
625 |
interpret v: measure_space ?N |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
626 |
where "space ?N = space M" and "sets ?N = sets M" and "measure ?N = \<nu>" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
627 |
by fact auto |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
628 |
let ?Q = "{Q\<in>sets M. \<nu> Q \<noteq> \<infinity>}" |
38656 | 629 |
let ?a = "SUP Q:?Q. \<mu> Q" |
630 |
have "{} \<in> ?Q" using v.empty_measure by auto |
|
631 |
then have Q_not_empty: "?Q \<noteq> {}" by blast |
|
632 |
have "?a \<le> \<mu> (space M)" using sets_into_space |
|
633 |
by (auto intro!: SUP_leI measure_mono top) |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
634 |
then have "?a \<noteq> \<infinity>" using finite_measure_of_space |
38656 | 635 |
by auto |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
636 |
from SUPR_countable_SUPR[OF Q_not_empty, of \<mu>] |
38656 | 637 |
obtain Q'' where "range Q'' \<subseteq> \<mu> ` ?Q" and a: "?a = (SUP i::nat. Q'' i)" |
638 |
by auto |
|
639 |
then have "\<forall>i. \<exists>Q'. Q'' i = \<mu> Q' \<and> Q' \<in> ?Q" by auto |
|
640 |
from choice[OF this] obtain Q' where Q': "\<And>i. Q'' i = \<mu> (Q' i)" "\<And>i. Q' i \<in> ?Q" |
|
641 |
by auto |
|
642 |
then have a_Lim: "?a = (SUP i::nat. \<mu> (Q' i))" using a by simp |
|
643 |
let "?O n" = "\<Union>i\<le>n. Q' i" |
|
644 |
have Union: "(SUP i. \<mu> (?O i)) = \<mu> (\<Union>i. ?O i)" |
|
645 |
proof (rule continuity_from_below[of ?O]) |
|
646 |
show "range ?O \<subseteq> sets M" using Q' by (auto intro!: finite_UN) |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
647 |
show "incseq ?O" by (fastsimp intro!: incseq_SucI) |
38656 | 648 |
qed |
649 |
have Q'_sets: "\<And>i. Q' i \<in> sets M" using Q' by auto |
|
650 |
have O_sets: "\<And>i. ?O i \<in> sets M" |
|
651 |
using Q' by (auto intro!: finite_UN Un) |
|
652 |
then have O_in_G: "\<And>i. ?O i \<in> ?Q" |
|
653 |
proof (safe del: notI) |
|
654 |
fix i have "Q' ` {..i} \<subseteq> sets M" |
|
655 |
using Q' by (auto intro: finite_UN) |
|
656 |
with v.measure_finitely_subadditive[of "{.. i}" Q'] |
|
657 |
have "\<nu> (?O i) \<le> (\<Sum>i\<le>i. \<nu> (Q' i))" by auto |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
658 |
also have "\<dots> < \<infinity>" using Q' by (simp add: setsum_Pinfty) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
659 |
finally show "\<nu> (?O i) \<noteq> \<infinity>" by simp |
38656 | 660 |
qed auto |
661 |
have O_mono: "\<And>n. ?O n \<subseteq> ?O (Suc n)" by fastsimp |
|
662 |
have a_eq: "?a = \<mu> (\<Union>i. ?O i)" unfolding Union[symmetric] |
|
663 |
proof (rule antisym) |
|
664 |
show "?a \<le> (SUP i. \<mu> (?O i))" unfolding a_Lim |
|
665 |
using Q' by (auto intro!: SUP_mono measure_mono finite_UN) |
|
666 |
show "(SUP i. \<mu> (?O i)) \<le> ?a" unfolding SUPR_def |
|
667 |
proof (safe intro!: Sup_mono, unfold bex_simps) |
|
668 |
fix i |
|
669 |
have *: "(\<Union>Q' ` {..i}) = ?O i" by auto |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
670 |
then show "\<exists>x. (x \<in> sets M \<and> \<nu> x \<noteq> \<infinity>) \<and> |
38656 | 671 |
\<mu> (\<Union>Q' ` {..i}) \<le> \<mu> x" |
672 |
using O_in_G[of i] by (auto intro!: exI[of _ "?O i"]) |
|
673 |
qed |
|
674 |
qed |
|
675 |
let "?O_0" = "(\<Union>i. ?O i)" |
|
676 |
have "?O_0 \<in> sets M" using Q' by auto |
|
40859 | 677 |
def Q \<equiv> "\<lambda>i. case i of 0 \<Rightarrow> Q' 0 | Suc n \<Rightarrow> ?O (Suc n) - ?O n" |
38656 | 678 |
{ fix i have "Q i \<in> sets M" unfolding Q_def using Q'[of 0] by (cases i) (auto intro: O_sets) } |
679 |
note Q_sets = this |
|
40859 | 680 |
show ?thesis |
681 |
proof (intro bexI exI conjI ballI impI allI) |
|
682 |
show "disjoint_family Q" |
|
683 |
by (fastsimp simp: disjoint_family_on_def Q_def |
|
684 |
split: nat.split_asm) |
|
685 |
show "range Q \<subseteq> sets M" |
|
686 |
using Q_sets by auto |
|
687 |
{ fix A assume A: "A \<in> sets M" "A \<subseteq> space M - ?O_0" |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
688 |
show "\<mu> A = 0 \<and> \<nu> A = 0 \<or> 0 < \<mu> A \<and> \<nu> A = \<infinity>" |
40859 | 689 |
proof (rule disjCI, simp) |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
690 |
assume *: "0 < \<mu> A \<longrightarrow> \<nu> A \<noteq> \<infinity>" |
40859 | 691 |
show "\<mu> A = 0 \<and> \<nu> A = 0" |
692 |
proof cases |
|
693 |
assume "\<mu> A = 0" moreover with ac A have "\<nu> A = 0" |
|
694 |
unfolding absolutely_continuous_def by auto |
|
695 |
ultimately show ?thesis by simp |
|
696 |
next |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
697 |
assume "\<mu> A \<noteq> 0" with * have "\<nu> A \<noteq> \<infinity>" using positive_measure[OF A(1)] by auto |
40859 | 698 |
with A have "\<mu> ?O_0 + \<mu> A = \<mu> (?O_0 \<union> A)" |
699 |
using Q' by (auto intro!: measure_additive countable_UN) |
|
700 |
also have "\<dots> = (SUP i. \<mu> (?O i \<union> A))" |
|
701 |
proof (rule continuity_from_below[of "\<lambda>i. ?O i \<union> A", symmetric, simplified]) |
|
702 |
show "range (\<lambda>i. ?O i \<union> A) \<subseteq> sets M" |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
703 |
using `\<nu> A \<noteq> \<infinity>` O_sets A by auto |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
704 |
qed (fastsimp intro!: incseq_SucI) |
40859 | 705 |
also have "\<dots> \<le> ?a" |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
706 |
proof (safe intro!: SUP_leI) |
40859 | 707 |
fix i have "?O i \<union> A \<in> ?Q" |
708 |
proof (safe del: notI) |
|
709 |
show "?O i \<union> A \<in> sets M" using O_sets A by auto |
|
710 |
from O_in_G[of i] |
|
711 |
moreover have "\<nu> (?O i \<union> A) \<le> \<nu> (?O i) + \<nu> A" |
|
712 |
using v.measure_subadditive[of "?O i" A] A O_sets by auto |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
713 |
ultimately show "\<nu> (?O i \<union> A) \<noteq> \<infinity>" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
714 |
using `\<nu> A \<noteq> \<infinity>` by auto |
40859 | 715 |
qed |
716 |
then show "\<mu> (?O i \<union> A) \<le> ?a" by (rule le_SUPI) |
|
717 |
qed |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
718 |
finally have "\<mu> A = 0" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
719 |
unfolding a_eq using real_measure[OF `?O_0 \<in> sets M`] real_measure[OF A(1)] by auto |
40859 | 720 |
with `\<mu> A \<noteq> 0` show ?thesis by auto |
721 |
qed |
|
722 |
qed } |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
723 |
{ fix i show "\<nu> (Q i) \<noteq> \<infinity>" |
40859 | 724 |
proof (cases i) |
725 |
case 0 then show ?thesis |
|
726 |
unfolding Q_def using Q'[of 0] by simp |
|
727 |
next |
|
728 |
case (Suc n) |
|
729 |
then show ?thesis unfolding Q_def |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
730 |
using `?O n \<in> ?Q` `?O (Suc n) \<in> ?Q` |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
731 |
using v.measure_mono[OF O_mono, of n] v.positive_measure[of "?O n"] v.positive_measure[of "?O (Suc n)"] |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
732 |
using v.measure_Diff[of "?O n" "?O (Suc n)", OF _ _ _ O_mono] |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
733 |
by (cases rule: extreal2_cases[of "\<nu> (\<Union> x\<le>Suc n. Q' x)" "\<nu> (\<Union> i\<le>n. Q' i)"]) auto |
40859 | 734 |
qed } |
735 |
show "space M - ?O_0 \<in> sets M" using Q'_sets by auto |
|
736 |
{ fix j have "(\<Union>i\<le>j. ?O i) = (\<Union>i\<le>j. Q i)" |
|
737 |
proof (induct j) |
|
738 |
case 0 then show ?case by (simp add: Q_def) |
|
739 |
next |
|
740 |
case (Suc j) |
|
741 |
have eq: "\<And>j. (\<Union>i\<le>j. ?O i) = (\<Union>i\<le>j. Q' i)" by fastsimp |
|
742 |
have "{..j} \<union> {..Suc j} = {..Suc j}" by auto |
|
743 |
then have "(\<Union>i\<le>Suc j. Q' i) = (\<Union>i\<le>j. Q' i) \<union> Q (Suc j)" |
|
744 |
by (simp add: UN_Un[symmetric] Q_def del: UN_Un) |
|
745 |
then show ?case using Suc by (auto simp add: eq atMost_Suc) |
|
746 |
qed } |
|
747 |
then have "(\<Union>j. (\<Union>i\<le>j. ?O i)) = (\<Union>j. (\<Union>i\<le>j. Q i))" by simp |
|
748 |
then show "space M - ?O_0 = space M - (\<Union>i. Q i)" by fastsimp |
|
749 |
qed |
|
750 |
qed |
|
751 |
||
752 |
lemma (in finite_measure) Radon_Nikodym_finite_measure_infinite: |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
753 |
assumes "measure_space (M\<lparr>measure := \<nu>\<rparr>)" (is "measure_space ?N") |
40859 | 754 |
assumes "absolutely_continuous \<nu>" |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
755 |
shows "\<exists>f \<in> borel_measurable M. (\<forall>x. 0 \<le> f x) \<and> (\<forall>A\<in>sets M. \<nu> A = (\<integral>\<^isup>+x. f x * indicator A x \<partial>M))" |
40859 | 756 |
proof - |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
757 |
interpret v: measure_space ?N |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
758 |
where "space ?N = space M" and "sets ?N = sets M" and "measure ?N = \<nu>" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
759 |
by fact auto |
40859 | 760 |
from split_space_into_finite_sets_and_rest[OF assms] |
761 |
obtain Q0 and Q :: "nat \<Rightarrow> 'a set" |
|
762 |
where Q: "disjoint_family Q" "range Q \<subseteq> sets M" |
|
763 |
and Q0: "Q0 \<in> sets M" "Q0 = space M - (\<Union>i. Q i)" |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
764 |
and in_Q0: "\<And>A. A \<in> sets M \<Longrightarrow> A \<subseteq> Q0 \<Longrightarrow> \<mu> A = 0 \<and> \<nu> A = 0 \<or> 0 < \<mu> A \<and> \<nu> A = \<infinity>" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
765 |
and Q_fin: "\<And>i. \<nu> (Q i) \<noteq> \<infinity>" by force |
40859 | 766 |
from Q have Q_sets: "\<And>i. Q i \<in> sets M" by auto |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
767 |
have "\<forall>i. \<exists>f. f\<in>borel_measurable M \<and> (\<forall>x. 0 \<le> f x) \<and> (\<forall>A\<in>sets M. |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
768 |
\<nu> (Q i \<inter> A) = (\<integral>\<^isup>+x. f x * indicator (Q i \<inter> A) x \<partial>M))" |
38656 | 769 |
proof |
770 |
fix i |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
771 |
have indicator_eq: "\<And>f x A. (f x :: extreal) * indicator (Q i \<inter> A) x * indicator (Q i) x |
38656 | 772 |
= (f x * indicator (Q i) x) * indicator A x" |
773 |
unfolding indicator_def by auto |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
774 |
have fm: "finite_measure (restricted_space (Q i))" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
775 |
(is "finite_measure ?R") by (rule restricted_finite_measure[OF Q_sets[of i]]) |
38656 | 776 |
then interpret R: finite_measure ?R . |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
777 |
have fmv: "finite_measure (restricted_space (Q i) \<lparr> measure := \<nu>\<rparr>)" (is "finite_measure ?Q") |
38656 | 778 |
unfolding finite_measure_def finite_measure_axioms_def |
779 |
proof |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
780 |
show "measure_space ?Q" |
38656 | 781 |
using v.restricted_measure_space Q_sets[of i] by auto |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
782 |
show "measure ?Q (space ?Q) \<noteq> \<infinity>" using Q_fin by simp |
38656 | 783 |
qed |
784 |
have "R.absolutely_continuous \<nu>" |
|
785 |
using `absolutely_continuous \<nu>` `Q i \<in> sets M` |
|
786 |
by (auto simp: R.absolutely_continuous_def absolutely_continuous_def) |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
787 |
from R.Radon_Nikodym_finite_measure[OF fmv this] |
38656 | 788 |
obtain f where f: "(\<lambda>x. f x * indicator (Q i) x) \<in> borel_measurable M" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
789 |
and f_int: "\<And>A. A\<in>sets M \<Longrightarrow> \<nu> (Q i \<inter> A) = (\<integral>\<^isup>+x. (f x * indicator (Q i) x) * indicator A x \<partial>M)" |
38656 | 790 |
unfolding Bex_def borel_measurable_restricted[OF `Q i \<in> sets M`] |
791 |
positive_integral_restricted[OF `Q i \<in> sets M`] by (auto simp: indicator_eq) |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
792 |
then show "\<exists>f. f\<in>borel_measurable M \<and> (\<forall>x. 0 \<le> f x) \<and> (\<forall>A\<in>sets M. |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
793 |
\<nu> (Q i \<inter> A) = (\<integral>\<^isup>+x. f x * indicator (Q i \<inter> A) x \<partial>M))" |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
794 |
by (auto intro!: exI[of _ "\<lambda>x. max 0 (f x * indicator (Q i) x)"] positive_integral_cong_pos |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
795 |
split: split_indicator split_if_asm simp: max_def) |
38656 | 796 |
qed |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
797 |
from choice[OF this] obtain f where borel: "\<And>i. f i \<in> borel_measurable M" "\<And>i x. 0 \<le> f i x" |
38656 | 798 |
and f: "\<And>A i. A \<in> sets M \<Longrightarrow> |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
799 |
\<nu> (Q i \<inter> A) = (\<integral>\<^isup>+x. f i x * indicator (Q i \<inter> A) x \<partial>M)" |
38656 | 800 |
by auto |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
801 |
let "?f x" = "(\<Sum>i. f i x * indicator (Q i) x) + \<infinity> * indicator Q0 x" |
38656 | 802 |
show ?thesis |
803 |
proof (safe intro!: bexI[of _ ?f]) |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
804 |
show "?f \<in> borel_measurable M" using Q0 borel Q_sets |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
805 |
by (auto intro!: measurable_If) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
806 |
show "\<And>x. 0 \<le> ?f x" using borel by (auto intro!: suminf_0_le simp: indicator_def) |
38656 | 807 |
fix A assume "A \<in> sets M" |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
808 |
have Qi: "\<And>i. Q i \<in> sets M" using Q by auto |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
809 |
have [intro,simp]: "\<And>i. (\<lambda>x. f i x * indicator (Q i \<inter> A) x) \<in> borel_measurable M" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
810 |
"\<And>i. AE x. 0 \<le> f i x * indicator (Q i \<inter> A) x" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
811 |
using borel Qi Q0(1) `A \<in> sets M` by (auto intro!: borel_measurable_extreal_times) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
812 |
have "(\<integral>\<^isup>+x. ?f x * indicator A x \<partial>M) = (\<integral>\<^isup>+x. (\<Sum>i. f i x * indicator (Q i \<inter> A) x) + \<infinity> * indicator (Q0 \<inter> A) x \<partial>M)" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
813 |
using borel by (intro positive_integral_cong) (auto simp: indicator_def) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
814 |
also have "\<dots> = (\<integral>\<^isup>+x. (\<Sum>i. f i x * indicator (Q i \<inter> A) x) \<partial>M) + \<infinity> * \<mu> (Q0 \<inter> A)" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
815 |
using borel Qi Q0(1) `A \<in> sets M` |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
816 |
by (subst positive_integral_add) (auto simp del: extreal_infty_mult |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
817 |
simp add: positive_integral_cmult_indicator Int intro!: suminf_0_le) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
818 |
also have "\<dots> = (\<Sum>i. \<nu> (Q i \<inter> A)) + \<infinity> * \<mu> (Q0 \<inter> A)" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
819 |
by (subst f[OF `A \<in> sets M`], subst positive_integral_suminf) auto |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
820 |
finally have "(\<integral>\<^isup>+x. ?f x * indicator A x \<partial>M) = (\<Sum>i. \<nu> (Q i \<inter> A)) + \<infinity> * \<mu> (Q0 \<inter> A)" . |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
821 |
moreover have "(\<Sum>i. \<nu> (Q i \<inter> A)) = \<nu> ((\<Union>i. Q i) \<inter> A)" |
40859 | 822 |
using Q Q_sets `A \<in> sets M` |
823 |
by (intro v.measure_countably_additive[of "\<lambda>i. Q i \<inter> A", unfolded comp_def, simplified]) |
|
824 |
(auto simp: disjoint_family_on_def) |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
825 |
moreover have "\<infinity> * \<mu> (Q0 \<inter> A) = \<nu> (Q0 \<inter> A)" |
40859 | 826 |
proof - |
827 |
have "Q0 \<inter> A \<in> sets M" using Q0(1) `A \<in> sets M` by blast |
|
828 |
from in_Q0[OF this] show ?thesis by auto |
|
38656 | 829 |
qed |
40859 | 830 |
moreover have "Q0 \<inter> A \<in> sets M" "((\<Union>i. Q i) \<inter> A) \<in> sets M" |
831 |
using Q_sets `A \<in> sets M` Q0(1) by (auto intro!: countable_UN) |
|
832 |
moreover have "((\<Union>i. Q i) \<inter> A) \<union> (Q0 \<inter> A) = A" "((\<Union>i. Q i) \<inter> A) \<inter> (Q0 \<inter> A) = {}" |
|
833 |
using `A \<in> sets M` sets_into_space Q0 by auto |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
834 |
ultimately show "\<nu> A = (\<integral>\<^isup>+x. ?f x * indicator A x \<partial>M)" |
40859 | 835 |
using v.measure_additive[simplified, of "(\<Union>i. Q i) \<inter> A" "Q0 \<inter> A"] |
836 |
by simp |
|
38656 | 837 |
qed |
838 |
qed |
|
839 |
||
840 |
lemma (in sigma_finite_measure) Radon_Nikodym: |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
841 |
assumes "measure_space (M\<lparr>measure := \<nu>\<rparr>)" (is "measure_space ?N") |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
842 |
assumes ac: "absolutely_continuous \<nu>" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
843 |
shows "\<exists>f \<in> borel_measurable M. (\<forall>x. 0 \<le> f x) \<and> (\<forall>A\<in>sets M. \<nu> A = (\<integral>\<^isup>+x. f x * indicator A x \<partial>M))" |
38656 | 844 |
proof - |
845 |
from Ex_finite_integrable_function |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
846 |
obtain h where finite: "integral\<^isup>P M h \<noteq> \<infinity>" and |
38656 | 847 |
borel: "h \<in> borel_measurable M" and |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
848 |
nn: "\<And>x. 0 \<le> h x" and |
38656 | 849 |
pos: "\<And>x. x \<in> space M \<Longrightarrow> 0 < h x" and |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
850 |
"\<And>x. x \<in> space M \<Longrightarrow> h x < \<infinity>" by auto |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
851 |
let "?T A" = "(\<integral>\<^isup>+x. h x * indicator A x \<partial>M)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
852 |
let ?MT = "M\<lparr> measure := ?T \<rparr>" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
853 |
interpret T: finite_measure ?MT |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
854 |
where "space ?MT = space M" and "sets ?MT = sets M" and "measure ?MT = ?T" |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
855 |
unfolding finite_measure_def finite_measure_axioms_def using borel finite nn |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
856 |
by (auto intro!: measure_space_density cong: positive_integral_cong) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
857 |
have "T.absolutely_continuous \<nu>" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
858 |
proof (unfold T.absolutely_continuous_def, safe) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
859 |
fix N assume "N \<in> sets M" "(\<integral>\<^isup>+x. h x * indicator N x \<partial>M) = 0" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
860 |
with borel ac pos have "AE x. x \<notin> N" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
861 |
by (subst (asm) positive_integral_0_iff_AE) (auto split: split_indicator simp: not_le) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
862 |
then have "N \<in> null_sets" using `N \<in> sets M` sets_into_space |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
863 |
by (subst (asm) AE_iff_measurable[OF `N \<in> sets M`]) auto |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
864 |
then show "\<nu> N = 0" using ac by (auto simp: absolutely_continuous_def) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
865 |
qed |
38656 | 866 |
from T.Radon_Nikodym_finite_measure_infinite[simplified, OF assms(1) this] |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
867 |
obtain f where f_borel: "f \<in> borel_measurable M" "\<And>x. 0 \<le> f x" and |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
868 |
fT: "\<And>A. A \<in> sets M \<Longrightarrow> \<nu> A = (\<integral>\<^isup>+ x. f x * indicator A x \<partial>?MT)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
869 |
by (auto simp: measurable_def) |
38656 | 870 |
show ?thesis |
871 |
proof (safe intro!: bexI[of _ "\<lambda>x. h x * f x"]) |
|
872 |
show "(\<lambda>x. h x * f x) \<in> borel_measurable M" |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
873 |
using borel f_borel by (auto intro: borel_measurable_extreal_times) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
874 |
show "\<And>x. 0 \<le> h x * f x" using nn f_borel by auto |
38656 | 875 |
fix A assume "A \<in> sets M" |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
876 |
then show "\<nu> A = (\<integral>\<^isup>+x. h x * f x * indicator A x \<partial>M)" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
877 |
unfolding fT[OF `A \<in> sets M`] mult_assoc using nn borel f_borel |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
878 |
by (intro positive_integral_translated_density) auto |
38656 | 879 |
qed |
880 |
qed |
|
881 |
||
40859 | 882 |
section "Uniqueness of densities" |
883 |
||
884 |
lemma (in measure_space) finite_density_unique: |
|
885 |
assumes borel: "f \<in> borel_measurable M" "g \<in> borel_measurable M" |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
886 |
assumes pos: "AE x. 0 \<le> f x" "AE x. 0 \<le> g x" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
887 |
and fin: "integral\<^isup>P M f \<noteq> \<infinity>" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
888 |
shows "(\<forall>A\<in>sets M. (\<integral>\<^isup>+x. f x * indicator A x \<partial>M) = (\<integral>\<^isup>+x. g x * indicator A x \<partial>M)) |
40859 | 889 |
\<longleftrightarrow> (AE x. f x = g x)" |
890 |
(is "(\<forall>A\<in>sets M. ?P f A = ?P g A) \<longleftrightarrow> _") |
|
891 |
proof (intro iffI ballI) |
|
892 |
fix A assume eq: "AE x. f x = g x" |
|
41705 | 893 |
then show "?P f A = ?P g A" |
894 |
by (auto intro: positive_integral_cong_AE) |
|
40859 | 895 |
next |
896 |
assume eq: "\<forall>A\<in>sets M. ?P f A = ?P g A" |
|
897 |
from this[THEN bspec, OF top] fin |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
898 |
have g_fin: "integral\<^isup>P M g \<noteq> \<infinity>" by (simp cong: positive_integral_cong) |
40859 | 899 |
{ fix f g assume borel: "f \<in> borel_measurable M" "g \<in> borel_measurable M" |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
900 |
and pos: "AE x. 0 \<le> f x" "AE x. 0 \<le> g x" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
901 |
and g_fin: "integral\<^isup>P M g \<noteq> \<infinity>" and eq: "\<forall>A\<in>sets M. ?P f A = ?P g A" |
40859 | 902 |
let ?N = "{x\<in>space M. g x < f x}" |
903 |
have N: "?N \<in> sets M" using borel by simp |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
904 |
have "?P g ?N \<le> integral\<^isup>P M g" using pos |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
905 |
by (intro positive_integral_mono_AE) (auto split: split_indicator) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
906 |
then have Pg_fin: "?P g ?N \<noteq> \<infinity>" using g_fin by auto |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
907 |
have "?P (\<lambda>x. (f x - g x)) ?N = (\<integral>\<^isup>+x. f x * indicator ?N x - g x * indicator ?N x \<partial>M)" |
40859 | 908 |
by (auto intro!: positive_integral_cong simp: indicator_def) |
909 |
also have "\<dots> = ?P f ?N - ?P g ?N" |
|
910 |
proof (rule positive_integral_diff) |
|
911 |
show "(\<lambda>x. f x * indicator ?N x) \<in> borel_measurable M" "(\<lambda>x. g x * indicator ?N x) \<in> borel_measurable M" |
|
912 |
using borel N by auto |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
913 |
show "AE x. g x * indicator ?N x \<le> f x * indicator ?N x" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
914 |
"AE x. 0 \<le> g x * indicator ?N x" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
915 |
using pos by (auto split: split_indicator) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
916 |
qed fact |
40859 | 917 |
also have "\<dots> = 0" |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
918 |
unfolding eq[THEN bspec, OF N] using positive_integral_positive Pg_fin by auto |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
919 |
finally have "AE x. f x \<le> g x" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
920 |
using pos borel positive_integral_PInf_AE[OF borel(2) g_fin] |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
921 |
by (subst (asm) positive_integral_0_iff_AE) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
922 |
(auto split: split_indicator simp: not_less extreal_minus_le_iff) } |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
923 |
from this[OF borel pos g_fin eq] this[OF borel(2,1) pos(2,1) fin] eq |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
924 |
show "AE x. f x = g x" by auto |
40859 | 925 |
qed |
926 |
||
927 |
lemma (in finite_measure) density_unique_finite_measure: |
|
928 |
assumes borel: "f \<in> borel_measurable M" "f' \<in> borel_measurable M" |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
929 |
assumes pos: "AE x. 0 \<le> f x" "AE x. 0 \<le> f' x" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
930 |
assumes f: "\<And>A. A \<in> sets M \<Longrightarrow> (\<integral>\<^isup>+x. f x * indicator A x \<partial>M) = (\<integral>\<^isup>+x. f' x * indicator A x \<partial>M)" |
40859 | 931 |
(is "\<And>A. A \<in> sets M \<Longrightarrow> ?P f A = ?P f' A") |
932 |
shows "AE x. f x = f' x" |
|
933 |
proof - |
|
934 |
let "?\<nu> A" = "?P f A" and "?\<nu>' A" = "?P f' A" |
|
935 |
let "?f A x" = "f x * indicator A x" and "?f' A x" = "f' x * indicator A x" |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
936 |
interpret M: measure_space "M\<lparr> measure := ?\<nu>\<rparr>" |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
937 |
using borel(1) pos(1) by (rule measure_space_density) simp |
40859 | 938 |
have ac: "absolutely_continuous ?\<nu>" |
939 |
using f by (rule density_is_absolutely_continuous) |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
940 |
from split_space_into_finite_sets_and_rest[OF `measure_space (M\<lparr> measure := ?\<nu>\<rparr>)` ac] |
40859 | 941 |
obtain Q0 and Q :: "nat \<Rightarrow> 'a set" |
942 |
where Q: "disjoint_family Q" "range Q \<subseteq> sets M" |
|
943 |
and Q0: "Q0 \<in> sets M" "Q0 = space M - (\<Union>i. Q i)" |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
944 |
and in_Q0: "\<And>A. A \<in> sets M \<Longrightarrow> A \<subseteq> Q0 \<Longrightarrow> \<mu> A = 0 \<and> ?\<nu> A = 0 \<or> 0 < \<mu> A \<and> ?\<nu> A = \<infinity>" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
945 |
and Q_fin: "\<And>i. ?\<nu> (Q i) \<noteq> \<infinity>" by force |
40859 | 946 |
from Q have Q_sets: "\<And>i. Q i \<in> sets M" by auto |
947 |
let ?N = "{x\<in>space M. f x \<noteq> f' x}" |
|
948 |
have "?N \<in> sets M" using borel by auto |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
949 |
have *: "\<And>i x A. \<And>y::extreal. y * indicator (Q i) x * indicator A x = y * indicator (Q i \<inter> A) x" |
40859 | 950 |
unfolding indicator_def by auto |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
951 |
have "\<forall>i. AE x. ?f (Q i) x = ?f' (Q i) x" using borel Q_fin Q pos |
40859 | 952 |
by (intro finite_density_unique[THEN iffD1] allI) |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
953 |
(auto intro!: borel_measurable_extreal_times f Int simp: *) |
41705 | 954 |
moreover have "AE x. ?f Q0 x = ?f' Q0 x" |
40859 | 955 |
proof (rule AE_I') |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
956 |
{ fix f :: "'a \<Rightarrow> extreal" assume borel: "f \<in> borel_measurable M" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
957 |
and eq: "\<And>A. A \<in> sets M \<Longrightarrow> ?\<nu> A = (\<integral>\<^isup>+x. f x * indicator A x \<partial>M)" |
40859 | 958 |
let "?A i" = "Q0 \<inter> {x \<in> space M. f x < of_nat i}" |
959 |
have "(\<Union>i. ?A i) \<in> null_sets" |
|
960 |
proof (rule null_sets_UN) |
|
961 |
fix i have "?A i \<in> sets M" |
|
962 |
using borel Q0(1) by auto |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
963 |
have "?\<nu> (?A i) \<le> (\<integral>\<^isup>+x. of_nat i * indicator (?A i) x \<partial>M)" |
40859 | 964 |
unfolding eq[OF `?A i \<in> sets M`] |
965 |
by (auto intro!: positive_integral_mono simp: indicator_def) |
|
966 |
also have "\<dots> = of_nat i * \<mu> (?A i)" |
|
967 |
using `?A i \<in> sets M` by (auto intro!: positive_integral_cmult_indicator) |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
968 |
also have "\<dots> < \<infinity>" |
40859 | 969 |
using `?A i \<in> sets M`[THEN finite_measure] by auto |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
970 |
finally have "?\<nu> (?A i) \<noteq> \<infinity>" by simp |
40859 | 971 |
then show "?A i \<in> null_sets" using in_Q0[OF `?A i \<in> sets M`] `?A i \<in> sets M` by auto |
972 |
qed |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
973 |
also have "(\<Union>i. ?A i) = Q0 \<inter> {x\<in>space M. f x \<noteq> \<infinity>}" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
974 |
by (auto simp: less_PInf_Ex_of_nat real_eq_of_nat) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
975 |
finally have "Q0 \<inter> {x\<in>space M. f x \<noteq> \<infinity>} \<in> null_sets" by simp } |
40859 | 976 |
from this[OF borel(1) refl] this[OF borel(2) f] |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
977 |
have "Q0 \<inter> {x\<in>space M. f x \<noteq> \<infinity>} \<in> null_sets" "Q0 \<inter> {x\<in>space M. f' x \<noteq> \<infinity>} \<in> null_sets" by simp_all |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
978 |
then show "(Q0 \<inter> {x\<in>space M. f x \<noteq> \<infinity>}) \<union> (Q0 \<inter> {x\<in>space M. f' x \<noteq> \<infinity>}) \<in> null_sets" by (rule null_sets_Un) |
40859 | 979 |
show "{x \<in> space M. ?f Q0 x \<noteq> ?f' Q0 x} \<subseteq> |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
980 |
(Q0 \<inter> {x\<in>space M. f x \<noteq> \<infinity>}) \<union> (Q0 \<inter> {x\<in>space M. f' x \<noteq> \<infinity>})" by (auto simp: indicator_def) |
40859 | 981 |
qed |
41705 | 982 |
moreover have "\<And>x. (?f Q0 x = ?f' Q0 x) \<longrightarrow> (\<forall>i. ?f (Q i) x = ?f' (Q i) x) \<longrightarrow> |
40859 | 983 |
?f (space M) x = ?f' (space M) x" |
984 |
by (auto simp: indicator_def Q0) |
|
41705 | 985 |
ultimately have "AE x. ?f (space M) x = ?f' (space M) x" |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
986 |
by (auto simp: AE_all_countable[symmetric]) |
41705 | 987 |
then show "AE x. f x = f' x" by auto |
40859 | 988 |
qed |
989 |
||
990 |
lemma (in sigma_finite_measure) density_unique: |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
991 |
assumes f: "f \<in> borel_measurable M" "AE x. 0 \<le> f x" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
992 |
assumes f': "f' \<in> borel_measurable M" "AE x. 0 \<le> f' x" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
993 |
assumes eq: "\<And>A. A \<in> sets M \<Longrightarrow> (\<integral>\<^isup>+x. f x * indicator A x \<partial>M) = (\<integral>\<^isup>+x. f' x * indicator A x \<partial>M)" |
40859 | 994 |
(is "\<And>A. A \<in> sets M \<Longrightarrow> ?P f A = ?P f' A") |
995 |
shows "AE x. f x = f' x" |
|
996 |
proof - |
|
997 |
obtain h where h_borel: "h \<in> borel_measurable M" |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
998 |
and fin: "integral\<^isup>P M h \<noteq> \<infinity>" and pos: "\<And>x. x \<in> space M \<Longrightarrow> 0 < h x \<and> h x < \<infinity>" "\<And>x. 0 \<le> h x" |
40859 | 999 |
using Ex_finite_integrable_function by auto |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1000 |
then have h_nn: "AE x. 0 \<le> h x" by auto |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1001 |
let ?H = "M\<lparr> measure := \<lambda>A. (\<integral>\<^isup>+x. h x * indicator A x \<partial>M) \<rparr>" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1002 |
have H: "measure_space ?H" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1003 |
using h_borel h_nn by (rule measure_space_density) simp |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1004 |
then interpret h: measure_space ?H . |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1005 |
interpret h: finite_measure "M\<lparr> measure := \<lambda>A. (\<integral>\<^isup>+x. h x * indicator A x \<partial>M) \<rparr>" |
40859 | 1006 |
by default (simp cong: positive_integral_cong add: fin) |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1007 |
let ?fM = "M\<lparr>measure := \<lambda>A. (\<integral>\<^isup>+x. f x * indicator A x \<partial>M)\<rparr>" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1008 |
interpret f: measure_space ?fM |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1009 |
using f by (rule measure_space_density) simp |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1010 |
let ?f'M = "M\<lparr>measure := \<lambda>A. (\<integral>\<^isup>+x. f' x * indicator A x \<partial>M)\<rparr>" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1011 |
interpret f': measure_space ?f'M |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1012 |
using f' by (rule measure_space_density) simp |
40859 | 1013 |
{ fix A assume "A \<in> sets M" |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1014 |
then have "{x \<in> space M. h x * indicator A x \<noteq> 0} = A" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1015 |
using pos(1) sets_into_space by (force simp: indicator_def) |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1016 |
then have "(\<integral>\<^isup>+x. h x * indicator A x \<partial>M) = 0 \<longleftrightarrow> A \<in> null_sets" |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1017 |
using h_borel `A \<in> sets M` h_nn by (subst positive_integral_0_iff) auto } |
40859 | 1018 |
note h_null_sets = this |
1019 |
{ fix A assume "A \<in> sets M" |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1020 |
have "(\<integral>\<^isup>+x. f x * (h x * indicator A x) \<partial>M) = (\<integral>\<^isup>+x. h x * indicator A x \<partial>?fM)" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1021 |
using `A \<in> sets M` h_borel h_nn f f' |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1022 |
by (intro positive_integral_translated_density[symmetric]) auto |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1023 |
also have "\<dots> = (\<integral>\<^isup>+x. h x * indicator A x \<partial>?f'M)" |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1024 |
by (rule f'.positive_integral_cong_measure) (simp_all add: eq) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1025 |
also have "\<dots> = (\<integral>\<^isup>+x. f' x * (h x * indicator A x) \<partial>M)" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1026 |
using `A \<in> sets M` h_borel h_nn f f' |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1027 |
by (intro positive_integral_translated_density) auto |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1028 |
finally have "(\<integral>\<^isup>+x. h x * (f x * indicator A x) \<partial>M) = (\<integral>\<^isup>+x. h x * (f' x * indicator A x) \<partial>M)" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1029 |
by (simp add: ac_simps) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1030 |
then have "(\<integral>\<^isup>+x. (f x * indicator A x) \<partial>?H) = (\<integral>\<^isup>+x. (f' x * indicator A x) \<partial>?H)" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1031 |
using `A \<in> sets M` h_borel h_nn f f' |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1032 |
by (subst (asm) (1 2) positive_integral_translated_density[symmetric]) auto } |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1033 |
then have "AE x in ?H. f x = f' x" using h_borel h_nn f f' |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1034 |
by (intro h.density_unique_finite_measure absolutely_continuous_AE[OF H] density_is_absolutely_continuous) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1035 |
simp_all |
40859 | 1036 |
then show "AE x. f x = f' x" |
1037 |
unfolding h.almost_everywhere_def almost_everywhere_def |
|
1038 |
by (auto simp add: h_null_sets) |
|
1039 |
qed |
|
1040 |
||
1041 |
lemma (in sigma_finite_measure) sigma_finite_iff_density_finite: |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1042 |
assumes \<nu>: "measure_space (M\<lparr>measure := \<nu>\<rparr>)" (is "measure_space ?N") |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1043 |
and f: "f \<in> borel_measurable M" "AE x. 0 \<le> f x" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1044 |
and eq: "\<And>A. A \<in> sets M \<Longrightarrow> \<nu> A = (\<integral>\<^isup>+x. f x * indicator A x \<partial>M)" |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1045 |
shows "sigma_finite_measure (M\<lparr>measure := \<nu>\<rparr>) \<longleftrightarrow> (AE x. f x \<noteq> \<infinity>)" |
40859 | 1046 |
proof |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1047 |
assume "sigma_finite_measure ?N" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1048 |
then interpret \<nu>: sigma_finite_measure ?N |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1049 |
where "borel_measurable ?N = borel_measurable M" and "measure ?N = \<nu>" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1050 |
and "sets ?N = sets M" and "space ?N = space M" by (auto simp: measurable_def) |
40859 | 1051 |
from \<nu>.Ex_finite_integrable_function obtain h where |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1052 |
h: "h \<in> borel_measurable M" "integral\<^isup>P ?N h \<noteq> \<infinity>" and |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1053 |
h_nn: "\<And>x. 0 \<le> h x" and |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1054 |
fin: "\<forall>x\<in>space M. 0 < h x \<and> h x < \<infinity>" by auto |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1055 |
have "AE x. f x * h x \<noteq> \<infinity>" |
40859 | 1056 |
proof (rule AE_I') |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1057 |
have "integral\<^isup>P ?N h = (\<integral>\<^isup>+x. f x * h x \<partial>M)" using f h h_nn |
41705 | 1058 |
by (subst \<nu>.positive_integral_cong_measure[symmetric, |
1059 |
of "M\<lparr> measure := \<lambda> A. \<integral>\<^isup>+x. f x * indicator A x \<partial>M \<rparr>"]) |
|
1060 |
(auto intro!: positive_integral_translated_density simp: eq) |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1061 |
then have "(\<integral>\<^isup>+x. f x * h x \<partial>M) \<noteq> \<infinity>" |
40859 | 1062 |
using h(2) by simp |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1063 |
then show "(\<lambda>x. f x * h x) -` {\<infinity>} \<inter> space M \<in> null_sets" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1064 |
using f h(1) by (auto intro!: positive_integral_PInf borel_measurable_vimage) |
40859 | 1065 |
qed auto |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1066 |
then show "AE x. f x \<noteq> \<infinity>" |
41705 | 1067 |
using fin by (auto elim!: AE_Ball_mp) |
40859 | 1068 |
next |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1069 |
assume AE: "AE x. f x \<noteq> \<infinity>" |
40859 | 1070 |
from sigma_finite guess Q .. note Q = this |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1071 |
interpret \<nu>: measure_space ?N |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1072 |
where "borel_measurable ?N = borel_measurable M" and "measure ?N = \<nu>" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1073 |
and "sets ?N = sets M" and "space ?N = space M" using \<nu> by (auto simp: measurable_def) |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1074 |
def A \<equiv> "\<lambda>i. f -` (case i of 0 \<Rightarrow> {\<infinity>} | Suc n \<Rightarrow> {.. of_nat (Suc n)}) \<inter> space M" |
40859 | 1075 |
{ fix i j have "A i \<inter> Q j \<in> sets M" |
1076 |
unfolding A_def using f Q |
|
1077 |
apply (rule_tac Int) |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1078 |
by (cases i) (auto intro: measurable_sets[OF f(1)]) } |
40859 | 1079 |
note A_in_sets = this |
1080 |
let "?A n" = "case prod_decode n of (i,j) \<Rightarrow> A i \<inter> Q j" |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1081 |
show "sigma_finite_measure ?N" |
40859 | 1082 |
proof (default, intro exI conjI subsetI allI) |
1083 |
fix x assume "x \<in> range ?A" |
|
1084 |
then obtain n where n: "x = ?A n" by auto |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1085 |
then show "x \<in> sets ?N" using A_in_sets by (cases "prod_decode n") auto |
40859 | 1086 |
next |
1087 |
have "(\<Union>i. ?A i) = (\<Union>i j. A i \<inter> Q j)" |
|
1088 |
proof safe |
|
1089 |
fix x i j assume "x \<in> A i" "x \<in> Q j" |
|
1090 |
then show "x \<in> (\<Union>i. case prod_decode i of (i, j) \<Rightarrow> A i \<inter> Q j)" |
|
1091 |
by (intro UN_I[of "prod_encode (i,j)"]) auto |
|
1092 |
qed auto |
|
1093 |
also have "\<dots> = (\<Union>i. A i) \<inter> space M" using Q by auto |
|
1094 |
also have "(\<Union>i. A i) = space M" |
|
1095 |
proof safe |
|
1096 |
fix x assume x: "x \<in> space M" |
|
1097 |
show "x \<in> (\<Union>i. A i)" |
|
1098 |
proof (cases "f x") |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1099 |
case PInf with x show ?thesis unfolding A_def by (auto intro: exI[of _ 0]) |
40859 | 1100 |
next |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1101 |
case (real r) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1102 |
with less_PInf_Ex_of_nat[of "f x"] obtain n where "f x < of_nat n" by (auto simp: real_eq_of_nat) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1103 |
then show ?thesis using x real unfolding A_def by (auto intro!: exI[of _ "Suc n"]) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1104 |
next |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1105 |
case MInf with x show ?thesis |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1106 |
unfolding A_def by (auto intro!: exI[of _ "Suc 0"]) |
40859 | 1107 |
qed |
1108 |
qed (auto simp: A_def) |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1109 |
finally show "(\<Union>i. ?A i) = space ?N" by simp |
40859 | 1110 |
next |
1111 |
fix n obtain i j where |
|
1112 |
[simp]: "prod_decode n = (i, j)" by (cases "prod_decode n") auto |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1113 |
have "(\<integral>\<^isup>+x. f x * indicator (A i \<inter> Q j) x \<partial>M) \<noteq> \<infinity>" |
40859 | 1114 |
proof (cases i) |
1115 |
case 0 |
|
1116 |
have "AE x. f x * indicator (A i \<inter> Q j) x = 0" |
|
41705 | 1117 |
using AE by (auto simp: A_def `i = 0`) |
1118 |
from positive_integral_cong_AE[OF this] show ?thesis by simp |
|
40859 | 1119 |
next |
1120 |
case (Suc n) |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1121 |
then have "(\<integral>\<^isup>+x. f x * indicator (A i \<inter> Q j) x \<partial>M) \<le> |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1122 |
(\<integral>\<^isup>+x. of_nat (Suc n) * indicator (Q j) x \<partial>M)" |
40859 | 1123 |
by (auto intro!: positive_integral_mono simp: indicator_def A_def) |
1124 |
also have "\<dots> = of_nat (Suc n) * \<mu> (Q j)" |
|
1125 |
using Q by (auto intro!: positive_integral_cmult_indicator) |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1126 |
also have "\<dots> < \<infinity>" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1127 |
using Q by (auto simp: real_eq_of_nat[symmetric]) |
40859 | 1128 |
finally show ?thesis by simp |
1129 |
qed |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1130 |
then show "measure ?N (?A n) \<noteq> \<infinity>" |
40859 | 1131 |
using A_in_sets Q eq by auto |
1132 |
qed |
|
1133 |
qed |
|
1134 |
||
40871 | 1135 |
section "Radon-Nikodym derivative" |
38656 | 1136 |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1137 |
definition |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1138 |
"RN_deriv M \<nu> \<equiv> SOME f. f \<in> borel_measurable M \<and> (\<forall>x. 0 \<le> f x) \<and> |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1139 |
(\<forall>A \<in> sets M. \<nu> A = (\<integral>\<^isup>+x. f x * indicator A x \<partial>M))" |
38656 | 1140 |
|
40859 | 1141 |
lemma (in sigma_finite_measure) RN_deriv_cong: |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1142 |
assumes cong: "\<And>A. A \<in> sets M \<Longrightarrow> measure M' A = \<mu> A" "sets M' = sets M" "space M' = space M" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1143 |
and \<nu>: "\<And>A. A \<in> sets M \<Longrightarrow> \<nu>' A = \<nu> A" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1144 |
shows "RN_deriv M' \<nu>' x = RN_deriv M \<nu> x" |
40859 | 1145 |
proof - |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1146 |
interpret \<mu>': sigma_finite_measure M' |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1147 |
using cong by (rule sigma_finite_measure_cong) |
40859 | 1148 |
show ?thesis |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1149 |
unfolding RN_deriv_def |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1150 |
by (simp add: cong \<nu> positive_integral_cong_measure[OF cong] measurable_def) |
40859 | 1151 |
qed |
1152 |
||
38656 | 1153 |
lemma (in sigma_finite_measure) RN_deriv: |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1154 |
assumes "measure_space (M\<lparr>measure := \<nu>\<rparr>)" |
38656 | 1155 |
assumes "absolutely_continuous \<nu>" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1156 |
shows "RN_deriv M \<nu> \<in> borel_measurable M" (is ?borel) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1157 |
and "\<And>A. A \<in> sets M \<Longrightarrow> \<nu> A = (\<integral>\<^isup>+x. RN_deriv M \<nu> x * indicator A x \<partial>M)" |
38656 | 1158 |
(is "\<And>A. _ \<Longrightarrow> ?int A") |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1159 |
and "0 \<le> RN_deriv M \<nu> x" |
38656 | 1160 |
proof - |
1161 |
note Ex = Radon_Nikodym[OF assms, unfolded Bex_def] |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1162 |
then show ?borel unfolding RN_deriv_def by (rule someI2_ex) auto |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1163 |
from Ex show "0 \<le> RN_deriv M \<nu> x" unfolding RN_deriv_def |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1164 |
by (rule someI2_ex) simp |
38656 | 1165 |
fix A assume "A \<in> sets M" |
1166 |
from Ex show "?int A" unfolding RN_deriv_def |
|
1167 |
by (rule someI2_ex) (simp add: `A \<in> sets M`) |
|
1168 |
qed |
|
1169 |
||
40859 | 1170 |
lemma (in sigma_finite_measure) RN_deriv_positive_integral: |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1171 |
assumes \<nu>: "measure_space (M\<lparr>measure := \<nu>\<rparr>)" "absolutely_continuous \<nu>" |
40859 | 1172 |
and f: "f \<in> borel_measurable M" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1173 |
shows "integral\<^isup>P (M\<lparr>measure := \<nu>\<rparr>) f = (\<integral>\<^isup>+x. RN_deriv M \<nu> x * f x \<partial>M)" |
40859 | 1174 |
proof - |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1175 |
interpret \<nu>: measure_space "M\<lparr>measure := \<nu>\<rparr>" by fact |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1176 |
note RN = RN_deriv[OF \<nu>] |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1177 |
have "integral\<^isup>P (M\<lparr>measure := \<nu>\<rparr>) f = (\<integral>\<^isup>+x. max 0 (f x) \<partial>M\<lparr>measure := \<nu>\<rparr>)" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1178 |
unfolding positive_integral_max_0 .. |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1179 |
also have "(\<integral>\<^isup>+x. max 0 (f x) \<partial>M\<lparr>measure := \<nu>\<rparr>) = |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1180 |
(\<integral>\<^isup>+x. max 0 (f x) \<partial>M\<lparr>measure := \<lambda>A. (\<integral>\<^isup>+x. RN_deriv M \<nu> x * indicator A x \<partial>M)\<rparr>)" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1181 |
by (intro \<nu>.positive_integral_cong_measure[symmetric]) (simp_all add: RN(2)) |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1182 |
also have "\<dots> = (\<integral>\<^isup>+x. RN_deriv M \<nu> x * max 0 (f x) \<partial>M)" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1183 |
by (intro positive_integral_translated_density) (auto simp add: RN f) |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1184 |
also have "\<dots> = (\<integral>\<^isup>+x. RN_deriv M \<nu> x * f x \<partial>M)" |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1185 |
using RN_deriv(3)[OF \<nu>] |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1186 |
by (auto intro!: positive_integral_cong_pos split: split_if_asm |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1187 |
simp: max_def extreal_mult_le_0_iff) |
40859 | 1188 |
finally show ?thesis . |
1189 |
qed |
|
1190 |
||
1191 |
lemma (in sigma_finite_measure) RN_deriv_unique: |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1192 |
assumes \<nu>: "measure_space (M\<lparr>measure := \<nu>\<rparr>)" "absolutely_continuous \<nu>" |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1193 |
and f: "f \<in> borel_measurable M" "AE x. 0 \<le> f x" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1194 |
and eq: "\<And>A. A \<in> sets M \<Longrightarrow> \<nu> A = (\<integral>\<^isup>+x. f x * indicator A x \<partial>M)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1195 |
shows "AE x. f x = RN_deriv M \<nu> x" |
40859 | 1196 |
proof (rule density_unique[OF f RN_deriv(1)[OF \<nu>]]) |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1197 |
show "AE x. 0 \<le> RN_deriv M \<nu> x" using RN_deriv[OF \<nu>] by auto |
40859 | 1198 |
fix A assume A: "A \<in> sets M" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1199 |
show "(\<integral>\<^isup>+x. f x * indicator A x \<partial>M) = (\<integral>\<^isup>+x. RN_deriv M \<nu> x * indicator A x \<partial>M)" |
40859 | 1200 |
unfolding eq[OF A, symmetric] RN_deriv(2)[OF \<nu> A, symmetric] .. |
1201 |
qed |
|
1202 |
||
41832 | 1203 |
lemma (in sigma_finite_measure) RN_deriv_vimage: |
1204 |
assumes T: "T \<in> measure_preserving M M'" |
|
1205 |
and T': "T' \<in> measure_preserving (M'\<lparr> measure := \<nu>' \<rparr>) (M\<lparr> measure := \<nu> \<rparr>)" |
|
1206 |
and inv: "\<And>x. x \<in> space M \<Longrightarrow> T' (T x) = x" |
|
1207 |
and \<nu>': "measure_space (M'\<lparr>measure := \<nu>'\<rparr>)" "measure_space.absolutely_continuous M' \<nu>'" |
|
1208 |
shows "AE x. RN_deriv M' \<nu>' (T x) = RN_deriv M \<nu> x" |
|
1209 |
proof (rule RN_deriv_unique) |
|
1210 |
interpret \<nu>': measure_space "M'\<lparr>measure := \<nu>'\<rparr>" by fact |
|
1211 |
show "measure_space (M\<lparr> measure := \<nu>\<rparr>)" |
|
1212 |
by (rule \<nu>'.measure_space_vimage[OF _ T'], simp) default |
|
1213 |
interpret M': measure_space M' |
|
1214 |
proof (rule measure_space_vimage) |
|
1215 |
have "sigma_algebra (M'\<lparr> measure := \<nu>'\<rparr>)" by default |
|
1216 |
then show "sigma_algebra M'" by simp |
|
1217 |
qed fact |
|
1218 |
show "absolutely_continuous \<nu>" unfolding absolutely_continuous_def |
|
1219 |
proof safe |
|
1220 |
fix N assume N: "N \<in> sets M" and N_0: "\<mu> N = 0" |
|
1221 |
then have N': "T' -` N \<inter> space M' \<in> sets M'" |
|
1222 |
using T' by (auto simp: measurable_def measure_preserving_def) |
|
1223 |
have "T -` (T' -` N \<inter> space M') \<inter> space M = N" |
|
1224 |
using inv T N sets_into_space[OF N] by (auto simp: measurable_def measure_preserving_def) |
|
1225 |
then have "measure M' (T' -` N \<inter> space M') = 0" |
|
1226 |
using measure_preservingD[OF T N'] N_0 by auto |
|
1227 |
with \<nu>'(2) N' show "\<nu> N = 0" using measure_preservingD[OF T', of N] N |
|
1228 |
unfolding M'.absolutely_continuous_def measurable_def by auto |
|
1229 |
qed |
|
1230 |
interpret M': sigma_finite_measure M' |
|
1231 |
proof |
|
1232 |
from sigma_finite guess F .. note F = this |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1233 |
show "\<exists>A::nat \<Rightarrow> 'c set. range A \<subseteq> sets M' \<and> (\<Union>i. A i) = space M' \<and> (\<forall>i. M'.\<mu> (A i) \<noteq> \<infinity>)" |
41832 | 1234 |
proof (intro exI conjI allI) |
1235 |
show *: "range (\<lambda>i. T' -` F i \<inter> space M') \<subseteq> sets M'" |
|
1236 |
using F T' by (auto simp: measurable_def measure_preserving_def) |
|
1237 |
show "(\<Union>i. T' -` F i \<inter> space M') = space M'" |
|
1238 |
using F T' by (force simp: measurable_def measure_preserving_def) |
|
1239 |
fix i |
|
1240 |
have "T' -` F i \<inter> space M' \<in> sets M'" using * by auto |
|
1241 |
note measure_preservingD[OF T this, symmetric] |
|
1242 |
moreover |
|
1243 |
have Fi: "F i \<in> sets M" using F by auto |
|
1244 |
then have "T -` (T' -` F i \<inter> space M') \<inter> space M = F i" |
|
1245 |
using T inv sets_into_space[OF Fi] |
|
1246 |
by (auto simp: measurable_def measure_preserving_def) |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1247 |
ultimately show "measure M' (T' -` F i \<inter> space M') \<noteq> \<infinity>" |
41832 | 1248 |
using F by simp |
1249 |
qed |
|
1250 |
qed |
|
1251 |
have "(RN_deriv M' \<nu>') \<circ> T \<in> borel_measurable M" |
|
1252 |
by (intro measurable_comp[where b=M'] M'.RN_deriv(1) measure_preservingD2[OF T]) fact+ |
|
1253 |
then show "(\<lambda>x. RN_deriv M' \<nu>' (T x)) \<in> borel_measurable M" |
|
1254 |
by (simp add: comp_def) |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1255 |
show "AE x. 0 \<le> RN_deriv M' \<nu>' (T x)" using M'.RN_deriv(3)[OF \<nu>'] by auto |
41832 | 1256 |
fix A let ?A = "T' -` A \<inter> space M'" |
1257 |
assume A: "A \<in> sets M" |
|
1258 |
then have A': "?A \<in> sets M'" using T' unfolding measurable_def measure_preserving_def |
|
1259 |
by auto |
|
1260 |
from A have "\<nu> A = \<nu>' ?A" using T'[THEN measure_preservingD] by simp |
|
1261 |
also have "\<dots> = \<integral>\<^isup>+ x. RN_deriv M' \<nu>' x * indicator ?A x \<partial>M'" |
|
1262 |
using A' by (rule M'.RN_deriv(2)[OF \<nu>']) |
|
1263 |
also have "\<dots> = \<integral>\<^isup>+ x. RN_deriv M' \<nu>' (T x) * indicator ?A (T x) \<partial>M" |
|
1264 |
proof (rule positive_integral_vimage) |
|
1265 |
show "sigma_algebra M'" by default |
|
1266 |
show "(\<lambda>x. RN_deriv M' \<nu>' x * indicator (T' -` A \<inter> space M') x) \<in> borel_measurable M'" |
|
1267 |
by (auto intro!: A' M'.RN_deriv(1)[OF \<nu>']) |
|
1268 |
qed fact |
|
1269 |
also have "\<dots> = \<integral>\<^isup>+ x. RN_deriv M' \<nu>' (T x) * indicator A x \<partial>M" |
|
1270 |
using T inv by (auto intro!: positive_integral_cong simp: measure_preserving_def measurable_def indicator_def) |
|
1271 |
finally show "\<nu> A = \<integral>\<^isup>+ x. RN_deriv M' \<nu>' (T x) * indicator A x \<partial>M" . |
|
1272 |
qed |
|
1273 |
||
40859 | 1274 |
lemma (in sigma_finite_measure) RN_deriv_finite: |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1275 |
assumes sfm: "sigma_finite_measure (M\<lparr>measure := \<nu>\<rparr>)" and ac: "absolutely_continuous \<nu>" |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1276 |
shows "AE x. RN_deriv M \<nu> x \<noteq> \<infinity>" |
40859 | 1277 |
proof - |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1278 |
interpret \<nu>: sigma_finite_measure "M\<lparr>measure := \<nu>\<rparr>" by fact |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1279 |
have \<nu>: "measure_space (M\<lparr>measure := \<nu>\<rparr>)" by default |
40859 | 1280 |
from sfm show ?thesis |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1281 |
using sigma_finite_iff_density_finite[OF \<nu> RN_deriv(1)[OF \<nu> ac]] RN_deriv(2,3)[OF \<nu> ac] by simp |
40859 | 1282 |
qed |
1283 |
||
1284 |
lemma (in sigma_finite_measure) |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1285 |
assumes \<nu>: "sigma_finite_measure (M\<lparr>measure := \<nu>\<rparr>)" "absolutely_continuous \<nu>" |
40859 | 1286 |
and f: "f \<in> borel_measurable M" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1287 |
shows RN_deriv_integrable: "integrable (M\<lparr>measure := \<nu>\<rparr>) f \<longleftrightarrow> |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1288 |
integrable M (\<lambda>x. real (RN_deriv M \<nu> x) * f x)" (is ?integrable) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1289 |
and RN_deriv_integral: "integral\<^isup>L (M\<lparr>measure := \<nu>\<rparr>) f = |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1290 |
(\<integral>x. real (RN_deriv M \<nu> x) * f x \<partial>M)" (is ?integral) |
40859 | 1291 |
proof - |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1292 |
interpret \<nu>: sigma_finite_measure "M\<lparr>measure := \<nu>\<rparr>" by fact |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1293 |
have ms: "measure_space (M\<lparr>measure := \<nu>\<rparr>)" by default |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1294 |
have minus_cong: "\<And>A B A' B'::extreal. A = A' \<Longrightarrow> B = B' \<Longrightarrow> real A - real B = real A' - real B'" by simp |
40859 | 1295 |
have f': "(\<lambda>x. - f x) \<in> borel_measurable M" using f by auto |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1296 |
have Nf: "f \<in> borel_measurable (M\<lparr>measure := \<nu>\<rparr>)" using f by simp |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1297 |
{ fix f :: "'a \<Rightarrow> real" |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1298 |
{ fix x assume *: "RN_deriv M \<nu> x \<noteq> \<infinity>" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1299 |
have "extreal (real (RN_deriv M \<nu> x)) * extreal (f x) = extreal (real (RN_deriv M \<nu> x) * f x)" |
40859 | 1300 |
by (simp add: mult_le_0_iff) |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1301 |
then have "RN_deriv M \<nu> x * extreal (f x) = extreal (real (RN_deriv M \<nu> x) * f x)" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1302 |
using RN_deriv(3)[OF ms \<nu>(2)] * by (auto simp add: extreal_real split: split_if_asm) } |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1303 |
then have "(\<integral>\<^isup>+x. extreal (real (RN_deriv M \<nu> x) * f x) \<partial>M) = (\<integral>\<^isup>+x. RN_deriv M \<nu> x * extreal (f x) \<partial>M)" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1304 |
"(\<integral>\<^isup>+x. extreal (- (real (RN_deriv M \<nu> x) * f x)) \<partial>M) = (\<integral>\<^isup>+x. RN_deriv M \<nu> x * extreal (- f x) \<partial>M)" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1305 |
using RN_deriv_finite[OF \<nu>] unfolding extreal_mult_minus_right uminus_extreal.simps(1)[symmetric] |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1306 |
by (auto intro!: positive_integral_cong_AE) } |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1307 |
note * = this |
40859 | 1308 |
show ?integral ?integrable |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1309 |
unfolding lebesgue_integral_def integrable_def * |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1310 |
using f RN_deriv(1)[OF ms \<nu>(2)] |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1311 |
by (auto simp: RN_deriv_positive_integral[OF ms \<nu>(2)]) |
40859 | 1312 |
qed |
1313 |
||
38656 | 1314 |
lemma (in sigma_finite_measure) RN_deriv_singleton: |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1315 |
assumes "measure_space (M\<lparr>measure := \<nu>\<rparr>)" |
38656 | 1316 |
and ac: "absolutely_continuous \<nu>" |
1317 |
and "{x} \<in> sets M" |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1318 |
shows "\<nu> {x} = RN_deriv M \<nu> x * \<mu> {x}" |
38656 | 1319 |
proof - |
1320 |
note deriv = RN_deriv[OF assms(1, 2)] |
|
1321 |
from deriv(2)[OF `{x} \<in> sets M`] |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1322 |
have "\<nu> {x} = (\<integral>\<^isup>+w. RN_deriv M \<nu> x * indicator {x} w \<partial>M)" |
38656 | 1323 |
by (auto simp: indicator_def intro!: positive_integral_cong) |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41832
diff
changeset
|
1324 |
thus ?thesis using positive_integral_cmult_indicator[OF _ `{x} \<in> sets M`] deriv(3) |
38656 | 1325 |
by auto |
1326 |
qed |
|
1327 |
||
1328 |
theorem (in finite_measure_space) RN_deriv_finite_measure: |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1329 |
assumes "measure_space (M\<lparr>measure := \<nu>\<rparr>)" |
38656 | 1330 |
and ac: "absolutely_continuous \<nu>" |
1331 |
and "x \<in> space M" |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1332 |
shows "\<nu> {x} = RN_deriv M \<nu> x * \<mu> {x}" |
38656 | 1333 |
proof - |
1334 |
have "{x} \<in> sets M" using sets_eq_Pow `x \<in> space M` by auto |
|
1335 |
from RN_deriv_singleton[OF assms(1,2) this] show ?thesis . |
|
1336 |
qed |
|
1337 |
||
1338 |
end |