diff -r b4cccce25d9a -r c335d880ff82 src/HOL/Probability/Information.thy --- a/src/HOL/Probability/Information.thy Wed Dec 08 18:07:04 2010 +0100 +++ b/src/HOL/Probability/Information.thy Wed Dec 08 16:15:14 2010 +0100 @@ -188,7 +188,7 @@ using f by (rule \.measure_space_isomorphic) let ?RN = "sigma_finite_measure.RN_deriv ?M ?\ ?\" - from RN_deriv_vimage[OF f \] + from RN_deriv_vimage[OF f[THEN bij_inv_the_inv_into] \] have *: "\.almost_everywhere (\x. ?RN (the_inv_into S f x) = RN_deriv \ x)" by (rule absolutely_continuous_AE[OF \])