diff -r e905fb37467f -r a8407aa7f916 src/HOL/Analysis/Set_Integral.thy --- a/src/HOL/Analysis/Set_Integral.thy Fri Feb 16 09:24:45 2024 +0100 +++ b/src/HOL/Analysis/Set_Integral.thy Fri Feb 16 11:22:29 2024 +0000 @@ -23,7 +23,7 @@ syntax "_ascii_set_lebesgue_integral" :: "pttrn \ 'a set \ 'a measure \ real \ real" - ("(4LINT (_):(_)/|(_)./ _)" [0,60,110,61] 10) + ("(4LINT (_):(_)/|(_)./ _)" [0,0,0,10] 10) translations "LINT x:A|M. f" == "CONST set_lebesgue_integral M A (\x. f)" @@ -39,11 +39,11 @@ syntax "_lebesgue_borel_integral" :: "pttrn \ real \ real" - ("(2LBINT _./ _)" [0,60] 10) + ("(2LBINT _./ _)" [0,10] 10) syntax "_set_lebesgue_borel_integral" :: "pttrn \ real set \ real \ real" - ("(3LBINT _:_./ _)" [0,60,61] 10) + ("(3LBINT _:_./ _)" [0,0,10] 10) (* Basic properties @@ -570,14 +570,14 @@ syntax "_complex_lebesgue_integral" :: "pttrn \ complex \ 'a measure \ complex" - ("\\<^sup>C _. _ \_" [60,61] 110) + ("\\<^sup>C _. _ \_" [0,0] 110) translations "\\<^sup>Cx. f \M" == "CONST complex_lebesgue_integral M (\x. f)" syntax "_ascii_complex_lebesgue_integral" :: "pttrn \ 'a measure \ real \ real" - ("(3CLINT _|_. _)" [0,110,60] 10) + ("(3CLINT _|_. _)" [0,0,10] 10) translations "CLINT x|M. f" == "CONST complex_lebesgue_integral M (\x. f)" @@ -611,7 +611,7 @@ syntax "_ascii_complex_set_lebesgue_integral" :: "pttrn \ 'a set \ 'a measure \ real \ real" -("(4CLINT _:_|_. _)" [0,60,110,61] 10) +("(4CLINT _:_|_. _)" [0,0,0,10] 10) translations "CLINT x:A|M. f" == "CONST complex_set_lebesgue_integral M A (\x. f)" @@ -630,10 +630,10 @@ syntax "_set_nn_integral" :: "pttrn => 'a set => 'a measure => ereal => ereal" -("(\\<^sup>+((_)\(_)./ _)/\_)" [0,60,110,61] 10) +("(\\<^sup>+((_)\(_)./ _)/\_)" [0,0,0,110] 10) "_set_lebesgue_integral" :: "pttrn => 'a set => 'a measure => ereal => ereal" -("(\((_)\(_)./ _)/\_)" [0,60,110,61] 10) +("(\((_)\(_)./ _)/\_)" [0,0,0,110] 10) translations "\\<^sup>+x \ A. f \M" == "CONST set_nn_integral M A (\x. f)"