author | wenzelm |
Tue, 21 Jun 2022 15:56:31 +0200 | |
changeset 75575 | 06f8b072f28e |
parent 74362 | 0135a0c77b64 |
permissions | -rw-r--r-- |
63627 | 1 |
(* Title: HOL/Analysis/Caratheodory.thy |
42067 | 2 |
Author: Lawrence C Paulson |
3 |
Author: Johannes Hölzl, TU München |
|
4 |
*) |
|
5 |
||
69722
b5163b2132c5
minor tagging updates in 13 theories
Angeliki KoutsoukouArgyraki <ak2110@cam.ac.uk>
parents:
69712
diff
changeset
|
6 |
section \<open>Caratheodory Extension Theorem\<close> |
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
7 |
|
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
8 |
theory Caratheodory |
69517 | 9 |
imports Measure_Space |
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
10 |
begin |
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
11 |
|
61808 | 12 |
text \<open> |
42067 | 13 |
Originally from the Hurd/Coble measure theory development, translated by Lawrence Paulson. |
61808 | 14 |
\<close> |
42067 | 15 |
|
69652
3417a8f154eb
updated tagging first 5
Angeliki KoutsoukouArgyraki <ak2110@cam.ac.uk>
parents:
69546
diff
changeset
|
16 |
lemma suminf_ennreal_2dimen: |
62975
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
17 |
fixes f:: "nat \<times> nat \<Rightarrow> ennreal" |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41689
diff
changeset
|
18 |
assumes "\<And>m. g m = (\<Sum>n. f (m,n))" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41689
diff
changeset
|
19 |
shows "(\<Sum>i. f (prod_decode i)) = suminf g" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41689
diff
changeset
|
20 |
proof - |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41689
diff
changeset
|
21 |
have g_def: "g = (\<lambda>m. (\<Sum>n. f (m,n)))" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41689
diff
changeset
|
22 |
using assms by (simp add: fun_eq_iff) |
64267 | 23 |
have reindex: "\<And>B. (\<Sum>x\<in>B. f (prod_decode x)) = sum f (prod_decode ` B)" |
24 |
by (simp add: sum.reindex[OF inj_prod_decode] comp_def) |
|
69260
0a9688695a1b
removed relics of ASCII syntax for indexed big operators
haftmann
parents:
69164
diff
changeset
|
25 |
have "(SUP n. \<Sum>i<n. f (prod_decode i)) = (SUP p \<in> UNIV \<times> UNIV. \<Sum>i<fst p. \<Sum>n<snd p. f (i, n))" |
64267 | 26 |
proof (intro SUP_eq; clarsimp simp: sum.cartesian_product reindex) |
62975
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
27 |
fix n |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41689
diff
changeset
|
28 |
let ?M = "\<lambda>f. Suc (Max (f ` prod_decode ` {..<n}))" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41689
diff
changeset
|
29 |
{ fix a b x assume "x < n" and [symmetric]: "(a, b) = prod_decode x" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41689
diff
changeset
|
30 |
then have "a < ?M fst" "b < ?M snd" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41689
diff
changeset
|
31 |
by (auto intro!: Max_ge le_imp_less_Suc image_eqI) } |
64267 | 32 |
then have "sum f (prod_decode ` {..<n}) \<le> sum f ({..<?M fst} \<times> {..<?M snd})" |
65680
378a2f11bec9
Simplification of some proofs. Also key lemmas using !! rather than ! in premises
paulson <lp15@cam.ac.uk>
parents:
64267
diff
changeset
|
33 |
by (auto intro!: sum_mono2) |
64267 | 34 |
then show "\<exists>a b. sum f (prod_decode ` {..<n}) \<le> sum f ({..<a} \<times> {..<b})" by auto |
62975
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
35 |
next |
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
36 |
fix a b |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41689
diff
changeset
|
37 |
let ?M = "prod_decode ` {..<Suc (Max (prod_encode ` ({..<a} \<times> {..<b})))}" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41689
diff
changeset
|
38 |
{ fix a' b' assume "a' < a" "b' < b" then have "(a', b') \<in> ?M" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41689
diff
changeset
|
39 |
by (auto intro!: Max_ge le_imp_less_Suc image_eqI[where x="prod_encode (a', b')"]) } |
64267 | 40 |
then have "sum f ({..<a} \<times> {..<b}) \<le> sum f ?M" |
65680
378a2f11bec9
Simplification of some proofs. Also key lemmas using !! rather than ! in premises
paulson <lp15@cam.ac.uk>
parents:
64267
diff
changeset
|
41 |
by (auto intro!: sum_mono2) |
64267 | 42 |
then show "\<exists>n. sum f ({..<a} \<times> {..<b}) \<le> sum f (prod_decode ` {..<n})" |
62975
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
43 |
by auto |
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
44 |
qed |
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
45 |
also have "\<dots> = (SUP p. \<Sum>i<p. \<Sum>n. f (i, n))" |
64267 | 46 |
unfolding suminf_sum[OF summableI, symmetric] |
66804
3f9bb52082c4
avoid name clashes on interpretation of abstract locales
haftmann
parents:
65680
diff
changeset
|
47 |
by (simp add: suminf_eq_SUP SUP_pair sum.swap[of _ "{..< fst _}"]) |
62975
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
48 |
finally show ?thesis unfolding g_def |
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
49 |
by (simp add: suminf_eq_SUP) |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41689
diff
changeset
|
50 |
qed |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41689
diff
changeset
|
51 |
|
69683 | 52 |
subsection \<open>Characterizations of Measures\<close> |
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
53 |
|
70136 | 54 |
definition\<^marker>\<open>tag important\<close> outer_measure_space where |
61273 | 55 |
"outer_measure_space M f \<longleftrightarrow> positive M f \<and> increasing M f \<and> countably_subadditive M f" |
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
56 |
|
70136 | 57 |
subsubsection\<^marker>\<open>tag important\<close> \<open>Lambda Systems\<close> |
56994 | 58 |
|
70136 | 59 |
definition\<^marker>\<open>tag important\<close> lambda_system :: "'a set \<Rightarrow> 'a set set \<Rightarrow> ('a set \<Rightarrow> ennreal) \<Rightarrow> 'a set set" |
62975
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
60 |
where |
61273 | 61 |
"lambda_system \<Omega> M f = {l \<in> M. \<forall>x \<in> M. f (l \<inter> x) + f ((\<Omega> - l) \<inter> x) = f x}" |
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
62 |
|
69652
3417a8f154eb
updated tagging first 5
Angeliki KoutsoukouArgyraki <ak2110@cam.ac.uk>
parents:
69546
diff
changeset
|
63 |
lemma (in algebra) lambda_system_eq: |
61273 | 64 |
"lambda_system \<Omega> M f = {l \<in> M. \<forall>x \<in> M. f (x \<inter> l) + f (x - l) = f x}" |
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
65 |
proof - |
61273 | 66 |
have [simp]: "\<And>l x. l \<in> M \<Longrightarrow> x \<in> M \<Longrightarrow> (\<Omega> - l) \<inter> x = x - l" |
37032 | 67 |
by (metis Int_Diff Int_absorb1 Int_commute sets_into_space) |
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
68 |
show ?thesis |
37032 | 69 |
by (auto simp add: lambda_system_def) (metis Int_commute)+ |
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
70 |
qed |
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
71 |
|
69652
3417a8f154eb
updated tagging first 5
Angeliki KoutsoukouArgyraki <ak2110@cam.ac.uk>
parents:
69546
diff
changeset
|
72 |
lemma (in algebra) lambda_system_empty: "positive M f \<Longrightarrow> {} \<in> lambda_system \<Omega> M f" |
42066
6db76c88907a
generalized Caratheodory from algebra to ring_of_sets
hoelzl
parents:
42065
diff
changeset
|
73 |
by (auto simp add: positive_def lambda_system_eq) |
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
74 |
|
69652
3417a8f154eb
updated tagging first 5
Angeliki KoutsoukouArgyraki <ak2110@cam.ac.uk>
parents:
69546
diff
changeset
|
75 |
lemma lambda_system_sets: "x \<in> lambda_system \<Omega> M f \<Longrightarrow> x \<in> M" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
76 |
by (simp add: lambda_system_def) |
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
77 |
|
69652
3417a8f154eb
updated tagging first 5
Angeliki KoutsoukouArgyraki <ak2110@cam.ac.uk>
parents:
69546
diff
changeset
|
78 |
lemma (in algebra) lambda_system_Compl: |
62975
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
79 |
fixes f:: "'a set \<Rightarrow> ennreal" |
47694 | 80 |
assumes x: "x \<in> lambda_system \<Omega> M f" |
81 |
shows "\<Omega> - x \<in> lambda_system \<Omega> M f" |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
82 |
proof - |
47694 | 83 |
have "x \<subseteq> \<Omega>" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
84 |
by (metis sets_into_space lambda_system_sets x) |
47694 | 85 |
hence "\<Omega> - (\<Omega> - x) = x" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
86 |
by (metis double_diff equalityE) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
87 |
with x show ?thesis |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
88 |
by (force simp add: lambda_system_def ac_simps) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
89 |
qed |
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
90 |
|
69652
3417a8f154eb
updated tagging first 5
Angeliki KoutsoukouArgyraki <ak2110@cam.ac.uk>
parents:
69546
diff
changeset
|
91 |
lemma (in algebra) lambda_system_Int: |
62975
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
92 |
fixes f:: "'a set \<Rightarrow> ennreal" |
47694 | 93 |
assumes xl: "x \<in> lambda_system \<Omega> M f" and yl: "y \<in> lambda_system \<Omega> M f" |
94 |
shows "x \<inter> y \<in> lambda_system \<Omega> M f" |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
95 |
proof - |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
96 |
from xl yl show ?thesis |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
97 |
proof (auto simp add: positive_def lambda_system_eq Int) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
98 |
fix u |
47694 | 99 |
assume x: "x \<in> M" and y: "y \<in> M" and u: "u \<in> M" |
100 |
and fx: "\<forall>z\<in>M. f (z \<inter> x) + f (z - x) = f z" |
|
101 |
and fy: "\<forall>z\<in>M. f (z \<inter> y) + f (z - y) = f z" |
|
102 |
have "u - x \<inter> y \<in> M" |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
103 |
by (metis Diff Diff_Int Un u x y) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
104 |
moreover |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
105 |
have "(u - (x \<inter> y)) \<inter> y = u \<inter> y - x" by blast |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
106 |
moreover |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
107 |
have "u - x \<inter> y - y = u - y" by blast |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
108 |
ultimately |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
109 |
have ey: "f (u - x \<inter> y) = f (u \<inter> y - x) + f (u - y)" using fy |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
110 |
by force |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
111 |
have "f (u \<inter> (x \<inter> y)) + f (u - x \<inter> y) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
112 |
= (f (u \<inter> (x \<inter> y)) + f (u \<inter> y - x)) + f (u - y)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
113 |
by (simp add: ey ac_simps) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
114 |
also have "... = (f ((u \<inter> y) \<inter> x) + f (u \<inter> y - x)) + f (u - y)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
115 |
by (simp add: Int_ac) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
116 |
also have "... = f (u \<inter> y) + f (u - y)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
117 |
using fx [THEN bspec, of "u \<inter> y"] Int y u |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
118 |
by force |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
119 |
also have "... = f u" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
120 |
by (metis fy u) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
121 |
finally show "f (u \<inter> (x \<inter> y)) + f (u - x \<inter> y) = f u" . |
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
122 |
qed |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
123 |
qed |
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
124 |
|
69652
3417a8f154eb
updated tagging first 5
Angeliki KoutsoukouArgyraki <ak2110@cam.ac.uk>
parents:
69546
diff
changeset
|
125 |
lemma (in algebra) lambda_system_Un: |
62975
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
126 |
fixes f:: "'a set \<Rightarrow> ennreal" |
47694 | 127 |
assumes xl: "x \<in> lambda_system \<Omega> M f" and yl: "y \<in> lambda_system \<Omega> M f" |
128 |
shows "x \<union> y \<in> lambda_system \<Omega> M f" |
|
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
129 |
proof - |
47694 | 130 |
have "(\<Omega> - x) \<inter> (\<Omega> - y) \<in> M" |
38656 | 131 |
by (metis Diff_Un Un compl_sets lambda_system_sets xl yl) |
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
132 |
moreover |
47694 | 133 |
have "x \<union> y = \<Omega> - ((\<Omega> - x) \<inter> (\<Omega> - y))" |
46731 | 134 |
by auto (metis subsetD lambda_system_sets sets_into_space xl yl)+ |
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
135 |
ultimately show ?thesis |
38656 | 136 |
by (metis lambda_system_Compl lambda_system_Int xl yl) |
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
137 |
qed |
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
138 |
|
69652
3417a8f154eb
updated tagging first 5
Angeliki KoutsoukouArgyraki <ak2110@cam.ac.uk>
parents:
69546
diff
changeset
|
139 |
lemma (in algebra) lambda_system_algebra: |
47694 | 140 |
"positive M f \<Longrightarrow> algebra \<Omega> (lambda_system \<Omega> M f)" |
42065
2b98b4c2e2f1
add ring_of_sets and subset_class as basis for algebra
hoelzl
parents:
41981
diff
changeset
|
141 |
apply (auto simp add: algebra_iff_Un) |
69712 | 142 |
apply (metis lambda_system_sets subsetD sets_into_space) |
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
143 |
apply (metis lambda_system_empty) |
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
144 |
apply (metis lambda_system_Compl) |
38656 | 145 |
apply (metis lambda_system_Un) |
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
146 |
done |
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
147 |
|
69652
3417a8f154eb
updated tagging first 5
Angeliki KoutsoukouArgyraki <ak2110@cam.ac.uk>
parents:
69546
diff
changeset
|
148 |
lemma (in algebra) lambda_system_strong_additive: |
47694 | 149 |
assumes z: "z \<in> M" and disj: "x \<inter> y = {}" |
150 |
and xl: "x \<in> lambda_system \<Omega> M f" and yl: "y \<in> lambda_system \<Omega> M f" |
|
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
151 |
shows "f (z \<inter> (x \<union> y)) = f (z \<inter> x) + f (z \<inter> y)" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
152 |
proof - |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
153 |
have "z \<inter> x = (z \<inter> (x \<union> y)) \<inter> x" using disj by blast |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
154 |
moreover |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
155 |
have "z \<inter> y = (z \<inter> (x \<union> y)) - x" using disj by blast |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
156 |
moreover |
47694 | 157 |
have "(z \<inter> (x \<union> y)) \<in> M" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
158 |
by (metis Int Un lambda_system_sets xl yl z) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
159 |
ultimately show ?thesis using xl yl |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
160 |
by (simp add: lambda_system_eq) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
161 |
qed |
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
162 |
|
69652
3417a8f154eb
updated tagging first 5
Angeliki KoutsoukouArgyraki <ak2110@cam.ac.uk>
parents:
69546
diff
changeset
|
163 |
lemma (in algebra) lambda_system_additive: "additive (lambda_system \<Omega> M f) f" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
164 |
proof (auto simp add: additive_def) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
165 |
fix x and y |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
166 |
assume disj: "x \<inter> y = {}" |
47694 | 167 |
and xl: "x \<in> lambda_system \<Omega> M f" and yl: "y \<in> lambda_system \<Omega> M f" |
168 |
hence "x \<in> M" "y \<in> M" by (blast intro: lambda_system_sets)+ |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
169 |
thus "f (x \<union> y) = f x + f y" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
170 |
using lambda_system_strong_additive [OF top disj xl yl] |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
171 |
by (simp add: Un) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
172 |
qed |
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
173 |
|
69652
3417a8f154eb
updated tagging first 5
Angeliki KoutsoukouArgyraki <ak2110@cam.ac.uk>
parents:
69546
diff
changeset
|
174 |
lemma lambda_system_increasing: "increasing M f \<Longrightarrow> increasing (lambda_system \<Omega> M f) f" |
38656 | 175 |
by (simp add: increasing_def lambda_system_def) |
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
176 |
|
69652
3417a8f154eb
updated tagging first 5
Angeliki KoutsoukouArgyraki <ak2110@cam.ac.uk>
parents:
69546
diff
changeset
|
177 |
lemma lambda_system_positive: "positive M f \<Longrightarrow> positive (lambda_system \<Omega> M f) f" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
178 |
by (simp add: positive_def lambda_system_def) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
179 |
|
69652
3417a8f154eb
updated tagging first 5
Angeliki KoutsoukouArgyraki <ak2110@cam.ac.uk>
parents:
69546
diff
changeset
|
180 |
lemma (in algebra) lambda_system_strong_sum: |
62975
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
181 |
fixes A:: "nat \<Rightarrow> 'a set" and f :: "'a set \<Rightarrow> ennreal" |
47694 | 182 |
assumes f: "positive M f" and a: "a \<in> M" |
183 |
and A: "range A \<subseteq> lambda_system \<Omega> M f" |
|
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
184 |
and disj: "disjoint_family A" |
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
185 |
shows "(\<Sum>i = 0..<n. f (a \<inter>A i)) = f (a \<inter> (\<Union>i\<in>{0..<n}. A i))" |
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
186 |
proof (induct n) |
38656 | 187 |
case 0 show ?case using f by (simp add: positive_def) |
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
188 |
next |
38656 | 189 |
case (Suc n) |
69325 | 190 |
have 2: "A n \<inter> \<Union> (A ` {0..<n}) = {}" using disj |
38656 | 191 |
by (force simp add: disjoint_family_on_def neq_iff) |
47694 | 192 |
have 3: "A n \<in> lambda_system \<Omega> M f" using A |
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
193 |
by blast |
47694 | 194 |
interpret l: algebra \<Omega> "lambda_system \<Omega> M f" |
42065
2b98b4c2e2f1
add ring_of_sets and subset_class as basis for algebra
hoelzl
parents:
41981
diff
changeset
|
195 |
using f by (rule lambda_system_algebra) |
69325 | 196 |
have 4: "\<Union> (A ` {0..<n}) \<in> lambda_system \<Omega> M f" |
42065
2b98b4c2e2f1
add ring_of_sets and subset_class as basis for algebra
hoelzl
parents:
41981
diff
changeset
|
197 |
using A l.UNION_in_sets by simp |
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
198 |
from Suc.hyps show ?case |
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
199 |
by (simp add: atLeastLessThanSuc lambda_system_strong_additive [OF a 2 3 4]) |
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
200 |
qed |
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
201 |
|
69652
3417a8f154eb
updated tagging first 5
Angeliki KoutsoukouArgyraki <ak2110@cam.ac.uk>
parents:
69546
diff
changeset
|
202 |
proposition (in sigma_algebra) lambda_system_caratheodory: |
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
203 |
assumes oms: "outer_measure_space M f" |
47694 | 204 |
and A: "range A \<subseteq> lambda_system \<Omega> M f" |
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
205 |
and disj: "disjoint_family A" |
47694 | 206 |
shows "(\<Union>i. A i) \<in> lambda_system \<Omega> M f \<and> (\<Sum>i. f (A i)) = f (\<Union>i. A i)" |
69652
3417a8f154eb
updated tagging first 5
Angeliki KoutsoukouArgyraki <ak2110@cam.ac.uk>
parents:
69546
diff
changeset
|
207 |
proof - |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
208 |
have pos: "positive M f" and inc: "increasing M f" |
38656 | 209 |
and csa: "countably_subadditive M f" |
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
210 |
by (metis oms outer_measure_space_def)+ |
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
211 |
have sa: "subadditive M f" |
38656 | 212 |
by (metis countably_subadditive_subadditive csa pos) |
47694 | 213 |
have A': "\<And>S. A`S \<subseteq> (lambda_system \<Omega> M f)" using A |
214 |
by auto |
|
215 |
interpret ls: algebra \<Omega> "lambda_system \<Omega> M f" |
|
42065
2b98b4c2e2f1
add ring_of_sets and subset_class as basis for algebra
hoelzl
parents:
41981
diff
changeset
|
216 |
using pos by (rule lambda_system_algebra) |
47694 | 217 |
have A'': "range A \<subseteq> M" |
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
218 |
by (metis A image_subset_iff lambda_system_sets) |
38656 | 219 |
|
47694 | 220 |
have U_in: "(\<Union>i. A i) \<in> M" |
37032 | 221 |
by (metis A'' countable_UN) |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41689
diff
changeset
|
222 |
have U_eq: "f (\<Union>i. A i) = (\<Sum>i. f (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:
41023
diff
changeset
|
223 |
proof (rule antisym) |
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41689
diff
changeset
|
224 |
show "f (\<Union>i. A i) \<le> (\<Sum>i. f (A i))" |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41689
diff
changeset
|
225 |
using csa[unfolded countably_subadditive_def] A'' disj U_in by auto |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41689
diff
changeset
|
226 |
have dis: "\<And>N. disjoint_family_on A {..<N}" by (intro disjoint_family_on_mono[OF _ disj]) auto |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41689
diff
changeset
|
227 |
show "(\<Sum>i. f (A i)) \<le> f (\<Union>i. A i)" |
61273 | 228 |
using ls.additive_sum [OF lambda_system_positive[OF pos] lambda_system_additive _ A' dis] A'' |
62975
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
229 |
by (intro suminf_le_const[OF summableI]) (auto intro!: increasingD[OF inc] 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:
41023
diff
changeset
|
230 |
qed |
61273 | 231 |
have "f (a \<inter> (\<Union>i. A i)) + f (a - (\<Union>i. A i)) = f a" |
232 |
if a [iff]: "a \<in> M" for a |
|
233 |
proof (rule antisym) |
|
234 |
have "range (\<lambda>i. a \<inter> A i) \<subseteq> M" using A'' |
|
235 |
by blast |
|
236 |
moreover |
|
237 |
have "disjoint_family (\<lambda>i. a \<inter> A i)" using disj |
|
238 |
by (auto simp add: disjoint_family_on_def) |
|
239 |
moreover |
|
240 |
have "a \<inter> (\<Union>i. A i) \<in> M" |
|
241 |
by (metis Int U_in a) |
|
242 |
ultimately |
|
243 |
have "f (a \<inter> (\<Union>i. A i)) \<le> (\<Sum>i. f (a \<inter> A i))" |
|
244 |
using csa[unfolded countably_subadditive_def, rule_format, of "(\<lambda>i. a \<inter> A i)"] |
|
245 |
by (simp add: o_def) |
|
246 |
hence "f (a \<inter> (\<Union>i. A i)) + f (a - (\<Union>i. A i)) \<le> (\<Sum>i. f (a \<inter> A i)) + f (a - (\<Union>i. A i))" |
|
247 |
by (rule add_right_mono) |
|
248 |
also have "\<dots> \<le> f a" |
|
62975
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
249 |
proof (intro ennreal_suminf_bound_add) |
61273 | 250 |
fix n |
251 |
have UNION_in: "(\<Union>i\<in>{0..<n}. A i) \<in> M" |
|
252 |
by (metis A'' UNION_in_sets) |
|
69325 | 253 |
have le_fa: "f (\<Union> (A ` {0..<n}) \<inter> a) \<le> f a" using A'' |
61273 | 254 |
by (blast intro: increasingD [OF inc] A'' UNION_in_sets) |
255 |
have ls: "(\<Union>i\<in>{0..<n}. A i) \<in> lambda_system \<Omega> M f" |
|
256 |
using ls.UNION_in_sets by (simp add: A) |
|
257 |
hence eq_fa: "f a = f (a \<inter> (\<Union>i\<in>{0..<n}. A i)) + f (a - (\<Union>i\<in>{0..<n}. A i))" |
|
258 |
by (simp add: lambda_system_eq UNION_in) |
|
259 |
have "f (a - (\<Union>i. A i)) \<le> f (a - (\<Union>i\<in>{0..<n}. A i))" |
|
260 |
by (blast intro: increasingD [OF inc] UNION_in U_in) |
|
261 |
thus "(\<Sum>i<n. f (a \<inter> A i)) + f (a - (\<Union>i. A i)) \<le> f a" |
|
262 |
by (simp add: lambda_system_strong_sum pos A disj eq_fa add_left_mono atLeast0LessThan[symmetric]) |
|
263 |
qed |
|
62975
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
264 |
finally show "f (a \<inter> (\<Union>i. A i)) + f (a - (\<Union>i. A i)) \<le> f a" |
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
265 |
by simp |
61273 | 266 |
next |
267 |
have "f a \<le> f (a \<inter> (\<Union>i. A i) \<union> (a - (\<Union>i. A i)))" |
|
268 |
by (blast intro: increasingD [OF inc] U_in) |
|
269 |
also have "... \<le> f (a \<inter> (\<Union>i. A i)) + f (a - (\<Union>i. A i))" |
|
270 |
by (blast intro: subadditiveD [OF sa] U_in) |
|
271 |
finally show "f a \<le> f (a \<inter> (\<Union>i. A i)) + f (a - (\<Union>i. A i))" . |
|
272 |
qed |
|
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
273 |
thus ?thesis |
38656 | 274 |
by (simp add: lambda_system_eq sums_iff U_eq U_in) |
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
275 |
qed |
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
276 |
|
69652
3417a8f154eb
updated tagging first 5
Angeliki KoutsoukouArgyraki <ak2110@cam.ac.uk>
parents:
69546
diff
changeset
|
277 |
proposition (in sigma_algebra) caratheodory_lemma: |
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
278 |
assumes oms: "outer_measure_space M f" |
47694 | 279 |
defines "L \<equiv> lambda_system \<Omega> M f" |
280 |
shows "measure_space \<Omega> L f" |
|
69652
3417a8f154eb
updated tagging first 5
Angeliki KoutsoukouArgyraki <ak2110@cam.ac.uk>
parents:
69546
diff
changeset
|
281 |
proof - |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
282 |
have pos: "positive M f" |
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
283 |
by (metis oms outer_measure_space_def) |
47694 | 284 |
have alg: "algebra \<Omega> L" |
38656 | 285 |
using lambda_system_algebra [of f, OF pos] |
47694 | 286 |
by (simp add: algebra_iff_Un L_def) |
42065
2b98b4c2e2f1
add ring_of_sets and subset_class as basis for algebra
hoelzl
parents:
41981
diff
changeset
|
287 |
then |
47694 | 288 |
have "sigma_algebra \<Omega> L" |
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
289 |
using lambda_system_caratheodory [OF oms] |
47694 | 290 |
by (simp add: sigma_algebra_disjoint_iff L_def) |
38656 | 291 |
moreover |
47694 | 292 |
have "countably_additive L f" "positive L f" |
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
293 |
using pos lambda_system_caratheodory [OF oms] |
47694 | 294 |
by (auto simp add: lambda_system_sets L_def countably_additive_def positive_def) |
38656 | 295 |
ultimately |
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
296 |
show ?thesis |
47694 | 297 |
using pos by (simp add: measure_space_def) |
38656 | 298 |
qed |
299 |
||
70136 | 300 |
definition\<^marker>\<open>tag important\<close> outer_measure :: "'a set set \<Rightarrow> ('a set \<Rightarrow> ennreal) \<Rightarrow> 'a set \<Rightarrow> ennreal" where |
61273 | 301 |
"outer_measure M f X = |
69260
0a9688695a1b
removed relics of ASCII syntax for indexed big operators
haftmann
parents:
69164
diff
changeset
|
302 |
(INF A\<in>{A. range A \<subseteq> M \<and> disjoint_family A \<and> X \<subseteq> (\<Union>i. A i)}. \<Sum>i. f (A i))" |
39096 | 303 |
|
69652
3417a8f154eb
updated tagging first 5
Angeliki KoutsoukouArgyraki <ak2110@cam.ac.uk>
parents:
69546
diff
changeset
|
304 |
lemma (in ring_of_sets) outer_measure_agrees: |
61273 | 305 |
assumes posf: "positive M f" and ca: "countably_additive M f" and s: "s \<in> M" |
306 |
shows "outer_measure M f s = f s" |
|
307 |
unfolding outer_measure_def |
|
308 |
proof (safe intro!: antisym INF_greatest) |
|
309 |
fix A :: "nat \<Rightarrow> 'a set" assume A: "range A \<subseteq> M" and dA: "disjoint_family A" and sA: "s \<subseteq> (\<Union>x. A x)" |
|
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
310 |
have inc: "increasing M f" |
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
311 |
by (metis additive_increasing ca countably_additive_additive posf) |
61273 | 312 |
have "f s = f (\<Union>i. A i \<inter> s)" |
313 |
using sA by (auto simp: Int_absorb1) |
|
314 |
also have "\<dots> = (\<Sum>i. f (A i \<inter> s))" |
|
315 |
using sA dA A s |
|
316 |
by (intro ca[unfolded countably_additive_def, rule_format, symmetric]) |
|
317 |
(auto simp: Int_absorb1 disjoint_family_on_def) |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41689
diff
changeset
|
318 |
also have "... \<le> (\<Sum>i. f (A i))" |
62975
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
319 |
using A s by (auto intro!: suminf_le increasingD[OF inc]) |
61273 | 320 |
finally show "f s \<le> (\<Sum>i. f (A i))" . |
321 |
next |
|
322 |
have "(\<Sum>i. f (if i = 0 then s else {})) \<le> f s" |
|
323 |
using positiveD1[OF posf] by (subst suminf_finite[of "{0}"]) auto |
|
69313 | 324 |
with s show "(INF A\<in>{A. range A \<subseteq> M \<and> disjoint_family A \<and> s \<subseteq> \<Union>(A ` UNIV)}. \<Sum>i. f (A i)) \<le> f s" |
61273 | 325 |
by (intro INF_lower2[of "\<lambda>i. if i = 0 then s else {}"]) |
326 |
(auto simp: disjoint_family_on_def) |
|
41981
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41689
diff
changeset
|
327 |
qed |
cdf7693bbe08
reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl
parents:
41689
diff
changeset
|
328 |
|
69652
3417a8f154eb
updated tagging first 5
Angeliki KoutsoukouArgyraki <ak2110@cam.ac.uk>
parents:
69546
diff
changeset
|
329 |
lemma outer_measure_empty: |
62975
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
330 |
"positive M f \<Longrightarrow> {} \<in> M \<Longrightarrow> outer_measure M f {} = 0" |
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
331 |
unfolding outer_measure_def |
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
332 |
by (intro antisym INF_lower2[of "\<lambda>_. {}"]) (auto simp: disjoint_family_on_def positive_def) |
61273 | 333 |
|
69652
3417a8f154eb
updated tagging first 5
Angeliki KoutsoukouArgyraki <ak2110@cam.ac.uk>
parents:
69546
diff
changeset
|
334 |
lemma (in ring_of_sets) positive_outer_measure: |
61273 | 335 |
assumes "positive M f" shows "positive (Pow \<Omega>) (outer_measure M f)" |
62975
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
336 |
unfolding positive_def by (auto simp: assms outer_measure_empty) |
61273 | 337 |
|
69652
3417a8f154eb
updated tagging first 5
Angeliki KoutsoukouArgyraki <ak2110@cam.ac.uk>
parents:
69546
diff
changeset
|
338 |
lemma (in ring_of_sets) increasing_outer_measure: "increasing (Pow \<Omega>) (outer_measure M f)" |
61273 | 339 |
by (force simp: increasing_def outer_measure_def intro!: INF_greatest intro: INF_lower) |
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
340 |
|
69652
3417a8f154eb
updated tagging first 5
Angeliki KoutsoukouArgyraki <ak2110@cam.ac.uk>
parents:
69546
diff
changeset
|
341 |
lemma (in ring_of_sets) outer_measure_le: |
61273 | 342 |
assumes pos: "positive M f" and inc: "increasing M f" and A: "range A \<subseteq> M" and X: "X \<subseteq> (\<Union>i. A i)" |
343 |
shows "outer_measure M f X \<le> (\<Sum>i. f (A i))" |
|
344 |
unfolding outer_measure_def |
|
345 |
proof (safe intro!: INF_lower2[of "disjointed A"] del: subsetI) |
|
346 |
show dA: "range (disjointed A) \<subseteq> M" |
|
347 |
by (auto intro!: A range_disjointed_sets) |
|
348 |
have "\<forall>n. f (disjointed A n) \<le> f (A n)" |
|
349 |
by (metis increasingD [OF inc] UNIV_I dA image_subset_iff disjointed_subset A) |
|
62975
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
350 |
then show "(\<Sum>i. f (disjointed A i)) \<le> (\<Sum>i. f (A i))" |
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
351 |
by (blast intro!: suminf_le) |
61273 | 352 |
qed (auto simp: X UN_disjointed_eq disjoint_family_disjointed) |
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
353 |
|
69652
3417a8f154eb
updated tagging first 5
Angeliki KoutsoukouArgyraki <ak2110@cam.ac.uk>
parents:
69546
diff
changeset
|
354 |
lemma (in ring_of_sets) outer_measure_close: |
62975
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
355 |
"outer_measure M f X < e \<Longrightarrow> \<exists>A. range A \<subseteq> M \<and> disjoint_family A \<and> X \<subseteq> (\<Union>i. A i) \<and> (\<Sum>i. f (A i)) < e" |
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
356 |
unfolding outer_measure_def INF_less_iff by auto |
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
357 |
|
69652
3417a8f154eb
updated tagging first 5
Angeliki KoutsoukouArgyraki <ak2110@cam.ac.uk>
parents:
69546
diff
changeset
|
358 |
lemma (in ring_of_sets) countably_subadditive_outer_measure: |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
359 |
assumes posf: "positive M f" and inc: "increasing M f" |
61273 | 360 |
shows "countably_subadditive (Pow \<Omega>) (outer_measure M f)" |
42066
6db76c88907a
generalized Caratheodory from algebra to ring_of_sets
hoelzl
parents:
42065
diff
changeset
|
361 |
proof (simp add: countably_subadditive_def, safe) |
61273 | 362 |
fix A :: "nat \<Rightarrow> _" assume A: "range A \<subseteq> Pow (\<Omega>)" and sb: "(\<Union>i. A i) \<subseteq> \<Omega>" |
363 |
let ?O = "outer_measure M f" |
|
62975
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
364 |
show "?O (\<Union>i. A i) \<le> (\<Sum>n. ?O (A n))" |
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
365 |
proof (rule ennreal_le_epsilon) |
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
366 |
fix b and e :: real assume "0 < e" "(\<Sum>n. outer_measure M f (A n)) < top" |
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
367 |
then have *: "\<And>n. outer_measure M f (A n) < outer_measure M f (A n) + e * (1/2)^Suc n" |
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
368 |
by (auto simp add: less_top dest!: ennreal_suminf_lessD) |
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
369 |
obtain B |
61273 | 370 |
where B: "\<And>n. range (B n) \<subseteq> M" |
371 |
and sbB: "\<And>n. A n \<subseteq> (\<Union>i. B n i)" |
|
372 |
and Ble: "\<And>n. (\<Sum>i. f (B n i)) \<le> ?O (A n) + e * (1/2)^(Suc n)" |
|
62975
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
373 |
by (metis less_imp_le outer_measure_close[OF *]) |
61273 | 374 |
|
63040 | 375 |
define C where "C = case_prod B o prod_decode" |
61273 | 376 |
from B have B_in_M: "\<And>i j. B i j \<in> M" |
61032
b57df8eecad6
standardized some occurences of ancient "split" alias
haftmann
parents:
60585
diff
changeset
|
377 |
by (rule range_subsetD) |
61273 | 378 |
then have C: "range C \<subseteq> M" |
379 |
by (auto simp add: C_def split_def) |
|
380 |
have A_C: "(\<Union>i. A i) \<subseteq> (\<Union>i. C i)" |
|
381 |
using sbB by (auto simp add: C_def subset_eq) (metis prod.case prod_encode_inverse) |
|
42066
6db76c88907a
generalized Caratheodory from algebra to ring_of_sets
hoelzl
parents:
42065
diff
changeset
|
382 |
|
62975
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
383 |
have "?O (\<Union>i. A i) \<le> ?O (\<Union>i. C i)" |
61273 | 384 |
using A_C A C by (intro increasing_outer_measure[THEN increasingD]) (auto dest!: sets_into_space) |
385 |
also have "\<dots> \<le> (\<Sum>i. f (C i))" |
|
386 |
using C by (intro outer_measure_le[OF posf inc]) auto |
|
387 |
also have "\<dots> = (\<Sum>n. \<Sum>i. f (B n i))" |
|
62975
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
388 |
using B_in_M unfolding C_def comp_def by (intro suminf_ennreal_2dimen) auto |
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
389 |
also have "\<dots> \<le> (\<Sum>n. ?O (A n) + e * (1/2) ^ Suc n)" |
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
390 |
using B_in_M by (intro suminf_le suminf_nonneg allI Ble) auto |
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
391 |
also have "... = (\<Sum>n. ?O (A n)) + (\<Sum>n. ennreal e * ennreal ((1/2) ^ Suc n))" |
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
392 |
using \<open>0 < e\<close> by (subst suminf_add[symmetric]) |
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
393 |
(auto simp del: ennreal_suminf_cmult simp add: ennreal_mult[symmetric]) |
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
394 |
also have "\<dots> = (\<Sum>n. ?O (A n)) + e" |
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
395 |
unfolding ennreal_suminf_cmult |
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
396 |
by (subst suminf_ennreal_eq[OF zero_le_power power_half_series]) auto |
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
397 |
finally show "?O (\<Union>i. A i) \<le> (\<Sum>n. ?O (A n)) + e" . |
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
398 |
qed |
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
399 |
qed |
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
400 |
|
69652
3417a8f154eb
updated tagging first 5
Angeliki KoutsoukouArgyraki <ak2110@cam.ac.uk>
parents:
69546
diff
changeset
|
401 |
lemma (in ring_of_sets) outer_measure_space_outer_measure: |
61273 | 402 |
"positive M f \<Longrightarrow> increasing M f \<Longrightarrow> outer_measure_space (Pow \<Omega>) (outer_measure M f)" |
403 |
by (simp add: outer_measure_space_def |
|
404 |
positive_outer_measure increasing_outer_measure countably_subadditive_outer_measure) |
|
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
405 |
|
69652
3417a8f154eb
updated tagging first 5
Angeliki KoutsoukouArgyraki <ak2110@cam.ac.uk>
parents:
69546
diff
changeset
|
406 |
lemma (in ring_of_sets) algebra_subset_lambda_system: |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
407 |
assumes posf: "positive M f" and inc: "increasing M f" |
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
408 |
and add: "additive M f" |
61273 | 409 |
shows "M \<subseteq> lambda_system \<Omega> (Pow \<Omega>) (outer_measure M f)" |
38656 | 410 |
proof (auto dest: sets_into_space |
411 |
simp add: algebra.lambda_system_eq [OF algebra_Pow]) |
|
61273 | 412 |
fix x s assume x: "x \<in> M" and s: "s \<subseteq> \<Omega>" |
413 |
have [simp]: "\<And>x. x \<in> M \<Longrightarrow> s \<inter> (\<Omega> - x) = s - x" using s |
|
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
414 |
by blast |
61273 | 415 |
have "outer_measure M f (s \<inter> x) + outer_measure M f (s - x) \<le> outer_measure M f s" |
416 |
unfolding outer_measure_def[of M f s] |
|
417 |
proof (safe intro!: INF_greatest) |
|
418 |
fix A :: "nat \<Rightarrow> 'a set" assume A: "disjoint_family A" "range A \<subseteq> M" "s \<subseteq> (\<Union>i. A i)" |
|
419 |
have "outer_measure M f (s \<inter> x) \<le> (\<Sum>i. f (A i \<inter> x))" |
|
420 |
unfolding outer_measure_def |
|
421 |
proof (safe intro!: INF_lower2[of "\<lambda>i. A i \<inter> x"]) |
|
422 |
from A(1) show "disjoint_family (\<lambda>i. A i \<inter> x)" |
|
423 |
by (rule disjoint_family_on_bisimulation) auto |
|
424 |
qed (insert x A, auto) |
|
425 |
moreover |
|
426 |
have "outer_measure M f (s - x) \<le> (\<Sum>i. f (A i - x))" |
|
427 |
unfolding outer_measure_def |
|
428 |
proof (safe intro!: INF_lower2[of "\<lambda>i. A i - x"]) |
|
429 |
from A(1) show "disjoint_family (\<lambda>i. A i - x)" |
|
430 |
by (rule disjoint_family_on_bisimulation) auto |
|
431 |
qed (insert x A, auto) |
|
432 |
ultimately have "outer_measure M f (s \<inter> x) + outer_measure M f (s - x) \<le> |
|
433 |
(\<Sum>i. f (A i \<inter> x)) + (\<Sum>i. f (A i - x))" by (rule add_mono) |
|
434 |
also have "\<dots> = (\<Sum>i. f (A i \<inter> x) + f (A i - x))" |
|
62975
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
435 |
using A(2) x posf by (subst suminf_add) (auto simp: positive_def) |
61273 | 436 |
also have "\<dots> = (\<Sum>i. f (A i))" |
437 |
using A x |
|
438 |
by (subst add[THEN additiveD, symmetric]) |
|
439 |
(auto intro!: arg_cong[where f=suminf] arg_cong[where f=f]) |
|
440 |
finally show "outer_measure M f (s \<inter> x) + outer_measure M f (s - x) \<le> (\<Sum>i. f (A i))" . |
|
42066
6db76c88907a
generalized Caratheodory from algebra to ring_of_sets
hoelzl
parents:
42065
diff
changeset
|
441 |
qed |
38656 | 442 |
moreover |
61273 | 443 |
have "outer_measure M f s \<le> outer_measure M f (s \<inter> x) + outer_measure M f (s - x)" |
42145 | 444 |
proof - |
61273 | 445 |
have "outer_measure M f s = outer_measure M f ((s \<inter> x) \<union> (s - x))" |
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
446 |
by (metis Un_Diff_Int Un_commute) |
61273 | 447 |
also have "... \<le> outer_measure M f (s \<inter> x) + outer_measure M f (s - x)" |
38656 | 448 |
apply (rule subadditiveD) |
42145 | 449 |
apply (rule ring_of_sets.countably_subadditive_subadditive [OF ring_of_sets_Pow]) |
62975
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
450 |
apply (simp add: positive_def outer_measure_empty[OF posf]) |
61273 | 451 |
apply (rule countably_subadditive_outer_measure) |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
452 |
using s by (auto intro!: posf inc) |
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
453 |
finally show ?thesis . |
42145 | 454 |
qed |
38656 | 455 |
ultimately |
61273 | 456 |
show "outer_measure M f (s \<inter> x) + outer_measure M f (s - x) = outer_measure M f s" |
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
457 |
by (rule order_antisym) |
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
458 |
qed |
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
459 |
|
69652
3417a8f154eb
updated tagging first 5
Angeliki KoutsoukouArgyraki <ak2110@cam.ac.uk>
parents:
69546
diff
changeset
|
460 |
lemma measure_down: "measure_space \<Omega> N \<mu> \<Longrightarrow> sigma_algebra \<Omega> M \<Longrightarrow> M \<subseteq> N \<Longrightarrow> measure_space \<Omega> M \<mu>" |
57446
06e195515deb
some lemmas about the indicator function; removed lemma sums_def2
hoelzl
parents:
57418
diff
changeset
|
461 |
by (auto simp add: measure_space_def positive_def countably_additive_def subset_eq) |
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
462 |
|
69683 | 463 |
subsection \<open>Caratheodory's theorem\<close> |
56994 | 464 |
|
69652
3417a8f154eb
updated tagging first 5
Angeliki KoutsoukouArgyraki <ak2110@cam.ac.uk>
parents:
69546
diff
changeset
|
465 |
theorem (in ring_of_sets) caratheodory': |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
466 |
assumes posf: "positive M f" and ca: "countably_additive M f" |
62975
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
467 |
shows "\<exists>\<mu> :: 'a set \<Rightarrow> ennreal. (\<forall>s \<in> M. \<mu> s = f s) \<and> measure_space \<Omega> (sigma_sets \<Omega> M) \<mu>" |
69652
3417a8f154eb
updated tagging first 5
Angeliki KoutsoukouArgyraki <ak2110@cam.ac.uk>
parents:
69546
diff
changeset
|
468 |
proof - |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
469 |
have inc: "increasing M f" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
470 |
by (metis additive_increasing ca countably_additive_additive posf) |
61273 | 471 |
let ?O = "outer_measure M f" |
63040 | 472 |
define ls where "ls = lambda_system \<Omega> (Pow \<Omega>) ?O" |
61273 | 473 |
have mls: "measure_space \<Omega> ls ?O" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
474 |
using sigma_algebra.caratheodory_lemma |
61273 | 475 |
[OF sigma_algebra_Pow outer_measure_space_outer_measure [OF posf inc]] |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
476 |
by (simp add: ls_def) |
47694 | 477 |
hence sls: "sigma_algebra \<Omega> ls" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
478 |
by (simp add: measure_space_def) |
47694 | 479 |
have "M \<subseteq> ls" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
480 |
by (simp add: ls_def) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
481 |
(metis ca posf inc countably_additive_additive algebra_subset_lambda_system) |
47694 | 482 |
hence sgs_sb: "sigma_sets (\<Omega>) (M) \<subseteq> ls" |
483 |
using sigma_algebra.sigma_sets_subset [OF sls, of "M"] |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
484 |
by simp |
61273 | 485 |
have "measure_space \<Omega> (sigma_sets \<Omega> M) ?O" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
486 |
by (rule measure_down [OF mls], rule sigma_algebra_sigma_sets) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
487 |
(simp_all add: sgs_sb space_closed) |
61273 | 488 |
thus ?thesis using outer_measure_agrees [OF posf ca] |
489 |
by (intro exI[of _ ?O]) auto |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41023
diff
changeset
|
490 |
qed |
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
491 |
|
69652
3417a8f154eb
updated tagging first 5
Angeliki KoutsoukouArgyraki <ak2110@cam.ac.uk>
parents:
69546
diff
changeset
|
492 |
lemma (in ring_of_sets) caratheodory_empty_continuous: |
47694 | 493 |
assumes f: "positive M f" "additive M f" and fin: "\<And>A. A \<in> M \<Longrightarrow> f A \<noteq> \<infinity>" |
61969 | 494 |
assumes cont: "\<And>A. range A \<subseteq> M \<Longrightarrow> decseq A \<Longrightarrow> (\<Inter>i. A i) = {} \<Longrightarrow> (\<lambda>i. f (A i)) \<longlonglongrightarrow> 0" |
62975
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
495 |
shows "\<exists>\<mu> :: 'a set \<Rightarrow> ennreal. (\<forall>s \<in> M. \<mu> s = f s) \<and> measure_space \<Omega> (sigma_sets \<Omega> M) \<mu>" |
69652
3417a8f154eb
updated tagging first 5
Angeliki KoutsoukouArgyraki <ak2110@cam.ac.uk>
parents:
69546
diff
changeset
|
496 |
proof (intro caratheodory' empty_continuous_imp_countably_additive f) |
47694 | 497 |
show "\<forall>A\<in>M. f A \<noteq> \<infinity>" using fin by auto |
42145 | 498 |
qed (rule cont) |
499 |
||
69683 | 500 |
subsection \<open>Volumes\<close> |
47762 | 501 |
|
70136 | 502 |
definition\<^marker>\<open>tag important\<close> volume :: "'a set set \<Rightarrow> ('a set \<Rightarrow> ennreal) \<Rightarrow> bool" where |
47762 | 503 |
"volume M f \<longleftrightarrow> |
504 |
(f {} = 0) \<and> (\<forall>a\<in>M. 0 \<le> f a) \<and> |
|
505 |
(\<forall>C\<subseteq>M. disjoint C \<longrightarrow> finite C \<longrightarrow> \<Union>C \<in> M \<longrightarrow> f (\<Union>C) = (\<Sum>c\<in>C. f c))" |
|
506 |
||
69652
3417a8f154eb
updated tagging first 5
Angeliki KoutsoukouArgyraki <ak2110@cam.ac.uk>
parents:
69546
diff
changeset
|
507 |
lemma volumeI: |
47762 | 508 |
assumes "f {} = 0" |
509 |
assumes "\<And>a. a \<in> M \<Longrightarrow> 0 \<le> f a" |
|
510 |
assumes "\<And>C. C \<subseteq> M \<Longrightarrow> disjoint C \<Longrightarrow> finite C \<Longrightarrow> \<Union>C \<in> M \<Longrightarrow> f (\<Union>C) = (\<Sum>c\<in>C. f c)" |
|
511 |
shows "volume M f" |
|
512 |
using assms by (auto simp: volume_def) |
|
513 |
||
69652
3417a8f154eb
updated tagging first 5
Angeliki KoutsoukouArgyraki <ak2110@cam.ac.uk>
parents:
69546
diff
changeset
|
514 |
lemma volume_positive: |
47762 | 515 |
"volume M f \<Longrightarrow> a \<in> M \<Longrightarrow> 0 \<le> f a" |
516 |
by (auto simp: volume_def) |
|
517 |
||
69652
3417a8f154eb
updated tagging first 5
Angeliki KoutsoukouArgyraki <ak2110@cam.ac.uk>
parents:
69546
diff
changeset
|
518 |
lemma volume_empty: |
47762 | 519 |
"volume M f \<Longrightarrow> f {} = 0" |
520 |
by (auto simp: volume_def) |
|
521 |
||
69652
3417a8f154eb
updated tagging first 5
Angeliki KoutsoukouArgyraki <ak2110@cam.ac.uk>
parents:
69546
diff
changeset
|
522 |
proposition volume_finite_additive: |
62975
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
523 |
assumes "volume M f" |
69313 | 524 |
assumes A: "\<And>i. i \<in> I \<Longrightarrow> A i \<in> M" "disjoint_family_on A I" "finite I" "\<Union>(A ` I) \<in> M" |
525 |
shows "f (\<Union>(A ` I)) = (\<Sum>i\<in>I. f (A i))" |
|
47762 | 526 |
proof - |
52141
eff000cab70f
weaker precendence of syntax for big intersection and union on sets
haftmann
parents:
51329
diff
changeset
|
527 |
have "A`I \<subseteq> M" "disjoint (A`I)" "finite (A`I)" "\<Union>(A`I) \<in> M" |
62343
24106dc44def
prefer abbreviations for compound operators INFIMUM and SUPREMUM
haftmann
parents:
61969
diff
changeset
|
528 |
using A by (auto simp: disjoint_family_on_disjoint_image) |
61808 | 529 |
with \<open>volume M f\<close> have "f (\<Union>(A`I)) = (\<Sum>a\<in>A`I. f a)" |
47762 | 530 |
unfolding volume_def by blast |
531 |
also have "\<dots> = (\<Sum>i\<in>I. f (A i))" |
|
64267 | 532 |
proof (subst sum.reindex_nontrivial) |
47762 | 533 |
fix i j assume "i \<in> I" "j \<in> I" "i \<noteq> j" "A i = A j" |
61808 | 534 |
with \<open>disjoint_family_on A I\<close> have "A i = {}" |
47762 | 535 |
by (auto simp: disjoint_family_on_def) |
536 |
then show "f (A i) = 0" |
|
61808 | 537 |
using volume_empty[OF \<open>volume M f\<close>] by simp |
538 |
qed (auto intro: \<open>finite I\<close>) |
|
69313 | 539 |
finally show "f (\<Union>(A ` I)) = (\<Sum>i\<in>I. f (A i))" |
47762 | 540 |
by simp |
541 |
qed |
|
542 |
||
69652
3417a8f154eb
updated tagging first 5
Angeliki KoutsoukouArgyraki <ak2110@cam.ac.uk>
parents:
69546
diff
changeset
|
543 |
lemma (in ring_of_sets) volume_additiveI: |
62975
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
544 |
assumes pos: "\<And>a. a \<in> M \<Longrightarrow> 0 \<le> \<mu> a" |
47762 | 545 |
assumes [simp]: "\<mu> {} = 0" |
546 |
assumes add: "\<And>a b. a \<in> M \<Longrightarrow> b \<in> M \<Longrightarrow> a \<inter> b = {} \<Longrightarrow> \<mu> (a \<union> b) = \<mu> a + \<mu> b" |
|
547 |
shows "volume M \<mu>" |
|
548 |
proof (unfold volume_def, safe) |
|
549 |
fix C assume "finite C" "C \<subseteq> M" "disjoint C" |
|
64267 | 550 |
then show "\<mu> (\<Union>C) = sum \<mu> C" |
47762 | 551 |
proof (induct C) |
552 |
case (insert c C) |
|
69745 | 553 |
from insert(1,2,4,5) have "\<mu> (\<Union>(insert c C)) = \<mu> c + \<mu> (\<Union>C)" |
47762 | 554 |
by (auto intro!: add simp: disjoint_def) |
555 |
with insert show ?case |
|
556 |
by (simp add: disjoint_def) |
|
557 |
qed simp |
|
558 |
qed fact+ |
|
559 |
||
69652
3417a8f154eb
updated tagging first 5
Angeliki KoutsoukouArgyraki <ak2110@cam.ac.uk>
parents:
69546
diff
changeset
|
560 |
proposition (in semiring_of_sets) extend_volume: |
47762 | 561 |
assumes "volume M \<mu>" |
562 |
shows "\<exists>\<mu>'. volume generated_ring \<mu>' \<and> (\<forall>a\<in>M. \<mu>' a = \<mu> a)" |
|
69652
3417a8f154eb
updated tagging first 5
Angeliki KoutsoukouArgyraki <ak2110@cam.ac.uk>
parents:
69546
diff
changeset
|
563 |
proof - |
47762 | 564 |
let ?R = generated_ring |
565 |
have "\<forall>a\<in>?R. \<exists>m. \<exists>C\<subseteq>M. a = \<Union>C \<and> finite C \<and> disjoint C \<and> m = (\<Sum>c\<in>C. \<mu> c)" |
|
566 |
by (auto simp: generated_ring_def) |
|
74362 | 567 |
from bchoice[OF this] obtain \<mu>' |
568 |
where \<mu>'_spec: "\<forall>x\<in>generated_ring. \<exists>C\<subseteq>M. x = \<Union> C \<and> finite C \<and> disjoint C \<and> \<mu>' x = sum \<mu> C" |
|
569 |
by blast |
|
47762 | 570 |
{ fix C assume C: "C \<subseteq> M" "finite C" "disjoint C" |
571 |
fix D assume D: "D \<subseteq> M" "finite D" "disjoint D" |
|
572 |
assume "\<Union>C = \<Union>D" |
|
573 |
have "(\<Sum>d\<in>D. \<mu> d) = (\<Sum>d\<in>D. \<Sum>c\<in>C. \<mu> (c \<inter> d))" |
|
64267 | 574 |
proof (intro sum.cong refl) |
47762 | 575 |
fix d assume "d \<in> D" |
576 |
have Un_eq_d: "(\<Union>c\<in>C. c \<inter> d) = d" |
|
61808 | 577 |
using \<open>d \<in> D\<close> \<open>\<Union>C = \<Union>D\<close> by auto |
47762 | 578 |
moreover have "\<mu> (\<Union>c\<in>C. c \<inter> d) = (\<Sum>c\<in>C. \<mu> (c \<inter> d))" |
579 |
proof (rule volume_finite_additive) |
|
580 |
{ fix c assume "c \<in> C" then show "c \<inter> d \<in> M" |
|
61808 | 581 |
using C D \<open>d \<in> D\<close> by auto } |
47762 | 582 |
show "(\<Union>a\<in>C. a \<inter> d) \<in> M" |
61808 | 583 |
unfolding Un_eq_d using \<open>d \<in> D\<close> D by auto |
47762 | 584 |
show "disjoint_family_on (\<lambda>a. a \<inter> d) C" |
61808 | 585 |
using \<open>disjoint C\<close> by (auto simp: disjoint_family_on_def disjoint_def) |
47762 | 586 |
qed fact+ |
587 |
ultimately show "\<mu> d = (\<Sum>c\<in>C. \<mu> (c \<inter> d))" by simp |
|
588 |
qed } |
|
589 |
note split_sum = this |
|
590 |
||
591 |
{ fix C assume C: "C \<subseteq> M" "finite C" "disjoint C" |
|
592 |
fix D assume D: "D \<subseteq> M" "finite D" "disjoint D" |
|
593 |
assume "\<Union>C = \<Union>D" |
|
594 |
with split_sum[OF C D] split_sum[OF D C] |
|
595 |
have "(\<Sum>d\<in>D. \<mu> d) = (\<Sum>c\<in>C. \<mu> c)" |
|
66804
3f9bb52082c4
avoid name clashes on interpretation of abstract locales
haftmann
parents:
65680
diff
changeset
|
596 |
by (simp, subst sum.swap, simp add: ac_simps) } |
47762 | 597 |
note sum_eq = this |
598 |
||
599 |
{ fix C assume C: "C \<subseteq> M" "finite C" "disjoint C" |
|
600 |
then have "\<Union>C \<in> ?R" by (auto simp: generated_ring_def) |
|
601 |
with \<mu>'_spec[THEN bspec, of "\<Union>C"] |
|
602 |
obtain D where |
|
603 |
D: "D \<subseteq> M" "finite D" "disjoint D" "\<Union>C = \<Union>D" and "\<mu>' (\<Union>C) = (\<Sum>d\<in>D. \<mu> d)" |
|
61427
3c69ea85f8dd
Fixed nonterminating "blast" proof
paulson <lp15@cam.ac.uk>
parents:
61424
diff
changeset
|
604 |
by auto |
47762 | 605 |
with sum_eq[OF C D] have "\<mu>' (\<Union>C) = (\<Sum>c\<in>C. \<mu> c)" by simp } |
606 |
note \<mu>' = this |
|
607 |
||
608 |
show ?thesis |
|
609 |
proof (intro exI conjI ring_of_sets.volume_additiveI[OF generating_ring] ballI) |
|
610 |
fix a assume "a \<in> M" with \<mu>'[of "{a}"] show "\<mu>' a = \<mu> a" |
|
611 |
by (simp add: disjoint_def) |
|
612 |
next |
|
74362 | 613 |
fix a assume "a \<in> ?R" |
614 |
then obtain Ca where Ca: "finite Ca" "disjoint Ca" "Ca \<subseteq> M" "a = \<Union> Ca" .. |
|
61808 | 615 |
with \<mu>'[of Ca] \<open>volume M \<mu>\<close>[THEN volume_positive] |
47762 | 616 |
show "0 \<le> \<mu>' a" |
64267 | 617 |
by (auto intro!: sum_nonneg) |
47762 | 618 |
next |
619 |
show "\<mu>' {} = 0" using \<mu>'[of "{}"] by auto |
|
620 |
next |
|
74362 | 621 |
fix a b assume "a \<in> ?R" "b \<in> ?R" |
622 |
then obtain Ca Cb |
|
623 |
where Ca: "finite Ca" "disjoint Ca" "Ca \<subseteq> M" "a = \<Union> Ca" |
|
624 |
and Cb: "finite Cb" "disjoint Cb" "Cb \<subseteq> M" "b = \<Union> Cb" |
|
625 |
by (meson generated_ringE) |
|
47762 | 626 |
assume "a \<inter> b = {}" |
627 |
with Ca Cb have "Ca \<inter> Cb \<subseteq> {{}}" by auto |
|
628 |
then have C_Int_cases: "Ca \<inter> Cb = {{}} \<or> Ca \<inter> Cb = {}" by auto |
|
629 |
||
61808 | 630 |
from \<open>a \<inter> b = {}\<close> have "\<mu>' (\<Union>(Ca \<union> Cb)) = (\<Sum>c\<in>Ca \<union> Cb. \<mu> c)" |
47762 | 631 |
using Ca Cb by (intro \<mu>') (auto intro!: disjoint_union) |
632 |
also have "\<dots> = (\<Sum>c\<in>Ca \<union> Cb. \<mu> c) + (\<Sum>c\<in>Ca \<inter> Cb. \<mu> c)" |
|
61808 | 633 |
using C_Int_cases volume_empty[OF \<open>volume M \<mu>\<close>] by (elim disjE) simp_all |
47762 | 634 |
also have "\<dots> = (\<Sum>c\<in>Ca. \<mu> c) + (\<Sum>c\<in>Cb. \<mu> c)" |
64267 | 635 |
using Ca Cb by (simp add: sum.union_inter) |
47762 | 636 |
also have "\<dots> = \<mu>' a + \<mu>' b" |
637 |
using Ca Cb by (simp add: \<mu>') |
|
638 |
finally show "\<mu>' (a \<union> b) = \<mu>' a + \<mu>' b" |
|
639 |
using Ca Cb by simp |
|
640 |
qed |
|
641 |
qed |
|
642 |
||
70136 | 643 |
subsubsection\<^marker>\<open>tag important\<close> \<open>Caratheodory on semirings\<close> |
47762 | 644 |
|
69652
3417a8f154eb
updated tagging first 5
Angeliki KoutsoukouArgyraki <ak2110@cam.ac.uk>
parents:
69546
diff
changeset
|
645 |
theorem (in semiring_of_sets) caratheodory: |
47762 | 646 |
assumes pos: "positive M \<mu>" and ca: "countably_additive M \<mu>" |
62975
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
647 |
shows "\<exists>\<mu>' :: 'a set \<Rightarrow> ennreal. (\<forall>s \<in> M. \<mu>' s = \<mu> s) \<and> measure_space \<Omega> (sigma_sets \<Omega> M) \<mu>'" |
69652
3417a8f154eb
updated tagging first 5
Angeliki KoutsoukouArgyraki <ak2110@cam.ac.uk>
parents:
69546
diff
changeset
|
648 |
proof - |
47762 | 649 |
have "volume M \<mu>" |
650 |
proof (rule volumeI) |
|
651 |
{ fix a assume "a \<in> M" then show "0 \<le> \<mu> a" |
|
652 |
using pos unfolding positive_def by auto } |
|
653 |
note p = this |
|
654 |
||
655 |
fix C assume sets_C: "C \<subseteq> M" "\<Union>C \<in> M" and "disjoint C" "finite C" |
|
656 |
have "\<exists>F'. bij_betw F' {..<card C} C" |
|
61808 | 657 |
by (rule finite_same_card_bij[OF _ \<open>finite C\<close>]) auto |
74362 | 658 |
then obtain F' where "bij_betw F' {..<card C} C" .. |
47762 | 659 |
then have F': "C = F' ` {..< card C}" "inj_on F' {..< card C}" |
660 |
by (auto simp: bij_betw_def) |
|
661 |
{ fix i j assume *: "i < card C" "j < card C" "i \<noteq> j" |
|
662 |
with F' have "F' i \<in> C" "F' j \<in> C" "F' i \<noteq> F' j" |
|
663 |
unfolding inj_on_def by auto |
|
61808 | 664 |
with \<open>disjoint C\<close>[THEN disjointD] |
47762 | 665 |
have "F' i \<inter> F' j = {}" |
666 |
by auto } |
|
667 |
note F'_disj = this |
|
63040 | 668 |
define F where "F i = (if i < card C then F' i else {})" for i |
47762 | 669 |
then have "disjoint_family F" |
670 |
using F'_disj by (auto simp: disjoint_family_on_def) |
|
671 |
moreover from F' have "(\<Union>i. F i) = \<Union>C" |
|
69661 | 672 |
by (auto simp add: F_def split: if_split_asm cong del: SUP_cong) |
47762 | 673 |
moreover have sets_F: "\<And>i. F i \<in> M" |
674 |
using F' sets_C by (auto simp: F_def) |
|
675 |
moreover note sets_C |
|
676 |
ultimately have "\<mu> (\<Union>C) = (\<Sum>i. \<mu> (F i))" |
|
677 |
using ca[unfolded countably_additive_def, THEN spec, of F] by auto |
|
678 |
also have "\<dots> = (\<Sum>i<card C. \<mu> (F' i))" |
|
679 |
proof - |
|
680 |
have "(\<lambda>i. if i \<in> {..< card C} then \<mu> (F' i) else 0) sums (\<Sum>i<card C. \<mu> (F' i))" |
|
681 |
by (rule sums_If_finite_set) auto |
|
682 |
also have "(\<lambda>i. if i \<in> {..< card C} then \<mu> (F' i) else 0) = (\<lambda>i. \<mu> (F i))" |
|
683 |
using pos by (auto simp: positive_def F_def) |
|
684 |
finally show "(\<Sum>i. \<mu> (F i)) = (\<Sum>i<card C. \<mu> (F' i))" |
|
685 |
by (simp add: sums_iff) |
|
686 |
qed |
|
687 |
also have "\<dots> = (\<Sum>c\<in>C. \<mu> c)" |
|
64267 | 688 |
using F'(2) by (subst (2) F') (simp add: sum.reindex) |
47762 | 689 |
finally show "\<mu> (\<Union>C) = (\<Sum>c\<in>C. \<mu> c)" . |
690 |
next |
|
691 |
show "\<mu> {} = 0" |
|
61808 | 692 |
using \<open>positive M \<mu>\<close> by (rule positiveD1) |
47762 | 693 |
qed |
694 |
from extend_volume[OF this] obtain \<mu>_r where |
|
695 |
V: "volume generated_ring \<mu>_r" "\<And>a. a \<in> M \<Longrightarrow> \<mu> a = \<mu>_r a" |
|
696 |
by auto |
|
697 |
||
698 |
interpret G: ring_of_sets \<Omega> generated_ring |
|
699 |
by (rule generating_ring) |
|
700 |
||
701 |
have pos: "positive generated_ring \<mu>_r" |
|
702 |
using V unfolding positive_def by (auto simp: positive_def intro!: volume_positive volume_empty) |
|
703 |
||
704 |
have "countably_additive generated_ring \<mu>_r" |
|
705 |
proof (rule countably_additiveI) |
|
74362 | 706 |
fix A' :: "nat \<Rightarrow> 'a set" |
707 |
assume A': "range A' \<subseteq> generated_ring" "disjoint_family A'" |
|
47762 | 708 |
and Un_A: "(\<Union>i. A' i) \<in> generated_ring" |
709 |
||
74362 | 710 |
obtain C' where C': "finite C'" "disjoint C'" "C' \<subseteq> M" "\<Union> (range A') = \<Union> C'" |
711 |
using generated_ringE[OF Un_A] by auto |
|
47762 | 712 |
|
713 |
{ fix c assume "c \<in> C'" |
|
63040 | 714 |
moreover define A where [abs_def]: "A i = A' i \<inter> c" for i |
47762 | 715 |
ultimately have A: "range A \<subseteq> generated_ring" "disjoint_family A" |
716 |
and Un_A: "(\<Union>i. A i) \<in> generated_ring" |
|
717 |
using A' C' |
|
718 |
by (auto intro!: G.Int G.finite_Union intro: generated_ringI_Basic simp: disjoint_family_on_def) |
|
61808 | 719 |
from A C' \<open>c \<in> C'\<close> have UN_eq: "(\<Union>i. A i) = c" |
47762 | 720 |
by (auto simp: A_def) |
721 |
||
69745 | 722 |
have "\<forall>i::nat. \<exists>f::nat \<Rightarrow> 'a set. \<mu>_r (A i) = (\<Sum>j. \<mu>_r (f j)) \<and> disjoint_family f \<and> \<Union>(range f) = A i \<and> (\<forall>j. f j \<in> M)" |
47762 | 723 |
(is "\<forall>i. ?P i") |
724 |
proof |
|
725 |
fix i |
|
726 |
from A have Ai: "A i \<in> generated_ring" by auto |
|
74362 | 727 |
from generated_ringE[OF this] obtain C |
728 |
where C: "finite C" "disjoint C" "C \<subseteq> M" "A i = \<Union> C" by auto |
|
47762 | 729 |
have "\<exists>F'. bij_betw F' {..<card C} C" |
61808 | 730 |
by (rule finite_same_card_bij[OF _ \<open>finite C\<close>]) auto |
74362 | 731 |
then obtain F where F: "bij_betw F {..<card C} C" .. |
63040 | 732 |
define f where [abs_def]: "f i = (if i < card C then F i else {})" for i |
47762 | 733 |
then have f: "bij_betw f {..< card C} C" |
734 |
by (intro bij_betw_cong[THEN iffD1, OF _ F]) auto |
|
735 |
with C have "\<forall>j. f j \<in> M" |
|
736 |
by (auto simp: Pi_iff f_def dest!: bij_betw_imp_funcset) |
|
737 |
moreover |
|
738 |
from f C have d_f: "disjoint_family_on f {..<card C}" |
|
739 |
by (intro disjoint_image_disjoint_family_on) (auto simp: bij_betw_def) |
|
740 |
then have "disjoint_family f" |
|
741 |
by (auto simp: disjoint_family_on_def f_def) |
|
742 |
moreover |
|
60585 | 743 |
have Ai_eq: "A i = (\<Union>x<card C. f x)" |
62343
24106dc44def
prefer abbreviations for compound operators INFIMUM and SUPREMUM
haftmann
parents:
61969
diff
changeset
|
744 |
using f C Ai unfolding bij_betw_def by auto |
69745 | 745 |
then have "\<Union>(range f) = A i" |
69768 | 746 |
using f by (auto simp add: f_def) |
62975
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
747 |
moreover |
47762 | 748 |
{ have "(\<Sum>j. \<mu>_r (f j)) = (\<Sum>j. if j \<in> {..< card C} then \<mu>_r (f j) else 0)" |
749 |
using volume_empty[OF V(1)] by (auto intro!: arg_cong[where f=suminf] simp: f_def) |
|
750 |
also have "\<dots> = (\<Sum>j<card C. \<mu>_r (f j))" |
|
751 |
by (rule sums_If_finite_set[THEN sums_unique, symmetric]) simp |
|
752 |
also have "\<dots> = \<mu>_r (A i)" |
|
753 |
using C f[THEN bij_betw_imp_funcset] unfolding Ai_eq |
|
754 |
by (intro volume_finite_additive[OF V(1) _ d_f, symmetric]) |
|
755 |
(auto simp: Pi_iff Ai_eq intro: generated_ringI_Basic) |
|
756 |
finally have "\<mu>_r (A i) = (\<Sum>j. \<mu>_r (f j))" .. } |
|
757 |
ultimately show "?P i" |
|
758 |
by blast |
|
759 |
qed |
|
74362 | 760 |
from choice[OF this] obtain f |
761 |
where f: "\<forall>x. \<mu>_r (A x) = (\<Sum>j. \<mu>_r (f x j)) \<and> disjoint_family (f x) \<and> \<Union> (range (f x)) = A x \<and> (\<forall>j. f x j \<in> M)" |
|
762 |
.. |
|
61424
c3658c18b7bc
prod_case as canonical name for product type eliminator
haftmann
parents:
61273
diff
changeset
|
763 |
then have UN_f_eq: "(\<Union>i. case_prod f (prod_decode i)) = (\<Union>i. A i)" |
47762 | 764 |
unfolding UN_extend_simps surj_prod_decode by (auto simp: set_eq_iff) |
765 |
||
61424
c3658c18b7bc
prod_case as canonical name for product type eliminator
haftmann
parents:
61273
diff
changeset
|
766 |
have d: "disjoint_family (\<lambda>i. case_prod f (prod_decode i))" |
47762 | 767 |
unfolding disjoint_family_on_def |
768 |
proof (intro ballI impI) |
|
769 |
fix m n :: nat assume "m \<noteq> n" |
|
770 |
then have neq: "prod_decode m \<noteq> prod_decode n" |
|
771 |
using inj_prod_decode[of UNIV] by (auto simp: inj_on_def) |
|
61424
c3658c18b7bc
prod_case as canonical name for product type eliminator
haftmann
parents:
61273
diff
changeset
|
772 |
show "case_prod f (prod_decode m) \<inter> case_prod f (prod_decode n) = {}" |
47762 | 773 |
proof cases |
774 |
assume "fst (prod_decode m) = fst (prod_decode n)" |
|
775 |
then show ?thesis |
|
776 |
using neq f by (fastforce simp: disjoint_family_on_def) |
|
777 |
next |
|
778 |
assume neq: "fst (prod_decode m) \<noteq> fst (prod_decode n)" |
|
61424
c3658c18b7bc
prod_case as canonical name for product type eliminator
haftmann
parents:
61273
diff
changeset
|
779 |
have "case_prod f (prod_decode m) \<subseteq> A (fst (prod_decode m))" |
c3658c18b7bc
prod_case as canonical name for product type eliminator
haftmann
parents:
61273
diff
changeset
|
780 |
"case_prod f (prod_decode n) \<subseteq> A (fst (prod_decode n))" |
47762 | 781 |
using f[THEN spec, of "fst (prod_decode m)"] |
782 |
using f[THEN spec, of "fst (prod_decode n)"] |
|
783 |
by (auto simp: set_eq_iff) |
|
784 |
with f A neq show ?thesis |
|
785 |
by (fastforce simp: disjoint_family_on_def subset_eq set_eq_iff) |
|
786 |
qed |
|
787 |
qed |
|
61424
c3658c18b7bc
prod_case as canonical name for product type eliminator
haftmann
parents:
61273
diff
changeset
|
788 |
from f have "(\<Sum>n. \<mu>_r (A n)) = (\<Sum>n. \<mu>_r (case_prod f (prod_decode n)))" |
62975
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
789 |
by (intro suminf_ennreal_2dimen[symmetric] generated_ringI_Basic) |
47762 | 790 |
(auto split: prod.split) |
61424
c3658c18b7bc
prod_case as canonical name for product type eliminator
haftmann
parents:
61273
diff
changeset
|
791 |
also have "\<dots> = (\<Sum>n. \<mu> (case_prod f (prod_decode n)))" |
47762 | 792 |
using f V(2) by (auto intro!: arg_cong[where f=suminf] split: prod.split) |
61424
c3658c18b7bc
prod_case as canonical name for product type eliminator
haftmann
parents:
61273
diff
changeset
|
793 |
also have "\<dots> = \<mu> (\<Union>i. case_prod f (prod_decode i))" |
61808 | 794 |
using f \<open>c \<in> C'\<close> C' |
47762 | 795 |
by (intro ca[unfolded countably_additive_def, rule_format]) |
796 |
(auto split: prod.split simp: UN_f_eq d UN_eq) |
|
797 |
finally have "(\<Sum>n. \<mu>_r (A' n \<inter> c)) = \<mu> c" |
|
798 |
using UN_f_eq UN_eq by (simp add: A_def) } |
|
799 |
note eq = this |
|
800 |
||
801 |
have "(\<Sum>n. \<mu>_r (A' n)) = (\<Sum>n. \<Sum>c\<in>C'. \<mu>_r (A' n \<inter> c))" |
|
49394
52e636ace94e
removing find_theorems commands that were left in the developments accidently
bulwahn
parents:
47762
diff
changeset
|
802 |
using C' A' |
47762 | 803 |
by (subst volume_finite_additive[symmetric, OF V(1)]) |
62343
24106dc44def
prefer abbreviations for compound operators INFIMUM and SUPREMUM
haftmann
parents:
61969
diff
changeset
|
804 |
(auto simp: disjoint_def disjoint_family_on_def |
47762 | 805 |
intro!: G.Int G.finite_Union arg_cong[where f="\<lambda>X. suminf (\<lambda>i. \<mu>_r (X i))"] ext |
806 |
intro: generated_ringI_Basic) |
|
807 |
also have "\<dots> = (\<Sum>c\<in>C'. \<Sum>n. \<mu>_r (A' n \<inter> c))" |
|
808 |
using C' A' |
|
64267 | 809 |
by (intro suminf_sum G.Int G.finite_Union) (auto intro: generated_ringI_Basic) |
47762 | 810 |
also have "\<dots> = (\<Sum>c\<in>C'. \<mu>_r c)" |
64267 | 811 |
using eq V C' by (auto intro!: sum.cong) |
47762 | 812 |
also have "\<dots> = \<mu>_r (\<Union>C')" |
813 |
using C' Un_A |
|
814 |
by (subst volume_finite_additive[symmetric, OF V(1)]) |
|
62343
24106dc44def
prefer abbreviations for compound operators INFIMUM and SUPREMUM
haftmann
parents:
61969
diff
changeset
|
815 |
(auto simp: disjoint_family_on_def disjoint_def |
47762 | 816 |
intro: generated_ringI_Basic) |
817 |
finally show "(\<Sum>n. \<mu>_r (A' n)) = \<mu>_r (\<Union>i. A' i)" |
|
818 |
using C' by simp |
|
819 |
qed |
|
74362 | 820 |
obtain \<mu>' where "(\<forall>s\<in>generated_ring. \<mu>' s = \<mu>_r s) \<and> measure_space \<Omega> (sigma_sets \<Omega> generated_ring) \<mu>'" |
821 |
using G.caratheodory'[OF pos \<open>countably_additive generated_ring \<mu>_r\<close>] by auto |
|
47762 | 822 |
with V show ?thesis |
823 |
unfolding sigma_sets_generated_ring_eq |
|
824 |
by (intro exI[of _ \<mu>']) (auto intro: generated_ringI_Basic) |
|
825 |
qed |
|
826 |
||
69652
3417a8f154eb
updated tagging first 5
Angeliki KoutsoukouArgyraki <ak2110@cam.ac.uk>
parents:
69546
diff
changeset
|
827 |
lemma extend_measure_caratheodory: |
57447
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
828 |
fixes G :: "'i \<Rightarrow> 'a set" |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
829 |
assumes M: "M = extend_measure \<Omega> I G \<mu>" |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
830 |
assumes "i \<in> I" |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
831 |
assumes "semiring_of_sets \<Omega> (G ` I)" |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
832 |
assumes empty: "\<And>i. i \<in> I \<Longrightarrow> G i = {} \<Longrightarrow> \<mu> i = 0" |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
833 |
assumes inj: "\<And>i j. i \<in> I \<Longrightarrow> j \<in> I \<Longrightarrow> G i = G j \<Longrightarrow> \<mu> i = \<mu> j" |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
834 |
assumes nonneg: "\<And>i. i \<in> I \<Longrightarrow> 0 \<le> \<mu> i" |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
835 |
assumes add: "\<And>A::nat \<Rightarrow> 'i. \<And>j. A \<in> UNIV \<rightarrow> I \<Longrightarrow> j \<in> I \<Longrightarrow> disjoint_family (G \<circ> A) \<Longrightarrow> |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
836 |
(\<Union>i. G (A i)) = G j \<Longrightarrow> (\<Sum>n. \<mu> (A n)) = \<mu> j" |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
837 |
shows "emeasure M (G i) = \<mu> i" |
68833
fde093888c16
tagged 21 theories in the Analysis library for the manual
Angeliki KoutsoukouArgyraki <ak2110@cam.ac.uk>
parents:
67682
diff
changeset
|
838 |
|
69652
3417a8f154eb
updated tagging first 5
Angeliki KoutsoukouArgyraki <ak2110@cam.ac.uk>
parents:
69546
diff
changeset
|
839 |
proof - |
57447
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
840 |
interpret semiring_of_sets \<Omega> "G ` I" |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
841 |
by fact |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
842 |
have "\<forall>g\<in>G`I. \<exists>i\<in>I. g = G i" |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
843 |
by auto |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
844 |
then obtain sel where sel: "\<And>g. g \<in> G ` I \<Longrightarrow> sel g \<in> I" "\<And>g. g \<in> G ` I \<Longrightarrow> G (sel g) = g" |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
845 |
by metis |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
846 |
|
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
847 |
have "\<exists>\<mu>'. (\<forall>s\<in>G ` I. \<mu>' s = \<mu> (sel s)) \<and> measure_space \<Omega> (sigma_sets \<Omega> (G ` I)) \<mu>'" |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
848 |
proof (rule caratheodory) |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
849 |
show "positive (G ` I) (\<lambda>s. \<mu> (sel s))" |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
850 |
by (auto simp: positive_def intro!: empty sel nonneg) |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
851 |
show "countably_additive (G ` I) (\<lambda>s. \<mu> (sel s))" |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
852 |
proof (rule countably_additiveI) |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
853 |
fix A :: "nat \<Rightarrow> 'a set" assume "range A \<subseteq> G ` I" "disjoint_family A" "(\<Union>i. A i) \<in> G ` I" |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
854 |
then show "(\<Sum>i. \<mu> (sel (A i))) = \<mu> (sel (\<Union>i. A i))" |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
855 |
by (intro add) (auto simp: sel image_subset_iff_funcset comp_def Pi_iff intro!: sel) |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
856 |
qed |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
857 |
qed |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
858 |
then obtain \<mu>' where \<mu>': "\<forall>s\<in>G ` I. \<mu>' s = \<mu> (sel s)" "measure_space \<Omega> (sigma_sets \<Omega> (G ` I)) \<mu>'" |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
859 |
by metis |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
860 |
|
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
861 |
show ?thesis |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
862 |
proof (rule emeasure_extend_measure[OF M]) |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
863 |
{ fix i assume "i \<in> I" then show "\<mu>' (G i) = \<mu> i" |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
864 |
using \<mu>' by (auto intro!: inj sel) } |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
865 |
show "G ` I \<subseteq> Pow \<Omega>" |
67682
00c436488398
tuned proofs -- prefer explicit names for facts from 'interpret';
wenzelm
parents:
66804
diff
changeset
|
866 |
by (rule space_closed) |
57447
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
867 |
then show "positive (sets M) \<mu>'" "countably_additive (sets M) \<mu>'" |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
868 |
using \<mu>' by (simp_all add: M sets_extend_measure measure_space_def) |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
869 |
qed fact |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
870 |
qed |
62975
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
hoelzl
parents:
62390
diff
changeset
|
871 |
|
69652
3417a8f154eb
updated tagging first 5
Angeliki KoutsoukouArgyraki <ak2110@cam.ac.uk>
parents:
69546
diff
changeset
|
872 |
proposition extend_measure_caratheodory_pair: |
57447
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
873 |
fixes G :: "'i \<Rightarrow> 'j \<Rightarrow> 'a set" |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
874 |
assumes M: "M = extend_measure \<Omega> {(a, b). P a b} (\<lambda>(a, b). G a b) (\<lambda>(a, b). \<mu> a b)" |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
875 |
assumes "P i j" |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
876 |
assumes semiring: "semiring_of_sets \<Omega> {G a b | a b. P a b}" |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
877 |
assumes empty: "\<And>i j. P i j \<Longrightarrow> G i j = {} \<Longrightarrow> \<mu> i j = 0" |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
878 |
assumes inj: "\<And>i j k l. P i j \<Longrightarrow> P k l \<Longrightarrow> G i j = G k l \<Longrightarrow> \<mu> i j = \<mu> k l" |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
879 |
assumes nonneg: "\<And>i j. P i j \<Longrightarrow> 0 \<le> \<mu> i j" |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
880 |
assumes add: "\<And>A::nat \<Rightarrow> 'i. \<And>B::nat \<Rightarrow> 'j. \<And>j k. |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
881 |
(\<And>n. P (A n) (B n)) \<Longrightarrow> P j k \<Longrightarrow> disjoint_family (\<lambda>n. G (A n) (B n)) \<Longrightarrow> |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
882 |
(\<Union>i. G (A i) (B i)) = G j k \<Longrightarrow> (\<Sum>n. \<mu> (A n) (B n)) = \<mu> j k" |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
883 |
shows "emeasure M (G i j) = \<mu> i j" |
69652
3417a8f154eb
updated tagging first 5
Angeliki KoutsoukouArgyraki <ak2110@cam.ac.uk>
parents:
69546
diff
changeset
|
884 |
proof - |
57447
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
885 |
have "emeasure M ((\<lambda>(a, b). G a b) (i, j)) = (\<lambda>(a, b). \<mu> a b) (i, j)" |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
886 |
proof (rule extend_measure_caratheodory[OF M]) |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
887 |
show "semiring_of_sets \<Omega> ((\<lambda>(a, b). G a b) ` {(a, b). P a b})" |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
888 |
using semiring by (simp add: image_def conj_commute) |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
889 |
next |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
890 |
fix A :: "nat \<Rightarrow> ('i \<times> 'j)" and j assume "A \<in> UNIV \<rightarrow> {(a, b). P a b}" "j \<in> {(a, b). P a b}" |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
891 |
"disjoint_family ((\<lambda>(a, b). G a b) \<circ> A)" |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
892 |
"(\<Union>i. case A i of (a, b) \<Rightarrow> G a b) = (case j of (a, b) \<Rightarrow> G a b)" |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
893 |
then show "(\<Sum>n. case A n of (a, b) \<Rightarrow> \<mu> a b) = (case j of (a, b) \<Rightarrow> \<mu> a b)" |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
894 |
using add[of "\<lambda>i. fst (A i)" "\<lambda>i. snd (A i)" "fst j" "snd j"] |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
895 |
by (simp add: split_beta' comp_def Pi_iff) |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
896 |
qed (auto split: prod.splits intro: assms) |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
897 |
then show ?thesis by simp |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
898 |
qed |
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents:
57446
diff
changeset
|
899 |
|
33271
7be66dee1a5a
New theory Probability, which contains a development of measure theory
paulson
parents:
diff
changeset
|
900 |
end |