src/HOL/Probability/Probability_Measure.thy
changeset 57275 0ddb5b755cdc
parent 57235 b0b9a10e4bf4
child 57418 6ab1c7cb0b8d
--- a/src/HOL/Probability/Probability_Measure.thy	Wed Jun 18 15:23:40 2014 +0200
+++ b/src/HOL/Probability/Probability_Measure.thy	Wed Jun 18 07:31:12 2014 +0200
@@ -745,6 +745,11 @@
   finally show ?thesis .
 qed
 
+lemma distributed_integrable_var:
+  fixes X :: "'a \<Rightarrow> real"
+  shows "distributed M lborel X (\<lambda>x. ereal (f x)) \<Longrightarrow> integrable lborel (\<lambda>x. f x * x) \<Longrightarrow> integrable M X"
+  using distributed_integrable[of M lborel X f "\<lambda>x. x"] by simp
+
 lemma (in prob_space) distributed_variance:
   fixes f::"real \<Rightarrow> real"
   assumes D: "distributed M lborel X f"