| author | wenzelm | 
| Thu, 11 Jan 2018 13:48:17 +0100 | |
| changeset 67405 | e9ab4ad7bd15 | 
| parent 64267 | b9a1486e79be | 
| child 68046 | 6aba668aea78 | 
| permissions | -rw-r--r-- | 
| 63627 | 1 | (* Title: HOL/Analysis/Regularity.thy | 
| 50087 | 2 | Author: Fabian Immler, TU München | 
| 3 | *) | |
| 4 | ||
| 61808 | 5 | section \<open>Regularity of Measures\<close> | 
| 50089 
1badf63e5d97
generalized to copy of countable types instead of instantiation of nat for discrete topology
 immler parents: 
50087diff
changeset | 6 | |
| 50087 | 7 | theory Regularity | 
| 8 | imports Measure_Space Borel_Space | |
| 9 | begin | |
| 10 | ||
| 11 | lemma | |
| 50881 
ae630bab13da
renamed countable_basis_space to second_countable_topology
 hoelzl parents: 
50530diff
changeset | 12 |   fixes M::"'a::{second_countable_topology, complete_space} measure"
 | 
| 50087 | 13 | assumes sb: "sets M = sets borel" | 
| 14 | assumes "emeasure M (space M) \<noteq> \<infinity>" | |
| 15 | assumes "B \<in> sets borel" | |
| 16 | shows inner_regular: "emeasure M B = | |
| 17 |     (SUP K : {K. K \<subseteq> B \<and> compact K}. emeasure M K)" (is "?inner B")
 | |
| 18 | and outer_regular: "emeasure M B = | |
| 19 |     (INF U : {U. B \<subseteq> U \<and> open U}. emeasure M U)" (is "?outer B")
 | |
| 20 | proof - | |
| 21 | have Us: "UNIV = space M" by (metis assms(1) sets_eq_imp_space_eq space_borel) | |
| 22 | hence sU: "space M = UNIV" by simp | |
| 23 | interpret finite_measure M by rule fact | |
| 24 | have approx_inner: "\<And>A. A \<in> sets M \<Longrightarrow> | |
| 62975 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 25 | (\<And>e. e > 0 \<Longrightarrow> \<exists>K. K \<subseteq> A \<and> compact K \<and> emeasure M A \<le> emeasure M K + ennreal e) \<Longrightarrow> ?inner A" | 
| 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 26 | by (rule ennreal_approx_SUP) | 
| 50087 | 27 | (force intro!: emeasure_mono simp: compact_imp_closed emeasure_eq_measure)+ | 
| 28 | have approx_outer: "\<And>A. A \<in> sets M \<Longrightarrow> | |
| 62975 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 29 | (\<And>e. e > 0 \<Longrightarrow> \<exists>B. A \<subseteq> B \<and> open B \<and> emeasure M B \<le> emeasure M A + ennreal e) \<Longrightarrow> ?outer A" | 
| 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 30 | by (rule ennreal_approx_INF) | 
| 50087 | 31 | (force intro!: emeasure_mono simp: emeasure_eq_measure sb)+ | 
| 50245 
dea9363887a6
based countable topological basis on Countable_Set
 immler parents: 
50244diff
changeset | 32 | from countable_dense_setE guess X::"'a set" . note X = this | 
| 50087 | 33 |   {
 | 
| 34 |     fix r::real assume "r > 0" hence "\<And>y. open (ball y r)" "\<And>y. ball y r \<noteq> {}" by auto
 | |
| 50245 
dea9363887a6
based countable topological basis on Countable_Set
 immler parents: 
50244diff
changeset | 35 | with X(2)[OF this] | 
| 
dea9363887a6
based countable topological basis on Countable_Set
 immler parents: 
50244diff
changeset | 36 | have x: "space M = (\<Union>x\<in>X. cball x r)" | 
| 50087 | 37 | by (auto simp add: sU) (metis dist_commute order_less_imp_le) | 
| 50245 
dea9363887a6
based countable topological basis on Countable_Set
 immler parents: 
50244diff
changeset | 38 |     let ?U = "\<Union>k. (\<Union>n\<in>{0..k}. cball (from_nat_into X n) r)"
 | 
| 61969 | 39 |     have "(\<lambda>k. emeasure M (\<Union>n\<in>{0..k}. cball (from_nat_into X n) r)) \<longlonglongrightarrow> M ?U"
 | 
| 62975 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 40 | by (rule Lim_emeasure_incseq) (auto intro!: borel_closed bexI simp: incseq_def Us sb) | 
| 50245 
dea9363887a6
based countable topological basis on Countable_Set
 immler parents: 
50244diff
changeset | 41 | also have "?U = space M" | 
| 
dea9363887a6
based countable topological basis on Countable_Set
 immler parents: 
50244diff
changeset | 42 | proof safe | 
| 61808 | 43 | fix x from X(2)[OF open_ball[of x r]] \<open>r > 0\<close> obtain d where d: "d\<in>X" "d \<in> ball x r" by auto | 
| 50245 
dea9363887a6
based countable topological basis on Countable_Set
 immler parents: 
50244diff
changeset | 44 | show "x \<in> ?U" | 
| 62343 
24106dc44def
prefer abbreviations for compound operators INFIMUM and SUPREMUM
 haftmann parents: 
61969diff
changeset | 45 | using X(1) d | 
| 
24106dc44def
prefer abbreviations for compound operators INFIMUM and SUPREMUM
 haftmann parents: 
61969diff
changeset | 46 | by simp (auto intro!: exI [where x = "to_nat_on X d"] simp: dist_commute Bex_def) | 
| 50245 
dea9363887a6
based countable topological basis on Countable_Set
 immler parents: 
50244diff
changeset | 47 | qed (simp add: sU) | 
| 61969 | 48 |     finally have "(\<lambda>k. M (\<Union>n\<in>{0..k}. cball (from_nat_into X n) r)) \<longlonglongrightarrow> M (space M)" .
 | 
| 50087 | 49 | } note M_space = this | 
| 50 |   {
 | |
| 51 | fix e ::real and n :: nat assume "e > 0" "n > 0" | |
| 56544 | 52 | hence "1/n > 0" "e * 2 powr - n > 0" by (auto) | 
| 61808 | 53 | from M_space[OF \<open>1/n>0\<close>] | 
| 61969 | 54 |     have "(\<lambda>k. measure M (\<Union>i\<in>{0..k}. cball (from_nat_into X i) (1/real n))) \<longlonglongrightarrow> measure M (space M)"
 | 
| 62975 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 55 | unfolding emeasure_eq_measure by (auto simp: measure_nonneg) | 
| 61808 | 56 | from metric_LIMSEQ_D[OF this \<open>0 < e * 2 powr -n\<close>] | 
| 50245 
dea9363887a6
based countable topological basis on Countable_Set
 immler parents: 
50244diff
changeset | 57 |     obtain k where "dist (measure M (\<Union>i\<in>{0..k}. cball (from_nat_into X i) (1/real n))) (measure M (space M)) <
 | 
| 50087 | 58 | e * 2 powr -n" | 
| 59 | by auto | |
| 50245 
dea9363887a6
based countable topological basis on Countable_Set
 immler parents: 
50244diff
changeset | 60 |     hence "measure M (\<Union>i\<in>{0..k}. cball (from_nat_into X i) (1/real n)) \<ge>
 | 
| 50087 | 61 | measure M (space M) - e * 2 powr -real n" | 
| 62 | by (auto simp: dist_real_def) | |
| 50245 
dea9363887a6
based countable topological basis on Countable_Set
 immler parents: 
50244diff
changeset | 63 |     hence "\<exists>k. measure M (\<Union>i\<in>{0..k}. cball (from_nat_into X i) (1/real n)) \<ge>
 | 
| 50087 | 64 | measure M (space M) - e * 2 powr - real n" .. | 
| 65 | } note k=this | |
| 66 |   hence "\<forall>e\<in>{0<..}. \<forall>(n::nat)\<in>{0<..}. \<exists>k.
 | |
