Merge
authorpaulson <lp15@cam.ac.uk>
Tue, 15 Dec 2015 14:41:47 +0000
changeset 61849 f8741f200f91
parent 61848 9250e546ab23 (current diff)
parent 61847 9e38cde3d672 (diff)
child 61855 32a530a5c54c
Merge
--- 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: