# HG changeset patch # User hoelzl # Date 1322744637 -3600 # Node ID 10192f9616195159ba0c7d028bfb09b7d628f7a3 # Parent 7c8bed80301f08f0ff71ecd67a27e8ae092e91e8 remove duplicate theorem setsum_real_distribution diff -r 7c8bed80301f -r 10192f961619 src/HOL/Probability/Information.thy --- a/src/HOL/Probability/Information.thy Thu Dec 01 13:34:16 2011 +0100 +++ b/src/HOL/Probability/Information.thy Thu Dec 01 14:03:57 2011 +0100 @@ -1020,13 +1020,6 @@ using setsum_joint_distribution[OF assms, of "\ space = UNIV, sets = Pow UNIV \" "\x. ()" "{()}"] using sigma_algebra_Pow[of "UNIV::unit set" "()"] by simp -lemma (in prob_space) setsum_real_distribution: - fixes MX :: "('c, 'd) measure_space_scheme" - assumes X: "finite_random_variable MX X" shows "(\a\space MX. distribution X {a}) = 1" - using setsum_joint_distribution[OF assms, of "\ space = UNIV, sets = Pow UNIV, measure = undefined \" "\x. ()" "{()}"] - using sigma_algebra_Pow[of "UNIV::unit set" "\ measure = undefined \"] - by auto - lemma (in information_space) conditional_mutual_information_generic_positive: assumes X: "finite_random_variable MX X" and Y: "finite_random_variable MY Y" and Z: "finite_random_variable MZ Z" shows "0 \ conditional_mutual_information b MX MY MZ X Y Z" @@ -1101,7 +1094,7 @@ setsum_joint_distribution_singleton[OF Y Z] intro!: setsum_cong) also have "log b (\z\space MZ. ?dZ {z}) = 0" - unfolding setsum_real_distribution[OF Z] by simp + unfolding setsum_distribution[OF Z] by simp finally show ?thesis by simp qed