src/HOL/Probability/Finite_Product_Measure.thy
changeset 56994 8d5e5ec1cac3
parent 56993 e5366291d6aa
child 56996 891e992e510f
--- a/src/HOL/Probability/Finite_Product_Measure.thy	Mon May 19 12:04:45 2014 +0200
+++ b/src/HOL/Probability/Finite_Product_Measure.thy	Mon May 19 13:44:13 2014 +0200
@@ -11,7 +11,7 @@
 lemma split_const: "(\<lambda>(i, j). c) = (\<lambda>_. c)"
   by auto
 
-subsubsection {* Merge two extensional functions *}
+subsubsection {* More about Function restricted by @{const extensional}  *}
 
 definition
   "merge I J = (\<lambda>(x, y) i. if i \<in> I then x i else if i \<in> J then y i else undefined)"
@@ -105,9 +105,9 @@
   "I \<inter> J = {} \<Longrightarrow> merge I J -` Pi\<^sub>E (I \<union> J) E = Pi I E \<times> Pi J E"
   by (auto simp: restrict_Pi_cancel PiE_def)
 
-section "Finite product spaces"
+subsection {* Finite product spaces *}
 
-section "Products"
+subsubsection {* Products *}
 
 definition prod_emb where
   "prod_emb I M K X = (\<lambda>x. restrict x K) -` X \<inter> (PIE i:I. space (M i))"