| 50245 
dea9363887a6
based countable topological basis on Countable_Set
 immler parents: 
50244diff
changeset | 67 |     measure M (\<Union>i\<in>{0..k}. cball (from_nat_into X i) (1/real n)) \<ge> measure M (space M) - e * 2 powr - real n"
 | 
| 50087 | 68 | by blast | 
| 69 |   then obtain k where k: "\<forall>e\<in>{0<..}. \<forall>n\<in>{0<..}. measure M (space M) - e * 2 powr - real (n::nat)
 | |
| 50245 
dea9363887a6
based countable topological basis on Countable_Set
 immler parents: 
50244diff
changeset | 70 |     \<le> measure M (\<Union>i\<in>{0..k e n}. cball (from_nat_into X i) (1 / n))"
 | 
| 58184 
db1381d811ab
cleanup Wfrec; introduce dependent_wf/wellorder_choice
 hoelzl parents: 
56544diff
changeset | 71 | by metis | 
| 50087 | 72 | hence k: "\<And>e n. e > 0 \<Longrightarrow> n > 0 \<Longrightarrow> measure M (space M) - e * 2 powr - n | 
| 50245 
dea9363887a6
based countable topological basis on Countable_Set
 immler parents: 
50244diff
changeset | 73 |     \<le> measure M (\<Union>i\<in>{0..k e n}. cball (from_nat_into X i) (1 / n))"
 | 
| 50087 | 74 | unfolding Ball_def by blast | 
| 75 | have approx_space: | |
| 62975 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 76 |     "\<exists>K \<in> {K. K \<subseteq> space M \<and> compact K}. emeasure M (space M) \<le> emeasure M K + ennreal e"
 | 
| 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 77 | (is "?thesis e") if "0 < e" for e :: real | 
| 50087 | 78 | proof - | 
| 63040 | 79 | define B where [abs_def]: | 
| 80 |       "B n = (\<Union>i\<in>{0..k e (Suc n)}. cball (from_nat_into X i) (1 / Suc n))" for n
 | |
| 62975 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 81 | have "\<And>n. closed (B n)" by (auto simp: B_def) | 
| 50087 | 82 | hence [simp]: "\<And>n. B n \<in> sets M" by (simp add: sb) | 
| 61808 | 83 | from k[OF \<open>e > 0\<close> zero_less_Suc] | 
| 50087 | 84 | have "\<And>n. measure M (space M) - measure M (B n) \<le> e * 2 powr - real (Suc n)" | 
| 85 | by (simp add: algebra_simps B_def finite_measure_compl) | |
| 86 | hence B_compl_le: "\<And>n::nat. measure M (space M - B n) \<le> e * 2 powr - real (Suc n)" | |
| 87 | by (simp add: finite_measure_compl) | |
| 63040 | 88 | define K where "K = (\<Inter>n. B n)" | 
| 61808 | 89 | from \<open>closed (B _)\<close> have "closed K" by (auto simp: K_def) | 
| 50087 | 90 | hence [simp]: "K \<in> sets M" by (simp add: sb) | 
| 91 | have "measure M (space M) - measure M K = measure M (space M - K)" | |
| 92 | by (simp add: finite_measure_compl) | |
| 93 | also have "\<dots> = emeasure M (\<Union>n. space M - B n)" by (auto simp: K_def emeasure_eq_measure) | |
| 94 | also have "\<dots> \<le> (\<Sum>n. emeasure M (space M - B n))" | |
| 95 | by (rule emeasure_subadditive_countably) (auto simp: summable_def) | |
| 62975 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 96 | also have "\<dots> \<le> (\<Sum>n. ennreal (e*2 powr - real (Suc n)))" | 
| 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 97 | using B_compl_le by (intro suminf_le) (simp_all add: measure_nonneg emeasure_eq_measure ennreal_leI) | 
| 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 98 | also have "\<dots> \<le> (\<Sum>n. ennreal (e * (1 / 2) ^ Suc n))" | 
| 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 99 | by (simp add: powr_minus powr_realpow field_simps del: of_nat_Suc) | 
| 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 100 | also have "\<dots> = ennreal e * (\<Sum>n. ennreal ((1 / 2) ^ Suc n))" | 
| 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 101 | unfolding ennreal_power[symmetric] | 
| 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 102 | using \<open>0 < e\<close> | 
| 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 103 | by (simp add: ac_simps ennreal_mult' divide_ennreal[symmetric] divide_ennreal_def | 
| 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 104 | ennreal_power[symmetric]) | 
| 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 105 | also have "\<dots> = e" | 
| 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 106 | by (subst suminf_ennreal_eq[OF zero_le_power power_half_series]) auto | 
| 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 107 | finally have "measure M (space M) \<le> measure M K + e" | 
| 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 108 | using \<open>0 < e\<close> by simp | 
| 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 109 | hence "emeasure M (space M) \<le> emeasure M K + e" | 
| 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 110 | using \<open>0 < e\<close> by (simp add: emeasure_eq_measure measure_nonneg ennreal_plus[symmetric] del: ennreal_plus) | 
| 50087 | 111 | moreover have "compact K" | 
| 112 | unfolding compact_eq_totally_bounded | |
| 113 | proof safe | |
| 61808 | 114 | show "complete K" using \<open>closed K\<close> by (simp add: complete_eq_closed) | 
| 50087 | 115 | fix e'::real assume "0 < e'" | 
| 116 | from nat_approx_posE[OF this] guess n . note n = this | |
| 50245 
dea9363887a6
based countable topological basis on Countable_Set
 immler parents: 
