src/HOL/Probability/Independent_Family.thy
changeset 50021 d96a3f468203
parent 50003 8c213922ed49
child 50087 635d73673b5e
--- a/src/HOL/Probability/Independent_Family.thy	Tue Nov 06 15:15:33 2012 +0100
+++ b/src/HOL/Probability/Independent_Family.thy	Tue Nov 06 19:18:35 2012 +0100
@@ -1004,9 +1004,6 @@
   "A \<in> sets N \<Longrightarrow> f \<in> measurable M N \<Longrightarrow> (\<lambda>x. indicator A (f x)) \<in> borel_measurable M"
   using measurable_comp[OF _ borel_measurable_indicator, of f M N A] by (auto simp add: comp_def)
 
-lemma measurable_id_prod[measurable (raw)]: "i = j \<Longrightarrow> (\<lambda>x. x) \<in> measurable (M i) (M j)"
-  by simp
-
 lemma (in product_sigma_finite) distr_component:
   "distr (M i) (Pi\<^isub>M {i} M) (\<lambda>x. \<lambda>i\<in>{i}. x) = Pi\<^isub>M {i} M" (is "?D = ?P")
 proof (intro measure_eqI[symmetric])