src/HOL/Probability/Information.thy
changeset 63040 eb4ddd18d635
parent 62975 1d066f6ab25d
child 63566 e5abbdee461a
equal deleted inserted replaced
63039:1a20fd9cf281 63040:eb4ddd18d635
  1669 
  1669 
  1670 lemma (in information_space) conditional_mutual_information_eq_conditional_entropy:
  1670 lemma (in information_space) conditional_mutual_information_eq_conditional_entropy:
  1671   assumes X: "simple_function M X" and Y: "simple_function M Y"
  1671   assumes X: "simple_function M X" and Y: "simple_function M Y"
  1672   shows "\<I>(X ; X | Y) = \<H>(X | Y)"
  1672   shows "\<I>(X ; X | Y) = \<H>(X | Y)"
  1673 proof -
  1673 proof -
  1674   def Py \<equiv> "\<lambda>x. if x \<in> Y`space M then measure M (Y -` {x} \<inter> space M) else 0"
  1674   define Py where "Py x = (if x \<in> Y`space M then measure M (Y -` {x} \<inter> space M) else 0)" for x
  1675   def Pxy \<equiv> "\<lambda>x. if x \<in> (\<lambda>x. (X x, Y x))`space M then measure M ((\<lambda>x. (X x, Y x)) -` {x} \<inter> space M) else 0"
  1675   define Pxy where "Pxy x =
  1676   def Pxxy \<equiv> "\<lambda>x. if x \<in> (\<lambda>x. (X x, X x, Y x))`space M then measure M ((\<lambda>x. (X x, X x, Y x)) -` {x} \<inter> space M) else 0"
  1676       (if x \<in> (\<lambda>x. (X x, Y x))`space M then measure M ((\<lambda>x. (X x, Y x)) -` {x} \<inter> space M) else 0)"
       
  1677     for x
       
  1678   define Pxxy where "Pxxy x =
       
  1679       (if x \<in> (\<lambda>x. (X x, X x, Y x))`space M then measure M ((\<lambda>x. (X x, X x, Y x)) -` {x} \<inter> space M)
       
  1680        else 0)"
       
  1681     for x
  1677   let ?M = "X`space M \<times> X`space M \<times> Y`space M"
  1682   let ?M = "X`space M \<times> X`space M \<times> Y`space M"
  1678 
  1683 
  1679   note XY = simple_function_Pair[OF X Y]
  1684   note XY = simple_function_Pair[OF X Y]
  1680   note XXY = simple_function_Pair[OF X XY]
  1685   note XXY = simple_function_Pair[OF X XY]
  1681   have Py: "simple_distributed M Y Py"
  1686   have Py: "simple_distributed M Y Py"