50244diff
changeset | 117 |       let ?k = "from_nat_into X ` {0..k e (Suc n)}"
 | 
| 50087 | 118 | have "finite ?k" by simp | 
| 58184 
db1381d811ab
cleanup Wfrec; introduce dependent_wf/wellorder_choice
 hoelzl parents: 
56544diff
changeset | 119 | moreover have "K \<subseteq> (\<Union>x\<in>?k. ball x e')" unfolding K_def B_def using n by force | 
| 
db1381d811ab
cleanup Wfrec; introduce dependent_wf/wellorder_choice
 hoelzl parents: 
56544diff
changeset | 120 | ultimately show "\<exists>k. finite k \<and> K \<subseteq> (\<Union>x\<in>k. ball x e')" by blast | 
| 50087 | 121 | qed | 
| 122 | ultimately | |
| 62975 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 123 | show ?thesis by (auto simp: sU) | 
| 50087 | 124 | qed | 
| 50125 
4319691be975
tuned: use induction rule sigma_sets_induct_disjoint
 hoelzl parents: 
50089diff
changeset | 125 |   { fix A::"'a set" assume "closed A" hence "A \<in> sets borel" by (simp add: compact_imp_closed)
 | 
| 50087 | 126 | hence [simp]: "A \<in> sets M" by (simp add: sb) | 
| 50125 
4319691be975
tuned: use induction rule sigma_sets_induct_disjoint
 hoelzl parents: 
50089diff
changeset | 127 | have "?inner A" | 
| 50087 | 128 | proof (rule approx_inner) | 
| 129 | fix e::real assume "e > 0" | |
| 130 | from approx_space[OF this] obtain K where | |
| 131 | K: "K \<subseteq> space M" "compact K" "emeasure M (space M) \<le> emeasure M K + e" | |
| 132 | by (auto simp: emeasure_eq_measure) | |
| 133 | hence [simp]: "K \<in> sets M" by (simp add: sb compact_imp_closed) | |
| 62975 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 134 | have "measure M A - measure M (A \<inter> K) = measure M (A - A \<inter> K)" | 
| 50087 | 135 | by (subst finite_measure_Diff) auto | 
| 136 | also have "A - A \<inter> K = A \<union> K - K" by auto | |
| 137 | also have "measure M \<dots> = measure M (A \<union> K) - measure M K" | |
| 138 | by (subst finite_measure_Diff) auto | |
| 139 | also have "\<dots> \<le> measure M (space M) - measure M K" | |
| 140 | by (simp add: emeasure_eq_measure sU sb finite_measure_mono) | |
| 62975 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 141 | also have "\<dots> \<le> e" | 
| 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 142 | using K \<open>0 < e\<close> by (simp add: emeasure_eq_measure ennreal_plus[symmetric] measure_nonneg del: ennreal_plus) | 
| 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 143 | finally have "emeasure M A \<le> emeasure M (A \<inter> K) + ennreal e" | 
| 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 144 | using \<open>0<e\<close> by (simp add: emeasure_eq_measure algebra_simps ennreal_plus[symmetric] measure_nonneg del: ennreal_plus) | 
| 61808 | 145 | moreover have "A \<inter> K \<subseteq> A" "compact (A \<inter> K)" using \<open>closed A\<close> \<open>compact K\<close> by auto | 
| 62975 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 146 | ultimately show "\<exists>K \<subseteq> A. compact K \<and> emeasure M A \<le> emeasure M K + ennreal e" | 
| 50087 | 147 | by blast | 
| 148 | qed simp | |
| 50125 
4319691be975
tuned: use induction rule sigma_sets_induct_disjoint
 hoelzl parents: 
50089diff
changeset | 149 | have "?outer A" | 
| 50087 | 150 | proof cases | 
| 151 |       assume "A \<noteq> {}"
 | |
| 152 |       let ?G = "\<lambda>d. {x. infdist x A < d}"
 | |
| 153 |       {
 | |
| 154 | fix d | |
| 155 |         have "?G d = (\<lambda>x. infdist x A) -` {..<d}" by auto
 | |
| 156 | also have "open \<dots>" | |
| 62533 
bc25f3916a99
new material to Blochj's theorem, as well as supporting lemmas
 paulson <lp15@cam.ac.uk> parents: 
62343diff
changeset | 157 | by (intro continuous_open_vimage) (auto intro!: continuous_infdist continuous_ident) | 
| 50087 | 158 | finally have "open (?G d)" . | 
| 159 | } note open_G = this | |
| 61808 | 160 |       from in_closed_iff_infdist_zero[OF \<open>closed A\<close> \<open>A \<noteq> {}\<close>]
 | 
| 50087 | 161 |       have "A = {x. infdist x A = 0}" by auto
 | 
| 162 | also have "\<dots> = (\<Inter>i. ?G (1/real (Suc i)))" | |
| 61609 
77b453bd616f
Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
 paulson <lp15@cam.ac.uk> parents: 
61284diff
changeset | 163 | proof (auto simp del: of_nat_Suc, rule ccontr) | 
| 50087 | 164 | fix x | 
| 165 | assume "infdist x A \<noteq> 0" | |
| 166 | hence pos: "infdist x A > 0" using infdist_nonneg[of x A] by simp | |
| 167 | from nat_approx_posE[OF this] guess n . | |
| 168 | moreover | |
| 169 | assume "\<forall>i. infdist x A < 1 / real (Suc i)" | |
| 170 | hence "infdist x A < 1 / real (Suc n)" by auto | |
| 61609 
77b453bd616f
Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
 paulson <lp15@cam.ac.uk> parents: 
61284diff
changeset | 171 | ultimately show False by simp | 
| 50087 | 172 | qed | 
| 173 | also have "M \<dots> = (INF n. emeasure M (?G (1 / real (Suc n))))" | |
| 174 | proof (rule INF_emeasure_decseq[symmetric], safe) | |
| 175 | fix i::nat | |
| 176 | from open_G[of "1 / real (Suc i)"] | |
| 177 | show "?G (1 / real (Suc i)) \<in> sets M" by (simp add: sb borel_open) | |
| 178 | next | |
| 179 |         show "decseq (\<lambda>i. {x. infdist x A < 1 / real (Suc i)})"
 | |
| 56544 | 180 | by (auto intro: less_trans intro!: divide_strict_left_mono | 
| 50087 | 181 | simp: decseq_def le_eq_less_or_eq) | 
| 182 | qed simp | |
| 183 | finally | |
| 184 |       have "emeasure M A = (INF n. emeasure M {x. infdist x A < 1 / real (Suc n)})" .
 | |
| 185 | moreover | |
| 186 |       have "\<dots> \<ge> (INF U:{U. A \<subseteq> U \<and> open U}. emeasure M U)"
 | |
| 187 | proof (intro INF_mono) | |
| 188 | fix m | |
| 189 |         have "?G (1 / real (Suc m)) \<in> {U. A \<subseteq> U \<and> open U}" using open_G by auto
 | |
| 190 | moreover have "M (?G (1 / real (Suc m))) \<le> M (?G (1 / real (Suc m)))" by simp | |
| 191 |         ultimately show "\<exists>U\<in>{U. A \<subseteq> U \<and> open U}.
 | |
| 192 |           emeasure M U \<le> emeasure M {x. infdist x A < 1 / real (Suc m)}"
 | |
| 193 | by blast | |
| 194 | qed | |
| 195 | moreover | |
| 196 |       have "emeasure M A \<le> (INF U:{U. A \<subseteq> U \<and> open U}. emeasure M U)"
 | |
| 197 | by (rule INF_greatest) (auto intro!: emeasure_mono simp: sb) | |
| 198 | ultimately show ?thesis by simp | |
| 51000 | 199 | qed (auto intro!: INF_eqI) | 
| 61808 | 200 | note \<open>?inner A\<close> \<open>?outer A\<close> } | 
| 50125 
4319691be975
tuned: use induction rule sigma_sets_induct_disjoint
 hoelzl parents: 
50089diff
changeset | 201 | note closed_in_D = this | 
| 61808 | 202 | from \<open>B \<in> sets borel\<close> | 
| 61609 
77b453bd616f
Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
 paulson <lp15@cam.ac.uk> parents: 
61284diff
changeset | 203 | have "Int_stable (Collect closed)" "Collect closed \<subseteq> Pow UNIV" "B \<in> sigma_sets UNIV (Collect closed)" | 
| 50125 
4319691be975
tuned: use induction rule sigma_sets_induct_disjoint
 hoelzl parents: 
50089diff
changeset | 204 | by (auto simp: Int_stable_def borel_eq_closed) | 
| 
4319691be975
tuned: use induction rule sigma_sets_induct_disjoint
 hoelzl parents: 
50089diff
changeset | 205 | then show "?inner B" "?outer B" | 
| 
4319691be975
tuned: use induction rule sigma_sets_induct_disjoint
 hoelzl parents: 
50089diff
changeset | 206 | proof (induct B rule: sigma_sets_induct_disjoint) | 
| 
4319691be975
tuned: use induction rule sigma_sets_induct_disjoint
 hoelzl parents: 
50089diff
changeset | 207 | case empty | 
| 51000 | 208 |     { case 1 show ?case by (intro SUP_eqI[symmetric]) auto }
 | 
| 209 |     { case 2 show ?case by (intro INF_eqI[symmetric]) (auto elim!: meta_allE[of _ "{}"]) }
 | |
| 50087 | 210 | next | 
| 50125 
4319691be975
tuned: use induction rule sigma_sets_induct_disjoint
 hoelzl parents: 
50089diff
changeset | 211 | case (basic B) | 
| 
4319691be975
tuned: use induction rule sigma_sets_induct_disjoint
 hoelzl parents: 
50089diff
changeset | 212 |     { case 1 from basic closed_in_D show ?case by auto }
 | 
| 
4319691be975
tuned: use induction rule sigma_sets_induct_disjoint
 hoelzl parents: 
50089diff
changeset | 213 |     { case 2 from basic closed_in_D show ?case by auto }
 | 
| 
4319691be975
tuned: use induction rule sigma_sets_induct_disjoint
 hoelzl parents: 
50089diff
changeset | 214 | next | 
| 
4319691be975
tuned: use induction rule sigma_sets_induct_disjoint
 hoelzl parents: 
50089diff
changeset | 215 | case (compl B) | 
| 
4319691be975
tuned: use induction rule sigma_sets_induct_disjoint
 hoelzl parents: 
50089diff
changeset | 216 | note inner = compl(2) and outer = compl(3) | 
| 
4319691be975
tuned: use induction rule sigma_sets_induct_disjoint
 hoelzl parents: 
50089diff
changeset | 217 | from compl have [simp]: "B \<in> sets M" by (auto simp: sb borel_eq_closed) | 
| 
4319691be975
tuned: use induction rule sigma_sets_induct_disjoint
 hoelzl parents: 
50089diff
changeset | 218 | case 2 | 
| 50087 | 219 | have "M (space M - B) = M (space M) - emeasure M B" by (auto simp: emeasure_compl) | 
| 220 |     also have "\<dots> = (INF K:{K. K \<subseteq> B \<and> compact K}. M (space M) -  M K)"
 | |
| 62975 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 221 | by (subst ennreal_SUP_const_minus) (auto simp: less_top[symmetric] inner) | 
| 50087 | 222 |     also have "\<dots> = (INF U:{U. U \<subseteq> B \<and> compact U}. M (space M - U))"
 | 
| 223 | by (rule INF_cong) (auto simp add: emeasure_compl sb compact_imp_closed) | |
| 224 |     also have "\<dots> \<ge> (INF U:{U. U \<subseteq> B \<and> closed U}. M (space M - U))"
 | |
| 225 | by (rule INF_superset_mono) (auto simp add: compact_imp_closed) | |
| 226 |     also have "(INF U:{U. U \<subseteq> B \<and> closed U}. M (space M - U)) =
 | |
| 50125 
4319691be975
tuned: use induction rule sigma_sets_induct_disjoint
 hoelzl parents: 
50089diff
changeset | 227 |         (INF U:{U. space M - B \<subseteq> U \<and> open U}. emeasure M U)"
 | 
| 62343 
24106dc44def
prefer abbreviations for compound operators INFIMUM and SUPREMUM
 haftmann parents: 
61969diff
changeset | 228 | unfolding INF_image [of _ "\<lambda>u. space M - u" _, symmetric, unfolded comp_def] | 
| 62975 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 229 | by (rule INF_cong) (auto simp add: sU Compl_eq_Diff_UNIV [symmetric, simp]) | 
| 50087 | 230 | finally have | 
| 231 |       "(INF U:{U. space M - B \<subseteq> U \<and> open U}. emeasure M U) \<le> emeasure M (space M - B)" .
 | |
| 232 | moreover have | |
| 233 |       "(INF U:{U. space M - B \<subseteq> U \<and> open U}. emeasure M U) \<ge> emeasure M (space M - B)"
 | |
| 234 | by (auto simp: sb sU intro!: INF_greatest emeasure_mono) | |
| 50125 
4319691be975
tuned: use induction rule sigma_sets_induct_disjoint
 hoelzl parents: 
50089diff
changeset | 235 | ultimately show ?case by (auto intro!: antisym simp: sets_eq_imp_space_eq[OF sb]) | 
| 
4319691be975
tuned: use induction rule sigma_sets_induct_disjoint
 hoelzl parents: 
50089diff
changeset | 236 | |
| 
4319691be975
tuned: use induction rule sigma_sets_induct_disjoint
 hoelzl parents: 
50089diff
changeset | 237 | case 1 | 
| 
4319691be975
tuned: use induction rule sigma_sets_induct_disjoint
 hoelzl parents: 
50089diff
changeset | 238 | have "M (space M - B) = M (space M) - emeasure M B" by (auto simp: emeasure_compl) | 
| 
4319691be975
tuned: use induction rule sigma_sets_induct_disjoint
 hoelzl parents: 
50089diff
changeset | 239 |     also have "\<dots> = (SUP U: {U. B \<subseteq> U \<and> open U}. M (space M) -  M U)"
 | 
| 62975 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 240 | unfolding outer by (subst ennreal_INF_const_minus) auto | 
| 50125 
4319691be975
tuned: use induction rule sigma_sets_induct_disjoint
 hoelzl parents: 
50089diff
changeset | 241 |     also have "\<dots> = (SUP U:{U. B \<subseteq> U \<and> open U}. M (space M - U))"
 | 
| 
4319691be975
tuned: use induction rule sigma_sets_induct_disjoint
 hoelzl parents: 
50089diff
changeset | 242 | by (rule SUP_cong) (auto simp add: emeasure_compl sb compact_imp_closed) | 
| 
4319691be975
tuned: use induction rule sigma_sets_induct_disjoint
 hoelzl parents: 
50089diff
changeset | 243 |     also have "\<dots> = (SUP K:{K. K \<subseteq> space M - B \<and> closed K}. emeasure M K)"
 | 
| 62343 
24106dc44def
prefer abbreviations for compound operators INFIMUM and SUPREMUM
 haftmann parents: 
61969diff
changeset | 244 | unfolding SUP_image [of _ "\<lambda>u. space M - u" _, symmetric, unfolded comp_def] | 
| 
24106dc44def
prefer abbreviations for compound operators INFIMUM and SUPREMUM
 haftmann parents: 
61969diff
changeset | 245 | by (rule SUP_cong) (auto simp add: sU) | 
| 50125 
4319691be975
tuned: use induction rule sigma_sets_induct_disjoint
 hoelzl parents: 
50089diff
changeset | 246 |     also have "\<dots> = (SUP K:{K. K \<subseteq> space M - B \<and> compact K}. emeasure M K)"
 | 
| 
4319691be975
tuned: use induction rule sigma_sets_induct_disjoint
 hoelzl parents: 
50089diff
changeset | 247 | proof (safe intro!: antisym SUP_least) | 
| 
4319691be975
tuned: use induction rule sigma_sets_induct_disjoint
 hoelzl parents: 
50089diff
changeset | 248 | fix K assume "closed K" "K \<subseteq> space M - B" | 
| 61808 | 249 | from closed_in_D[OF \<open>closed K\<close>] | 
| 50125 
4319691be975
tuned: use induction rule sigma_sets_induct_disjoint
 hoelzl parents: 
50089diff
changeset | 250 |       have K_inner: "emeasure M K = (SUP K:{Ka. Ka \<subseteq> K \<and> compact Ka}. emeasure M K)" by simp
 | 
| 
4319691be975
tuned: use induction rule sigma_sets_induct_disjoint
 hoelzl parents: 
50089diff
changeset | 251 |       show "emeasure M K \<le> (SUP K:{K. K \<subseteq> space M - B \<and> compact K}. emeasure M K)"
 | 
| 61808 | 252 | unfolding K_inner using \<open>K \<subseteq> space M - B\<close> | 
| 50125 
4319691be975
tuned: use induction rule sigma_sets_induct_disjoint
 hoelzl parents: 
50089diff
changeset | 253 | by (auto intro!: SUP_upper SUP_least) | 
| 
4319691be975
tuned: use induction rule sigma_sets_induct_disjoint
 hoelzl parents: 
50089diff
changeset | 254 | qed (fastforce intro!: SUP_least SUP_upper simp: compact_imp_closed) | 
| 
4319691be975
tuned: use induction rule sigma_sets_induct_disjoint
 hoelzl parents: 
50089diff
changeset | 255 | finally show ?case by (auto intro!: antisym simp: sets_eq_imp_space_eq[OF sb]) | 
| 50087 | 256 | next | 
| 50125 
4319691be975
tuned: use induction rule sigma_sets_induct_disjoint
 hoelzl parents: 
50089diff
changeset | 257 | case (union D) | 
| 
4319691be975
tuned: use induction rule sigma_sets_induct_disjoint
 hoelzl parents: 
50089diff
changeset | 258 | then have "range D \<subseteq> sets M" by (auto simp: sb borel_eq_closed) | 
| 
4319691be975
tuned: use induction rule sigma_sets_induct_disjoint
 hoelzl parents: 
50089diff
changeset | 259 | with union have M[symmetric]: "(\<Sum>i. M (D i)) = M (\<Union>i. D i)" by (intro suminf_emeasure) | 
| 61969 | 260 | also have "(\<lambda>n. \<Sum>i<n. M (D i)) \<longlonglongrightarrow> (\<Sum>i. M (D i))" | 
| 62975 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 261 | by (intro summable_LIMSEQ) auto | 
| 61969 | 262 | finally have measure_LIMSEQ: "(\<lambda>n. \<Sum>i<n. measure M (D i)) \<longlonglongrightarrow> measure M (\<Union>i. D i)" | 
| 64267 | 263 | by (simp add: emeasure_eq_measure measure_nonneg sum_nonneg) | 
| 61808 | 264 | have "(\<Union>i. D i) \<in> sets M" using \<open>range D \<subseteq> sets M\<close> by auto | 
| 61609 
77b453bd616f
Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
 paulson <lp15@cam.ac.uk> parents: 
61284diff
changeset | 265 | |
| 50125 
4319691be975
tuned: use induction rule sigma_sets_induct_disjoint
 hoelzl parents: 
50089diff
changeset | 266 | case 1 | 
| 
4319691be975
tuned: use induction rule sigma_sets_induct_disjoint
 hoelzl parents: 
50089diff
changeset | 267 | show ?case | 
| 50087 | 268 | proof (rule approx_inner) | 
| 269 | fix e::real assume "e > 0" | |
| 270 | with measure_LIMSEQ | |
| 56193 
c726ecfb22b6
cleanup Series: sorted according to typeclass hierarchy, use {..<_} instead of {0..<_}
 hoelzl parents: 
56166diff
changeset | 271 | have "\<exists>no. \<forall>n\<ge>no. \<bar>(\<Sum>i<n. measure M (D i)) -measure M (\<Union>x. D x)\<bar> < e/2" | 
| 60017 
b785d6d06430
Overloading of ln and powr, but "approximation" no longer works for powr. Code generation also fails due to type ambiguity in scala.
 paulson <lp15@cam.ac.uk> parents: 
59452diff
changeset | 272 | by (auto simp: lim_sequentially dist_real_def simp del: less_divide_eq_numeral1) | 
| 56193 
c726ecfb22b6
cleanup Series: sorted according to typeclass hierarchy, use {..<_} instead of {0..<_}
 hoelzl parents: 
56166diff
changeset | 273 | hence "\<exists>n0. \<bar>(\<Sum>i<n0. measure M (D i)) - measure M (\<Union>x. D x)\<bar> < e/2" by auto | 
| 
c726ecfb22b6
cleanup Series: sorted according to typeclass hierarchy, use {..<_} instead of {0..<_}
 hoelzl parents: 
56166diff
changeset | 274 | then obtain n0 where n0: "\<bar>(\<Sum>i<n0. measure M (D i)) - measure M (\<Union>i. D i)\<bar> < e/2" | 
| 50087 | 275 | unfolding choice_iff by blast | 
| 62975 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 276 | have "ennreal (\<Sum>i<n0. measure M (D i)) = (\<Sum>i<n0. M (D i))" | 
| 64267 | 277 | by (auto simp add: emeasure_eq_measure sum_nonneg measure_nonneg) | 
| 278 | also have "\<dots> \<le> (\<Sum>i. M (D i))" by (rule sum_le_suminf) auto | |
| 50087 | 279 | also have "\<dots> = M (\<Union>i. D i)" by (simp add: M) | 
| 280 | also have "\<dots> = measure M (\<Union>i. D i)" by (simp add: emeasure_eq_measure) | |
| 56193 
c726ecfb22b6
cleanup Series: sorted according to typeclass hierarchy, use {..<_} instead of {0..<_}
 hoelzl parents: 
56166diff
changeset | 281 | finally have n0: "measure M (\<Union>i. D i) - (\<Sum>i<n0. measure M (D i)) < e/2" | 
| 64267 | 282 | using n0 by (auto simp: measure_nonneg sum_nonneg) | 
| 50087 | 283 | have "\<forall>i. \<exists>K. K \<subseteq> D i \<and> compact K \<and> emeasure M (D i) \<le> emeasure M K + e/(2*Suc n0)" | 
| 284 | proof | |
| 285 | fix i | |
| 61808 | 286 | from \<open>0 < e\<close> have "0 < e/(2*Suc n0)" by simp | 
| 50087 | 287 |         have "emeasure M (D i) = (SUP K:{K. K \<subseteq> (D i) \<and> compact K}. emeasure M K)"
 | 
| 50125 
4319691be975
tuned: use induction rule sigma_sets_induct_disjoint
 hoelzl parents: 
50089diff
changeset | 288 | using union by blast | 
| 62975 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 289 | from SUP_approx_ennreal[OF \<open>0 < e/(2*Suc n0)\<close> _ this] | 
| 50087 | 290 | show "\<exists>K. K \<subseteq> D i \<and> compact K \<and> emeasure M (D i) \<le> emeasure M K + e/(2*Suc n0)" | 
| 62975 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 291 | by (auto simp: emeasure_eq_measure intro: less_imp_le compact_empty) | 
| 50087 | 292 | qed | 
| 293 | then obtain K where K: "\<And>i. K i \<subseteq> D i" "\<And>i. compact (K i)" | |
| 294 | "\<And>i. emeasure M (D i) \<le> emeasure M (K i) + e/(2*Suc n0)" | |
| 295 | unfolding choice_iff by blast | |
| 56193 
c726ecfb22b6
cleanup Series: sorted according to typeclass hierarchy, use {..<_} instead of {0..<_}
 hoelzl parents: 
56166diff
changeset | 296 |       let ?K = "\<Union>i\<in>{..<n0}. K i"
 | 
| 61808 | 297 |       have "disjoint_family_on K {..<n0}" using K \<open>disjoint_family D\<close>
 | 
| 50087 | 298 | unfolding disjoint_family_on_def by blast | 
| 56193 
c726ecfb22b6
cleanup Series: sorted according to typeclass hierarchy, use {..<_} instead of {0..<_}
 hoelzl parents: 
56166diff
changeset | 299 | hence mK: "measure M ?K = (\<Sum>i<n0. measure M (K i))" using K | 
| 50087 | 300 | by (intro finite_measure_finite_Union) (auto simp: sb compact_imp_closed) | 
| 56193 
c726ecfb22b6
cleanup Series: sorted according to typeclass hierarchy, use {..<_} instead of {0..<_}
 hoelzl parents: 
56166diff
changeset | 301 | have "measure M (\<Union>i. D i) < (\<Sum>i<n0. measure M (D i)) + e/2" using n0 by simp | 
| 
c726ecfb22b6
cleanup Series: sorted according to typeclass hierarchy, use {..<_} instead of {0..<_}
 hoelzl parents: 
56166diff
changeset | 302 | also have "(\<Sum>i<n0. measure M (D i)) \<le> (\<Sum>i<n0. measure M (K i) + e/(2*Suc n0))" | 
| 62975 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 303 | using K \<open>0 < e\<close> | 
| 64267 | 304 | by (auto intro: sum_mono simp: emeasure_eq_measure measure_nonneg ennreal_plus[symmetric] simp del: ennreal_plus) | 
| 56193 
c726ecfb22b6
cleanup Series: sorted according to typeclass hierarchy, use {..<_} instead of {0..<_}
 hoelzl parents: 
56166diff
changeset | 305 | also have "\<dots> = (\<Sum>i<n0. measure M (K i)) + (\<Sum>i<n0. e/(2*Suc n0))" | 
| 64267 | 306 | by (simp add: sum.distrib) | 
| 61808 | 307 | also have "\<dots> \<le> (\<Sum>i<n0. measure M (K i)) + e / 2" using \<open>0 < e\<close> | 
| 61609 
77b453bd616f
Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
 paulson <lp15@cam.ac.uk> parents: 
61284diff
changeset | 308 | by (auto simp: field_simps intro!: mult_left_mono) | 
| 50087 | 309 | finally | 
| 56193 
c726ecfb22b6
cleanup Series: sorted according to typeclass hierarchy, use {..<_} instead of {0..<_}
 hoelzl parents: 
56166diff
changeset | 310 | have "measure M (\<Union>i. D i) < (\<Sum>i<n0. measure M (K i)) + e / 2 + e / 2" | 
| 50087 | 311 | by auto | 
| 62975 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 312 | hence "M (\<Union>i. D i) < M ?K + e" | 
| 64267 | 313 | using \<open>0<e\<close> by (auto simp: mK emeasure_eq_measure measure_nonneg sum_nonneg ennreal_less_iff ennreal_plus[symmetric] simp del: ennreal_plus) | 
| 50087 | 314 | moreover | 
| 315 | have "?K \<subseteq> (\<Union>i. D i)" using K by auto | |
| 316 | moreover | |
| 317 | have "compact ?K" using K by auto | |
| 318 | ultimately | |
| 62975 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 319 | have "?K\<subseteq>(\<Union>i. D i) \<and> compact ?K \<and> emeasure M (\<Union>i. D i) \<le> emeasure M ?K + ennreal e" by simp | 
| 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 320 | thus "\<exists>K\<subseteq>\<Union>i. D i. compact K \<and> emeasure M (\<Union>i. D i) \<le> emeasure M K + ennreal e" .. | 
| 50125 
4319691be975
tuned: use induction rule sigma_sets_induct_disjoint
 hoelzl parents: 
50089diff
changeset | 321 | qed fact | 
| 
4319691be975
tuned: use induction rule sigma_sets_induct_disjoint
 hoelzl parents: 
50089diff
changeset | 322 | case 2 | 
| 
4319691be975
tuned: use induction rule sigma_sets_induct_disjoint
 hoelzl parents: 
