--- a/src/HOL/Probability/Sigma_Algebra.thy Tue Dec 15 14:40:36 2015 +0000
+++ b/src/HOL/Probability/Sigma_Algebra.thy Tue Dec 15 14:41:47 2015 +0000
@@ -1700,7 +1700,7 @@
subsubsection \<open>Measurable functions\<close>
-definition measurable :: "'a measure \<Rightarrow> 'b measure \<Rightarrow> ('a \<Rightarrow> 'b) set" where
+definition measurable :: "'a measure \<Rightarrow> 'b measure \<Rightarrow> ('a \<Rightarrow> 'b) set" (infixr "\<rightarrow>\<^sub>M" 60) where
"measurable A B = {f \<in> space A \<rightarrow> space B. \<forall>y \<in> sets B. f -` y \<inter> space A \<in> sets A}"
lemma measurableI: