src/HOL/Probability/Independent_Family.thy
changeset 49795 9f2fb9b25a77
parent 49794 3c7b5988e094
child 50003 8c213922ed49
equal deleted inserted replaced
49794:3c7b5988e094 49795:9f2fb9b25a77
  1168         using rvs ab by (simp add: emeasure_eq_measure emeasure_distr)
  1168         using rvs ab by (simp add: emeasure_eq_measure emeasure_distr)
  1169     qed
  1169     qed
  1170   qed
  1170   qed
  1171 qed
  1171 qed
  1172 
  1172 
       
  1173 lemma (in prob_space) distributed_joint_indep:
       
  1174   assumes S: "sigma_finite_measure S" and T: "sigma_finite_measure T"
       
  1175   assumes X: "distributed M S X Px" and Y: "distributed M T Y Py"
       
  1176   assumes indep: "indep_var S X T Y"
       
  1177   shows "distributed M (S \<Otimes>\<^isub>M T) (\<lambda>x. (X x, Y x)) (\<lambda>(x, y). Px x * Py y)"
       
  1178   using indep_var_distribution_eq[of S X T Y] indep
       
  1179   by (intro distributed_joint_indep'[OF S T X Y]) auto
       
  1180 
  1173 end
  1181 end