diff -r 01b8c8d17f13 -r 2a77bc3b4eac src/ZF/OrdQuant.thy --- a/src/ZF/OrdQuant.thy Fri Sep 20 23:36:33 2024 +0200 +++ b/src/ZF/OrdQuant.thy Fri Sep 20 23:37:00 2024 +0200 @@ -23,9 +23,9 @@ "OUnion(i,B) \ {z: \x\i. B(x). Ord(i)}" syntax - "_oall" :: "[idt, i, o] \ o" (\(3\_<_./ _)\ 10) - "_oex" :: "[idt, i, o] \ o" (\(3\_<_./ _)\ 10) - "_OUNION" :: "[idt, i, i] \ i" (\(3\_<_./ _)\ 10) + "_oall" :: "[idt, i, o] \ o" (\(\indent=3 notation=\binder \<\\\_<_./ _)\ 10) + "_oex" :: "[idt, i, o] \ o" (\(\indent=3 notation=\binder \<\\\_<_./ _)\ 10) + "_OUNION" :: "[idt, i, i] \ i" (\(\indent=3 notation=\binder \<\\\_<_./ _)\ 10) syntax_consts "_oall" \ oall and "_oex" \ oex and @@ -196,8 +196,8 @@ "rex(M, P) \ \x. M(x) \ P(x)" syntax - "_rall" :: "[pttrn, i\o, o] \ o" (\(3\_[_]./ _)\ 10) - "_rex" :: "[pttrn, i\o, o] \ o" (\(3\_[_]./ _)\ 10) + "_rall" :: "[pttrn, i\o, o] \ o" (\(\indent=3 notation=\binder \[]\\\_[_]./ _)\ 10) + "_rex" :: "[pttrn, i\o, o] \ o" (\(\indent=3 notation=\binder \[]\\\_[_]./ _)\ 10) syntax_consts "_rall" \ rall and "_rex" \ rex