author | hoelzl |
Wed, 23 Feb 2011 11:40:12 +0100 | |
changeset 41831 | 91a2b435dd7a |
parent 41706 | a207a858d1f6 |
child 41981 | cdf7693bbe08 |
permissions | -rw-r--r-- |
35833 | 1 |
theory Product_Measure |
38656 | 2 |
imports Lebesgue_Integration |
35833 | 3 |
begin |
4 |
||
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
5 |
lemma sigma_sets_subseteq: assumes "A \<subseteq> B" shows "sigma_sets X A \<subseteq> sigma_sets X B" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
6 |
proof |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
7 |
fix x assume "x \<in> sigma_sets X A" then show "x \<in> sigma_sets X B" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
8 |
by induct (insert `A \<subseteq> B`, auto intro: sigma_sets.intros) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
9 |
qed |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
10 |
|
40859 | 11 |
lemma times_Int_times: "A \<times> B \<inter> C \<times> D = (A \<inter> C) \<times> (B \<inter> D)" |
12 |
by auto |
|
13 |
||
14 |
lemma Pair_vimage_times[simp]: "\<And>A B x. Pair x -` (A \<times> B) = (if x \<in> A then B else {})" |
|
15 |
by auto |
|
16 |
||
17 |
lemma rev_Pair_vimage_times[simp]: "\<And>A B y. (\<lambda>x. (x, y)) -` (A \<times> B) = (if y \<in> B then A else {})" |
|
18 |
by auto |
|
19 |
||
20 |
lemma case_prod_distrib: "f (case x of (x, y) \<Rightarrow> g x y) = (case x of (x, y) \<Rightarrow> f (g x y))" |
|
21 |
by (cases x) simp |
|
22 |
||
41026
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
23 |
lemma split_beta': "(\<lambda>(x,y). f x y) = (\<lambda>x. f (fst x) (snd x))" |
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
24 |
by (auto simp: fun_eq_iff) |
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
25 |
|
40859 | 26 |
abbreviation |
27 |
"Pi\<^isub>E A B \<equiv> Pi A B \<inter> extensional A" |
|
39094 | 28 |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
29 |
syntax |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
30 |
"_PiE" :: "[pttrn, 'a set, 'b set] => ('a => 'b) set" ("(3PIE _:_./ _)" 10) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
31 |
|
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
32 |
syntax (xsymbols) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
33 |
"_PiE" :: "[pttrn, 'a set, 'b set] => ('a => 'b) set" ("(3\<Pi>\<^isub>E _\<in>_./ _)" 10) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
34 |
|
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
35 |
syntax (HTML output) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
36 |
"_PiE" :: "[pttrn, 'a set, 'b set] => ('a => 'b) set" ("(3\<Pi>\<^isub>E _\<in>_./ _)" 10) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
37 |
|
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
38 |
translations |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
39 |
"PIE x:A. B" == "CONST Pi\<^isub>E A (%x. B)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
40 |
|
40859 | 41 |
abbreviation |
42 |
funcset_extensional :: "['a set, 'b set] => ('a => 'b) set" |
|
43 |
(infixr "->\<^isub>E" 60) where |
|
44 |
"A ->\<^isub>E B \<equiv> Pi\<^isub>E A (%_. B)" |
|
45 |
||
46 |
notation (xsymbols) |
|
47 |
funcset_extensional (infixr "\<rightarrow>\<^isub>E" 60) |
|
48 |
||
49 |
lemma extensional_empty[simp]: "extensional {} = {\<lambda>x. undefined}" |
|
50 |
by safe (auto simp add: extensional_def fun_eq_iff) |
|
51 |
||
52 |
lemma extensional_insert[intro, simp]: |
|
53 |
assumes "a \<in> extensional (insert i I)" |
|
54 |
shows "a(i := b) \<in> extensional (insert i I)" |
|
55 |
using assms unfolding extensional_def by auto |
|
56 |
||
57 |
lemma extensional_Int[simp]: |
|
58 |
"extensional I \<inter> extensional I' = extensional (I \<inter> I')" |
|
59 |
unfolding extensional_def by auto |
|
38656 | 60 |
|
35833 | 61 |
definition |
40859 | 62 |
"merge I x J y = (\<lambda>i. if i \<in> I then x i else if i \<in> J then y i else undefined)" |
63 |
||
64 |
lemma merge_apply[simp]: |
|
65 |
"I \<inter> J = {} \<Longrightarrow> i \<in> I \<Longrightarrow> merge I x J y i = x i" |
|
66 |
"I \<inter> J = {} \<Longrightarrow> i \<in> J \<Longrightarrow> merge I x J y i = y i" |
|
67 |
"J \<inter> I = {} \<Longrightarrow> i \<in> I \<Longrightarrow> merge I x J y i = x i" |
|
68 |
"J \<inter> I = {} \<Longrightarrow> i \<in> J \<Longrightarrow> merge I x J y i = y i" |
|
69 |
"i \<notin> I \<Longrightarrow> i \<notin> J \<Longrightarrow> merge I x J y i = undefined" |
|
70 |
unfolding merge_def by auto |
|
71 |
||
72 |
lemma merge_commute: |
|
73 |
"I \<inter> J = {} \<Longrightarrow> merge I x J y = merge J y I x" |
|
74 |
by (auto simp: merge_def intro!: ext) |
|
75 |
||
76 |
lemma Pi_cancel_merge_range[simp]: |
|
77 |
"I \<inter> J = {} \<Longrightarrow> x \<in> Pi I (merge I A J B) \<longleftrightarrow> x \<in> Pi I A" |
|
78 |
"I \<inter> J = {} \<Longrightarrow> x \<in> Pi I (merge J B I A) \<longleftrightarrow> x \<in> Pi I A" |
|
79 |
"J \<inter> I = {} \<Longrightarrow> x \<in> Pi I (merge I A J B) \<longleftrightarrow> x \<in> Pi I A" |
|
80 |
"J \<inter> I = {} \<Longrightarrow> x \<in> Pi I (merge J B I A) \<longleftrightarrow> x \<in> Pi I A" |
|
81 |
by (auto simp: Pi_def) |
|
82 |
||
83 |
lemma Pi_cancel_merge[simp]: |
|
84 |
"I \<inter> J = {} \<Longrightarrow> merge I x J y \<in> Pi I B \<longleftrightarrow> x \<in> Pi I B" |
|
85 |
"J \<inter> I = {} \<Longrightarrow> merge I x J y \<in> Pi I B \<longleftrightarrow> x \<in> Pi I B" |
|
86 |
"I \<inter> J = {} \<Longrightarrow> merge I x J y \<in> Pi J B \<longleftrightarrow> y \<in> Pi J B" |
|
87 |
"J \<inter> I = {} \<Longrightarrow> merge I x J y \<in> Pi J B \<longleftrightarrow> y \<in> Pi J B" |
|
88 |
by (auto simp: Pi_def) |
|
89 |
||
90 |
lemma extensional_merge[simp]: "merge I x J y \<in> extensional (I \<union> J)" |
|
91 |
by (auto simp: extensional_def) |
|
92 |
||
93 |
lemma restrict_Pi_cancel: "restrict x I \<in> Pi I A \<longleftrightarrow> x \<in> Pi I A" |
|
94 |
by (auto simp: restrict_def Pi_def) |
|
95 |
||
96 |
lemma restrict_merge[simp]: |
|
97 |
"I \<inter> J = {} \<Longrightarrow> restrict (merge I x J y) I = restrict x I" |
|
98 |
"I \<inter> J = {} \<Longrightarrow> restrict (merge I x J y) J = restrict y J" |
|
99 |
"J \<inter> I = {} \<Longrightarrow> restrict (merge I x J y) I = restrict x I" |
|
100 |
"J \<inter> I = {} \<Longrightarrow> restrict (merge I x J y) J = restrict y J" |
|
101 |
by (auto simp: restrict_def intro!: ext) |
|
102 |
||
103 |
lemma extensional_insert_undefined[intro, simp]: |
|
104 |
assumes "a \<in> extensional (insert i I)" |
|
105 |
shows "a(i := undefined) \<in> extensional I" |
|
106 |
using assms unfolding extensional_def by auto |
|
107 |
||
108 |
lemma extensional_insert_cancel[intro, simp]: |
|
109 |
assumes "a \<in> extensional I" |
|
110 |
shows "a \<in> extensional (insert i I)" |
|
111 |
using assms unfolding extensional_def by auto |
|
112 |
||
41095 | 113 |
lemma merge_singleton[simp]: "i \<notin> I \<Longrightarrow> merge I x {i} y = restrict (x(i := y i)) (insert i I)" |
114 |
unfolding merge_def by (auto simp: fun_eq_iff) |
|
115 |
||
116 |
lemma Pi_Int: "Pi I E \<inter> Pi I F = (\<Pi> i\<in>I. E i \<inter> F i)" |
|
117 |
by auto |
|
118 |
||
40859 | 119 |
lemma PiE_Int: "(Pi\<^isub>E I A) \<inter> (Pi\<^isub>E I B) = Pi\<^isub>E I (\<lambda>x. A x \<inter> B x)" |
120 |
by auto |
|
121 |
||
122 |
lemma Pi_cancel_fupd_range[simp]: "i \<notin> I \<Longrightarrow> x \<in> Pi I (B(i := b)) \<longleftrightarrow> x \<in> Pi I B" |
|
123 |
by (auto simp: Pi_def) |
|
124 |
||
125 |
lemma Pi_split_insert_domain[simp]: "x \<in> Pi (insert i I) X \<longleftrightarrow> x \<in> Pi I X \<and> x i \<in> X i" |
|
126 |
by (auto simp: Pi_def) |
|
39088
ca17017c10e6
Measurable on product space is equiv. to measurable components
hoelzl
parents:
39082
diff
changeset
|
127 |
|
40859 | 128 |
lemma Pi_split_domain[simp]: "x \<in> Pi (I \<union> J) X \<longleftrightarrow> x \<in> Pi I X \<and> x \<in> Pi J X" |
129 |
by (auto simp: Pi_def) |
|
130 |
||
131 |
lemma Pi_cancel_fupd[simp]: "i \<notin> I \<Longrightarrow> x(i := a) \<in> Pi I B \<longleftrightarrow> x \<in> Pi I B" |
|
132 |
by (auto simp: Pi_def) |
|
133 |
||
41095 | 134 |
lemma restrict_vimage: |
135 |
assumes "I \<inter> J = {}" |
|
136 |
shows "(\<lambda>x. (restrict x I, restrict x J)) -` (Pi\<^isub>E I E \<times> Pi\<^isub>E J F) = Pi (I \<union> J) (merge I E J F)" |
|
137 |
using assms by (auto simp: restrict_Pi_cancel) |
|
138 |
||
139 |
lemma merge_vimage: |
|
140 |
assumes "I \<inter> J = {}" |
|
141 |
shows "(\<lambda>(x,y). merge I x J y) -` Pi\<^isub>E (I \<union> J) E = Pi I E \<times> Pi J E" |
|
142 |
using assms by (auto simp: restrict_Pi_cancel) |
|
143 |
||
144 |
lemma restrict_fupd[simp]: "i \<notin> I \<Longrightarrow> restrict (f (i := x)) I = restrict f I" |
|
145 |
by (auto simp: restrict_def intro!: ext) |
|
146 |
||
147 |
lemma merge_restrict[simp]: |
|
148 |
"merge I (restrict x I) J y = merge I x J y" |
|
149 |
"merge I x J (restrict y J) = merge I x J y" |
|
150 |
unfolding merge_def by (auto intro!: ext) |
|
151 |
||
152 |
lemma merge_x_x_eq_restrict[simp]: |
|
153 |
"merge I x J x = restrict x (I \<union> J)" |
|
154 |
unfolding merge_def by (auto intro!: ext) |
|
155 |
||
156 |
lemma Pi_fupd_iff: "i \<in> I \<Longrightarrow> f \<in> Pi I (B(i := A)) \<longleftrightarrow> f \<in> Pi (I - {i}) B \<and> f i \<in> A" |
|
157 |
apply auto |
|
158 |
apply (drule_tac x=x in Pi_mem) |
|
159 |
apply (simp_all split: split_if_asm) |
|
160 |
apply (drule_tac x=i in Pi_mem) |
|
161 |
apply (auto dest!: Pi_mem) |
|
162 |
done |
|
163 |
||
164 |
lemma Pi_UN: |
|
165 |
fixes A :: "nat \<Rightarrow> 'i \<Rightarrow> 'a set" |
|
166 |
assumes "finite I" and mono: "\<And>i n m. i \<in> I \<Longrightarrow> n \<le> m \<Longrightarrow> A n i \<subseteq> A m i" |
|
167 |
shows "(\<Union>n. Pi I (A n)) = (\<Pi> i\<in>I. \<Union>n. A n i)" |
|
168 |
proof (intro set_eqI iffI) |
|
169 |
fix f assume "f \<in> (\<Pi> i\<in>I. \<Union>n. A n i)" |
|
170 |
then have "\<forall>i\<in>I. \<exists>n. f i \<in> A n i" by auto |
|
171 |
from bchoice[OF this] obtain n where n: "\<And>i. i \<in> I \<Longrightarrow> f i \<in> (A (n i) i)" by auto |
|
172 |
obtain k where k: "\<And>i. i \<in> I \<Longrightarrow> n i \<le> k" |
|
173 |
using `finite I` finite_nat_set_iff_bounded_le[of "n`I"] by auto |
|
174 |
have "f \<in> Pi I (A k)" |
|
175 |
proof (intro Pi_I) |
|
176 |
fix i assume "i \<in> I" |
|
177 |
from mono[OF this, of "n i" k] k[OF this] n[OF this] |
|
178 |
show "f i \<in> A k i" by auto |
|
179 |
qed |
|
180 |
then show "f \<in> (\<Union>n. Pi I (A n))" by auto |
|
181 |
qed auto |
|
182 |
||
183 |
lemma PiE_cong: |
|
184 |
assumes "\<And>i. i\<in>I \<Longrightarrow> A i = B i" |
|
185 |
shows "Pi\<^isub>E I A = Pi\<^isub>E I B" |
|
186 |
using assms by (auto intro!: Pi_cong) |
|
187 |
||
188 |
lemma restrict_upd[simp]: |
|
189 |
"i \<notin> I \<Longrightarrow> (restrict f I)(i := y) = restrict (f(i := y)) (insert i I)" |
|
190 |
by (auto simp: fun_eq_iff) |
|
191 |
||
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
192 |
lemma Pi_eq_subset: |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
193 |
assumes ne: "\<And>i. i \<in> I \<Longrightarrow> F i \<noteq> {}" "\<And>i. i \<in> I \<Longrightarrow> F' i \<noteq> {}" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
194 |
assumes eq: "Pi\<^isub>E I F = Pi\<^isub>E I F'" and "i \<in> I" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
195 |
shows "F i \<subseteq> F' i" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
196 |
proof |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
197 |
fix x assume "x \<in> F i" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
198 |
with ne have "\<forall>j. \<exists>y. ((j \<in> I \<longrightarrow> y \<in> F j \<and> (i = j \<longrightarrow> x = y)) \<and> (j \<notin> I \<longrightarrow> y = undefined))" by auto |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
199 |
from choice[OF this] guess f .. note f = this |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
200 |
then have "f \<in> Pi\<^isub>E I F" by (auto simp: extensional_def) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
201 |
then have "f \<in> Pi\<^isub>E I F'" using assms by simp |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
202 |
then show "x \<in> F' i" using f `i \<in> I` by auto |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
203 |
qed |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
204 |
|
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
205 |
lemma Pi_eq_iff_not_empty: |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
206 |
assumes ne: "\<And>i. i \<in> I \<Longrightarrow> F i \<noteq> {}" "\<And>i. i \<in> I \<Longrightarrow> F' i \<noteq> {}" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
207 |
shows "Pi\<^isub>E I F = Pi\<^isub>E I F' \<longleftrightarrow> (\<forall>i\<in>I. F i = F' i)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
208 |
proof (intro iffI ballI) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
209 |
fix i assume eq: "Pi\<^isub>E I F = Pi\<^isub>E I F'" and i: "i \<in> I" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
210 |
show "F i = F' i" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
211 |
using Pi_eq_subset[of I F F', OF ne eq i] |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
212 |
using Pi_eq_subset[of I F' F, OF ne(2,1) eq[symmetric] i] |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
213 |
by auto |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
214 |
qed auto |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
215 |
|
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
216 |
lemma Pi_eq_empty_iff: |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
217 |
"Pi\<^isub>E I F = {} \<longleftrightarrow> (\<exists>i\<in>I. F i = {})" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
218 |
proof |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
219 |
assume "Pi\<^isub>E I F = {}" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
220 |
show "\<exists>i\<in>I. F i = {}" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
221 |
proof (rule ccontr) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
222 |
assume "\<not> ?thesis" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
223 |
then have "\<forall>i. \<exists>y. (i \<in> I \<longrightarrow> y \<in> F i) \<and> (i \<notin> I \<longrightarrow> y = undefined)" by auto |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
224 |
from choice[OF this] guess f .. |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
225 |
then have "f \<in> Pi\<^isub>E I F" by (auto simp: extensional_def) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
226 |
with `Pi\<^isub>E I F = {}` show False by auto |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
227 |
qed |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
228 |
qed auto |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
229 |
|
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
230 |
lemma Pi_eq_iff: |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
231 |
"Pi\<^isub>E I F = Pi\<^isub>E I F' \<longleftrightarrow> (\<forall>i\<in>I. F i = F' i) \<or> ((\<exists>i\<in>I. F i = {}) \<and> (\<exists>i\<in>I. F' i = {}))" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
232 |
proof (intro iffI disjCI) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
233 |
assume eq[simp]: "Pi\<^isub>E I F = Pi\<^isub>E I F'" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
234 |
assume "\<not> ((\<exists>i\<in>I. F i = {}) \<and> (\<exists>i\<in>I. F' i = {}))" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
235 |
then have "(\<forall>i\<in>I. F i \<noteq> {}) \<and> (\<forall>i\<in>I. F' i \<noteq> {})" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
236 |
using Pi_eq_empty_iff[of I F] Pi_eq_empty_iff[of I F'] by auto |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
237 |
with Pi_eq_iff_not_empty[of I F F'] show "\<forall>i\<in>I. F i = F' i" by auto |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
238 |
next |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
239 |
assume "(\<forall>i\<in>I. F i = F' i) \<or> (\<exists>i\<in>I. F i = {}) \<and> (\<exists>i\<in>I. F' i = {})" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
240 |
then show "Pi\<^isub>E I F = Pi\<^isub>E I F'" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
241 |
using Pi_eq_empty_iff[of I F] Pi_eq_empty_iff[of I F'] by auto |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
242 |
qed |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
243 |
|
40859 | 244 |
section "Binary products" |
245 |
||
246 |
definition |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
247 |
"pair_measure_generator A B = |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
248 |
\<lparr> space = space A \<times> space B, |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
249 |
sets = {a \<times> b | a b. a \<in> sets A \<and> b \<in> sets B}, |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
250 |
measure = \<lambda>X. \<integral>\<^isup>+x. (\<integral>\<^isup>+y. indicator X (x,y) \<partial>B) \<partial>A \<rparr>" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
251 |
|
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
252 |
definition pair_measure (infixr "\<Otimes>\<^isub>M" 80) where |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
253 |
"A \<Otimes>\<^isub>M B = sigma (pair_measure_generator A B)" |
40859 | 254 |
|
255 |
locale pair_sigma_algebra = M1: sigma_algebra M1 + M2: sigma_algebra M2 |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
256 |
for M1 :: "('a, 'c) measure_space_scheme" and M2 :: "('b, 'd) measure_space_scheme" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
257 |
|
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
258 |
abbreviation (in pair_sigma_algebra) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
259 |
"E \<equiv> pair_measure_generator M1 M2" |
40859 | 260 |
|
261 |
abbreviation (in pair_sigma_algebra) |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
262 |
"P \<equiv> M1 \<Otimes>\<^isub>M M2" |
40859 | 263 |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
264 |
lemma sigma_algebra_pair_measure: |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
265 |
"sets M1 \<subseteq> Pow (space M1) \<Longrightarrow> sets M2 \<subseteq> Pow (space M2) \<Longrightarrow> sigma_algebra (pair_measure M1 M2)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
266 |
by (force simp: pair_measure_def pair_measure_generator_def intro!: sigma_algebra_sigma) |
40859 | 267 |
|
268 |
sublocale pair_sigma_algebra \<subseteq> sigma_algebra P |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
269 |
using M1.space_closed M2.space_closed |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
270 |
by (rule sigma_algebra_pair_measure) |
40859 | 271 |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
272 |
lemma pair_measure_generatorI[intro, simp]: |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
273 |
"x \<in> sets A \<Longrightarrow> y \<in> sets B \<Longrightarrow> x \<times> y \<in> sets (pair_measure_generator A B)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
274 |
by (auto simp add: pair_measure_generator_def) |
40859 | 275 |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
276 |
lemma pair_measureI[intro, simp]: |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
277 |
"x \<in> sets A \<Longrightarrow> y \<in> sets B \<Longrightarrow> x \<times> y \<in> sets (A \<Otimes>\<^isub>M B)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
278 |
by (auto simp add: pair_measure_def) |
40859 | 279 |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
280 |
lemma space_pair_measure: |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
281 |
"space (A \<Otimes>\<^isub>M B) = space A \<times> space B" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
282 |
by (simp add: pair_measure_def pair_measure_generator_def) |
41095 | 283 |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
284 |
lemma sets_pair_measure_generator: |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
285 |
"sets (pair_measure_generator N M) = (\<lambda>(x, y). x \<times> y) ` (sets N \<times> sets M)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
286 |
unfolding pair_measure_generator_def by auto |
41095 | 287 |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
288 |
lemma pair_measure_generator_sets_into_space: |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
289 |
assumes "sets M \<subseteq> Pow (space M)" "sets N \<subseteq> Pow (space N)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
290 |
shows "sets (pair_measure_generator M N) \<subseteq> Pow (space (pair_measure_generator M N))" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
291 |
using assms by (auto simp: pair_measure_generator_def) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
292 |
|
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
293 |
lemma pair_measure_generator_Int_snd: |
40859 | 294 |
assumes "sets S1 \<subseteq> Pow (space S1)" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
295 |
shows "sets (pair_measure_generator S1 (algebra.restricted_space S2 A)) = |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
296 |
sets (algebra.restricted_space (pair_measure_generator S1 S2) (space S1 \<times> A))" |
40859 | 297 |
(is "?L = ?R") |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
298 |
apply (auto simp: pair_measure_generator_def image_iff) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
299 |
using assms |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
300 |
apply (rule_tac x="a \<times> xa" in exI) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
301 |
apply force |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
302 |
using assms |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
303 |
apply (rule_tac x="a" in exI) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
304 |
apply (rule_tac x="b \<inter> A" in exI) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
305 |
apply auto |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
306 |
done |
40859 | 307 |
|
308 |
lemma (in pair_sigma_algebra) |
|
309 |
shows measurable_fst[intro!, simp]: |
|
310 |
"fst \<in> measurable P M1" (is ?fst) |
|
311 |
and measurable_snd[intro!, simp]: |
|
312 |
"snd \<in> measurable P M2" (is ?snd) |
|
39088
ca17017c10e6
Measurable on product space is equiv. to measurable components
hoelzl
parents:
39082
diff
changeset
|
313 |
proof - |
ca17017c10e6
Measurable on product space is equiv. to measurable components
hoelzl
parents:
39082
diff
changeset
|
314 |
{ fix X assume "X \<in> sets M1" |
ca17017c10e6
Measurable on product space is equiv. to measurable components
hoelzl
parents:
39082
diff
changeset
|
315 |
then have "\<exists>X1\<in>sets M1. \<exists>X2\<in>sets M2. fst -` X \<inter> space M1 \<times> space M2 = X1 \<times> X2" |
ca17017c10e6
Measurable on product space is equiv. to measurable components
hoelzl
parents:
39082
diff
changeset
|
316 |
apply - apply (rule bexI[of _ X]) apply (rule bexI[of _ "space M2"]) |
ca17017c10e6
Measurable on product space is equiv. to measurable components
hoelzl
parents:
39082
diff
changeset
|
317 |
using M1.sets_into_space by force+ } |
ca17017c10e6
Measurable on product space is equiv. to measurable components
hoelzl
parents:
39082
diff
changeset
|
318 |
moreover |
ca17017c10e6
Measurable on product space is equiv. to measurable components
hoelzl
parents:
39082
diff
changeset
|
319 |
{ fix X assume "X \<in> sets M2" |
ca17017c10e6
Measurable on product space is equiv. to measurable components
hoelzl
parents:
39082
diff
changeset
|
320 |
then have "\<exists>X1\<in>sets M1. \<exists>X2\<in>sets M2. snd -` X \<inter> space M1 \<times> space M2 = X1 \<times> X2" |
ca17017c10e6
Measurable on product space is equiv. to measurable components
hoelzl
parents:
39082
diff
changeset
|
321 |
apply - apply (rule bexI[of _ "space M1"]) apply (rule bexI[of _ X]) |
ca17017c10e6
Measurable on product space is equiv. to measurable components
hoelzl
parents:
39082
diff
changeset
|
322 |
using M2.sets_into_space by force+ } |
40859 | 323 |
ultimately have "?fst \<and> ?snd" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
324 |
by (fastsimp simp: measurable_def sets_sigma space_pair_measure |
40859 | 325 |
intro!: sigma_sets.Basic) |
326 |
then show ?fst ?snd by auto |
|
327 |
qed |
|
328 |
||
41095 | 329 |
lemma (in pair_sigma_algebra) measurable_pair_iff: |
40859 | 330 |
assumes "sigma_algebra M" |
331 |
shows "f \<in> measurable M P \<longleftrightarrow> |
|
332 |
(fst \<circ> f) \<in> measurable M M1 \<and> (snd \<circ> f) \<in> measurable M M2" |
|
333 |
proof - |
|
334 |
interpret M: sigma_algebra M by fact |
|
335 |
from assms show ?thesis |
|
336 |
proof (safe intro!: measurable_comp[where b=P]) |
|
337 |
assume f: "(fst \<circ> f) \<in> measurable M M1" and s: "(snd \<circ> f) \<in> measurable M M2" |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
338 |
show "f \<in> measurable M P" unfolding pair_measure_def |
40859 | 339 |
proof (rule M.measurable_sigma) |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
340 |
show "sets (pair_measure_generator M1 M2) \<subseteq> Pow (space E)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
341 |
unfolding pair_measure_generator_def using M1.sets_into_space M2.sets_into_space by auto |
40859 | 342 |
show "f \<in> space M \<rightarrow> space E" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
343 |
using f s by (auto simp: mem_Times_iff measurable_def comp_def space_sigma pair_measure_generator_def) |
40859 | 344 |
fix A assume "A \<in> sets E" |
345 |
then obtain B C where "B \<in> sets M1" "C \<in> sets M2" "A = B \<times> C" |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
346 |
unfolding pair_measure_generator_def by auto |
40859 | 347 |
moreover have "(fst \<circ> f) -` B \<inter> space M \<in> sets M" |
348 |
using f `B \<in> sets M1` unfolding measurable_def by auto |
|
349 |
moreover have "(snd \<circ> f) -` C \<inter> space M \<in> sets M" |
|
350 |
using s `C \<in> sets M2` unfolding measurable_def by auto |
|
351 |
moreover have "f -` A \<inter> space M = ((fst \<circ> f) -` B \<inter> space M) \<inter> ((snd \<circ> f) -` C \<inter> space M)" |
|
352 |
unfolding `A = B \<times> C` by (auto simp: vimage_Times) |
|
353 |
ultimately show "f -` A \<inter> space M \<in> sets M" by auto |
|
354 |
qed |
|
355 |
qed |
|
356 |
qed |
|
357 |
||
41095 | 358 |
lemma (in pair_sigma_algebra) measurable_pair: |
40859 | 359 |
assumes "sigma_algebra M" |
41095 | 360 |
assumes "(fst \<circ> f) \<in> measurable M M1" "(snd \<circ> f) \<in> measurable M M2" |
40859 | 361 |
shows "f \<in> measurable M P" |
41095 | 362 |
unfolding measurable_pair_iff[OF assms(1)] using assms(2,3) by simp |
40859 | 363 |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
364 |
lemma pair_measure_generatorE: |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
365 |
assumes "X \<in> sets (pair_measure_generator M1 M2)" |
40859 | 366 |
obtains A B where "X = A \<times> B" "A \<in> sets M1" "B \<in> sets M2" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
367 |
using assms unfolding pair_measure_generator_def by auto |
40859 | 368 |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
369 |
lemma (in pair_sigma_algebra) pair_measure_generator_swap: |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
370 |
"(\<lambda>X. (\<lambda>(x,y). (y,x)) -` X \<inter> space M2 \<times> space M1) ` sets E = sets (pair_measure_generator M2 M1)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
371 |
proof (safe elim!: pair_measure_generatorE) |
40859 | 372 |
fix A B assume "A \<in> sets M1" "B \<in> sets M2" |
373 |
moreover then have "(\<lambda>(x, y). (y, x)) -` (A \<times> B) \<inter> space M2 \<times> space M1 = B \<times> A" |
|
374 |
using M1.sets_into_space M2.sets_into_space by auto |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
375 |
ultimately show "(\<lambda>(x, y). (y, x)) -` (A \<times> B) \<inter> space M2 \<times> space M1 \<in> sets (pair_measure_generator M2 M1)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
376 |
by (auto intro: pair_measure_generatorI) |
40859 | 377 |
next |
378 |
fix A B assume "A \<in> sets M1" "B \<in> sets M2" |
|
379 |
then show "B \<times> A \<in> (\<lambda>X. (\<lambda>(x, y). (y, x)) -` X \<inter> space M2 \<times> space M1) ` sets E" |
|
380 |
using M1.sets_into_space M2.sets_into_space |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
381 |
by (auto intro!: image_eqI[where x="A \<times> B"] pair_measure_generatorI) |
40859 | 382 |
qed |
383 |
||
384 |
lemma (in pair_sigma_algebra) sets_pair_sigma_algebra_swap: |
|
385 |
assumes Q: "Q \<in> sets P" |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
386 |
shows "(\<lambda>(x,y). (y, x)) -` Q \<in> sets (M2 \<Otimes>\<^isub>M M1)" (is "_ \<in> sets ?Q") |
40859 | 387 |
proof - |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
388 |
let "?f Q" = "(\<lambda>(x,y). (y, x)) -` Q \<inter> space M2 \<times> space M1" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
389 |
have *: "(\<lambda>(x,y). (y, x)) -` Q = ?f Q" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
390 |
using sets_into_space[OF Q] by (auto simp: space_pair_measure) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
391 |
have "sets (M2 \<Otimes>\<^isub>M M1) = sets (sigma (pair_measure_generator M2 M1))" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
392 |
unfolding pair_measure_def .. |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
393 |
also have "\<dots> = sigma_sets (space M2 \<times> space M1) (?f ` sets E)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
394 |
unfolding sigma_def pair_measure_generator_swap[symmetric] |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
395 |
by (simp add: pair_measure_generator_def) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
396 |
also have "\<dots> = ?f ` sigma_sets (space M1 \<times> space M2) (sets E)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
397 |
using M1.sets_into_space M2.sets_into_space |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
398 |
by (intro sigma_sets_vimage) (auto simp: pair_measure_generator_def) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
399 |
also have "\<dots> = ?f ` sets P" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
400 |
unfolding pair_measure_def pair_measure_generator_def sigma_def by simp |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
401 |
finally show ?thesis |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
402 |
using Q by (subst *) auto |
40859 | 403 |
qed |
404 |
||
405 |
lemma (in pair_sigma_algebra) pair_sigma_algebra_swap_measurable: |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
406 |
shows "(\<lambda>(x,y). (y, x)) \<in> measurable P (M2 \<Otimes>\<^isub>M M1)" |
40859 | 407 |
(is "?f \<in> measurable ?P ?Q") |
408 |
unfolding measurable_def |
|
409 |
proof (intro CollectI conjI Pi_I ballI) |
|
410 |
fix x assume "x \<in> space ?P" then show "(case x of (x, y) \<Rightarrow> (y, x)) \<in> space ?Q" |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
411 |
unfolding pair_measure_generator_def pair_measure_def by auto |
40859 | 412 |
next |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
413 |
fix A assume "A \<in> sets (M2 \<Otimes>\<^isub>M M1)" |
40859 | 414 |
interpret Q: pair_sigma_algebra M2 M1 by default |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
415 |
with Q.sets_pair_sigma_algebra_swap[OF `A \<in> sets (M2 \<Otimes>\<^isub>M M1)`] |
40859 | 416 |
show "?f -` A \<inter> space ?P \<in> sets ?P" by simp |
417 |
qed |
|
418 |
||
419 |
lemma (in pair_sigma_algebra) measurable_cut_fst: |
|
420 |
assumes "Q \<in> sets P" shows "Pair x -` Q \<in> sets M2" |
|
421 |
proof - |
|
422 |
let ?Q' = "{Q. Q \<subseteq> space P \<and> Pair x -` Q \<in> sets M2}" |
|
423 |
let ?Q = "\<lparr> space = space P, sets = ?Q' \<rparr>" |
|
424 |
interpret Q: sigma_algebra ?Q |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
425 |
proof qed (auto simp: vimage_UN vimage_Diff space_pair_measure) |
40859 | 426 |
have "sets E \<subseteq> sets ?Q" |
427 |
using M1.sets_into_space M2.sets_into_space |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
428 |
by (auto simp: pair_measure_generator_def space_pair_measure) |
40859 | 429 |
then have "sets P \<subseteq> sets ?Q" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
430 |
apply (subst pair_measure_def, intro Q.sets_sigma_subset) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
431 |
by (simp add: pair_measure_def) |
40859 | 432 |
with assms show ?thesis by auto |
433 |
qed |
|
434 |
||
435 |
lemma (in pair_sigma_algebra) measurable_cut_snd: |
|
436 |
assumes Q: "Q \<in> sets P" shows "(\<lambda>x. (x, y)) -` Q \<in> sets M1" (is "?cut Q \<in> sets M1") |
|
437 |
proof - |
|
438 |
interpret Q: pair_sigma_algebra M2 M1 by default |
|
439 |
with Q.measurable_cut_fst[OF sets_pair_sigma_algebra_swap[OF Q], of y] |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
440 |
show ?thesis by (simp add: vimage_compose[symmetric] comp_def) |
40859 | 441 |
qed |
442 |
||
443 |
lemma (in pair_sigma_algebra) measurable_pair_image_snd: |
|
444 |
assumes m: "f \<in> measurable P M" and "x \<in> space M1" |
|
445 |
shows "(\<lambda>y. f (x, y)) \<in> measurable M2 M" |
|
446 |
unfolding measurable_def |
|
447 |
proof (intro CollectI conjI Pi_I ballI) |
|
448 |
fix y assume "y \<in> space M2" with `f \<in> measurable P M` `x \<in> space M1` |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
449 |
show "f (x, y) \<in> space M" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
450 |
unfolding measurable_def pair_measure_generator_def pair_measure_def by auto |
40859 | 451 |
next |
452 |
fix A assume "A \<in> sets M" |
|
453 |
then have "Pair x -` (f -` A \<inter> space P) \<in> sets M2" (is "?C \<in> _") |
|
454 |
using `f \<in> measurable P M` |
|
455 |
by (intro measurable_cut_fst) (auto simp: measurable_def) |
|
456 |
also have "?C = (\<lambda>y. f (x, y)) -` A \<inter> space M2" |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
457 |
using `x \<in> space M1` by (auto simp: pair_measure_generator_def pair_measure_def) |
40859 | 458 |
finally show "(\<lambda>y. f (x, y)) -` A \<inter> space M2 \<in> sets M2" . |
459 |
qed |
|
460 |
||
461 |
lemma (in pair_sigma_algebra) measurable_pair_image_fst: |
|
462 |
assumes m: "f \<in> measurable P M" and "y \<in> space M2" |
|
463 |
shows "(\<lambda>x. f (x, y)) \<in> measurable M1 M" |
|
464 |
proof - |
|
465 |
interpret Q: pair_sigma_algebra M2 M1 by default |
|
466 |
from Q.measurable_pair_image_snd[OF measurable_comp `y \<in> space M2`, |
|
467 |
OF Q.pair_sigma_algebra_swap_measurable m] |
|
468 |
show ?thesis by simp |
|
469 |
qed |
|
470 |
||
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
471 |
lemma (in pair_sigma_algebra) Int_stable_pair_measure_generator: "Int_stable E" |
40859 | 472 |
unfolding Int_stable_def |
473 |
proof (intro ballI) |
|
474 |
fix A B assume "A \<in> sets E" "B \<in> sets E" |
|
475 |
then obtain A1 A2 B1 B2 where "A = A1 \<times> A2" "B = B1 \<times> B2" |
|
476 |
"A1 \<in> sets M1" "A2 \<in> sets M2" "B1 \<in> sets M1" "B2 \<in> sets M2" |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
477 |
unfolding pair_measure_generator_def by auto |
40859 | 478 |
then show "A \<inter> B \<in> sets E" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
479 |
by (auto simp add: times_Int_times pair_measure_generator_def) |
40859 | 480 |
qed |
481 |
||
482 |
lemma finite_measure_cut_measurable: |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
483 |
fixes M1 :: "('a, 'c) measure_space_scheme" and M2 :: "('b, 'd) measure_space_scheme" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
484 |
assumes "sigma_finite_measure M1" "finite_measure M2" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
485 |
assumes "Q \<in> sets (M1 \<Otimes>\<^isub>M M2)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
486 |
shows "(\<lambda>x. measure M2 (Pair x -` Q)) \<in> borel_measurable M1" |
40859 | 487 |
(is "?s Q \<in> _") |
488 |
proof - |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
489 |
interpret M1: sigma_finite_measure M1 by fact |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
490 |
interpret M2: finite_measure M2 by fact |
40859 | 491 |
interpret pair_sigma_algebra M1 M2 by default |
492 |
have [intro]: "sigma_algebra M1" by fact |
|
493 |
have [intro]: "sigma_algebra M2" by fact |
|
494 |
let ?D = "\<lparr> space = space P, sets = {A\<in>sets P. ?s A \<in> borel_measurable M1} \<rparr>" |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
495 |
note space_pair_measure[simp] |
40859 | 496 |
interpret dynkin_system ?D |
497 |
proof (intro dynkin_systemI) |
|
498 |
fix A assume "A \<in> sets ?D" then show "A \<subseteq> space ?D" |
|
499 |
using sets_into_space by simp |
|
500 |
next |
|
501 |
from top show "space ?D \<in> sets ?D" |
|
502 |
by (auto simp add: if_distrib intro!: M1.measurable_If) |
|
503 |
next |
|
504 |
fix A assume "A \<in> sets ?D" |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
505 |
with sets_into_space have "\<And>x. measure M2 (Pair x -` (space M1 \<times> space M2 - A)) = |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
506 |
(if x \<in> space M1 then measure M2 (space M2) - ?s A x else 0)" |
40859 | 507 |
by (auto intro!: M2.finite_measure_compl measurable_cut_fst |
508 |
simp: vimage_Diff) |
|
509 |
with `A \<in> sets ?D` top show "space ?D - A \<in> sets ?D" |
|
41023
9118eb4eb8dc
it is known as the extended reals, not the infinite reals
hoelzl
parents:
40873
diff
changeset
|
510 |
by (auto intro!: Diff M1.measurable_If M1.borel_measurable_pextreal_diff) |
40859 | 511 |
next |
512 |
fix F :: "nat \<Rightarrow> ('a\<times>'b) set" assume "disjoint_family F" "range F \<subseteq> sets ?D" |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
513 |
moreover then have "\<And>x. measure M2 (\<Union>i. Pair x -` F i) = (\<Sum>\<^isub>\<infinity> i. ?s (F i) x)" |
40859 | 514 |
by (intro M2.measure_countably_additive[symmetric]) |
515 |
(auto intro!: measurable_cut_fst simp: disjoint_family_on_def) |
|
516 |
ultimately show "(\<Union>i. F i) \<in> sets ?D" |
|
517 |
by (auto simp: vimage_UN intro!: M1.borel_measurable_psuminf) |
|
518 |
qed |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
519 |
have "sets P = sets ?D" apply (subst pair_measure_def) |
40859 | 520 |
proof (intro dynkin_lemma) |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
521 |
show "Int_stable E" by (rule Int_stable_pair_measure_generator) |
40859 | 522 |
from M1.sets_into_space have "\<And>A. A \<in> sets M1 \<Longrightarrow> {x \<in> space M1. x \<in> A} = A" |
523 |
by auto |
|
524 |
then show "sets E \<subseteq> sets ?D" |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
525 |
by (auto simp: pair_measure_generator_def sets_sigma if_distrib |
40859 | 526 |
intro: sigma_sets.Basic intro!: M1.measurable_If) |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
527 |
qed (auto simp: pair_measure_def) |
40859 | 528 |
with `Q \<in> sets P` have "Q \<in> sets ?D" by simp |
529 |
then show "?s Q \<in> borel_measurable M1" by simp |
|
530 |
qed |
|
531 |
||
532 |
subsection {* Binary products of $\sigma$-finite measure spaces *} |
|
533 |
||
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
534 |
locale pair_sigma_finite = M1: sigma_finite_measure M1 + M2: sigma_finite_measure M2 |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
535 |
for M1 :: "('a, 'c) measure_space_scheme" and M2 :: "('b, 'd) measure_space_scheme" |
40859 | 536 |
|
537 |
sublocale pair_sigma_finite \<subseteq> pair_sigma_algebra M1 M2 |
|
538 |
by default |
|
539 |
||
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
540 |
lemma times_eq_iff: "A \<times> B = C \<times> D \<longleftrightarrow> A = C \<and> B = D \<or> ((A = {} \<or> B = {}) \<and> (C = {} \<or> D = {}))" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
541 |
by auto |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
542 |
|
40859 | 543 |
lemma (in pair_sigma_finite) measure_cut_measurable_fst: |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
544 |
assumes "Q \<in> sets P" shows "(\<lambda>x. measure M2 (Pair x -` Q)) \<in> borel_measurable M1" (is "?s Q \<in> _") |
40859 | 545 |
proof - |
546 |
have [intro]: "sigma_algebra M1" and [intro]: "sigma_algebra M2" by default+ |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
547 |
have M1: "sigma_finite_measure M1" by default |
40859 | 548 |
from M2.disjoint_sigma_finite guess F .. note F = this |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
549 |
then have "\<And>i. F i \<in> sets M2" by auto |
40859 | 550 |
let "?C x i" = "F i \<inter> Pair x -` Q" |
551 |
{ fix i |
|
552 |
let ?R = "M2.restricted_space (F i)" |
|
553 |
have [simp]: "space M1 \<times> F i \<inter> space M1 \<times> space M2 = space M1 \<times> F i" |
|
554 |
using F M2.sets_into_space by auto |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
555 |
let ?R2 = "M2.restricted_space (F i)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
556 |
have "(\<lambda>x. measure ?R2 (Pair x -` (space M1 \<times> space ?R2 \<inter> Q))) \<in> borel_measurable M1" |
40859 | 557 |
proof (intro finite_measure_cut_measurable[OF M1]) |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
558 |
show "finite_measure ?R2" |
40859 | 559 |
using F by (intro M2.restricted_to_finite_measure) auto |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
560 |
have "(space M1 \<times> space ?R2) \<inter> Q \<in> (op \<inter> (space M1 \<times> F i)) ` sets P" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
561 |
using `Q \<in> sets P` by (auto simp: image_iff) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
562 |
also have "\<dots> = sigma_sets (space M1 \<times> F i) ((op \<inter> (space M1 \<times> F i)) ` sets E)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
563 |
unfolding pair_measure_def pair_measure_generator_def sigma_def |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
564 |
using `F i \<in> sets M2` M2.sets_into_space |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
565 |
by (auto intro!: sigma_sets_Int sigma_sets.Basic) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
566 |
also have "\<dots> \<subseteq> sets (M1 \<Otimes>\<^isub>M ?R2)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
567 |
using M1.sets_into_space |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
568 |
apply (auto simp: times_Int_times pair_measure_def pair_measure_generator_def sigma_def |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
569 |
intro!: sigma_sets_subseteq) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
570 |
apply (rule_tac x="a" in exI) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
571 |
apply (rule_tac x="b \<inter> F i" in exI) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
572 |
by auto |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
573 |
finally show "(space M1 \<times> space ?R2) \<inter> Q \<in> sets (M1 \<Otimes>\<^isub>M ?R2)" . |
40859 | 574 |
qed |
575 |
moreover have "\<And>x. Pair x -` (space M1 \<times> F i \<inter> Q) = ?C x i" |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
576 |
using `Q \<in> sets P` sets_into_space by (auto simp: space_pair_measure) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
577 |
ultimately have "(\<lambda>x. measure M2 (?C x i)) \<in> borel_measurable M1" |
40859 | 578 |
by simp } |
579 |
moreover |
|
580 |
{ fix x |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
581 |
have "(\<Sum>\<^isub>\<infinity>i. measure M2 (?C x i)) = measure M2 (\<Union>i. ?C x i)" |
40859 | 582 |
proof (intro M2.measure_countably_additive) |
583 |
show "range (?C x) \<subseteq> sets M2" |
|
584 |
using F `Q \<in> sets P` by (auto intro!: M2.Int measurable_cut_fst) |
|
585 |
have "disjoint_family F" using F by auto |
|
586 |
show "disjoint_family (?C x)" |
|
587 |
by (rule disjoint_family_on_bisimulation[OF `disjoint_family F`]) auto |
|
588 |
qed |
|
589 |
also have "(\<Union>i. ?C x i) = Pair x -` Q" |
|
590 |
using F sets_into_space `Q \<in> sets P` |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
591 |
by (auto simp: space_pair_measure) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
592 |
finally have "measure M2 (Pair x -` Q) = (\<Sum>\<^isub>\<infinity>i. measure M2 (?C x i))" |
40859 | 593 |
by simp } |
594 |
ultimately show ?thesis |
|
595 |
by (auto intro!: M1.borel_measurable_psuminf) |
|
596 |
qed |
|
597 |
||
598 |
lemma (in pair_sigma_finite) measure_cut_measurable_snd: |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
599 |
assumes "Q \<in> sets P" shows "(\<lambda>y. M1.\<mu> ((\<lambda>x. (x, y)) -` Q)) \<in> borel_measurable M2" |
40859 | 600 |
proof - |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
601 |
interpret Q: pair_sigma_finite M2 M1 by default |
40859 | 602 |
note sets_pair_sigma_algebra_swap[OF assms] |
603 |
from Q.measure_cut_measurable_fst[OF this] |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
604 |
show ?thesis by (simp add: vimage_compose[symmetric] comp_def) |
40859 | 605 |
qed |
606 |
||
607 |
lemma (in pair_sigma_algebra) pair_sigma_algebra_measurable: |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
608 |
assumes "f \<in> measurable P M" shows "(\<lambda>(x,y). f (y, x)) \<in> measurable (M2 \<Otimes>\<^isub>M M1) M" |
40859 | 609 |
proof - |
610 |
interpret Q: pair_sigma_algebra M2 M1 by default |
|
611 |
have *: "(\<lambda>(x,y). f (y, x)) = f \<circ> (\<lambda>(x,y). (y, x))" by (simp add: fun_eq_iff) |
|
612 |
show ?thesis |
|
613 |
using Q.pair_sigma_algebra_swap_measurable assms |
|
614 |
unfolding * by (rule measurable_comp) |
|
39088
ca17017c10e6
Measurable on product space is equiv. to measurable components
hoelzl
parents:
39082
diff
changeset
|
615 |
qed |
ca17017c10e6
Measurable on product space is equiv. to measurable components
hoelzl
parents:
39082
diff
changeset
|
616 |
|
40859 | 617 |
lemma (in pair_sigma_finite) pair_measure_alt: |
618 |
assumes "A \<in> sets P" |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
619 |
shows "measure (M1 \<Otimes>\<^isub>M M2) A = (\<integral>\<^isup>+ x. measure M2 (Pair x -` A) \<partial>M1)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
620 |
apply (simp add: pair_measure_def pair_measure_generator_def) |
40859 | 621 |
proof (rule M1.positive_integral_cong) |
622 |
fix x assume "x \<in> space M1" |
|
41023
9118eb4eb8dc
it is known as the extended reals, not the infinite reals
hoelzl
parents:
40873
diff
changeset
|
623 |
have *: "\<And>y. indicator A (x, y) = (indicator (Pair x -` A) y :: pextreal)" |
40859 | 624 |
unfolding indicator_def by auto |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
625 |
show "(\<integral>\<^isup>+ y. indicator A (x, y) \<partial>M2) = measure M2 (Pair x -` A)" |
40859 | 626 |
unfolding * |
627 |
apply (subst M2.positive_integral_indicator) |
|
628 |
apply (rule measurable_cut_fst[OF assms]) |
|
629 |
by simp |
|
630 |
qed |
|
631 |
||
632 |
lemma (in pair_sigma_finite) pair_measure_times: |
|
633 |
assumes A: "A \<in> sets M1" and "B \<in> sets M2" |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
634 |
shows "measure (M1 \<Otimes>\<^isub>M M2) (A \<times> B) = M1.\<mu> A * measure M2 B" |
40859 | 635 |
proof - |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
636 |
have "measure (M1 \<Otimes>\<^isub>M M2) (A \<times> B) = (\<integral>\<^isup>+ x. measure M2 B * indicator A x \<partial>M1)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
637 |
using assms by (auto intro!: M1.positive_integral_cong simp: pair_measure_alt) |
40859 | 638 |
with assms show ?thesis |
639 |
by (simp add: M1.positive_integral_cmult_indicator ac_simps) |
|
640 |
qed |
|
641 |
||
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
642 |
lemma (in pair_sigma_finite) sigma_finite_up_in_pair_measure_generator: |
40859 | 643 |
"\<exists>F::nat \<Rightarrow> ('a \<times> 'b) set. range F \<subseteq> sets E \<and> F \<up> space E \<and> |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
644 |
(\<forall>i. measure (M1 \<Otimes>\<^isub>M M2) (F i) \<noteq> \<omega>)" |
40859 | 645 |
proof - |
646 |
obtain F1 :: "nat \<Rightarrow> 'a set" and F2 :: "nat \<Rightarrow> 'b set" where |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
647 |
F1: "range F1 \<subseteq> sets M1" "F1 \<up> space M1" "\<And>i. M1.\<mu> (F1 i) \<noteq> \<omega>" and |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
648 |
F2: "range F2 \<subseteq> sets M2" "F2 \<up> space M2" "\<And>i. M2.\<mu> (F2 i) \<noteq> \<omega>" |
40859 | 649 |
using M1.sigma_finite_up M2.sigma_finite_up by auto |
650 |
then have space: "space M1 = (\<Union>i. F1 i)" "space M2 = (\<Union>i. F2 i)" |
|
651 |
unfolding isoton_def by auto |
|
652 |
let ?F = "\<lambda>i. F1 i \<times> F2 i" |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
653 |
show ?thesis unfolding isoton_def space_pair_measure |
40859 | 654 |
proof (intro exI[of _ ?F] conjI allI) |
655 |
show "range ?F \<subseteq> sets E" using F1 F2 |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
656 |
by (fastsimp intro!: pair_measure_generatorI) |
40859 | 657 |
next |
658 |
have "space M1 \<times> space M2 \<subseteq> (\<Union>i. ?F i)" |
|
659 |
proof (intro subsetI) |
|
660 |
fix x assume "x \<in> space M1 \<times> space M2" |
|
661 |
then obtain i j where "fst x \<in> F1 i" "snd x \<in> F2 j" |
|
662 |
by (auto simp: space) |
|
663 |
then have "fst x \<in> F1 (max i j)" "snd x \<in> F2 (max j i)" |
|
664 |
using `F1 \<up> space M1` `F2 \<up> space M2` |
|
665 |
by (auto simp: max_def dest: isoton_mono_le) |
|
666 |
then have "(fst x, snd x) \<in> F1 (max i j) \<times> F2 (max i j)" |
|
667 |
by (intro SigmaI) (auto simp add: min_max.sup_commute) |
|
668 |
then show "x \<in> (\<Union>i. ?F i)" by auto |
|
669 |
qed |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
670 |
then show "(\<Union>i. ?F i) = space E" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
671 |
using space by (auto simp: space pair_measure_generator_def) |
40859 | 672 |
next |
673 |
fix i show "F1 i \<times> F2 i \<subseteq> F1 (Suc i) \<times> F2 (Suc i)" |
|
674 |
using `F1 \<up> space M1` `F2 \<up> space M2` unfolding isoton_def |
|
675 |
by auto |
|
676 |
next |
|
677 |
fix i |
|
678 |
from F1 F2 have "F1 i \<in> sets M1" "F2 i \<in> sets M2" by auto |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
679 |
with F1 F2 show "measure P (F1 i \<times> F2 i) \<noteq> \<omega>" |
40859 | 680 |
by (simp add: pair_measure_times) |
681 |
qed |
|
682 |
qed |
|
683 |
||
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
684 |
sublocale pair_sigma_finite \<subseteq> sigma_finite_measure P |
40859 | 685 |
proof |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
686 |
show "measure P {} = 0" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
687 |
unfolding pair_measure_def pair_measure_generator_def sigma_def by auto |
40859 | 688 |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
689 |
show "countably_additive P (measure P)" |
40859 | 690 |
unfolding countably_additive_def |
691 |
proof (intro allI impI) |
|
692 |
fix F :: "nat \<Rightarrow> ('a \<times> 'b) set" |
|
693 |
assume F: "range F \<subseteq> sets P" "disjoint_family F" |
|
694 |
from F have *: "\<And>i. F i \<in> sets P" "(\<Union>i. F i) \<in> sets P" by auto |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
695 |
moreover from F have "\<And>i. (\<lambda>x. measure M2 (Pair x -` F i)) \<in> borel_measurable M1" |
40859 | 696 |
by (intro measure_cut_measurable_fst) auto |
697 |
moreover have "\<And>x. disjoint_family (\<lambda>i. Pair x -` F i)" |
|
698 |
by (intro disjoint_family_on_bisimulation[OF F(2)]) auto |
|
699 |
moreover have "\<And>x. x \<in> space M1 \<Longrightarrow> range (\<lambda>i. Pair x -` F i) \<subseteq> sets M2" |
|
700 |
using F by (auto intro!: measurable_cut_fst) |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
701 |
ultimately show "(\<Sum>\<^isub>\<infinity>n. measure P (F n)) = measure P (\<Union>i. F i)" |
40859 | 702 |
by (simp add: pair_measure_alt vimage_UN M1.positive_integral_psuminf[symmetric] |
703 |
M2.measure_countably_additive |
|
704 |
cong: M1.positive_integral_cong) |
|
705 |
qed |
|
706 |
||
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
707 |
from sigma_finite_up_in_pair_measure_generator guess F :: "nat \<Rightarrow> ('a \<times> 'b) set" .. note F = this |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
708 |
show "\<exists>F::nat \<Rightarrow> ('a \<times> 'b) set. range F \<subseteq> sets P \<and> (\<Union>i. F i) = space P \<and> (\<forall>i. measure P (F i) \<noteq> \<omega>)" |
40859 | 709 |
proof (rule exI[of _ F], intro conjI) |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
710 |
show "range F \<subseteq> sets P" using F by (auto simp: pair_measure_def) |
40859 | 711 |
show "(\<Union>i. F i) = space P" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
712 |
using F by (auto simp: pair_measure_def pair_measure_generator_def isoton_def) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
713 |
show "\<forall>i. measure P (F i) \<noteq> \<omega>" using F by auto |
40859 | 714 |
qed |
715 |
qed |
|
39088
ca17017c10e6
Measurable on product space is equiv. to measurable components
hoelzl
parents:
39082
diff
changeset
|
716 |
|
41661 | 717 |
lemma (in pair_sigma_algebra) sets_swap: |
718 |
assumes "A \<in> sets P" |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
719 |
shows "(\<lambda>(x, y). (y, x)) -` A \<inter> space (M2 \<Otimes>\<^isub>M M1) \<in> sets (M2 \<Otimes>\<^isub>M M1)" |
41661 | 720 |
(is "_ -` A \<inter> space ?Q \<in> sets ?Q") |
721 |
proof - |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
722 |
have *: "(\<lambda>(x, y). (y, x)) -` A \<inter> space ?Q = (\<lambda>(x, y). (y, x)) -` A" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
723 |
using `A \<in> sets P` sets_into_space by (auto simp: space_pair_measure) |
41661 | 724 |
show ?thesis |
725 |
unfolding * using assms by (rule sets_pair_sigma_algebra_swap) |
|
726 |
qed |
|
727 |
||
40859 | 728 |
lemma (in pair_sigma_finite) pair_measure_alt2: |
41706
a207a858d1f6
prefer p2e before e2p; use measure_unique_Int_stable_vimage;
hoelzl
parents:
41705
diff
changeset
|
729 |
assumes A: "A \<in> sets P" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
730 |
shows "\<mu> A = (\<integral>\<^isup>+y. M1.\<mu> ((\<lambda>x. (x, y)) -` A) \<partial>M2)" |
40859 | 731 |
(is "_ = ?\<nu> A") |
732 |
proof - |
|
41706
a207a858d1f6
prefer p2e before e2p; use measure_unique_Int_stable_vimage;
hoelzl
parents:
41705
diff
changeset
|
733 |
interpret Q: pair_sigma_finite M2 M1 by default |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
734 |
from sigma_finite_up_in_pair_measure_generator guess F :: "nat \<Rightarrow> ('a \<times> 'b) set" .. note F = this |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
735 |
have [simp]: "\<And>m. \<lparr> space = space E, sets = sets (sigma E), measure = m \<rparr> = P\<lparr> measure := m \<rparr>" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
736 |
unfolding pair_measure_def by simp |
41706
a207a858d1f6
prefer p2e before e2p; use measure_unique_Int_stable_vimage;
hoelzl
parents:
41705
diff
changeset
|
737 |
|
a207a858d1f6
prefer p2e before e2p; use measure_unique_Int_stable_vimage;
hoelzl
parents:
41705
diff
changeset
|
738 |
have "\<mu> A = Q.\<mu> ((\<lambda>(y, x). (x, y)) -` A \<inter> space Q.P)" |
a207a858d1f6
prefer p2e before e2p; use measure_unique_Int_stable_vimage;
hoelzl
parents:
41705
diff
changeset
|
739 |
proof (rule measure_unique_Int_stable_vimage[OF Int_stable_pair_measure_generator]) |
a207a858d1f6
prefer p2e before e2p; use measure_unique_Int_stable_vimage;
hoelzl
parents:
41705
diff
changeset
|
740 |
show "measure_space P" "measure_space Q.P" by default |
a207a858d1f6
prefer p2e before e2p; use measure_unique_Int_stable_vimage;
hoelzl
parents:
41705
diff
changeset
|
741 |
show "(\<lambda>(y, x). (x, y)) \<in> measurable Q.P P" by (rule Q.pair_sigma_algebra_swap_measurable) |
a207a858d1f6
prefer p2e before e2p; use measure_unique_Int_stable_vimage;
hoelzl
parents:
41705
diff
changeset
|
742 |
show "sets (sigma E) = sets P" "space E = space P" "A \<in> sets (sigma E)" |
a207a858d1f6
prefer p2e before e2p; use measure_unique_Int_stable_vimage;
hoelzl
parents:
41705
diff
changeset
|
743 |
using assms unfolding pair_measure_def by auto |
a207a858d1f6
prefer p2e before e2p; use measure_unique_Int_stable_vimage;
hoelzl
parents:
41705
diff
changeset
|
744 |
show "range F \<subseteq> sets E" "F \<up> space E" "\<And>i. \<mu> (F i) \<noteq> \<omega>" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
745 |
using F `A \<in> sets P` by (auto simp: pair_measure_def) |
40859 | 746 |
fix X assume "X \<in> sets E" |
41706
a207a858d1f6
prefer p2e before e2p; use measure_unique_Int_stable_vimage;
hoelzl
parents:
41705
diff
changeset
|
747 |
then obtain A B where X[simp]: "X = A \<times> B" and AB: "A \<in> sets M1" "B \<in> sets M2" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
748 |
unfolding pair_measure_def pair_measure_generator_def by auto |
41706
a207a858d1f6
prefer p2e before e2p; use measure_unique_Int_stable_vimage;
hoelzl
parents:
41705
diff
changeset
|
749 |
then have "(\<lambda>(y, x). (x, y)) -` X \<inter> space Q.P = B \<times> A" |
a207a858d1f6
prefer p2e before e2p; use measure_unique_Int_stable_vimage;
hoelzl
parents:
41705
diff
changeset
|
750 |
using M1.sets_into_space M2.sets_into_space by (auto simp: space_pair_measure) |
a207a858d1f6
prefer p2e before e2p; use measure_unique_Int_stable_vimage;
hoelzl
parents:
41705
diff
changeset
|
751 |
then show "\<mu> X = Q.\<mu> ((\<lambda>(y, x). (x, y)) -` X \<inter> space Q.P)" |
a207a858d1f6
prefer p2e before e2p; use measure_unique_Int_stable_vimage;
hoelzl
parents:
41705
diff
changeset
|
752 |
using AB by (simp add: pair_measure_times Q.pair_measure_times ac_simps) |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
753 |
qed |
41706
a207a858d1f6
prefer p2e before e2p; use measure_unique_Int_stable_vimage;
hoelzl
parents:
41705
diff
changeset
|
754 |
then show ?thesis |
a207a858d1f6
prefer p2e before e2p; use measure_unique_Int_stable_vimage;
hoelzl
parents:
41705
diff
changeset
|
755 |
using sets_into_space[OF A] Q.pair_measure_alt[OF sets_swap[OF A]] |
a207a858d1f6
prefer p2e before e2p; use measure_unique_Int_stable_vimage;
hoelzl
parents:
41705
diff
changeset
|
756 |
by (auto simp add: Q.pair_measure_alt space_pair_measure |
a207a858d1f6
prefer p2e before e2p; use measure_unique_Int_stable_vimage;
hoelzl
parents:
41705
diff
changeset
|
757 |
intro!: M2.positive_integral_cong arg_cong[where f="M1.\<mu>"]) |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
758 |
qed |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
759 |
|
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
760 |
lemma pair_sigma_algebra_sigma: |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
761 |
assumes 1: "S1 \<up> (space E1)" "range S1 \<subseteq> sets E1" and E1: "sets E1 \<subseteq> Pow (space E1)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
762 |
assumes 2: "S2 \<up> (space E2)" "range S2 \<subseteq> sets E2" and E2: "sets E2 \<subseteq> Pow (space E2)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
763 |
shows "sets (sigma (pair_measure_generator (sigma E1) (sigma E2))) = sets (sigma (pair_measure_generator E1 E2))" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
764 |
(is "sets ?S = sets ?E") |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
765 |
proof - |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
766 |
interpret M1: sigma_algebra "sigma E1" using E1 by (rule sigma_algebra_sigma) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
767 |
interpret M2: sigma_algebra "sigma E2" using E2 by (rule sigma_algebra_sigma) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
768 |
have P: "sets (pair_measure_generator E1 E2) \<subseteq> Pow (space E1 \<times> space E2)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
769 |
using E1 E2 by (auto simp add: pair_measure_generator_def) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
770 |
interpret E: sigma_algebra ?E unfolding pair_measure_generator_def |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
771 |
using E1 E2 by (intro sigma_algebra_sigma) auto |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
772 |
{ fix A assume "A \<in> sets E1" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
773 |
then have "fst -` A \<inter> space ?E = A \<times> (\<Union>i. S2 i)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
774 |
using E1 2 unfolding isoton_def pair_measure_generator_def by auto |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
775 |
also have "\<dots> = (\<Union>i. A \<times> S2 i)" by auto |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
776 |
also have "\<dots> \<in> sets ?E" unfolding pair_measure_generator_def sets_sigma |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
777 |
using 2 `A \<in> sets E1` |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
778 |
by (intro sigma_sets.Union) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
779 |
(auto simp: image_subset_iff intro!: sigma_sets.Basic) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
780 |
finally have "fst -` A \<inter> space ?E \<in> sets ?E" . } |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
781 |
moreover |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
782 |
{ fix B assume "B \<in> sets E2" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
783 |
then have "snd -` B \<inter> space ?E = (\<Union>i. S1 i) \<times> B" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
784 |
using E2 1 unfolding isoton_def pair_measure_generator_def by auto |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
785 |
also have "\<dots> = (\<Union>i. S1 i \<times> B)" by auto |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
786 |
also have "\<dots> \<in> sets ?E" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
787 |
using 1 `B \<in> sets E2` unfolding pair_measure_generator_def sets_sigma |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
788 |
by (intro sigma_sets.Union) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
789 |
(auto simp: image_subset_iff intro!: sigma_sets.Basic) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
790 |
finally have "snd -` B \<inter> space ?E \<in> sets ?E" . } |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
791 |
ultimately have proj: |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
792 |
"fst \<in> measurable ?E (sigma E1) \<and> snd \<in> measurable ?E (sigma E2)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
793 |
using E1 E2 by (subst (1 2) E.measurable_iff_sigma) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
794 |
(auto simp: pair_measure_generator_def sets_sigma) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
795 |
{ fix A B assume A: "A \<in> sets (sigma E1)" and B: "B \<in> sets (sigma E2)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
796 |
with proj have "fst -` A \<inter> space ?E \<in> sets ?E" "snd -` B \<inter> space ?E \<in> sets ?E" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
797 |
unfolding measurable_def by simp_all |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
798 |
moreover have "A \<times> B = (fst -` A \<inter> space ?E) \<inter> (snd -` B \<inter> space ?E)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
799 |
using A B M1.sets_into_space M2.sets_into_space |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
800 |
by (auto simp: pair_measure_generator_def) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
801 |
ultimately have "A \<times> B \<in> sets ?E" by auto } |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
802 |
then have "sigma_sets (space ?E) (sets (pair_measure_generator (sigma E1) (sigma E2))) \<subseteq> sets ?E" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
803 |
by (intro E.sigma_sets_subset) (auto simp add: pair_measure_generator_def sets_sigma) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
804 |
then have subset: "sets ?S \<subseteq> sets ?E" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
805 |
by (simp add: sets_sigma pair_measure_generator_def) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
806 |
show "sets ?S = sets ?E" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
807 |
proof (intro set_eqI iffI) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
808 |
fix A assume "A \<in> sets ?E" then show "A \<in> sets ?S" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
809 |
unfolding sets_sigma |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
810 |
proof induct |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
811 |
case (Basic A) then show ?case |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
812 |
by (auto simp: pair_measure_generator_def sets_sigma intro: sigma_sets.Basic) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
813 |
qed (auto intro: sigma_sets.intros simp: pair_measure_generator_def) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
814 |
next |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
815 |
fix A assume "A \<in> sets ?S" then show "A \<in> sets ?E" using subset by auto |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
816 |
qed |
40859 | 817 |
qed |
818 |
||
819 |
section "Fubinis theorem" |
|
820 |
||
821 |
lemma (in pair_sigma_finite) simple_function_cut: |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
822 |
assumes f: "simple_function P f" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
823 |
shows "(\<lambda>x. \<integral>\<^isup>+y. f (x, y) \<partial>M2) \<in> borel_measurable M1" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
824 |
and "(\<integral>\<^isup>+ x. (\<integral>\<^isup>+ y. f (x, y) \<partial>M2) \<partial>M1) = integral\<^isup>P P f" |
40859 | 825 |
proof - |
826 |
have f_borel: "f \<in> borel_measurable P" |
|
827 |
using f by (rule borel_measurable_simple_function) |
|
828 |
let "?F z" = "f -` {z} \<inter> space P" |
|
829 |
let "?F' x z" = "Pair x -` ?F z" |
|
830 |
{ fix x assume "x \<in> space M1" |
|
831 |
have [simp]: "\<And>z y. indicator (?F z) (x, y) = indicator (?F' x z) y" |
|
832 |
by (auto simp: indicator_def) |
|
833 |
have "\<And>y. y \<in> space M2 \<Longrightarrow> (x, y) \<in> space P" using `x \<in> space M1` |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
834 |
by (simp add: space_pair_measure) |
40859 | 835 |
moreover have "\<And>x z. ?F' x z \<in> sets M2" using f_borel |
836 |
by (intro borel_measurable_vimage measurable_cut_fst) |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
837 |
ultimately have "simple_function M2 (\<lambda> y. f (x, y))" |
40859 | 838 |
apply (rule_tac M2.simple_function_cong[THEN iffD2, OF _]) |
839 |
apply (rule simple_function_indicator_representation[OF f]) |
|
840 |
using `x \<in> space M1` by (auto simp del: space_sigma) } |
|
841 |
note M2_sf = this |
|
842 |
{ fix x assume x: "x \<in> space M1" |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
843 |
then have "(\<integral>\<^isup>+y. f (x, y) \<partial>M2) = (\<Sum>z\<in>f ` space P. z * M2.\<mu> (?F' x z))" |
40859 | 844 |
unfolding M2.positive_integral_eq_simple_integral[OF M2_sf[OF x]] |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
845 |
unfolding simple_integral_def |
40859 | 846 |
proof (safe intro!: setsum_mono_zero_cong_left) |
847 |
from f show "finite (f ` space P)" by (rule simple_functionD) |
|
848 |
next |
|
849 |
fix y assume "y \<in> space M2" then show "f (x, y) \<in> f ` space P" |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
850 |
using `x \<in> space M1` by (auto simp: space_pair_measure) |
40859 | 851 |
next |
852 |
fix x' y assume "(x', y) \<in> space P" |
|
853 |
"f (x', y) \<notin> (\<lambda>y. f (x, y)) ` space M2" |
|
854 |
then have *: "?F' x (f (x', y)) = {}" |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
855 |
by (force simp: space_pair_measure) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
856 |
show "f (x', y) * M2.\<mu> (?F' x (f (x', y))) = 0" |
40859 | 857 |
unfolding * by simp |
858 |
qed (simp add: vimage_compose[symmetric] comp_def |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
859 |
space_pair_measure) } |
40859 | 860 |
note eq = this |
861 |
moreover have "\<And>z. ?F z \<in> sets P" |
|
862 |
by (auto intro!: f_borel borel_measurable_vimage simp del: space_sigma) |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
863 |
moreover then have "\<And>z. (\<lambda>x. M2.\<mu> (?F' x z)) \<in> borel_measurable M1" |
40859 | 864 |
by (auto intro!: measure_cut_measurable_fst simp del: vimage_Int) |
865 |
ultimately |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
866 |
show "(\<lambda>x. \<integral>\<^isup>+y. f (x, y) \<partial>M2) \<in> borel_measurable M1" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
867 |
and "(\<integral>\<^isup>+ x. (\<integral>\<^isup>+ y. f (x, y) \<partial>M2) \<partial>M1) = integral\<^isup>P P f" |
40859 | 868 |
by (auto simp del: vimage_Int cong: measurable_cong |
41023
9118eb4eb8dc
it is known as the extended reals, not the infinite reals
hoelzl
parents:
40873
diff
changeset
|
869 |
intro!: M1.borel_measurable_pextreal_setsum |
40859 | 870 |
simp add: M1.positive_integral_setsum simple_integral_def |
871 |
M1.positive_integral_cmult |
|
872 |
M1.positive_integral_cong[OF eq] |
|
873 |
positive_integral_eq_simple_integral[OF f] |
|
874 |
pair_measure_alt[symmetric]) |
|
875 |
qed |
|
876 |
||
877 |
lemma (in pair_sigma_finite) positive_integral_fst_measurable: |
|
878 |
assumes f: "f \<in> borel_measurable P" |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
879 |
shows "(\<lambda>x. \<integral>\<^isup>+ y. f (x, y) \<partial>M2) \<in> borel_measurable M1" |
40859 | 880 |
(is "?C f \<in> borel_measurable M1") |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
881 |
and "(\<integral>\<^isup>+ x. (\<integral>\<^isup>+ y. f (x, y) \<partial>M2) \<partial>M1) = integral\<^isup>P P f" |
40859 | 882 |
proof - |
883 |
from borel_measurable_implies_simple_function_sequence[OF f] |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
884 |
obtain F where F: "\<And>i. simple_function P (F i)" "F \<up> f" by auto |
40859 | 885 |
then have F_borel: "\<And>i. F i \<in> borel_measurable P" |
886 |
and F_mono: "\<And>i x. F i x \<le> F (Suc i) x" |
|
887 |
and F_SUPR: "\<And>x. (SUP i. F i x) = f x" |
|
41097
a1abfa4e2b44
use SUPR_ and INFI_apply instead of SUPR_, INFI_fun_expand
hoelzl
parents:
41096
diff
changeset
|
888 |
unfolding isoton_fun_expand unfolding isoton_def le_fun_def |
40859 | 889 |
by (auto intro: borel_measurable_simple_function) |
890 |
note sf = simple_function_cut[OF F(1)] |
|
41097
a1abfa4e2b44
use SUPR_ and INFI_apply instead of SUPR_, INFI_fun_expand
hoelzl
parents:
41096
diff
changeset
|
891 |
then have "(\<lambda>x. SUP i. ?C (F i) x) \<in> borel_measurable M1" |
a1abfa4e2b44
use SUPR_ and INFI_apply instead of SUPR_, INFI_fun_expand
hoelzl
parents:
41096
diff
changeset
|
892 |
using F(1) by auto |
40859 | 893 |
moreover |
894 |
{ fix x assume "x \<in> space M1" |
|
895 |
have isotone: "(\<lambda> i y. F i (x, y)) \<up> (\<lambda>y. f (x, y))" |
|
896 |
using `F \<up> f` unfolding isoton_fun_expand |
|
897 |
by (auto simp: isoton_def) |
|
898 |
note measurable_pair_image_snd[OF F_borel`x \<in> space M1`] |
|
899 |
from M2.positive_integral_isoton[OF isotone this] |
|
900 |
have "(SUP i. ?C (F i) x) = ?C f x" |
|
901 |
by (simp add: isoton_def) } |
|
902 |
note SUPR_C = this |
|
903 |
ultimately show "?C f \<in> borel_measurable M1" |
|
41097
a1abfa4e2b44
use SUPR_ and INFI_apply instead of SUPR_, INFI_fun_expand
hoelzl
parents:
41096
diff
changeset
|
904 |
by (simp cong: measurable_cong) |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
905 |
have "(\<integral>\<^isup>+x. (SUP i. F i x) \<partial>P) = (SUP i. integral\<^isup>P P (F i))" |
40859 | 906 |
using F_borel F_mono |
907 |
by (auto intro!: positive_integral_monotone_convergence_SUP[symmetric]) |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
908 |
also have "(SUP i. integral\<^isup>P P (F i)) = (SUP i. \<integral>\<^isup>+ x. (\<integral>\<^isup>+ y. F i (x, y) \<partial>M2) \<partial>M1)" |
40859 | 909 |
unfolding sf(2) by simp |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
910 |
also have "\<dots> = \<integral>\<^isup>+ x. (SUP i. \<integral>\<^isup>+ y. F i (x, y) \<partial>M2) \<partial>M1" |
40859 | 911 |
by (auto intro!: M1.positive_integral_monotone_convergence_SUP[OF _ sf(1)] |
912 |
M2.positive_integral_mono F_mono) |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
913 |
also have "\<dots> = \<integral>\<^isup>+ x. (\<integral>\<^isup>+ y. (SUP i. F i (x, y)) \<partial>M2) \<partial>M1" |
40859 | 914 |
using F_borel F_mono |
915 |
by (auto intro!: M2.positive_integral_monotone_convergence_SUP |
|
916 |
M1.positive_integral_cong measurable_pair_image_snd) |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
917 |
finally show "(\<integral>\<^isup>+ x. (\<integral>\<^isup>+ y. f (x, y) \<partial>M2) \<partial>M1) = integral\<^isup>P P f" |
40859 | 918 |
unfolding F_SUPR by simp |
919 |
qed |
|
920 |
||
41831 | 921 |
lemma (in pair_sigma_finite) measure_preserving_swap: |
922 |
"(\<lambda>(x,y). (y, x)) \<in> measure_preserving (M1 \<Otimes>\<^isub>M M2) (M2 \<Otimes>\<^isub>M M1)" |
|
923 |
proof |
|
924 |
interpret Q: pair_sigma_finite M2 M1 by default |
|
925 |
show *: "(\<lambda>(x,y). (y, x)) \<in> measurable (M1 \<Otimes>\<^isub>M M2) (M2 \<Otimes>\<^isub>M M1)" |
|
926 |
using pair_sigma_algebra_swap_measurable . |
|
927 |
fix X assume "X \<in> sets (M2 \<Otimes>\<^isub>M M1)" |
|
928 |
from measurable_sets[OF * this] this Q.sets_into_space[OF this] |
|
929 |
show "measure (M1 \<Otimes>\<^isub>M M2) ((\<lambda>(x, y). (y, x)) -` X \<inter> space P) = measure (M2 \<Otimes>\<^isub>M M1) X" |
|
930 |
by (auto intro!: M1.positive_integral_cong arg_cong[where f="M2.\<mu>"] |
|
931 |
simp: pair_measure_alt Q.pair_measure_alt2 space_pair_measure) |
|
932 |
qed |
|
933 |
||
41661 | 934 |
lemma (in pair_sigma_finite) positive_integral_product_swap: |
935 |
assumes f: "f \<in> borel_measurable P" |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
936 |
shows "(\<integral>\<^isup>+x. f (case x of (x,y)\<Rightarrow>(y,x)) \<partial>(M2 \<Otimes>\<^isub>M M1)) = integral\<^isup>P P f" |
41661 | 937 |
proof - |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
938 |
interpret Q: pair_sigma_finite M2 M1 by default |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
939 |
have "sigma_algebra P" by default |
41831 | 940 |
with f show ?thesis |
941 |
by (subst Q.positive_integral_vimage[OF _ Q.measure_preserving_swap]) auto |
|
41661 | 942 |
qed |
943 |
||
40859 | 944 |
lemma (in pair_sigma_finite) positive_integral_snd_measurable: |
945 |
assumes f: "f \<in> borel_measurable P" |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
946 |
shows "(\<integral>\<^isup>+ y. (\<integral>\<^isup>+ x. f (x, y) \<partial>M1) \<partial>M2) = integral\<^isup>P P f" |
40859 | 947 |
proof - |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
948 |
interpret Q: pair_sigma_finite M2 M1 by default |
40859 | 949 |
note pair_sigma_algebra_measurable[OF f] |
950 |
from Q.positive_integral_fst_measurable[OF this] |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
951 |
have "(\<integral>\<^isup>+ y. (\<integral>\<^isup>+ x. f (x, y) \<partial>M1) \<partial>M2) = (\<integral>\<^isup>+ (x, y). f (y, x) \<partial>Q.P)" |
40859 | 952 |
by simp |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
953 |
also have "(\<integral>\<^isup>+ (x, y). f (y, x) \<partial>Q.P) = integral\<^isup>P P f" |
41661 | 954 |
unfolding positive_integral_product_swap[OF f, symmetric] |
955 |
by (auto intro!: Q.positive_integral_cong) |
|
40859 | 956 |
finally show ?thesis . |
957 |
qed |
|
958 |
||
959 |
lemma (in pair_sigma_finite) Fubini: |
|
960 |
assumes f: "f \<in> borel_measurable P" |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
961 |
shows "(\<integral>\<^isup>+ y. (\<integral>\<^isup>+ x. f (x, y) \<partial>M1) \<partial>M2) = (\<integral>\<^isup>+ x. (\<integral>\<^isup>+ y. f (x, y) \<partial>M2) \<partial>M1)" |
40859 | 962 |
unfolding positive_integral_snd_measurable[OF assms] |
963 |
unfolding positive_integral_fst_measurable[OF assms] .. |
|
964 |
||
965 |
lemma (in pair_sigma_finite) AE_pair: |
|
966 |
assumes "almost_everywhere (\<lambda>x. Q x)" |
|
967 |
shows "M1.almost_everywhere (\<lambda>x. M2.almost_everywhere (\<lambda>y. Q (x, y)))" |
|
968 |
proof - |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
969 |
obtain N where N: "N \<in> sets P" "\<mu> N = 0" "{x\<in>space P. \<not> Q x} \<subseteq> N" |
40859 | 970 |
using assms unfolding almost_everywhere_def by auto |
971 |
show ?thesis |
|
972 |
proof (rule M1.AE_I) |
|
973 |
from N measure_cut_measurable_fst[OF `N \<in> sets P`] |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
974 |
show "M1.\<mu> {x\<in>space M1. M2.\<mu> (Pair x -` N) \<noteq> 0} = 0" |
40859 | 975 |
by (simp add: M1.positive_integral_0_iff pair_measure_alt vimage_def) |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
976 |
show "{x \<in> space M1. M2.\<mu> (Pair x -` N) \<noteq> 0} \<in> sets M1" |
41023
9118eb4eb8dc
it is known as the extended reals, not the infinite reals
hoelzl
parents:
40873
diff
changeset
|
977 |
by (intro M1.borel_measurable_pextreal_neq_const measure_cut_measurable_fst N) |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
978 |
{ fix x assume "x \<in> space M1" "M2.\<mu> (Pair x -` N) = 0" |
40859 | 979 |
have "M2.almost_everywhere (\<lambda>y. Q (x, y))" |
980 |
proof (rule M2.AE_I) |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
981 |
show "M2.\<mu> (Pair x -` N) = 0" by fact |
40859 | 982 |
show "Pair x -` N \<in> sets M2" by (intro measurable_cut_fst N) |
983 |
show "{y \<in> space M2. \<not> Q (x, y)} \<subseteq> Pair x -` N" |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
984 |
using N `x \<in> space M1` unfolding space_sigma space_pair_measure by auto |
40859 | 985 |
qed } |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
986 |
then show "{x \<in> space M1. \<not> M2.almost_everywhere (\<lambda>y. Q (x, y))} \<subseteq> {x \<in> space M1. M2.\<mu> (Pair x -` N) \<noteq> 0}" |
40859 | 987 |
by auto |
39088
ca17017c10e6
Measurable on product space is equiv. to measurable components
hoelzl
parents:
39082
diff
changeset
|
988 |
qed |
ca17017c10e6
Measurable on product space is equiv. to measurable components
hoelzl
parents:
39082
diff
changeset
|
989 |
qed |
35833 | 990 |
|
41026
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
991 |
lemma (in pair_sigma_algebra) measurable_product_swap: |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
992 |
"f \<in> measurable (M2 \<Otimes>\<^isub>M M1) M \<longleftrightarrow> (\<lambda>(x,y). f (y,x)) \<in> measurable P M" |
41026
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
993 |
proof - |
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
994 |
interpret Q: pair_sigma_algebra M2 M1 by default |
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
995 |
show ?thesis |
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
996 |
using pair_sigma_algebra_measurable[of "\<lambda>(x,y). f (y, x)"] |
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
997 |
by (auto intro!: pair_sigma_algebra_measurable Q.pair_sigma_algebra_measurable iffI) |
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
998 |
qed |
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
999 |
|
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1000 |
lemma (in pair_sigma_finite) integrable_product_swap: |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1001 |
assumes "integrable P f" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1002 |
shows "integrable (M2 \<Otimes>\<^isub>M M1) (\<lambda>(x,y). f (y,x))" |
41026
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1003 |
proof - |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1004 |
interpret Q: pair_sigma_finite M2 M1 by default |
41661 | 1005 |
have *: "(\<lambda>(x,y). f (y,x)) = (\<lambda>x. f (case x of (x,y)\<Rightarrow>(y,x)))" by (auto simp: fun_eq_iff) |
1006 |
show ?thesis unfolding * |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1007 |
using assms unfolding integrable_def |
41661 | 1008 |
apply (subst (1 2) positive_integral_product_swap) |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1009 |
using `integrable P f` unfolding integrable_def |
41661 | 1010 |
by (auto simp: *[symmetric] Q.measurable_product_swap[symmetric]) |
1011 |
qed |
|
1012 |
||
1013 |
lemma (in pair_sigma_finite) integrable_product_swap_iff: |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1014 |
"integrable (M2 \<Otimes>\<^isub>M M1) (\<lambda>(x,y). f (y,x)) \<longleftrightarrow> integrable P f" |
41661 | 1015 |
proof - |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1016 |
interpret Q: pair_sigma_finite M2 M1 by default |
41661 | 1017 |
from Q.integrable_product_swap[of "\<lambda>(x,y). f (y,x)"] integrable_product_swap[of f] |
1018 |
show ?thesis by auto |
|
41026
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1019 |
qed |
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1020 |
|
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1021 |
lemma (in pair_sigma_finite) integral_product_swap: |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1022 |
assumes "integrable P f" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1023 |
shows "(\<integral>(x,y). f (y,x) \<partial>(M2 \<Otimes>\<^isub>M M1)) = integral\<^isup>L P f" |
41026
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1024 |
proof - |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1025 |
interpret Q: pair_sigma_finite M2 M1 by default |
41661 | 1026 |
have *: "(\<lambda>(x,y). f (y,x)) = (\<lambda>x. f (case x of (x,y)\<Rightarrow>(y,x)))" by (auto simp: fun_eq_iff) |
41026
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1027 |
show ?thesis |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1028 |
unfolding lebesgue_integral_def * |
41661 | 1029 |
apply (subst (1 2) positive_integral_product_swap) |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1030 |
using `integrable P f` unfolding integrable_def |
41661 | 1031 |
by (auto simp: *[symmetric] Q.measurable_product_swap[symmetric]) |
41026
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1032 |
qed |
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1033 |
|
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1034 |
lemma (in pair_sigma_finite) integrable_fst_measurable: |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1035 |
assumes f: "integrable P f" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1036 |
shows "M1.almost_everywhere (\<lambda>x. integrable M2 (\<lambda> y. f (x, y)))" (is "?AE") |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1037 |
and "(\<integral>x. (\<integral>y. f (x, y) \<partial>M2) \<partial>M1) = integral\<^isup>L P f" (is "?INT") |
41026
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1038 |
proof - |
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1039 |
let "?pf x" = "Real (f x)" and "?nf x" = "Real (- f x)" |
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1040 |
have |
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1041 |
borel: "?nf \<in> borel_measurable P""?pf \<in> borel_measurable P" and |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1042 |
int: "integral\<^isup>P P ?nf \<noteq> \<omega>" "integral\<^isup>P P ?pf \<noteq> \<omega>" |
41026
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1043 |
using assms by auto |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1044 |
have "(\<integral>\<^isup>+x. (\<integral>\<^isup>+y. Real (f (x, y)) \<partial>M2) \<partial>M1) \<noteq> \<omega>" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1045 |
"(\<integral>\<^isup>+x. (\<integral>\<^isup>+y. Real (- f (x, y)) \<partial>M2) \<partial>M1) \<noteq> \<omega>" |
41026
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1046 |
using borel[THEN positive_integral_fst_measurable(1)] int |
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1047 |
unfolding borel[THEN positive_integral_fst_measurable(2)] by simp_all |
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1048 |
with borel[THEN positive_integral_fst_measurable(1)] |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1049 |
have AE: "M1.almost_everywhere (\<lambda>x. (\<integral>\<^isup>+y. Real (f (x, y)) \<partial>M2) \<noteq> \<omega>)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1050 |
"M1.almost_everywhere (\<lambda>x. (\<integral>\<^isup>+y. Real (- f (x, y)) \<partial>M2) \<noteq> \<omega>)" |
41026
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1051 |
by (auto intro!: M1.positive_integral_omega_AE) |
41705 | 1052 |
then show ?AE using assms |
1053 |
by (simp add: measurable_pair_image_snd integrable_def) |
|
1054 |
{ fix f assume borel: "(\<lambda>x. Real (f x)) \<in> borel_measurable P" |
|
1055 |
and int: "integral\<^isup>P P (\<lambda>x. Real (f x)) \<noteq> \<omega>" |
|
1056 |
and AE: "M1.almost_everywhere (\<lambda>x. (\<integral>\<^isup>+y. Real (f (x, y)) \<partial>M2) \<noteq> \<omega>)" |
|
1057 |
have "integrable M1 (\<lambda>x. real (\<integral>\<^isup>+y. Real (f (x, y)) \<partial>M2))" (is "integrable M1 ?f") |
|
1058 |
proof (intro integrable_def[THEN iffD2] conjI) |
|
1059 |
show "?f \<in> borel_measurable M1" |
|
1060 |
using borel by (auto intro!: M1.borel_measurable_real positive_integral_fst_measurable) |
|
1061 |
have "(\<integral>\<^isup>+x. Real (?f x) \<partial>M1) = (\<integral>\<^isup>+x. (\<integral>\<^isup>+y. Real (f (x, y)) \<partial>M2) \<partial>M1)" |
|
1062 |
using AE by (auto intro!: M1.positive_integral_cong_AE simp: Real_real) |
|
1063 |
then show "(\<integral>\<^isup>+x. Real (?f x) \<partial>M1) \<noteq> \<omega>" |
|
1064 |
using positive_integral_fst_measurable[OF borel] int by simp |
|
1065 |
have "(\<integral>\<^isup>+x. Real (- ?f x) \<partial>M1) = (\<integral>\<^isup>+x. 0 \<partial>M1)" |
|
1066 |
by (intro M1.positive_integral_cong) simp |
|
1067 |
then show "(\<integral>\<^isup>+x. Real (- ?f x) \<partial>M1) \<noteq> \<omega>" by simp |
|
1068 |
qed } |
|
1069 |
from this[OF borel(1) int(1) AE(2)] this[OF borel(2) int(2) AE(1)] |
|
1070 |
show ?INT |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1071 |
unfolding lebesgue_integral_def[of P] lebesgue_integral_def[of M2] |
41026
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1072 |
borel[THEN positive_integral_fst_measurable(2), symmetric] |
41705 | 1073 |
using AE by (simp add: M1.integral_real) |
41026
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1074 |
qed |
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1075 |
|
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1076 |
lemma (in pair_sigma_finite) integrable_snd_measurable: |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1077 |
assumes f: "integrable P f" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1078 |
shows "M2.almost_everywhere (\<lambda>y. integrable M1 (\<lambda>x. f (x, y)))" (is "?AE") |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1079 |
and "(\<integral>y. (\<integral>x. f (x, y) \<partial>M1) \<partial>M2) = integral\<^isup>L P f" (is "?INT") |
41026
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1080 |
proof - |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1081 |
interpret Q: pair_sigma_finite M2 M1 by default |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1082 |
have Q_int: "integrable Q.P (\<lambda>(x, y). f (y, x))" |
41661 | 1083 |
using f unfolding integrable_product_swap_iff . |
41026
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1084 |
show ?INT |
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1085 |
using Q.integrable_fst_measurable(2)[OF Q_int] |
41661 | 1086 |
using integral_product_swap[OF f] by simp |
41026
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1087 |
show ?AE |
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1088 |
using Q.integrable_fst_measurable(1)[OF Q_int] |
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1089 |
by simp |
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1090 |
qed |
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1091 |
|
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1092 |
lemma (in pair_sigma_finite) Fubini_integral: |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1093 |
assumes f: "integrable P f" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1094 |
shows "(\<integral>y. (\<integral>x. f (x, y) \<partial>M1) \<partial>M2) = (\<integral>x. (\<integral>y. f (x, y) \<partial>M2) \<partial>M1)" |
41026
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1095 |
unfolding integrable_snd_measurable[OF assms] |
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1096 |
unfolding integrable_fst_measurable[OF assms] .. |
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1097 |
|
40859 | 1098 |
section "Finite product spaces" |
1099 |
||
1100 |
section "Products" |
|
1101 |
||
1102 |
locale product_sigma_algebra = |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1103 |
fixes M :: "'i \<Rightarrow> ('a, 'b) measure_space_scheme" |
40859 | 1104 |
assumes sigma_algebras: "\<And>i. sigma_algebra (M i)" |
1105 |
||
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1106 |
locale finite_product_sigma_algebra = product_sigma_algebra M |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1107 |
for M :: "'i \<Rightarrow> ('a, 'b) measure_space_scheme" + |
40859 | 1108 |
fixes I :: "'i set" |
1109 |
assumes finite_index: "finite I" |
|
1110 |
||
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1111 |
definition |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1112 |
"product_algebra_generator I M = \<lparr> space = (\<Pi>\<^isub>E i \<in> I. space (M i)), |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1113 |
sets = Pi\<^isub>E I ` (\<Pi> i \<in> I. sets (M i)), |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1114 |
measure = \<lambda>A. (\<Prod>i\<in>I. measure (M i) ((SOME F. A = Pi\<^isub>E I F) i)) \<rparr>" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1115 |
|
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1116 |
definition product_algebra_def: |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1117 |
"Pi\<^isub>M I M = sigma (product_algebra_generator I M) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1118 |
\<lparr> measure := (SOME \<mu>. sigma_finite_measure (sigma (product_algebra_generator I M) \<lparr> measure := \<mu> \<rparr>) \<and> |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1119 |
(\<forall>A\<in>\<Pi> i\<in>I. sets (M i). \<mu> (Pi\<^isub>E I A) = (\<Prod>i\<in>I. measure (M i) (A i))))\<rparr>" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1120 |
|
40859 | 1121 |
syntax |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1122 |
"_PiM" :: "[pttrn, 'i set, ('a, 'b) measure_space_scheme] => |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1123 |
('i => 'a, 'b) measure_space_scheme" ("(3PIM _:_./ _)" 10) |
40859 | 1124 |
|
1125 |
syntax (xsymbols) |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1126 |
"_PiM" :: "[pttrn, 'i set, ('a, 'b) measure_space_scheme] => |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1127 |
('i => 'a, 'b) measure_space_scheme" ("(3\<Pi>\<^isub>M _\<in>_./ _)" 10) |
40859 | 1128 |
|
1129 |
syntax (HTML output) |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1130 |
"_PiM" :: "[pttrn, 'i set, ('a, 'b) measure_space_scheme] => |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1131 |
('i => 'a, 'b) measure_space_scheme" ("(3\<Pi>\<^isub>M _\<in>_./ _)" 10) |
40859 | 1132 |
|
1133 |
translations |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1134 |
"PIM x:I. M" == "CONST Pi\<^isub>M I (%x. M)" |
40859 | 1135 |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1136 |
abbreviation (in finite_product_sigma_algebra) "G \<equiv> product_algebra_generator I M" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1137 |
abbreviation (in finite_product_sigma_algebra) "P \<equiv> Pi\<^isub>M I M" |
40859 | 1138 |
|
1139 |
sublocale product_sigma_algebra \<subseteq> M: sigma_algebra "M i" for i by (rule sigma_algebras) |
|
1140 |
||
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1141 |
lemma sigma_into_space: |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1142 |
assumes "sets M \<subseteq> Pow (space M)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1143 |
shows "sets (sigma M) \<subseteq> Pow (space M)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1144 |
using sigma_sets_into_sp[OF assms] unfolding sigma_def by auto |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1145 |
|
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1146 |
lemma (in product_sigma_algebra) product_algebra_generator_into_space: |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1147 |
"sets (product_algebra_generator I M) \<subseteq> Pow (space (product_algebra_generator I M))" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1148 |
using M.sets_into_space unfolding product_algebra_generator_def |
40859 | 1149 |
by auto blast |
1150 |
||
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1151 |
lemma (in product_sigma_algebra) product_algebra_into_space: |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1152 |
"sets (Pi\<^isub>M I M) \<subseteq> Pow (space (Pi\<^isub>M I M))" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1153 |
using product_algebra_generator_into_space |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1154 |
by (auto intro!: sigma_into_space simp add: product_algebra_def) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1155 |
|
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1156 |
lemma (in product_sigma_algebra) sigma_algebra_product_algebra: "sigma_algebra (Pi\<^isub>M I M)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1157 |
using product_algebra_generator_into_space unfolding product_algebra_def |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1158 |
by (rule sigma_algebra.sigma_algebra_cong[OF sigma_algebra_sigma]) simp_all |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1159 |
|
40859 | 1160 |
sublocale finite_product_sigma_algebra \<subseteq> sigma_algebra P |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1161 |
using sigma_algebra_product_algebra . |
40859 | 1162 |
|
41095 | 1163 |
lemma product_algebraE: |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1164 |
assumes "A \<in> sets (product_algebra_generator I M)" |
41095 | 1165 |
obtains E where "A = Pi\<^isub>E I E" "E \<in> (\<Pi> i\<in>I. sets (M i))" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1166 |
using assms unfolding product_algebra_generator_def by auto |
41095 | 1167 |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1168 |
lemma product_algebra_generatorI[intro]: |
41095 | 1169 |
assumes "E \<in> (\<Pi> i\<in>I. sets (M i))" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1170 |
shows "Pi\<^isub>E I E \<in> sets (product_algebra_generator I M)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1171 |
using assms unfolding product_algebra_generator_def by auto |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1172 |
|
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1173 |
lemma space_product_algebra_generator[simp]: |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1174 |
"space (product_algebra_generator I M) = Pi\<^isub>E I (\<lambda>i. space (M i))" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1175 |
unfolding product_algebra_generator_def by simp |
41095 | 1176 |
|
40859 | 1177 |
lemma space_product_algebra[simp]: |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1178 |
"space (Pi\<^isub>M I M) = (\<Pi>\<^isub>E i\<in>I. space (M i))" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1179 |
unfolding product_algebra_def product_algebra_generator_def by simp |
40859 | 1180 |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1181 |
lemma sets_product_algebra: |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1182 |
"sets (Pi\<^isub>M I M) = sets (sigma (product_algebra_generator I M))" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1183 |
unfolding product_algebra_def sigma_def by simp |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1184 |
|
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1185 |
lemma product_algebra_generator_sets_into_space: |
41095 | 1186 |
assumes "\<And>i. i\<in>I \<Longrightarrow> sets (M i) \<subseteq> Pow (space (M i))" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1187 |
shows "sets (product_algebra_generator I M) \<subseteq> Pow (space (product_algebra_generator I M))" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1188 |
using assms by (auto simp: product_algebra_generator_def) blast |
40859 | 1189 |
|
1190 |
lemma (in finite_product_sigma_algebra) in_P[simp, intro]: |
|
1191 |
"\<lbrakk> \<And>i. i \<in> I \<Longrightarrow> A i \<in> sets (M i) \<rbrakk> \<Longrightarrow> Pi\<^isub>E I A \<in> sets P" |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1192 |
by (auto simp: sets_product_algebra) |
41026
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1193 |
|
40859 | 1194 |
section "Generating set generates also product algebra" |
1195 |
||
1196 |
lemma sigma_product_algebra_sigma_eq: |
|
1197 |
assumes "finite I" |
|
1198 |
assumes isotone: "\<And>i. i \<in> I \<Longrightarrow> (S i) \<up> (space (E i))" |
|
1199 |
assumes sets_into: "\<And>i. i \<in> I \<Longrightarrow> range (S i) \<subseteq> sets (E i)" |
|
1200 |
and E: "\<And>i. sets (E i) \<subseteq> Pow (space (E i))" |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1201 |
shows "sets (\<Pi>\<^isub>M i\<in>I. sigma (E i)) = sets (\<Pi>\<^isub>M i\<in>I. E i)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1202 |
(is "sets ?S = sets ?E") |
40859 | 1203 |
proof cases |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1204 |
assume "I = {}" then show ?thesis |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1205 |
by (simp add: product_algebra_def product_algebra_generator_def) |
40859 | 1206 |
next |
1207 |
assume "I \<noteq> {}" |
|
1208 |
interpret E: sigma_algebra "sigma (E i)" for i |
|
1209 |
using E by (rule sigma_algebra_sigma) |
|
1210 |
have into_space[intro]: "\<And>i x A. A \<in> sets (E i) \<Longrightarrow> x i \<in> A \<Longrightarrow> x i \<in> space (E i)" |
|
1211 |
using E by auto |
|
1212 |
interpret G: sigma_algebra ?E |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1213 |
unfolding product_algebra_def product_algebra_generator_def using E |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1214 |
by (intro sigma_algebra.sigma_algebra_cong[OF sigma_algebra_sigma]) (auto dest: Pi_mem) |
40859 | 1215 |
{ fix A i assume "i \<in> I" and A: "A \<in> sets (E i)" |
1216 |
then have "(\<lambda>x. x i) -` A \<inter> space ?E = (\<Pi>\<^isub>E j\<in>I. if j = i then A else \<Union>n. S j n) \<inter> space ?E" |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1217 |
using isotone unfolding isoton_def space_product_algebra |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1218 |
by (auto dest: Pi_mem) |
40859 | 1219 |
also have "\<dots> = (\<Union>n. (\<Pi>\<^isub>E j\<in>I. if j = i then A else S j n))" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1220 |
unfolding space_product_algebra |
40859 | 1221 |
apply simp |
1222 |
apply (subst Pi_UN[OF `finite I`]) |
|
1223 |
using isotone[THEN isoton_mono_le] apply simp |
|
1224 |
apply (simp add: PiE_Int) |
|
1225 |
apply (intro PiE_cong) |
|
1226 |
using A sets_into by (auto intro!: into_space) |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1227 |
also have "\<dots> \<in> sets ?E" |
40859 | 1228 |
using sets_into `A \<in> sets (E i)` |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1229 |
unfolding sets_product_algebra sets_sigma |
40859 | 1230 |
by (intro sigma_sets.Union) |
1231 |
(auto simp: image_subset_iff intro!: sigma_sets.Basic) |
|
1232 |
finally have "(\<lambda>x. x i) -` A \<inter> space ?E \<in> sets ?E" . } |
|
1233 |
then have proj: |
|
1234 |
"\<And>i. i\<in>I \<Longrightarrow> (\<lambda>x. x i) \<in> measurable ?E (sigma (E i))" |
|
1235 |
using E by (subst G.measurable_iff_sigma) |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1236 |
(auto simp: sets_product_algebra sets_sigma) |
40859 | 1237 |
{ fix A assume A: "\<And>i. i \<in> I \<Longrightarrow> A i \<in> sets (sigma (E i))" |
1238 |
with proj have basic: "\<And>i. i \<in> I \<Longrightarrow> (\<lambda>x. x i) -` (A i) \<inter> space ?E \<in> sets ?E" |
|
1239 |
unfolding measurable_def by simp |
|
1240 |
have "Pi\<^isub>E I A = (\<Inter>i\<in>I. (\<lambda>x. x i) -` (A i) \<inter> space ?E)" |
|
1241 |
using A E.sets_into_space `I \<noteq> {}` unfolding product_algebra_def by auto blast |
|
1242 |
then have "Pi\<^isub>E I A \<in> sets ?E" |
|
1243 |
using G.finite_INT[OF `finite I` `I \<noteq> {}` basic, of "\<lambda>i. i"] by simp } |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1244 |
then have "sigma_sets (space ?E) (sets (product_algebra_generator I (\<lambda>i. sigma (E i)))) \<subseteq> sets ?E" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1245 |
by (intro G.sigma_sets_subset) (auto simp add: product_algebra_generator_def) |
40859 | 1246 |
then have subset: "sets ?S \<subseteq> sets ?E" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1247 |
by (simp add: sets_sigma sets_product_algebra) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1248 |
show "sets ?S = sets ?E" |
40859 | 1249 |
proof (intro set_eqI iffI) |
1250 |
fix A assume "A \<in> sets ?E" then show "A \<in> sets ?S" |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1251 |
unfolding sets_sigma sets_product_algebra |
40859 | 1252 |
proof induct |
1253 |
case (Basic A) then show ?case |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1254 |
by (auto simp: sets_sigma product_algebra_generator_def intro: sigma_sets.Basic) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1255 |
qed (auto intro: sigma_sets.intros simp: product_algebra_generator_def) |
40859 | 1256 |
next |
1257 |
fix A assume "A \<in> sets ?S" then show "A \<in> sets ?E" using subset by auto |
|
1258 |
qed |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1259 |
qed |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1260 |
|
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1261 |
lemma product_algebraI[intro]: |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1262 |
"E \<in> (\<Pi> i\<in>I. sets (M i)) \<Longrightarrow> Pi\<^isub>E I E \<in> sets (Pi\<^isub>M I M)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1263 |
using assms unfolding product_algebra_def by (auto intro: product_algebra_generatorI) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1264 |
|
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1265 |
lemma (in product_sigma_algebra) measurable_component_update: |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1266 |
assumes "x \<in> space (Pi\<^isub>M I M)" and "i \<notin> I" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1267 |
shows "(\<lambda>v. x(i := v)) \<in> measurable (M i) (Pi\<^isub>M (insert i I) M)" (is "?f \<in> _") |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1268 |
unfolding product_algebra_def apply simp |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1269 |
proof (intro measurable_sigma) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1270 |
let ?G = "product_algebra_generator (insert i I) M" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1271 |
show "sets ?G \<subseteq> Pow (space ?G)" using product_algebra_generator_into_space . |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1272 |
show "?f \<in> space (M i) \<rightarrow> space ?G" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1273 |
using M.sets_into_space assms by auto |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1274 |
fix A assume "A \<in> sets ?G" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1275 |
from product_algebraE[OF this] guess E . note E = this |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1276 |
then have "?f -` A \<inter> space (M i) = E i \<or> ?f -` A \<inter> space (M i) = {}" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1277 |
using M.sets_into_space assms by auto |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1278 |
then show "?f -` A \<inter> space (M i) \<in> sets (M i)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1279 |
using E by (auto intro!: product_algebraI) |
40859 | 1280 |
qed |
1281 |
||
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1282 |
lemma (in product_sigma_algebra) measurable_add_dim: |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1283 |
assumes "i \<notin> I" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1284 |
shows "(\<lambda>(f, y). f(i := y)) \<in> measurable (Pi\<^isub>M I M \<Otimes>\<^isub>M M i) (Pi\<^isub>M (insert i I) M)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1285 |
proof - |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1286 |
let ?f = "(\<lambda>(f, y). f(i := y))" and ?G = "product_algebra_generator (insert i I) M" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1287 |
interpret Ii: pair_sigma_algebra "Pi\<^isub>M I M" "M i" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1288 |
unfolding pair_sigma_algebra_def |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1289 |
by (intro sigma_algebra_product_algebra sigma_algebras conjI) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1290 |
have "?f \<in> measurable Ii.P (sigma ?G)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1291 |
proof (rule Ii.measurable_sigma) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1292 |
show "sets ?G \<subseteq> Pow (space ?G)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1293 |
using product_algebra_generator_into_space . |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1294 |
show "?f \<in> space (Pi\<^isub>M I M \<Otimes>\<^isub>M M i) \<rightarrow> space ?G" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1295 |
by (auto simp: space_pair_measure) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1296 |
next |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1297 |
fix A assume "A \<in> sets ?G" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1298 |
then obtain F where "A = Pi\<^isub>E (insert i I) F" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1299 |
and F: "\<And>j. j \<in> I \<Longrightarrow> F j \<in> sets (M j)" "F i \<in> sets (M i)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1300 |
by (auto elim!: product_algebraE) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1301 |
then have "?f -` A \<inter> space (Pi\<^isub>M I M \<Otimes>\<^isub>M M i) = Pi\<^isub>E I F \<times> (F i)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1302 |
using sets_into_space `i \<notin> I` |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1303 |
by (auto simp add: space_pair_measure) blast+ |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1304 |
then show "?f -` A \<inter> space (Pi\<^isub>M I M \<Otimes>\<^isub>M M i) \<in> sets (Pi\<^isub>M I M \<Otimes>\<^isub>M M i)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1305 |
using F by (auto intro!: pair_measureI) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1306 |
qed |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1307 |
then show ?thesis |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1308 |
by (simp add: product_algebra_def) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1309 |
qed |
41095 | 1310 |
|
1311 |
lemma (in product_sigma_algebra) measurable_merge: |
|
1312 |
assumes [simp]: "I \<inter> J = {}" |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1313 |
shows "(\<lambda>(x, y). merge I x J y) \<in> measurable (Pi\<^isub>M I M \<Otimes>\<^isub>M Pi\<^isub>M J M) (Pi\<^isub>M (I \<union> J) M)" |
40859 | 1314 |
proof - |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1315 |
let ?I = "Pi\<^isub>M I M" and ?J = "Pi\<^isub>M J M" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1316 |
interpret P: sigma_algebra "?I \<Otimes>\<^isub>M ?J" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1317 |
by (intro sigma_algebra_pair_measure product_algebra_into_space) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1318 |
let ?f = "\<lambda>(x, y). merge I x J y" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1319 |
let ?G = "product_algebra_generator (I \<union> J) M" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1320 |
have "?f \<in> measurable (?I \<Otimes>\<^isub>M ?J) (sigma ?G)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1321 |
proof (rule P.measurable_sigma) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1322 |
fix A assume "A \<in> sets ?G" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1323 |
from product_algebraE[OF this] |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1324 |
obtain E where E: "A = Pi\<^isub>E (I \<union> J) E" "E \<in> (\<Pi> i\<in>I \<union> J. sets (M i))" . |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1325 |
then have *: "?f -` A \<inter> space (?I \<Otimes>\<^isub>M ?J) = Pi\<^isub>E I E \<times> Pi\<^isub>E J E" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1326 |
using sets_into_space `I \<inter> J = {}` |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1327 |
by (auto simp add: space_pair_measure) blast+ |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1328 |
then show "?f -` A \<inter> space (?I \<Otimes>\<^isub>M ?J) \<in> sets (?I \<Otimes>\<^isub>M ?J)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1329 |
using E unfolding * by (auto intro!: pair_measureI in_sigma product_algebra_generatorI |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1330 |
simp: product_algebra_def) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1331 |
qed (insert product_algebra_generator_into_space, auto simp: space_pair_measure) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1332 |
then show "?f \<in> measurable (?I \<Otimes>\<^isub>M ?J) (Pi\<^isub>M (I \<union> J) M)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1333 |
unfolding product_algebra_def[of "I \<union> J"] by simp |
40859 | 1334 |
qed |
1335 |
||
41095 | 1336 |
lemma (in product_sigma_algebra) measurable_component_singleton: |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1337 |
assumes "i \<in> I" shows "(\<lambda>x. x i) \<in> measurable (Pi\<^isub>M I M) (M i)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1338 |
proof (unfold measurable_def, intro CollectI conjI ballI) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1339 |
fix A assume "A \<in> sets (M i)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1340 |
then have "(\<lambda>x. x i) -` A \<inter> space (Pi\<^isub>M I M) = (\<Pi>\<^isub>E j\<in>I. if i = j then A else space (M j))" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1341 |
using M.sets_into_space `i \<in> I` by (fastsimp dest: Pi_mem split: split_if_asm) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1342 |
then show "(\<lambda>x. x i) -` A \<inter> space (Pi\<^isub>M I M) \<in> sets (Pi\<^isub>M I M)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1343 |
using `A \<in> sets (M i)` by (auto intro!: product_algebraI) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1344 |
qed (insert `i \<in> I`, auto) |
41661 | 1345 |
|
40859 | 1346 |
locale product_sigma_finite = |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1347 |
fixes M :: "'i \<Rightarrow> ('a,'b) measure_space_scheme" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1348 |
assumes sigma_finite_measures: "\<And>i. sigma_finite_measure (M i)" |
40859 | 1349 |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1350 |
locale finite_product_sigma_finite = product_sigma_finite M |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1351 |
for M :: "'i \<Rightarrow> ('a,'b) measure_space_scheme" + |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1352 |
fixes I :: "'i set" assumes finite_index'[intro]: "finite I" |
40859 | 1353 |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1354 |
sublocale product_sigma_finite \<subseteq> M: sigma_finite_measure "M i" for i |
40859 | 1355 |
by (rule sigma_finite_measures) |
1356 |
||
1357 |
sublocale product_sigma_finite \<subseteq> product_sigma_algebra |
|
1358 |
by default |
|
1359 |
||
1360 |
sublocale finite_product_sigma_finite \<subseteq> finite_product_sigma_algebra |
|
1361 |
by default (fact finite_index') |
|
1362 |
||
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1363 |
lemma (in finite_product_sigma_finite) product_algebra_generator_measure: |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1364 |
assumes "Pi\<^isub>E I F \<in> sets G" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1365 |
shows "measure G (Pi\<^isub>E I F) = (\<Prod>i\<in>I. M.\<mu> i (F i))" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1366 |
proof cases |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1367 |
assume ne: "\<forall>i\<in>I. F i \<noteq> {}" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1368 |
have "\<forall>i\<in>I. (SOME F'. Pi\<^isub>E I F = Pi\<^isub>E I F') i = F i" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1369 |
by (rule someI2[where P="\<lambda>F'. Pi\<^isub>E I F = Pi\<^isub>E I F'"]) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1370 |
(insert ne, auto simp: Pi_eq_iff) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1371 |
then show ?thesis |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1372 |
unfolding product_algebra_generator_def by simp |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1373 |
next |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1374 |
assume empty: "\<not> (\<forall>j\<in>I. F j \<noteq> {})" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1375 |
then have "(\<Prod>j\<in>I. M.\<mu> j (F j)) = 0" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1376 |
by (auto simp: setprod_pextreal_0 intro!: bexI) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1377 |
moreover |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1378 |
have "\<exists>j\<in>I. (SOME F'. Pi\<^isub>E I F = Pi\<^isub>E I F') j = {}" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1379 |
by (rule someI2[where P="\<lambda>F'. Pi\<^isub>E I F = Pi\<^isub>E I F'"]) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1380 |
(insert empty, auto simp: Pi_eq_empty_iff[symmetric]) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1381 |
then have "(\<Prod>j\<in>I. M.\<mu> j ((SOME F'. Pi\<^isub>E I F = Pi\<^isub>E I F') j)) = 0" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1382 |
by (auto simp: setprod_pextreal_0 intro!: bexI) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1383 |
ultimately show ?thesis |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1384 |
unfolding product_algebra_generator_def by simp |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1385 |
qed |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1386 |
|
40859 | 1387 |
lemma (in finite_product_sigma_finite) sigma_finite_pairs: |
1388 |
"\<exists>F::'i \<Rightarrow> nat \<Rightarrow> 'a set. |
|
1389 |
(\<forall>i\<in>I. range (F i) \<subseteq> sets (M i)) \<and> |
|
1390 |
(\<forall>k. \<forall>i\<in>I. \<mu> i (F i k) \<noteq> \<omega>) \<and> |
|
1391 |
(\<lambda>k. \<Pi>\<^isub>E i\<in>I. F i k) \<up> space G" |
|
1392 |
proof - |
|
1393 |
have "\<forall>i::'i. \<exists>F::nat \<Rightarrow> 'a set. range F \<subseteq> sets (M i) \<and> F \<up> space (M i) \<and> (\<forall>k. \<mu> i (F k) \<noteq> \<omega>)" |
|
1394 |
using M.sigma_finite_up by simp |
|
1395 |
from choice[OF this] guess F :: "'i \<Rightarrow> nat \<Rightarrow> 'a set" .. |
|
1396 |
then have "\<And>i. range (F i) \<subseteq> sets (M i)" "\<And>i. F i \<up> space (M i)" "\<And>i k. \<mu> i (F i k) \<noteq> \<omega>" |
|
1397 |
by auto |
|
1398 |
let ?F = "\<lambda>k. \<Pi>\<^isub>E i\<in>I. F i k" |
|
1399 |
note space_product_algebra[simp] |
|
1400 |
show ?thesis |
|
1401 |
proof (intro exI[of _ F] conjI allI isotoneI set_eqI iffI ballI) |
|
1402 |
fix i show "range (F i) \<subseteq> sets (M i)" by fact |
|
1403 |
next |
|
1404 |
fix i k show "\<mu> i (F i k) \<noteq> \<omega>" by fact |
|
1405 |
next |
|
1406 |
fix A assume "A \<in> (\<Union>i. ?F i)" then show "A \<in> space G" |
|
41831 | 1407 |
using `\<And>i. range (F i) \<subseteq> sets (M i)` M.sets_into_space |
1408 |
by (force simp: image_subset_iff) |
|
40859 | 1409 |
next |
1410 |
fix f assume "f \<in> space G" |
|
1411 |
with Pi_UN[OF finite_index, of "\<lambda>k i. F i k"] |
|
1412 |
`\<And>i. F i \<up> space (M i)`[THEN isotonD(2)] |
|
1413 |
`\<And>i. F i \<up> space (M i)`[THEN isoton_mono_le] |
|
1414 |
show "f \<in> (\<Union>i. ?F i)" by auto |
|
1415 |
next |
|
1416 |
fix i show "?F i \<subseteq> ?F (Suc i)" |
|
1417 |
using `\<And>i. F i \<up> space (M i)`[THEN isotonD(1)] by auto |
|
1418 |
qed |
|
1419 |
qed |
|
1420 |
||
41831 | 1421 |
lemma sets_pair_cancel_measure[simp]: |
1422 |
"sets (M1\<lparr>measure := m1\<rparr> \<Otimes>\<^isub>M M2) = sets (M1 \<Otimes>\<^isub>M M2)" |
|
1423 |
"sets (M1 \<Otimes>\<^isub>M M2\<lparr>measure := m2\<rparr>) = sets (M1 \<Otimes>\<^isub>M M2)" |
|
1424 |
unfolding pair_measure_def pair_measure_generator_def sets_sigma |
|
1425 |
by simp_all |
|
1426 |
||
1427 |
lemma measurable_pair_cancel_measure[simp]: |
|
1428 |
"measurable (M1\<lparr>measure := m1\<rparr> \<Otimes>\<^isub>M M2) M = measurable (M1 \<Otimes>\<^isub>M M2) M" |
|
1429 |
"measurable (M1 \<Otimes>\<^isub>M M2\<lparr>measure := m2\<rparr>) M = measurable (M1 \<Otimes>\<^isub>M M2) M" |
|
1430 |
"measurable M (M1\<lparr>measure := m3\<rparr> \<Otimes>\<^isub>M M2) = measurable M (M1 \<Otimes>\<^isub>M M2)" |
|
1431 |
"measurable M (M1 \<Otimes>\<^isub>M M2\<lparr>measure := m4\<rparr>) = measurable M (M1 \<Otimes>\<^isub>M M2)" |
|
1432 |
unfolding measurable_def by (auto simp add: space_pair_measure) |
|
1433 |
||
40859 | 1434 |
lemma (in product_sigma_finite) product_measure_exists: |
1435 |
assumes "finite I" |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1436 |
shows "\<exists>\<nu>. sigma_finite_measure (sigma (product_algebra_generator I M) \<lparr> measure := \<nu> \<rparr>) \<and> |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1437 |
(\<forall>A\<in>\<Pi> i\<in>I. sets (M i). \<nu> (Pi\<^isub>E I A) = (\<Prod>i\<in>I. M.\<mu> i (A i)))" |
40859 | 1438 |
using `finite I` proof induct |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1439 |
case empty |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1440 |
interpret finite_product_sigma_finite M "{}" by default simp |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1441 |
let ?\<nu> = "(\<lambda>A. if A = {} then 0 else 1) :: 'd set \<Rightarrow> pextreal" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1442 |
show ?case |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1443 |
proof (intro exI conjI ballI) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1444 |
have "sigma_algebra (sigma G \<lparr>measure := ?\<nu>\<rparr>)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1445 |
by (rule sigma_algebra_cong) (simp_all add: product_algebra_def) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1446 |
then have "measure_space (sigma G\<lparr>measure := ?\<nu>\<rparr>)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1447 |
by (rule finite_additivity_sufficient) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1448 |
(simp_all add: positive_def additive_def sets_sigma |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1449 |
product_algebra_generator_def image_constant) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1450 |
then show "sigma_finite_measure (sigma G\<lparr>measure := ?\<nu>\<rparr>)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1451 |
by (auto intro!: exI[of _ "\<lambda>i. {\<lambda>_. undefined}"] |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1452 |
simp: sigma_finite_measure_def sigma_finite_measure_axioms_def |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1453 |
product_algebra_generator_def) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1454 |
qed auto |
40859 | 1455 |
next |
1456 |
case (insert i I) |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1457 |
interpret finite_product_sigma_finite M I by default fact |
40859 | 1458 |
have "finite (insert i I)" using `finite I` by auto |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1459 |
interpret I': finite_product_sigma_finite M "insert i I" by default fact |
40859 | 1460 |
from insert obtain \<nu> where |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1461 |
prod: "\<And>A. A \<in> (\<Pi> i\<in>I. sets (M i)) \<Longrightarrow> \<nu> (Pi\<^isub>E I A) = (\<Prod>i\<in>I. M.\<mu> i (A i))" and |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1462 |
"sigma_finite_measure (sigma G\<lparr> measure := \<nu> \<rparr>)" by auto |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1463 |
then interpret I: sigma_finite_measure "P\<lparr> measure := \<nu>\<rparr>" unfolding product_algebra_def by simp |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1464 |
interpret P: pair_sigma_finite "P\<lparr> measure := \<nu>\<rparr>" "M i" .. |
41661 | 1465 |
let ?h = "(\<lambda>(f, y). f(i := y))" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1466 |
let ?\<nu> = "\<lambda>A. P.\<mu> (?h -` A \<inter> space P.P)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1467 |
have I': "sigma_algebra (I'.P\<lparr> measure := ?\<nu> \<rparr>)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1468 |
by (rule I'.sigma_algebra_cong) simp_all |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1469 |
interpret I'': measure_space "I'.P\<lparr> measure := ?\<nu> \<rparr>" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1470 |
using measurable_add_dim[OF `i \<notin> I`] |
41831 | 1471 |
by (intro P.measure_space_vimage[OF I']) (auto simp add: measure_preserving_def) |
40859 | 1472 |
show ?case |
1473 |
proof (intro exI[of _ ?\<nu>] conjI ballI) |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1474 |
let "?m A" = "measure (Pi\<^isub>M I M\<lparr>measure := \<nu>\<rparr> \<Otimes>\<^isub>M M i) (?h -` A \<inter> space P.P)" |
40859 | 1475 |
{ fix A assume A: "A \<in> (\<Pi> i\<in>insert i I. sets (M i))" |
41661 | 1476 |
then have *: "?h -` Pi\<^isub>E (insert i I) A \<inter> space P.P = Pi\<^isub>E I A \<times> A i" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1477 |
using `i \<notin> I` M.sets_into_space by (auto simp: space_pair_measure space_product_algebra) blast |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1478 |
show "?m (Pi\<^isub>E (insert i I) A) = (\<Prod>i\<in>insert i I. M.\<mu> i (A i))" |
41661 | 1479 |
unfolding * using A |
40859 | 1480 |
apply (subst P.pair_measure_times) |
41661 | 1481 |
using A apply fastsimp |
1482 |
using A apply fastsimp |
|
1483 |
using `i \<notin> I` `finite I` prod[of A] A by (auto simp: ac_simps) } |
|
40859 | 1484 |
note product = this |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1485 |
have *: "sigma I'.G\<lparr> measure := ?\<nu> \<rparr> = I'.P\<lparr> measure := ?\<nu> \<rparr>" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1486 |
by (simp add: product_algebra_def) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1487 |
show "sigma_finite_measure (sigma I'.G\<lparr> measure := ?\<nu> \<rparr>)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1488 |
proof (unfold *, default, simp) |
40859 | 1489 |
from I'.sigma_finite_pairs guess F :: "'i \<Rightarrow> nat \<Rightarrow> 'a set" .. |
1490 |
then have F: "\<And>j. j \<in> insert i I \<Longrightarrow> range (F j) \<subseteq> sets (M j)" |
|
1491 |
"(\<lambda>k. \<Pi>\<^isub>E j \<in> insert i I. F j k) \<up> space I'.G" |
|
1492 |
"\<And>k. \<And>j. j \<in> insert i I \<Longrightarrow> \<mu> j (F j k) \<noteq> \<omega>" |
|
1493 |
by blast+ |
|
1494 |
let "?F k" = "\<Pi>\<^isub>E j \<in> insert i I. F j k" |
|
1495 |
show "\<exists>F::nat \<Rightarrow> ('i \<Rightarrow> 'a) set. range F \<subseteq> sets I'.P \<and> |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1496 |
(\<Union>i. F i) = (\<Pi>\<^isub>E i\<in>insert i I. space (M i)) \<and> (\<forall>i. ?m (F i) \<noteq> \<omega>)" |
40859 | 1497 |
proof (intro exI[of _ ?F] conjI allI) |
1498 |
show "range ?F \<subseteq> sets I'.P" using F(1) by auto |
|
1499 |
next |
|
1500 |
from F(2)[THEN isotonD(2)] |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1501 |
show "(\<Union>i. ?F i) = (\<Pi>\<^isub>E i\<in>insert i I. space (M i))" by simp |
40859 | 1502 |
next |
1503 |
fix j |
|
1504 |
show "?\<nu> (?F j) \<noteq> \<omega>" |
|
1505 |
using F `finite I` |
|
1506 |
by (subst product) (auto simp: setprod_\<omega>) |
|
1507 |
qed |
|
1508 |
qed |
|
1509 |
qed |
|
1510 |
qed |
|
1511 |
||
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1512 |
sublocale finite_product_sigma_finite \<subseteq> sigma_finite_measure P |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1513 |
unfolding product_algebra_def |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1514 |
using product_measure_exists[OF finite_index] |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1515 |
by (rule someI2_ex) auto |
40859 | 1516 |
|
1517 |
lemma (in finite_product_sigma_finite) measure_times: |
|
1518 |
assumes "\<And>i. i \<in> I \<Longrightarrow> A i \<in> sets (M i)" |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1519 |
shows "\<mu> (Pi\<^isub>E I A) = (\<Prod>i\<in>I. M.\<mu> i (A i))" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1520 |
unfolding product_algebra_def |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1521 |
using product_measure_exists[OF finite_index] |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1522 |
proof (rule someI2_ex, elim conjE) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1523 |
fix \<nu> assume *: "\<forall>A\<in>\<Pi> i\<in>I. sets (M i). \<nu> (Pi\<^isub>E I A) = (\<Prod>i\<in>I. M.\<mu> i (A i))" |
40859 | 1524 |
have "Pi\<^isub>E I A = Pi\<^isub>E I (\<lambda>i\<in>I. A i)" by (auto dest: Pi_mem) |
1525 |
then have "\<nu> (Pi\<^isub>E I A) = \<nu> (Pi\<^isub>E I (\<lambda>i\<in>I. A i))" by simp |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1526 |
also have "\<dots> = (\<Prod>i\<in>I. M.\<mu> i ((\<lambda>i\<in>I. A i) i))" using assms * by auto |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1527 |
finally show "measure (sigma G\<lparr>measure := \<nu>\<rparr>) (Pi\<^isub>E I A) = (\<Prod>i\<in>I. M.\<mu> i (A i))" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1528 |
by (simp add: sigma_def) |
40859 | 1529 |
qed |
41096 | 1530 |
|
1531 |
lemma (in product_sigma_finite) product_measure_empty[simp]: |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1532 |
"measure (Pi\<^isub>M {} M) {\<lambda>x. undefined} = 1" |
41096 | 1533 |
proof - |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1534 |
interpret finite_product_sigma_finite M "{}" by default auto |
41096 | 1535 |
from measure_times[of "\<lambda>x. {}"] show ?thesis by simp |
1536 |
qed |
|
1537 |
||
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1538 |
lemma (in finite_product_sigma_algebra) P_empty: |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1539 |
assumes "I = {}" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1540 |
shows "space P = {\<lambda>k. undefined}" "sets P = { {}, {\<lambda>k. undefined} }" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1541 |
unfolding product_algebra_def product_algebra_generator_def `I = {}` |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1542 |
by (simp_all add: sigma_def image_constant) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1543 |
|
40859 | 1544 |
lemma (in product_sigma_finite) positive_integral_empty: |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1545 |
"integral\<^isup>P (Pi\<^isub>M {} M) f = f (\<lambda>k. undefined)" |
40859 | 1546 |
proof - |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1547 |
interpret finite_product_sigma_finite M "{}" by default (fact finite.emptyI) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1548 |
have "\<And>A. measure (Pi\<^isub>M {} M) (Pi\<^isub>E {} A) = 1" |
40859 | 1549 |
using assms by (subst measure_times) auto |
1550 |
then show ?thesis |
|
40873 | 1551 |
unfolding positive_integral_def simple_function_def simple_integral_def_raw |
40859 | 1552 |
proof (simp add: P_empty, intro antisym) |
1553 |
show "f (\<lambda>k. undefined) \<le> (SUP f:{g. g \<le> f}. f (\<lambda>k. undefined))" |
|
1554 |
by (intro le_SUPI) auto |
|
1555 |
show "(SUP f:{g. g \<le> f}. f (\<lambda>k. undefined)) \<le> f (\<lambda>k. undefined)" |
|
1556 |
by (intro SUP_leI) (auto simp: le_fun_def) |
|
1557 |
qed |
|
1558 |
qed |
|
1559 |
||
41026
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1560 |
lemma (in product_sigma_finite) measure_fold: |
40859 | 1561 |
assumes IJ[simp]: "I \<inter> J = {}" and fin: "finite I" "finite J" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1562 |
assumes A: "A \<in> sets (Pi\<^isub>M (I \<union> J) M)" |
41706
a207a858d1f6
prefer p2e before e2p; use measure_unique_Int_stable_vimage;
hoelzl
parents:
41705
diff
changeset
|
1563 |
shows "measure (Pi\<^isub>M (I \<union> J) M) A = |
a207a858d1f6
prefer p2e before e2p; use measure_unique_Int_stable_vimage;
hoelzl
parents:
41705
diff
changeset
|
1564 |
measure (Pi\<^isub>M I M \<Otimes>\<^isub>M Pi\<^isub>M J M) ((\<lambda>(x,y). merge I x J y) -` A \<inter> space (Pi\<^isub>M I M \<Otimes>\<^isub>M Pi\<^isub>M J M))" |
40859 | 1565 |
proof - |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1566 |
interpret I: finite_product_sigma_finite M I by default fact |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1567 |
interpret J: finite_product_sigma_finite M J by default fact |
40859 | 1568 |
have "finite (I \<union> J)" using fin by auto |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1569 |
interpret IJ: finite_product_sigma_finite M "I \<union> J" by default fact |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1570 |
interpret P: pair_sigma_finite I.P J.P by default |
41661 | 1571 |
let ?g = "\<lambda>(x,y). merge I x J y" |
1572 |
let "?X S" = "?g -` S \<inter> space P.P" |
|
1573 |
from IJ.sigma_finite_pairs obtain F where |
|
1574 |
F: "\<And>i. i\<in> I \<union> J \<Longrightarrow> range (F i) \<subseteq> sets (M i)" |
|
1575 |
"(\<lambda>k. \<Pi>\<^isub>E i\<in>I \<union> J. F i k) \<up> space IJ.G" |
|
1576 |
"\<And>k. \<forall>i\<in>I\<union>J. \<mu> i (F i k) \<noteq> \<omega>" |
|
1577 |
by auto |
|
1578 |
let ?F = "\<lambda>k. \<Pi>\<^isub>E i\<in>I \<union> J. F i k" |
|
41706
a207a858d1f6
prefer p2e before e2p; use measure_unique_Int_stable_vimage;
hoelzl
parents:
41705
diff
changeset
|
1579 |
show "IJ.\<mu> A = P.\<mu> (?X A)" |
a207a858d1f6
prefer p2e before e2p; use measure_unique_Int_stable_vimage;
hoelzl
parents:
41705
diff
changeset
|
1580 |
proof (rule measure_unique_Int_stable_vimage) |
a207a858d1f6
prefer p2e before e2p; use measure_unique_Int_stable_vimage;
hoelzl
parents:
41705
diff
changeset
|
1581 |
show "measure_space IJ.P" "measure_space P.P" by default |
a207a858d1f6
prefer p2e before e2p; use measure_unique_Int_stable_vimage;
hoelzl
parents:
41705
diff
changeset
|
1582 |
show "sets (sigma IJ.G) = sets IJ.P" "space IJ.G = space IJ.P" "A \<in> sets (sigma IJ.G)" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1583 |
using A unfolding product_algebra_def by auto |
41706
a207a858d1f6
prefer p2e before e2p; use measure_unique_Int_stable_vimage;
hoelzl
parents:
41705
diff
changeset
|
1584 |
next |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1585 |
show "Int_stable IJ.G" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1586 |
by (simp add: PiE_Int Int_stable_def product_algebra_def |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1587 |
product_algebra_generator_def) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1588 |
auto |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1589 |
show "range ?F \<subseteq> sets IJ.G" using F |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1590 |
by (simp add: image_subset_iff product_algebra_def |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1591 |
product_algebra_generator_def) |
41661 | 1592 |
show "?F \<up> space IJ.G " using F(2) by simp |
41706
a207a858d1f6
prefer p2e before e2p; use measure_unique_Int_stable_vimage;
hoelzl
parents:
41705
diff
changeset
|
1593 |
show "\<And>k. IJ.\<mu> (?F k) \<noteq> \<omega>" |
a207a858d1f6
prefer p2e before e2p; use measure_unique_Int_stable_vimage;
hoelzl
parents:
41705
diff
changeset
|
1594 |
using `finite I` F |
a207a858d1f6
prefer p2e before e2p; use measure_unique_Int_stable_vimage;
hoelzl
parents:
41705
diff
changeset
|
1595 |
by (subst IJ.measure_times) (auto simp add: setprod_\<omega>) |
a207a858d1f6
prefer p2e before e2p; use measure_unique_Int_stable_vimage;
hoelzl
parents:
41705
diff
changeset
|
1596 |
show "?g \<in> measurable P.P IJ.P" |
a207a858d1f6
prefer p2e before e2p; use measure_unique_Int_stable_vimage;
hoelzl
parents:
41705
diff
changeset
|
1597 |
using IJ by (rule measurable_merge) |
41661 | 1598 |
next |
1599 |
fix A assume "A \<in> sets IJ.G" |
|
41706
a207a858d1f6
prefer p2e before e2p; use measure_unique_Int_stable_vimage;
hoelzl
parents:
41705
diff
changeset
|
1600 |
then obtain F where A: "A = Pi\<^isub>E (I \<union> J) F" |
41661 | 1601 |
and F: "\<And>i. i \<in> I \<union> J \<Longrightarrow> F i \<in> sets (M i)" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1602 |
by (auto simp: product_algebra_generator_def) |
41706
a207a858d1f6
prefer p2e before e2p; use measure_unique_Int_stable_vimage;
hoelzl
parents:
41705
diff
changeset
|
1603 |
then have X: "?X A = (Pi\<^isub>E I F \<times> Pi\<^isub>E J F)" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1604 |
using sets_into_space by (auto simp: space_pair_measure) blast+ |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1605 |
then have "P.\<mu> (?X A) = (\<Prod>i\<in>I. \<mu> i (F i)) * (\<Prod>i\<in>J. \<mu> i (F i))" |
41661 | 1606 |
using `finite J` `finite I` F |
1607 |
by (simp add: P.pair_measure_times I.measure_times J.measure_times) |
|
1608 |
also have "\<dots> = (\<Prod>i\<in>I \<union> J. \<mu> i (F i))" |
|
1609 |
using `finite J` `finite I` `I \<inter> J = {}` by (simp add: setprod_Un_one) |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1610 |
also have "\<dots> = IJ.\<mu> A" |
41661 | 1611 |
using `finite J` `finite I` F unfolding A |
1612 |
by (intro IJ.measure_times[symmetric]) auto |
|
41706
a207a858d1f6
prefer p2e before e2p; use measure_unique_Int_stable_vimage;
hoelzl
parents:
41705
diff
changeset
|
1613 |
finally show "IJ.\<mu> A = P.\<mu> (?X A)" by (rule sym) |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1614 |
qed |
41661 | 1615 |
qed |
41026
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1616 |
|
41831 | 1617 |
lemma (in product_sigma_finite) measure_preserving_merge: |
1618 |
assumes IJ: "I \<inter> J = {}" and "finite I" "finite J" |
|
1619 |
shows "(\<lambda>(x,y). merge I x J y) \<in> measure_preserving (Pi\<^isub>M I M \<Otimes>\<^isub>M Pi\<^isub>M J M) (Pi\<^isub>M (I \<union> J) M)" |
|
1620 |
by (intro measure_preservingI measurable_merge[OF IJ] measure_fold[symmetric] assms) |
|
1621 |
||
41026
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1622 |
lemma (in product_sigma_finite) product_positive_integral_fold: |
41831 | 1623 |
assumes IJ[simp]: "I \<inter> J = {}" "finite I" "finite J" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1624 |
and f: "f \<in> borel_measurable (Pi\<^isub>M (I \<union> J) M)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1625 |
shows "integral\<^isup>P (Pi\<^isub>M (I \<union> J) M) f = |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1626 |
(\<integral>\<^isup>+ x. (\<integral>\<^isup>+ y. f (merge I x J y) \<partial>(Pi\<^isub>M J M)) \<partial>(Pi\<^isub>M I M))" |
41026
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1627 |
proof - |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1628 |
interpret I: finite_product_sigma_finite M I by default fact |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1629 |
interpret J: finite_product_sigma_finite M J by default fact |
41831 | 1630 |
interpret P: pair_sigma_finite "Pi\<^isub>M I M" "Pi\<^isub>M J M" by default |
1631 |
interpret IJ: finite_product_sigma_finite M "I \<union> J" by default simp |
|
41026
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1632 |
have P_borel: "(\<lambda>x. f (case x of (x, y) \<Rightarrow> merge I x J y)) \<in> borel_measurable P.P" |
41831 | 1633 |
using measurable_comp[OF measurable_merge[OF IJ(1)] f] by (simp add: comp_def) |
41661 | 1634 |
show ?thesis |
41026
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1635 |
unfolding P.positive_integral_fst_measurable[OF P_borel, simplified] |
41661 | 1636 |
proof (rule P.positive_integral_vimage) |
1637 |
show "sigma_algebra IJ.P" by default |
|
41831 | 1638 |
show "(\<lambda>(x, y). merge I x J y) \<in> measure_preserving P.P IJ.P" |
1639 |
using IJ by (rule measure_preserving_merge) |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1640 |
show "f \<in> borel_measurable IJ.P" using f by simp |
41661 | 1641 |
qed |
40859 | 1642 |
qed |
1643 |
||
41831 | 1644 |
lemma (in product_sigma_finite) measure_preserving_component_singelton: |
1645 |
"(\<lambda>x. x i) \<in> measure_preserving (Pi\<^isub>M {i} M) (M i)" |
|
1646 |
proof (intro measure_preservingI measurable_component_singleton) |
|
1647 |
interpret I: finite_product_sigma_finite M "{i}" by default simp |
|
1648 |
fix A let ?P = "(\<lambda>x. x i) -` A \<inter> space I.P" |
|
1649 |
assume A: "A \<in> sets (M i)" |
|
1650 |
then have *: "?P = {i} \<rightarrow>\<^isub>E A" using sets_into_space by auto |
|
1651 |
show "I.\<mu> ?P = M.\<mu> i A" unfolding * |
|
1652 |
using A I.measure_times[of "\<lambda>_. A"] by auto |
|
1653 |
qed auto |
|
1654 |
||
41026
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1655 |
lemma (in product_sigma_finite) product_positive_integral_singleton: |
40859 | 1656 |
assumes f: "f \<in> borel_measurable (M i)" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1657 |
shows "integral\<^isup>P (Pi\<^isub>M {i} M) (\<lambda>x. f (x i)) = integral\<^isup>P (M i) f" |
40859 | 1658 |
proof - |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1659 |
interpret I: finite_product_sigma_finite M "{i}" by default simp |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1660 |
show ?thesis |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1661 |
proof (rule I.positive_integral_vimage[symmetric]) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1662 |
show "sigma_algebra (M i)" by (rule sigma_algebras) |
41831 | 1663 |
show "(\<lambda>x. x i) \<in> measure_preserving (Pi\<^isub>M {i} M) (M i)" |
1664 |
by (rule measure_preserving_component_singelton) |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1665 |
show "f \<in> borel_measurable (M i)" by fact |
41661 | 1666 |
qed |
40859 | 1667 |
qed |
1668 |
||
41096 | 1669 |
lemma (in product_sigma_finite) product_positive_integral_insert: |
1670 |
assumes [simp]: "finite I" "i \<notin> I" |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1671 |
and f: "f \<in> borel_measurable (Pi\<^isub>M (insert i I) M)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1672 |
shows "integral\<^isup>P (Pi\<^isub>M (insert i I) M) f = (\<integral>\<^isup>+ x. (\<integral>\<^isup>+ y. f (x(i := y)) \<partial>(M i)) \<partial>(Pi\<^isub>M I M))" |
41096 | 1673 |
proof - |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1674 |
interpret I: finite_product_sigma_finite M I by default auto |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1675 |
interpret i: finite_product_sigma_finite M "{i}" by default auto |
41096 | 1676 |
interpret P: pair_sigma_algebra I.P i.P .. |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1677 |
have IJ: "I \<inter> {i} = {}" and insert: "I \<union> {i} = insert i I" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1678 |
using f by auto |
41096 | 1679 |
show ?thesis |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1680 |
unfolding product_positive_integral_fold[OF IJ, unfolded insert, simplified, OF f] |
41096 | 1681 |
proof (rule I.positive_integral_cong, subst product_positive_integral_singleton) |
1682 |
fix x assume x: "x \<in> space I.P" |
|
1683 |
let "?f y" = "f (restrict (x(i := y)) (insert i I))" |
|
1684 |
have f'_eq: "\<And>y. ?f y = f (x(i := y))" |
|
1685 |
using x by (auto intro!: arg_cong[where f=f] simp: fun_eq_iff extensional_def) |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1686 |
show "?f \<in> borel_measurable (M i)" unfolding f'_eq |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1687 |
using measurable_comp[OF measurable_component_update f] x `i \<notin> I` |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1688 |
by (simp add: comp_def) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1689 |
show "integral\<^isup>P (M i) ?f = \<integral>\<^isup>+ y. f (x(i:=y)) \<partial>M i" |
41096 | 1690 |
unfolding f'_eq by simp |
1691 |
qed |
|
1692 |
qed |
|
1693 |
||
1694 |
lemma (in product_sigma_finite) product_positive_integral_setprod: |
|
1695 |
fixes f :: "'i \<Rightarrow> 'a \<Rightarrow> pextreal" |
|
1696 |
assumes "finite I" and borel: "\<And>i. i \<in> I \<Longrightarrow> f i \<in> borel_measurable (M i)" |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1697 |
shows "(\<integral>\<^isup>+ x. (\<Prod>i\<in>I. f i (x i)) \<partial>Pi\<^isub>M I M) = (\<Prod>i\<in>I. integral\<^isup>P (M i) (f i))" |
41096 | 1698 |
using assms proof induct |
1699 |
case empty |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1700 |
interpret finite_product_sigma_finite M "{}" by default auto |
41096 | 1701 |
then show ?case by simp |
1702 |
next |
|
1703 |
case (insert i I) |
|
1704 |
note `finite I`[intro, simp] |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1705 |
interpret I: finite_product_sigma_finite M I by default auto |
41096 | 1706 |
have *: "\<And>x y. (\<Prod>j\<in>I. f j (if j = i then y else x j)) = (\<Prod>j\<in>I. f j (x j))" |
1707 |
using insert by (auto intro!: setprod_cong) |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1708 |
have prod: "\<And>J. J \<subseteq> insert i I \<Longrightarrow> (\<lambda>x. (\<Prod>i\<in>J. f i (x i))) \<in> borel_measurable (Pi\<^isub>M J M)" |
41096 | 1709 |
using sets_into_space insert |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1710 |
by (intro sigma_algebra.borel_measurable_pextreal_setprod sigma_algebra_product_algebra |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1711 |
measurable_comp[OF measurable_component_singleton, unfolded comp_def]) |
41096 | 1712 |
auto |
1713 |
show ?case |
|
1714 |
by (simp add: product_positive_integral_insert[OF insert(1,2) prod]) |
|
1715 |
(simp add: insert I.positive_integral_cmult M.positive_integral_multc * prod subset_insertI) |
|
1716 |
qed |
|
1717 |
||
41026
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1718 |
lemma (in product_sigma_finite) product_integral_singleton: |
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1719 |
assumes f: "f \<in> borel_measurable (M i)" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1720 |
shows "(\<integral>x. f (x i) \<partial>Pi\<^isub>M {i} M) = integral\<^isup>L (M i) f" |
41026
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1721 |
proof - |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1722 |
interpret I: finite_product_sigma_finite M "{i}" by default simp |
41026
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1723 |
have *: "(\<lambda>x. Real (f x)) \<in> borel_measurable (M i)" |
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1724 |
"(\<lambda>x. Real (- f x)) \<in> borel_measurable (M i)" |
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1725 |
using assms by auto |
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1726 |
show ?thesis |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1727 |
unfolding lebesgue_integral_def *[THEN product_positive_integral_singleton] .. |
41026
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1728 |
qed |
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1729 |
|
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1730 |
lemma (in product_sigma_finite) product_integral_fold: |
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1731 |
assumes IJ[simp]: "I \<inter> J = {}" and fin: "finite I" "finite J" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1732 |
and f: "integrable (Pi\<^isub>M (I \<union> J) M) f" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1733 |
shows "integral\<^isup>L (Pi\<^isub>M (I \<union> J) M) f = (\<integral>x. (\<integral>y. f (merge I x J y) \<partial>Pi\<^isub>M J M) \<partial>Pi\<^isub>M I M)" |
41026
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1734 |
proof - |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1735 |
interpret I: finite_product_sigma_finite M I by default fact |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1736 |
interpret J: finite_product_sigma_finite M J by default fact |
41026
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1737 |
have "finite (I \<union> J)" using fin by auto |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1738 |
interpret IJ: finite_product_sigma_finite M "I \<union> J" by default fact |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1739 |
interpret P: pair_sigma_finite I.P J.P by default |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1740 |
let ?M = "\<lambda>(x, y). merge I x J y" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1741 |
let ?f = "\<lambda>x. f (?M x)" |
41026
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1742 |
show ?thesis |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1743 |
proof (subst P.integrable_fst_measurable(2)[of ?f, simplified]) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1744 |
have 1: "sigma_algebra IJ.P" by default |
41831 | 1745 |
have 2: "?M \<in> measure_preserving P.P IJ.P" using measure_preserving_merge[OF assms(1,2,3)] . |
1746 |
have 3: "integrable (Pi\<^isub>M (I \<union> J) M) f" by fact |
|
1747 |
then have 4: "f \<in> borel_measurable (Pi\<^isub>M (I \<union> J) M)" |
|
1748 |
by (simp add: integrable_def) |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1749 |
show "integrable P.P ?f" |
41831 | 1750 |
by (rule P.integrable_vimage[where f=f, OF 1 2 3]) |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1751 |
show "integral\<^isup>L IJ.P f = integral\<^isup>L P.P ?f" |
41831 | 1752 |
by (rule P.integral_vimage[where f=f, OF 1 2 4]) |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1753 |
qed |
41026
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1754 |
qed |
bea75746dc9d
folding on arbitrary Lebesgue integrable functions
hoelzl
parents:
41023
diff
changeset
|
1755 |
|
41096 | 1756 |
lemma (in product_sigma_finite) product_integral_insert: |
1757 |
assumes [simp]: "finite I" "i \<notin> I" |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1758 |
and f: "integrable (Pi\<^isub>M (insert i I) M) f" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1759 |
shows "integral\<^isup>L (Pi\<^isub>M (insert i I) M) f = (\<integral>x. (\<integral>y. f (x(i:=y)) \<partial>M i) \<partial>Pi\<^isub>M I M)" |
41096 | 1760 |
proof - |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1761 |
interpret I: finite_product_sigma_finite M I by default auto |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1762 |
interpret I': finite_product_sigma_finite M "insert i I" by default auto |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1763 |
interpret i: finite_product_sigma_finite M "{i}" by default auto |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1764 |
interpret P: pair_sigma_finite I.P i.P .. |
41096 | 1765 |
have IJ: "I \<inter> {i} = {}" by auto |
1766 |
show ?thesis |
|
1767 |
unfolding product_integral_fold[OF IJ, simplified, OF f] |
|
1768 |
proof (rule I.integral_cong, subst product_integral_singleton) |
|
1769 |
fix x assume x: "x \<in> space I.P" |
|
1770 |
let "?f y" = "f (restrict (x(i := y)) (insert i I))" |
|
1771 |
have f'_eq: "\<And>y. ?f y = f (x(i := y))" |
|
1772 |
using x by (auto intro!: arg_cong[where f=f] simp: fun_eq_iff extensional_def) |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1773 |
have f: "f \<in> borel_measurable I'.P" using f unfolding integrable_def by auto |
41096 | 1774 |
show "?f \<in> borel_measurable (M i)" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1775 |
unfolding measurable_cong[OF f'_eq] |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1776 |
using measurable_comp[OF measurable_component_update f] x `i \<notin> I` |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1777 |
by (simp add: comp_def) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1778 |
show "integral\<^isup>L (M i) ?f = integral\<^isup>L (M i) (\<lambda>y. f (x(i := y)))" |
41096 | 1779 |
unfolding f'_eq by simp |
1780 |
qed |
|
1781 |
qed |
|
1782 |
||
1783 |
lemma (in product_sigma_finite) product_integrable_setprod: |
|
1784 |
fixes f :: "'i \<Rightarrow> 'a \<Rightarrow> real" |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1785 |
assumes [simp]: "finite I" and integrable: "\<And>i. i \<in> I \<Longrightarrow> integrable (M i) (f i)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1786 |
shows "integrable (Pi\<^isub>M I M) (\<lambda>x. (\<Prod>i\<in>I. f i (x i)))" (is "integrable _ ?f") |
41096 | 1787 |
proof - |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1788 |
interpret finite_product_sigma_finite M I by default fact |
41096 | 1789 |
have f: "\<And>i. i \<in> I \<Longrightarrow> f i \<in> borel_measurable (M i)" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1790 |
using integrable unfolding integrable_def by auto |
41096 | 1791 |
then have borel: "?f \<in> borel_measurable P" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1792 |
using measurable_comp[OF measurable_component_singleton f] |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1793 |
by (auto intro!: borel_measurable_setprod simp: comp_def) |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1794 |
moreover have "integrable (Pi\<^isub>M I M) (\<lambda>x. \<bar>\<Prod>i\<in>I. f i (x i)\<bar>)" |
41096 | 1795 |
proof (unfold integrable_def, intro conjI) |
1796 |
show "(\<lambda>x. abs (?f x)) \<in> borel_measurable P" |
|
1797 |
using borel by auto |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1798 |
have "(\<integral>\<^isup>+x. Real (abs (?f x)) \<partial>P) = (\<integral>\<^isup>+x. (\<Prod>i\<in>I. Real (abs (f i (x i)))) \<partial>P)" |
41096 | 1799 |
by (simp add: Real_setprod abs_setprod) |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1800 |
also have "\<dots> = (\<Prod>i\<in>I. (\<integral>\<^isup>+x. Real (abs (f i x)) \<partial>M i))" |
41096 | 1801 |
using f by (subst product_positive_integral_setprod) auto |
1802 |
also have "\<dots> < \<omega>" |
|
1803 |
using integrable[THEN M.integrable_abs] |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1804 |
unfolding pextreal_less_\<omega> setprod_\<omega> integrable_def by simp |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1805 |
finally show "(\<integral>\<^isup>+x. Real (abs (?f x)) \<partial>P) \<noteq> \<omega>" by auto |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1806 |
show "(\<integral>\<^isup>+x. Real (- abs (?f x)) \<partial>P) \<noteq> \<omega>" by simp |
41096 | 1807 |
qed |
1808 |
ultimately show ?thesis |
|
1809 |
by (rule integrable_abs_iff[THEN iffD1]) |
|
1810 |
qed |
|
1811 |
||
1812 |
lemma (in product_sigma_finite) product_integral_setprod: |
|
1813 |
fixes f :: "'i \<Rightarrow> 'a \<Rightarrow> real" |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1814 |
assumes "finite I" "I \<noteq> {}" and integrable: "\<And>i. i \<in> I \<Longrightarrow> integrable (M i) (f i)" |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1815 |
shows "(\<integral>x. (\<Prod>i\<in>I. f i (x i)) \<partial>Pi\<^isub>M I M) = (\<Prod>i\<in>I. integral\<^isup>L (M i) (f i))" |
41096 | 1816 |
using assms proof (induct rule: finite_ne_induct) |
1817 |
case (singleton i) |
|
1818 |
then show ?case by (simp add: product_integral_singleton integrable_def) |
|
1819 |
next |
|
1820 |
case (insert i I) |
|
1821 |
then have iI: "finite (insert i I)" by auto |
|
1822 |
then have prod: "\<And>J. J \<subseteq> insert i I \<Longrightarrow> |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1823 |
integrable (Pi\<^isub>M J M) (\<lambda>x. (\<Prod>i\<in>J. f i (x i)))" |
41096 | 1824 |
by (intro product_integrable_setprod insert(5)) (auto intro: finite_subset) |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1825 |
interpret I: finite_product_sigma_finite M I by default fact |
41096 | 1826 |
have *: "\<And>x y. (\<Prod>j\<in>I. f j (if j = i then y else x j)) = (\<Prod>j\<in>I. f j (x j))" |
1827 |
using `i \<notin> I` by (auto intro!: setprod_cong) |
|
1828 |
show ?case |
|
1829 |
unfolding product_integral_insert[OF insert(1,3) prod[OF subset_refl]] |
|
1830 |
by (simp add: * insert integral_multc I.integral_cmult[OF prod] subset_insertI) |
|
1831 |
qed |
|
1832 |
||
40859 | 1833 |
section "Products on finite spaces" |
1834 |
||
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1835 |
lemma sigma_sets_pair_measure_generator_finite: |
38656 | 1836 |
assumes "finite A" and "finite B" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1837 |
shows "sigma_sets (A \<times> B) { a \<times> b | a b. a \<in> Pow A \<and> b \<in> Pow B} = Pow (A \<times> B)" |
40859 | 1838 |
(is "sigma_sets ?prod ?sets = _") |
38656 | 1839 |
proof safe |
1840 |
have fin: "finite (A \<times> B)" using assms by (rule finite_cartesian_product) |
|
1841 |
fix x assume subset: "x \<subseteq> A \<times> B" |
|
1842 |
hence "finite x" using fin by (rule finite_subset) |
|
40859 | 1843 |
from this subset show "x \<in> sigma_sets ?prod ?sets" |
38656 | 1844 |
proof (induct x) |
1845 |
case empty show ?case by (rule sigma_sets.Empty) |
|
1846 |
next |
|
1847 |
case (insert a x) |
|
40859 | 1848 |
hence "{a} \<in> sigma_sets ?prod ?sets" |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1849 |
by (auto simp: pair_measure_generator_def intro!: sigma_sets.Basic) |
38656 | 1850 |
moreover have "x \<in> sigma_sets ?prod ?sets" using insert by auto |
1851 |
ultimately show ?case unfolding insert_is_Un[of a x] by (rule sigma_sets_Un) |
|
1852 |
qed |
|
1853 |
next |
|
1854 |
fix x a b |
|
40859 | 1855 |
assume "x \<in> sigma_sets ?prod ?sets" and "(a, b) \<in> x" |
38656 | 1856 |
from sigma_sets_into_sp[OF _ this(1)] this(2) |
40859 | 1857 |
show "a \<in> A" and "b \<in> B" by auto |
35833 | 1858 |
qed |
1859 |
||
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1860 |
locale pair_finite_sigma_algebra = M1: finite_sigma_algebra M1 + M2: finite_sigma_algebra M2 |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1861 |
for M1 :: "('a, 'c) measure_space_scheme" and M2 :: "('b, 'd) measure_space_scheme" |
40859 | 1862 |
|
1863 |
sublocale pair_finite_sigma_algebra \<subseteq> pair_sigma_algebra by default |
|
1864 |
||
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1865 |
lemma (in pair_finite_sigma_algebra) finite_pair_sigma_algebra: |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1866 |
shows "P = \<lparr> space = space M1 \<times> space M2, sets = Pow (space M1 \<times> space M2), \<dots> = algebra.more P \<rparr>" |
35977 | 1867 |
proof - |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1868 |
show ?thesis |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1869 |
using sigma_sets_pair_measure_generator_finite[OF M1.finite_space M2.finite_space] |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1870 |
by (intro algebra.equality) (simp_all add: pair_measure_def pair_measure_generator_def sigma_def) |
40859 | 1871 |
qed |
1872 |
||
1873 |
sublocale pair_finite_sigma_algebra \<subseteq> finite_sigma_algebra P |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1874 |
apply default |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1875 |
using M1.finite_space M2.finite_space |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1876 |
apply (subst finite_pair_sigma_algebra) apply simp |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1877 |
apply (subst (1 2) finite_pair_sigma_algebra) apply simp |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1878 |
done |
35833 | 1879 |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1880 |
locale pair_finite_space = M1: finite_measure_space M1 + M2: finite_measure_space M2 |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1881 |
for M1 M2 |
40859 | 1882 |
|
1883 |
sublocale pair_finite_space \<subseteq> pair_finite_sigma_algebra |
|
1884 |
by default |
|
35833 | 1885 |
|
40859 | 1886 |
sublocale pair_finite_space \<subseteq> pair_sigma_finite |
1887 |
by default |
|
38656 | 1888 |
|
40859 | 1889 |
lemma (in pair_finite_space) pair_measure_Pair[simp]: |
1890 |
assumes "a \<in> space M1" "b \<in> space M2" |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1891 |
shows "\<mu> {(a, b)} = M1.\<mu> {a} * M2.\<mu> {b}" |
40859 | 1892 |
proof - |
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1893 |
have "\<mu> ({a}\<times>{b}) = M1.\<mu> {a} * M2.\<mu> {b}" |
40859 | 1894 |
using M1.sets_eq_Pow M2.sets_eq_Pow assms |
1895 |
by (subst pair_measure_times) auto |
|
1896 |
then show ?thesis by simp |
|
38656 | 1897 |
qed |
1898 |
||
40859 | 1899 |
lemma (in pair_finite_space) pair_measure_singleton[simp]: |
1900 |
assumes "x \<in> space M1 \<times> space M2" |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1901 |
shows "\<mu> {x} = M1.\<mu> {fst x} * M2.\<mu> {snd x}" |
40859 | 1902 |
using pair_measure_Pair assms by (cases x) auto |
38656 | 1903 |
|
41689
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1904 |
sublocale pair_finite_space \<subseteq> finite_measure_space P |
3e39b0e730d6
the measure valuation is again part of the measure_space type, instead of an explicit parameter to the locale;
hoelzl
parents:
41661
diff
changeset
|
1905 |
by default (auto simp: space_pair_measure) |
39097 | 1906 |
|
40859 | 1907 |
end |