diff -r e6f5b1bbcb01 -r f366643536cd src/HOL/Probability/Nonnegative_Lebesgue_Integration.thy --- a/src/HOL/Probability/Nonnegative_Lebesgue_Integration.thy Wed Jan 14 09:59:12 2015 +0100 +++ b/src/HOL/Probability/Nonnegative_Lebesgue_Integration.thy Wed Jan 14 10:15:41 2015 +0100 @@ -740,7 +740,7 @@ "integral\<^sup>N M f = (SUP g : {g. simple_function M g \ g \ max 0 \ f}. integral\<^sup>S M g)" syntax - "_nn_integral" :: "pttrn \ ereal \ 'a measure \ ereal" ("\\<^sup>+ _. _ \_" [60,61] 110) + "_nn_integral" :: "pttrn \ ereal \ 'a measure \ ereal" ("\\<^sup>+((2 _./ _)/ \_)" [60,61] 110) translations "\\<^sup>+x. f \M" == "CONST nn_integral M (\x. f)"