50089diff
changeset | 323 | show ?case | 
| 61808 | 324 | proof (rule approx_outer[OF \<open>(\<Union>i. D i) \<in> sets M\<close>]) | 
| 50087 | 325 | fix e::real assume "e > 0" | 
| 326 | have "\<forall>i::nat. \<exists>U. D i \<subseteq> U \<and> open U \<and> e/(2 powr Suc i) > emeasure M U - emeasure M (D i)" | |
| 327 | proof | |
| 328 | fix i::nat | |
| 61808 | 329 | from \<open>0 < e\<close> have "0 < e/(2 powr Suc i)" by simp | 
| 50087 | 330 |         have "emeasure M (D i) = (INF U:{U. (D i) \<subseteq> U \<and> open U}. emeasure M U)"
 | 
| 50125 
4319691be975
tuned: use induction rule sigma_sets_induct_disjoint
 hoelzl parents: 
50089diff
changeset | 331 | using union by blast | 
| 62975 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 332 | from INF_approx_ennreal[OF \<open>0 < e/(2 powr Suc i)\<close> this] | 
| 50087 | 333 | show "\<exists>U. D i \<subseteq> U \<and> open U \<and> e/(2 powr Suc i) > emeasure M U - emeasure M (D i)" | 
| 62975 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 334 | using \<open>0<e\<close> | 
| 64267 | 335 | by (auto simp: emeasure_eq_measure measure_nonneg sum_nonneg ennreal_less_iff ennreal_plus[symmetric] ennreal_minus | 
| 62975 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 336 | finite_measure_mono sb | 
| 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 337 | simp del: ennreal_plus) | 
| 50087 | 338 | qed | 
| 339 | then obtain U where U: "\<And>i. D i \<subseteq> U i" "\<And>i. open (U i)" | |
| 340 | "\<And>i. e/(2 powr Suc i) > emeasure M (U i) - emeasure M (D i)" | |
| 341 | unfolding choice_iff by blast | |
| 342 | let ?U = "\<Union>i. U i" | |
| 62975 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 343 | have "ennreal (measure M ?U - measure M (\<Union>i. D i)) = M ?U - M (\<Union>i. D i)" | 
| 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 344 | using U(1,2) | 
| 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 345 | by (subst ennreal_minus[symmetric]) | 
| 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 346 | (auto intro!: finite_measure_mono simp: sb measure_nonneg emeasure_eq_measure) | 
| 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 347 | also have "\<dots> = M (?U - (\<Union>i. D i))" using U \<open>(\<Union>i. D i) \<in> sets M\<close> | 
| 50087 | 348 | by (subst emeasure_Diff) (auto simp: sb) | 
| 61808 | 349 | also have "\<dots> \<le> M (\<Union>i. U i - D i)" using U \<open>range D \<subseteq> sets M\<close> | 
| 50244 
de72bbe42190
qualified interpretation of sigma_algebra, to avoid name clashes
 immler parents: 
50125diff
changeset | 350 | by (intro emeasure_mono) (auto simp: sb intro!: sets.countable_nat_UN sets.Diff) | 
| 61808 | 351 | also have "\<dots> \<le> (\<Sum>i. M (U i - D i))" using U \<open>range D \<subseteq> sets M\<close> | 
| 50244 
de72bbe42190
qualified interpretation of sigma_algebra, to avoid name clashes
 immler parents: 
50125diff
changeset | 352 | by (intro emeasure_subadditive_countably) (auto intro!: sets.Diff simp: sb) | 
| 62975 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 353 | also have "\<dots> \<le> (\<Sum>i. ennreal e/(2 powr Suc i))" using U \<open>range D \<subseteq> sets M\<close> | 
| 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 354 | using \<open>0<e\<close> | 
| 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 355 | by (intro suminf_le, subst emeasure_Diff) | 
| 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 356 | (auto simp: emeasure_Diff emeasure_eq_measure sb measure_nonneg ennreal_minus | 
| 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 357 | finite_measure_mono divide_ennreal ennreal_less_iff | 
| 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 358 | intro: less_imp_le) | 
| 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 359 | also have "\<dots> \<le> (\<Sum>n. ennreal (e * (1 / 2) ^ Suc n))" | 
| 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 360 | using \<open>0<e\<close> | 
| 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 361 | by (simp add: powr_minus powr_realpow field_simps divide_ennreal del: of_nat_Suc) | 
| 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 362 | also have "\<dots> = ennreal e * (\<Sum>n. ennreal ((1 / 2) ^ Suc n))" | 
| 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 363 | unfolding ennreal_power[symmetric] | 
| 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 364 | using \<open>0 < e\<close> | 
| 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 365 | by (simp add: ac_simps ennreal_mult' divide_ennreal[symmetric] divide_ennreal_def | 
| 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 366 | ennreal_power[symmetric]) | 
| 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 367 | also have "\<dots> = ennreal e" | 
| 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 368 | by (subst suminf_ennreal_eq[OF zero_le_power power_half_series]) auto | 
| 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 369 | finally have "emeasure M ?U \<le> emeasure M (\<Union>i. D i) + ennreal e" | 
| 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 370 | using \<open>0<e\<close> by (simp add: emeasure_eq_measure ennreal_plus[symmetric] measure_nonneg del: ennreal_plus) | 
| 50087 | 371 | moreover | 
| 372 | have "(\<Union>i. D i) \<subseteq> ?U" using U by auto | |
| 373 | moreover | |
| 374 | have "open ?U" using U by auto | |
| 375 | ultimately | |
| 62975 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 376 | have "(\<Union>i. D i) \<subseteq> ?U \<and> open ?U \<and> emeasure M ?U \<le> emeasure M (\<Union>i. D i) + ennreal e" by simp | 
| 
1d066f6ab25d
Probability: move emeasure and nn_integral from ereal to ennreal
 hoelzl parents: 
62533diff
changeset | 377 | thus "\<exists>B. (\<Union>i. D i) \<subseteq> B \<and> open B \<and> emeasure M B \<le> emeasure M (\<Union>i. D i) + ennreal e" .. | 
| 50087 | 378 | qed | 
| 379 | qed | |
| 380 | qed | |
| 381 | ||
| 382 | end | |
| 383 |