src/HOL/Analysis/Nonnegative_Lebesgue_Integration.thy
changeset 64008 17a20ca86d62
parent 63918 6bf55e6e0b75
child 64267 b9a1486e79be
--- a/src/HOL/Analysis/Nonnegative_Lebesgue_Integration.thy	Mon Oct 03 14:09:26 2016 +0100
+++ b/src/HOL/Analysis/Nonnegative_Lebesgue_Integration.thy	Fri Sep 30 16:08:38 2016 +0200
@@ -1692,6 +1692,16 @@
     by (simp add: ** nn_integral_suminf from_nat_into)
 qed
 
+lemma of_bool_Bex_eq_nn_integral:
+  assumes unique: "\<And>x y. x \<in> X \<Longrightarrow> y \<in> X \<Longrightarrow> P x \<Longrightarrow> P y \<Longrightarrow> x = y"
+  shows "of_bool (\<exists>y\<in>X. P y) = (\<integral>\<^sup>+y. of_bool (P y) \<partial>count_space X)"
+proof cases
+  assume "\<exists>y\<in>X. P y"
+  then obtain y where "P y" "y \<in> X" by auto
+  then show ?thesis
+    by (subst nn_integral_count_space'[where A="{y}"]) (auto dest: unique)
+qed (auto cong: nn_integral_cong_simp)
+
 lemma emeasure_UN_countable:
   assumes sets[measurable]: "\<And>i. i \<in> I \<Longrightarrow> X i \<in> sets M" and I[simp]: "countable I"
   assumes disj: "disjoint_family_on X I"