src/HOL/Probability/Information.thy
changeset 39302 d7728f65b353
parent 39198 f967a16dfcdd
child 40859 de0b30e6c2d2
--- a/src/HOL/Probability/Information.thy	Mon Sep 13 08:43:48 2010 +0200
+++ b/src/HOL/Probability/Information.thy	Mon Sep 13 11:13:15 2010 +0200
@@ -505,7 +505,7 @@
     by auto
   also have "\<dots> = log b (\<Sum>x\<in>X`space M. if ?d x \<noteq> 0 then 1 else 0)"
     apply (rule arg_cong[where f="\<lambda>f. log b (\<Sum>x\<in>X`space M. f x)"])
-    using distribution_finite[of X] by (auto simp: ext_iff real_of_pinfreal_eq_0)
+    using distribution_finite[of X] by (auto simp: fun_eq_iff real_of_pinfreal_eq_0)
   finally show ?thesis
     using finite_space by (auto simp: setsum_cases real_eq_of_nat)
 qed
@@ -645,7 +645,7 @@
   let "?dZ A" = "real (distribution Z A)"
   let ?M = "X ` space M \<times> Y ` space M \<times> Z ` space M"
 
-  have split_beta: "\<And>f. split f = (\<lambda>x. f (fst x) (snd x))" by (simp add: ext_iff)
+  have split_beta: "\<And>f. split f = (\<lambda>x. f (fst x) (snd x))" by (simp add: fun_eq_iff)
 
   have "- (\<Sum>(x, y, z) \<in> ?M. ?dXYZ {(x, y, z)} *
     log b (?dXYZ {(x, y, z)} / (?dXZ {(x, z)} * ?dYZ {(y,z)} / ?dZ {z})))