diff -r ff2a637a449e -r fc5066122e68 src/Pure/Examples/Higher_Order_Logic.thy --- a/src/Pure/Examples/Higher_Order_Logic.thy Fri Oct 18 11:44:05 2024 +0200 +++ b/src/Pure/Examples/Higher_Order_Logic.thy Fri Oct 18 14:20:09 2024 +0200 @@ -401,7 +401,7 @@ axiomatization Eps :: "('a \ o) \ 'a" where someI: "P x \ P (Eps P)" -syntax "_Eps" :: "pttrn \ o \ 'a" (\(3SOME _./ _)\ [0, 10] 10) +syntax "_Eps" :: "pttrn \ o \ 'a" (\(\indent=3 notation=\binder SOME\\SOME _./ _)\ [0, 10] 10) syntax_consts "_Eps" \ Eps translations "SOME x. P" \ "CONST Eps (\x. P)"