src/HOL/Analysis/Binary_Product_Measure.thy
changeset 69683 8b3458ca0762
parent 69652 3417a8f154eb
child 69722 b5163b2132c5
--- a/src/HOL/Analysis/Binary_Product_Measure.thy	Thu Jan 17 16:37:06 2019 -0500
+++ b/src/HOL/Analysis/Binary_Product_Measure.thy	Thu Jan 17 16:38:00 2019 -0500
@@ -14,7 +14,7 @@
 lemma rev_Pair_vimage_times[simp]: "(\<lambda>x. (x, y)) -` (A \<times> B) = (if y \<in> B then A else {})"
   by auto
 
-subsection%important "Binary products"
+subsection "Binary products"
 
 definition%important pair_measure (infixr "\<Otimes>\<^sub>M" 80) where
   "A \<Otimes>\<^sub>M B = measure_of (space A \<times> space B)
@@ -336,7 +336,7 @@
     by (simp add: ac_simps)
 qed
 
-subsection%important \<open>Binary products of \<open>\<sigma>\<close>-finite emeasure spaces\<close>
+subsection \<open>Binary products of \<open>\<sigma>\<close>-finite emeasure spaces\<close>
 
 locale%unimportant pair_sigma_finite = M1?: sigma_finite_measure M1 + M2?: sigma_finite_measure M2
   for M1 :: "'a measure" and M2 :: "'b measure"
@@ -531,7 +531,7 @@
     done
 qed
 
-subsection%important "Fubinis theorem"
+subsection "Fubinis theorem"
 
 lemma measurable_compose_Pair1:
   "x \<in> space M1 \<Longrightarrow> g \<in> measurable (M1 \<Otimes>\<^sub>M M2) L \<Longrightarrow> (\<lambda>y. g (x, y)) \<in> measurable M2 L"
@@ -602,7 +602,7 @@
   shows "(\<integral>\<^sup>+ y. (\<integral>\<^sup>+ x. f x y \<partial>M1) \<partial>M2) = (\<integral>\<^sup>+ x. (\<integral>\<^sup>+ y. f x y \<partial>M2) \<partial>M1)"
   using Fubini[OF f] by simp
 
-subsection%important \<open>Products on counting spaces, densities and distributions\<close>
+subsection \<open>Products on counting spaces, densities and distributions\<close>
 
 proposition sigma_prod:
   assumes X_cover: "\<exists>E\<subseteq>A. countable E \<and> X = \<Union>E" and A: "A \<subseteq> Pow X"
@@ -1095,7 +1095,7 @@
 using _ _ assms(1)
 by(rule measurable_compose_countable'[where f="\<lambda>a b. f (a, snd b)" and g=fst and I=A, simplified])simp_all
 
-subsection%important \<open>Product of Borel spaces\<close>
+subsection \<open>Product of Borel spaces\<close>
 
 theorem borel_Times:
   fixes A :: "'a::topological_space set" and B :: "'b::topological_space set"