src/HOL/Probability/Giry_Monad.thy
changeset 67399 eab6ce8368fa
parent 67226 ec32cdaab97b
child 67649 1e1782c1aedf
--- a/src/HOL/Probability/Giry_Monad.thy	Wed Jan 10 15:21:49 2018 +0100
+++ b/src/HOL/Probability/Giry_Monad.thy	Wed Jan 10 15:25:09 2018 +0100
@@ -349,7 +349,7 @@
       (\<lambda>M'. emeasure M' (f -` A \<inter> space M)) \<in> borel_measurable (subprob_algebra M)"
       by (intro measurable_cong)
          (auto simp: emeasure_distr space_subprob_algebra
-               intro!: arg_cong2[where f=emeasure] sets_eq_imp_space_eq arg_cong2[where f="op \<inter>"])
+               intro!: arg_cong2[where f=emeasure] sets_eq_imp_space_eq arg_cong2[where f="(\<inter>)"])
     also have "\<dots>"
       using A by (intro measurable_emeasure_subprob_algebra) simp
     finally show "(\<lambda>M'. emeasure (distr M' N f) A) \<in> borel_measurable (subprob_algebra M)" .