# HG changeset patch # User wenzelm # Date 1726868220 -7200 # Node ID 2a77bc3b4eacc58661586bcb24138b9817be78f4 # Parent 01b8c8d17f1362a7b8c71ddc44d924cca13674ad more inner syntax markup: minor object-logics; diff -r 01b8c8d17f13 -r 2a77bc3b4eac src/CCL/CCL.thy --- a/src/CCL/CCL.thy Fri Sep 20 23:36:33 2024 +0200 +++ b/src/CCL/CCL.thy Fri Sep 20 23:37:00 2024 +0200 @@ -35,7 +35,7 @@ (*** Term Formers ***) true :: "i" false :: "i" - pair :: "[i,i]\i" (\(1<_,/_>)\) + pair :: "[i,i]\i" (\(\indent=1 notation=\mixfix pair\\<_,/_>)\) lambda :: "(i\i)\i" (binder \lam \ 55) "case" :: "[i,i,i,[i,i]\i,(i\i)\i]\i" "apply" :: "[i,i]\i" (infixl \`\ 56) diff -r 01b8c8d17f13 -r 2a77bc3b4eac src/CCL/Set.thy --- a/src/CCL/Set.thy Fri Sep 20 23:36:33 2024 +0200 +++ b/src/CCL/Set.thy Fri Sep 20 23:37:00 2024 +0200 @@ -18,7 +18,7 @@ and set_extension: "A = B \ (ALL x. x:A \ x:B)" syntax - "_Coll" :: "[idt, o] \ 'a set" (\(1{_./ _})\) + "_Coll" :: "[idt, o] \ 'a set" (\(\indent=1 notation=\mixfix Collect\\{_./ _})\) syntax_consts "_Coll" == Collect translations @@ -50,8 +50,8 @@ where "Bex(A, P) == EX x. x:A \ P(x)" syntax - "_Ball" :: "[idt, 'a set, o] \ o" (\(ALL _:_./ _)\ [0, 0, 0] 10) - "_Bex" :: "[idt, 'a set, o] \ o" (\(EX _:_./ _)\ [0, 0, 0] 10) + "_Ball" :: "[idt, 'a set, o] \ o" (\(\notation=\binder ALL:\\ALL _:_./ _)\ [0, 0, 0] 10) + "_Bex" :: "[idt, 'a set, o] \ o" (\(\notation=\binder EX:\\EX _:_./ _)\ [0, 0, 0] 10) syntax_consts "_Ball" == Ball and "_Bex" == Bex @@ -127,8 +127,8 @@ where "UNION(A, B) == {y. EX x:A. y: B(x)}" syntax - "_INTER" :: "[idt, 'a set, 'b set] \ 'b set" (\(INT _:_./ _)\ [0, 0, 0] 10) - "_UNION" :: "[idt, 'a set, 'b set] \ 'b set" (\(UN _:_./ _)\ [0, 0, 0] 10) + "_INTER" :: "[idt, 'a set, 'b set] \ 'b set" (\(\notation=\binder INT:\\INT _:_./ _)\ [0, 0, 0] 10) + "_UNION" :: "[idt, 'a set, 'b set] \ 'b set" (\(\notation=\binder UN:\\UN _:_./ _)\ [0, 0, 0] 10) syntax_consts "_INTER" == INTER and "_UNION" == UNION diff -r 01b8c8d17f13 -r 2a77bc3b4eac src/CCL/Term.thy --- a/src/CCL/Term.thy Fri Sep 20 23:36:33 2024 +0200 +++ b/src/CCL/Term.thy Fri Sep 20 23:37:00 2024 +0200 @@ -12,7 +12,8 @@ definition one :: "i" where "one == true" -definition "if" :: "[i,i,i]\i" (\(3if _/ then _/ else _)\ [0,0,60] 60) +definition "if" :: "[i,i,i]\i" + (\(\indent=3 notation=\mixfix if then else\\if _/ then _/ else _)\ [0,0,60] 60) where "if b then t else u == case(b, t, u, \ x y. bot, \v. bot)" definition inl :: "i\i" @@ -48,7 +49,8 @@ definition "let1" :: "[i,i\i]\i" where let_def: "let1(t, f) == case(t,f(true),f(false), \x y. f(), \u. f(lam x. u(x)))" -syntax "_let1" :: "[idt,i,i]\i" (\(3let _ be _/ in _)\ [0,0,60] 60) +syntax "_let1" :: "[idt,i,i]\i" + (\(\indent=3 notation=\mixfix let be in\\let _ be _/ in _)\ [0,0,60] 60) syntax_consts "_let1" == let1 translations "let x be a in e" == "CONST let1(a, \x. e)" @@ -65,9 +67,12 @@ \g'. f(\x y z. g'(>)))" syntax - "_letrec" :: "[idt,idt,i,i]\i" (\(3letrec _ _ be _/ in _)\ [0,0,0,60] 60) - "_letrec2" :: "[idt,idt,idt,i,i]\i" (\(3letrec _ _ _ be _/ in _)\ [0,0,0,0,60] 60) - "_letrec3" :: "[idt,idt,idt,idt,i,i]\i" (\(3letrec _ _ _ _ be _/ in _)\ [0,0,0,0,0,60] 60) + "_letrec" :: "[idt,idt,i,i]\i" + (\(\indent=3 notation=\mixfix letrec be in\\letrec _ _ be _/ in _)\ [0,0,0,60] 60) + "_letrec2" :: "[idt,idt,idt,i,i]\i" + (\(\indent=3 notation=\mixfix letrec be in\\letrec _ _ _ be _/ in _)\ [0,0,0,0,60] 60) + "_letrec3" :: "[idt,idt,idt,idt,i,i]\i" + (\(\indent=3 notation=\mixfix letrec be in\\letrec _ _ _ _ be _/ in _)\ [0,0,0,0,0,60] 60) syntax_consts "_letrec" == letrec and "_letrec2" == letrec2 and @@ -143,7 +148,7 @@ definition lrec :: "[i,i,[i,i,i]\i]\i" where "lrec(l,b,c) == letrec g x be lcase(x, b, \h t. c(h,t,g(t))) in g(l)" -definition napply :: "[i\i,i,i]\i" (\(_ ^ _ ` _)\ [56,56,56] 56) +definition napply :: "[i\i,i,i]\i" (\(\notation=\mixfix napply\\_ ^ _ ` _)\ [56,56,56] 56) where "f ^n` a == nrec(n,a,\x g. f(g))" lemmas simp_can_defs = one_def inl_def inr_def diff -r 01b8c8d17f13 -r 2a77bc3b4eac src/CCL/Trancl.thy --- a/src/CCL/Trancl.thy Fri Sep 20 23:36:33 2024 +0200 +++ b/src/CCL/Trancl.thy Fri Sep 20 23:37:00 2024 +0200 @@ -18,10 +18,10 @@ definition relcomp :: "[i set,i set] \ i set" (infixr \O\ 60) (*composition of relations*) where "r O s == {xz. EX x y z. xz = \ :s \ :r}" -definition rtrancl :: "i set \ i set" (\(_^*)\ [100] 100) +definition rtrancl :: "i set \ i set" (\(\notation=\postfix ^*\\_^*)\ [100] 100) where "r^* == lfp(\s. id Un (r O s))" -definition trancl :: "i set \ i set" (\(_^+)\ [100] 100) +definition trancl :: "i set \ i set" (\(\notation=\postfix ^+\\_^+)\ [100] 100) where "r^+ == r O rtrancl(r)" diff -r 01b8c8d17f13 -r 2a77bc3b4eac src/CCL/Type.thy --- a/src/CCL/Type.thy Fri Sep 20 23:36:33 2024 +0200 +++ b/src/CCL/Type.thy Fri Sep 20 23:37:00 2024 +0200 @@ -13,7 +13,7 @@ where "Subtype(A, P) == {x. x:A \ P(x)}" syntax - "_Subtype" :: "[idt, 'a set, o] \ 'a set" (\(1{_: _ ./ _})\) + "_Subtype" :: "[idt, 'a set, o] \ 'a set" (\(\indent=1 notation=\mixfix Subtype\\{_: _ ./ _})\) syntax_consts "_Subtype" == Subtype translations @@ -35,10 +35,10 @@ where "Sigma(A,B) == {x. EX a:A. EX b:B(a).x=}" syntax - "_Pi" :: "[idt, i set, i set] \ i set" (\(3PROD _:_./ _)\ [0,0,60] 60) - "_Sigma" :: "[idt, i set, i set] \ i set" (\(3SUM _:_./ _)\ [0,0,60] 60) - "_arrow" :: "[i set, i set] \ i set" (\(_ ->/ _)\ [54, 53] 53) - "_star" :: "[i set, i set] \ i set" (\(_ */ _)\ [56, 55] 55) + "_Pi" :: "[idt, i set, i set] \ i set" (\(\indent=3 notation=\binder PROD:\\PROD _:_./ _)\ [0,0,60] 60) + "_Sigma" :: "[idt, i set, i set] \ i set" (\(\indent=3 notation=\binder SUM:\\SUM _:_./ _)\ [0,0,60] 60) + "_arrow" :: "[i set, i set] \ i set" (\(\notation=\infix ->\\_ ->/ _)\ [54, 53] 53) + "_star" :: "[i set, i set] \ i set" (\(\notation=\infix *\\_ */ _)\ [56, 55] 55) syntax_consts "_Pi" "_arrow" \ Pi and "_Sigma" "_star" \ Sigma @@ -73,7 +73,7 @@ definition TEx :: "(i set \ i set) \ i set" (binder \TEX \ 55) where "TEX X. B(X) == Union({X. EX Y. X=B(Y)})" -definition Lift :: "i set \ i set" (\(3[_])\) +definition Lift :: "i set \ i set" (\(\indent=3 notation=\mixfix Lift\\[_])\) where "[A] == A Un {bot}" definition SPLIT :: "[i, [i, i] \ i set] \ i set" diff -r 01b8c8d17f13 -r 2a77bc3b4eac src/CTT/CTT.thy --- a/src/CTT/CTT.thy Fri Sep 20 23:36:33 2024 +0200 +++ b/src/CTT/CTT.thy Fri Sep 20 23:37:00 2024 +0200 @@ -18,10 +18,10 @@ consts \ \Judgments\ - Type :: "t \ prop" (\(_ type)\ [10] 5) - Eqtype :: "[t,t]\prop" (\(_ =/ _)\ [10,10] 5) - Elem :: "[i, t]\prop" (\(_ /: _)\ [10,10] 5) - Eqelem :: "[i,i,t]\prop" (\(_ =/ _ :/ _)\ [10,10,10] 5) + Type :: "t \ prop" (\(\notation=\postfix Type\\_ type)\ [10] 5) + Eqtype :: "[t,t]\prop" (\(\notation=\infix Eqtype\\_ =/ _)\ [10,10] 5) + Elem :: "[i, t]\prop" (\(\notation=\infix Elem\\_ /: _)\ [10,10] 5) + Eqelem :: "[i,i,t]\prop" (\(\notation=\mixfix Eqelem\\_ =/ _ :/ _)\ [10,10,10] 5) Reduce :: "[i,i]\prop" (\Reduce[_,_]\) \ \Types for truth values\ F :: "t" @@ -40,7 +40,7 @@ "when" :: "[i, i\i, i\i]\i" \ \General sum and binary product\ Sum :: "[t, i\t]\t" - pair :: "[i,i]\i" (\(1<_,/_>)\) + pair :: "[i,i]\i" (\(\indent=1 notation=\mixfix pair\\<_,/_>)\) fst :: "i\i" snd :: "i\i" split :: "[i, [i,i]\i] \i" @@ -56,8 +56,8 @@ must be introduced after the judgment forms.\ syntax - "_PROD" :: "[idt,t,t]\t" (\(3\_:_./ _)\ 10) - "_SUM" :: "[idt,t,t]\t" (\(3\_:_./ _)\ 10) + "_PROD" :: "[idt,t,t]\t" (\(\indent=3 notation=\binder \\\\_:_./ _)\ 10) + "_SUM" :: "[idt,t,t]\t" (\(\indent=3 notation=\binder \\\\_:_./ _)\ 10) syntax_consts "_PROD" \ Prod and "_SUM" \ Sum diff -r 01b8c8d17f13 -r 2a77bc3b4eac src/Cube/Cube.thy --- a/src/Cube/Cube.thy Fri Sep 20 23:36:33 2024 +0200 +++ b/src/Cube/Cube.thy Fri Sep 20 23:37:00 2024 +0200 @@ -29,15 +29,15 @@ nonterminal context' and typing' syntax - "_Trueprop" :: "[context', typing'] \ prop" (\(_/ \ _)\) - "_Trueprop1" :: "typing' \ prop" (\(_)\) + "_Trueprop" :: "[context', typing'] \ prop" (\(\notation=\infix Trueprop\\_/ \ _)\) + "_Trueprop1" :: "typing' \ prop" (\(\notation=\prefix Trueprop\\_)\) "" :: "id \ context'" (\_\) "" :: "var \ context'" (\_\) "_MT_context" :: "context'" (\\) "_Context" :: "[typing', context'] \ context'" (\_ _\) - "_Has_type" :: "[term, term] \ typing'" (\(_:/ _)\ [0, 0] 5) - "_Lam" :: "[idt, term, term] \ term" (\(3\<^bold>\_:_./ _)\ [0, 0, 0] 10) - "_Pi" :: "[idt, term, term] \ term" (\(3\_:_./ _)\ [0, 0] 10) + "_Has_type" :: "[term, term] \ typing'" (\(\notation=\infix Has_Type\\_:/ _)\ [0, 0] 5) + "_Lam" :: "[idt, term, term] \ term" (\(\indent=3 notation=\binder \<^bold>\\\\<^bold>\_:_./ _)\ [0, 0, 0] 10) + "_Pi" :: "[idt, term, term] \ term" (\(\indent=3 notation=\binder \\\\_:_./ _)\ [0, 0] 10) "_arrow" :: "[term, term] \ term" (infixr \\\ 10) syntax_consts "_Trueprop" \ Trueprop and diff -r 01b8c8d17f13 -r 2a77bc3b4eac src/FOL/IFOL.thy --- a/src/FOL/IFOL.thy Fri Sep 20 23:36:33 2024 +0200 +++ b/src/FOL/IFOL.thy Fri Sep 20 23:37:00 2024 +0200 @@ -101,7 +101,7 @@ abbreviation not_equal :: \['a, 'a] \ o\ (infixl \\\ 50) where \x \ y \ \ (x = y)\ -syntax "_Uniq" :: "pttrn \ o \ o" (\(2\\<^sub>\\<^sub>1 _./ _)\ [0, 10] 10) +syntax "_Uniq" :: "pttrn \ o \ o" (\(\indent=2 notation=\binder \\<^sub>\\<^sub>1\\\\<^sub>\\<^sub>1 _./ _)\ [0, 10] 10) syntax_consts "_Uniq" \ Uniq translations "\\<^sub>\\<^sub>1x. P" \ "CONST Uniq (\x. P)" @@ -743,10 +743,10 @@ where \Let(s, f) \ f(s)\ syntax - "_bind" :: \[pttrn, 'a] => letbind\ (\(2_ =/ _)\ 10) + "_bind" :: \[pttrn, 'a] => letbind\ (\(\indent=2 notation=\infix letbind\\_ =/ _)\ 10) "" :: \letbind => letbinds\ (\_\) "_binds" :: \[letbind, letbinds] => letbinds\ (\_;/ _\) - "_Let" :: \[letbinds, 'a] => 'a\ (\(let (_)/ in (_))\ 10) + "_Let" :: \[letbinds, 'a] => 'a\ (\(\notation=\mixfix let in\\let (_)/ in (_))\ 10) syntax_consts "_Let" \ Let translations "_Let(_binds(b, bs), e)" == "_Let(b, _Let(bs, e))" diff -r 01b8c8d17f13 -r 2a77bc3b4eac src/FOLP/IFOLP.thy --- a/src/FOLP/IFOLP.thy Fri Sep 20 23:36:33 2024 +0200 +++ b/src/FOLP/IFOLP.thy Fri Sep 20 23:37:00 2024 +0200 @@ -23,7 +23,7 @@ consts (*** Judgements ***) Proof :: "[o,p]=>prop" - EqProof :: "[p,p,o]=>prop" (\(3_ /= _ :/ _)\ [10,10,10] 5) + EqProof :: "[p,p,o]=>prop" (\(\indent=3 notation=\mixfix EqProof\\_ /= _ :/ _)\ [10,10,10] 5) (*** Logical Connectives -- Type Formers ***) eq :: "['a,'a] => o" (infixl \=\ 50) @@ -44,7 +44,7 @@ contr :: "p=>p" fst :: "p=>p" snd :: "p=>p" - pair :: "[p,p]=>p" (\(1<_,/_>)\) + pair :: "[p,p]=>p" (\(\indent=1 notation=\mixfix pair\\<_,/_>)\) split :: "[p, [p,p]=>p] =>p" inl :: "p=>p" inr :: "p=>p" @@ -53,14 +53,14 @@ App :: "[p,p]=>p" (infixl \`\ 60) alll :: "['a=>p]=>p" (binder \all \ 55) app :: "[p,'a]=>p" (infixl \^\ 55) - exists :: "['a,p]=>p" (\(1[_,/_])\) + exists :: "['a,p]=>p" (\(\indent=1 notation=\mixfix exists\\[_,/_])\) xsplit :: "[p,['a,p]=>p]=>p" ideq :: "'a=>p" idpeel :: "[p,'a=>p]=>p" nrm :: p NRM :: p -syntax "_Proof" :: "[p,o]=>prop" (\(_ /: _)\ [51, 10] 5) +syntax "_Proof" :: "[p,o]=>prop" (\(\notation=\infix Proof\\_ /: _)\ [51, 10] 5) parse_translation \ let fun proof_tr [p, P] = Syntax.const \<^const_syntax>\Proof\ $ P $ p diff -r 01b8c8d17f13 -r 2a77bc3b4eac src/LCF/LCF.thy --- a/src/LCF/LCF.thy Fri Sep 20 23:36:33 2024 +0200 +++ b/src/LCF/LCF.thy Fri Sep 20 23:37:00 2024 +0200 @@ -39,8 +39,8 @@ WHEN :: "['a\'c, 'b\'c, 'a+'b] \ 'c" adm :: "('a \ o) \ o" VOID :: "void" (\'(')\) - PAIR :: "['a,'b] \ 'a*'b" (\(1<_,/_>)\ [0,0] 100) - COND :: "[tr,'a,'a] \ 'a" (\(_ \/ (_ |/ _))\ [60,60,60] 60) + PAIR :: "['a,'b] \ 'a*'b" (\(\indent=1 notation=\mixfix PAIR\\<_,/_>)\ [0,0] 100) + COND :: "[tr,'a,'a] \ 'a" (\(\notation=\mixfix COND\\_ \/ (_ |/ _))\ [60,60,60] 60) less :: "['a,'a] \ o" (infixl \<<\ 50) axiomatization where diff -r 01b8c8d17f13 -r 2a77bc3b4eac src/Sequents/ILL.thy --- a/src/Sequents/ILL.thy Fri Sep 20 23:36:33 2024 +0200 +++ b/src/Sequents/ILL.thy Fri Sep 20 23:37:00 2024 +0200 @@ -29,8 +29,8 @@ PromAux :: "three_seqi" syntax - "_Trueprop" :: "single_seqe" (\((_)/ \ (_))\ [6,6] 5) - "_Context" :: "two_seqe" (\((_)/ :=: (_))\ [6,6] 5) + "_Trueprop" :: "single_seqe" (\(\notation=\infix Trueprop\\(_)/ \ (_))\ [6,6] 5) + "_Context" :: "two_seqe" (\(\notation=\infix Context\\(_)/ :=: (_))\ [6,6] 5) "_PromAux" :: "three_seqe" (\promaux {_||_||_}\) parse_translation \ diff -r 01b8c8d17f13 -r 2a77bc3b4eac src/Sequents/LK0.thy --- a/src/Sequents/LK0.thy Fri Sep 20 23:36:33 2024 +0200 +++ b/src/Sequents/LK0.thy Fri Sep 20 23:37:00 2024 +0200 @@ -34,7 +34,7 @@ Ex :: "('a \ o) \ o" (binder \\\ 10) syntax - "_Trueprop" :: "two_seqe" (\((_)/ \ (_))\ [6,6] 5) + "_Trueprop" :: "two_seqe" (\(\notation=\infix Trueprop\\(_)/ \ (_))\ [6,6] 5) parse_translation \[(\<^syntax_const>\_Trueprop\, K (two_seq_tr \<^const_syntax>\Trueprop\))]\ print_translation \[(\<^const_syntax>\Trueprop\, K (two_seq_tr' \<^syntax_const>\_Trueprop\))]\ @@ -104,7 +104,7 @@ The: "\$H \ $E, P(a), $F; \x.$H, P(x) \ $E, x=a, $F\ \ $H \ $E, P(THE x. P(x)), $F" -definition If :: "[o, 'a, 'a] \ 'a" (\(if (_)/ then (_)/ else (_))\ 10) +definition If :: "[o, 'a, 'a] \ 'a" (\(\notation=\mixfix if then else\\if (_)/ then (_)/ else (_))\ 10) where "If(P,x,y) \ THE z::'a. (P \ z = x) \ (\ P \ z = y)" diff -r 01b8c8d17f13 -r 2a77bc3b4eac src/ZF/Finite.thy --- a/src/ZF/Finite.thy Fri Sep 20 23:36:33 2024 +0200 +++ b/src/ZF/Finite.thy Fri Sep 20 23:37:00 2024 +0200 @@ -19,7 +19,7 @@ consts Fin :: "i\i" - FiniteFun :: "[i,i]\i" (\(_ -||>/ _)\ [61, 60] 60) + FiniteFun :: "[i,i]\i" (\(\notation=\infix -||>\\_ -||>/ _)\ [61, 60] 60) inductive domains "Fin(A)" \ "Pow(A)" diff -r 01b8c8d17f13 -r 2a77bc3b4eac src/ZF/Induct/Multiset.thy --- a/src/ZF/Induct/Multiset.thy Fri Sep 20 23:36:33 2024 +0200 +++ b/src/ZF/Induct/Multiset.thy Fri Sep 20 23:37:00 2024 +0200 @@ -70,11 +70,11 @@ "msize(M) \ setsum(\a. $# mcount(M,a), mset_of(M))" abbreviation - melem :: "[i,i] \ o" (\(_/ :# _)\ [50, 51] 50) where + melem :: "[i,i] \ o" (\(\notation=\infix :#\\_/ :# _)\ [50, 51] 50) where "a :# M \ a \ mset_of(M)" syntax - "_MColl" :: "[pttrn, i, o] \ i" (\(1{# _ \ _./ _#})\) + "_MColl" :: "[pttrn, i, o] \ i" (\(\indent=1 notation=\mixfix MCollect\\{# _ \ _./ _#})\) syntax_consts "_MColl" \ MCollect translations "{#x \ M. P#}" == "CONST MCollect(M, \x. P)" 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 diff -r 01b8c8d17f13 -r 2a77bc3b4eac src/ZF/Order.thy --- a/src/ZF/Order.thy Fri Sep 20 23:36:33 2024 +0200 +++ b/src/ZF/Order.thy Fri Sep 20 23:37:00 2024 +0200 @@ -49,7 +49,7 @@ {f \ A->B. \x\A. \y\A. \x,y\:r \ :s}" definition - ord_iso :: "[i,i,i,i]\i" (\(\_, _\ \/ \_, _\)\ 51) (*Order isomorphisms*) where + ord_iso :: "[i,i,i,i]\i" (\(\notation=\infix ord_iso\\\_, _\ \/ \_, _\)\ 51) (*Order isomorphisms*) where "\A,r\ \ \B,s\ \ {f \ bij(A,B). \x\A. \y\A. \x,y\:r \ :s}" diff -r 01b8c8d17f13 -r 2a77bc3b4eac src/ZF/QPair.thy --- a/src/ZF/QPair.thy Fri Sep 20 23:36:33 2024 +0200 +++ b/src/ZF/QPair.thy Fri Sep 20 23:37:00 2024 +0200 @@ -45,7 +45,7 @@ "QSigma(A,B) \ \x\A. \y\B(x). {}" syntax - "_QSUM" :: "[idt, i, i] \ i" (\(3QSUM _ \ _./ _)\ 10) + "_QSUM" :: "[idt, i, i] \ i" (\(\indent=3 notation=\binder QSUM\\\QSUM _ \ _./ _)\ 10) syntax_consts "_QSUM" \ QSigma translations diff -r 01b8c8d17f13 -r 2a77bc3b4eac src/ZF/Trancl.thy --- a/src/ZF/Trancl.thy Fri Sep 20 23:36:33 2024 +0200 +++ b/src/ZF/Trancl.thy Fri Sep 20 23:37:00 2024 +0200 @@ -37,11 +37,11 @@ \x,y\: r \ \y,z\: r \ \x,z\: r" definition - rtrancl :: "i\i" (\(_^*)\ [100] 100) (*refl/transitive closure*) where + rtrancl :: "i\i" (\(\notation=\postfix ^*\\_^*)\ [100] 100) (*refl/transitive closure*) where "r^* \ lfp(field(r)*field(r), \s. id(field(r)) \ (r O s))" definition - trancl :: "i\i" (\(_^+)\ [100] 100) (*transitive closure*) where + trancl :: "i\i" (\(\notation=\postfix ^+\\_^+)\ [100] 100) (*transitive closure*) where "r^+ \ r O r^*" definition diff -r 01b8c8d17f13 -r 2a77bc3b4eac src/ZF/UNITY/Follows.thy --- a/src/ZF/UNITY/Follows.thy Fri Sep 20 23:36:33 2024 +0200 +++ b/src/ZF/UNITY/Follows.thy Fri Sep 20 23:37:00 2024 +0200 @@ -39,7 +39,7 @@ abbreviation Follows' :: "[i\i, i\i, i, i] \ i" - (\(_ /Fols _ /Wrt (_ /'/ _))\ [60, 0, 0, 60] 60) where + (\(\notation=\mixfix Fols Wrt\\_ /Fols _ /Wrt (_ /'/ _))\ [60, 0, 0, 60] 60) where "f Fols g Wrt r/A \ Follows(A,r,f,g)" diff -r 01b8c8d17f13 -r 2a77bc3b4eac src/ZF/UNITY/Guar.thy --- a/src/ZF/UNITY/Guar.thy Fri Sep 20 23:36:33 2024 +0200 +++ b/src/ZF/UNITY/Guar.thy Fri Sep 20 23:37:00 2024 +0200 @@ -77,13 +77,13 @@ "welldef \ {F \ program. Init(F) \ 0}" definition - refines :: "[i, i, i] \ o" (\(3_ refines _ wrt _)\ [10,10,10] 10) where + refines :: "[i, i, i] \ o" (\(\indent=3 notation=\mixfix refines wrt\\_ refines _ wrt _)\ [10,10,10] 10) where "G refines F wrt X \ \H \ program. (F ok H \ G ok H \ F \ H \ welldef \ X) \ (G \ H \ welldef \ X)" definition - iso_refines :: "[i,i, i] \ o" (\(3_ iso'_refines _ wrt _)\ [10,10,10] 10) where + iso_refines :: "[i,i, i] \ o" (\(\indent=3 notation=\mixfix iso_refines wrt\\_ iso'_refines _ wrt _)\ [10,10,10] 10) where "G iso_refines F wrt X \ F \ welldef \ X \ G \ welldef \ X" diff -r 01b8c8d17f13 -r 2a77bc3b4eac src/ZF/UNITY/Increasing.thy --- a/src/ZF/UNITY/Increasing.thy Fri Sep 20 23:36:33 2024 +0200 +++ b/src/ZF/UNITY/Increasing.thy Fri Sep 20 23:37:00 2024 +0200 @@ -23,7 +23,7 @@ (\x \ state. f(x):A)}" abbreviation (input) - IncWrt :: "[i\i, i, i] \ i" (\(_ IncreasingWrt _ '/ _)\ [60, 0, 60] 60) where + IncWrt :: "[i\i, i, i] \ i" (\(\notation=\mixfix IncreasingWrt\\_ IncreasingWrt _ '/ _)\ [60, 0, 60] 60) where "f IncreasingWrt r/A \ Increasing[A](r,f)" diff -r 01b8c8d17f13 -r 2a77bc3b4eac src/ZF/UNITY/Union.thy --- a/src/ZF/UNITY/Union.thy Fri Sep 20 23:36:33 2024 +0200 +++ b/src/ZF/UNITY/Union.thy Fri Sep 20 23:37:00 2024 +0200 @@ -41,8 +41,8 @@ SKIP \ X \ (\G \ program. Acts(G) \ (\F \ X. Acts(F)) \ G \ X)" syntax - "_JOIN1" :: "[pttrns, i] \ i" (\(3\_./ _)\ 10) - "_JOIN" :: "[pttrn, i, i] \ i" (\(3\_ \ _./ _)\ 10) + "_JOIN1" :: "[pttrns, i] \ i" (\(\indent=3 notation=\binder \\\\_./ _)\ 10) + "_JOIN" :: "[pttrn, i, i] \ i" (\(\indent=3 notation=\binder \\\\\_ \ _./ _)\ 10) syntax_consts "_JOIN1" "_JOIN" == JOIN translations diff -r 01b8c8d17f13 -r 2a77bc3b4eac src/ZF/ZF.thy --- a/src/ZF/ZF.thy Fri Sep 20 23:36:33 2024 +0200 +++ b/src/ZF/ZF.thy Fri Sep 20 23:37:00 2024 +0200 @@ -7,14 +7,14 @@ subsection\Iteration of the function \<^term>\F\\ -consts iterates :: "[i\i,i,i] \ i" (\(_^_ '(_'))\ [60,1000,1000] 60) +consts iterates :: "[i\i,i,i] \ i" (\(\notation=\mixfix iterates\\_^_ '(_'))\ [60,1000,1000] 60) primrec "F^0 (x) = x" "F^(succ(n)) (x) = F(F^n (x))" definition - iterates_omega :: "[i\i,i] \ i" (\(_^\ '(_'))\ [60,1000] 60) where + iterates_omega :: "[i\i,i] \ i" (\(\notation=\mixfix iterates_omega\\_^\ '(_'))\ [60,1000] 60) where "F^\ (x) \ \n\nat. F^n (x)" lemma iterates_triv: diff -r 01b8c8d17f13 -r 2a77bc3b4eac src/ZF/ZF_Base.thy --- a/src/ZF/ZF_Base.thy Fri Sep 20 23:36:33 2024 +0200 +++ b/src/ZF/ZF_Base.thy Fri Sep 20 23:37:00 2024 +0200 @@ -36,8 +36,8 @@ where "Bex(A, P) \ \x. x\A \ P(x)" syntax - "_Ball" :: "[pttrn, i, o] \ o" (\(3\_\_./ _)\ 10) - "_Bex" :: "[pttrn, i, o] \ o" (\(3\_\_./ _)\ 10) + "_Ball" :: "[pttrn, i, o] \ o" (\(\indent=3 notation=\binder \\\\\_\_./ _)\ 10) + "_Bex" :: "[pttrn, i, o] \ o" (\(\indent=3 notation=\binder \\\\\_\_./ _)\ 10) syntax_consts "_Ball" \ Ball and "_Bex" \ Bex @@ -55,7 +55,7 @@ where "Replace(A,P) \ PrimReplace(A, \x y. (\!z. P(x,z)) \ P(x,y))" syntax - "_Replace" :: "[pttrn, pttrn, i, o] \ i" (\(1{_ ./ _ \ _, _})\) + "_Replace" :: "[pttrn, pttrn, i, o] \ i" (\(\indent=1 notation=\mixfix Replace\\{_ ./ _ \ _, _})\) syntax_consts "_Replace" \ Replace translations @@ -68,7 +68,7 @@ where "RepFun(A,f) \ {y . x\A, y=f(x)}" syntax - "_RepFun" :: "[i, pttrn, i] \ i" (\(1{_ ./ _ \ _})\ [51,0,51]) + "_RepFun" :: "[i, pttrn, i] \ i" (\(\indent=1 notation=\mixfix RepFun\\{_ ./ _ \ _})\ [51,0,51]) syntax_consts "_RepFun" \ RepFun translations @@ -80,7 +80,7 @@ where "Collect(A,P) \ {y . x\A, x=y \ P(x)}" syntax - "_Collect" :: "[pttrn, i, o] \ i" (\(1{_ \ _ ./ _})\) + "_Collect" :: "[pttrn, i, o] \ i" (\(\indent=1 notation=\mixfix Collect\\{_ \ _ ./ _})\) syntax_consts "_Collect" \ Collect translations @@ -93,8 +93,8 @@ where "\(A) \ { x\\(A) . \y\A. x\y}" syntax - "_UNION" :: "[pttrn, i, i] \ i" (\(3\_\_./ _)\ 10) - "_INTER" :: "[pttrn, i, i] \ i" (\(3\_\_./ _)\ 10) + "_UNION" :: "[pttrn, i, i] \ i" (\(\indent=3 notation=\binder \\\\\_\_./ _)\ 10) + "_INTER" :: "[pttrn, i, i] \ i" (\(\indent=3 notation=\binder \\\\\_\_./ _)\ 10) syntax_consts "_UNION" == Union and "_INTER" == Inter @@ -169,7 +169,7 @@ definition The :: "(i \ o) \ i" (binder \THE \ 10) where the_def: "The(P) \ \({y . x \ {0}, P(y)})" -definition If :: "[o, i, i] \ i" (\(if (_)/ then (_)/ else (_))\ [10] 10) +definition If :: "[o, i, i] \ i" (\(\notation=\mixfix if then else\\if (_)/ then (_)/ else (_))\ [10] 10) where if_def: "if P then a else b \ THE z. P \ z=a | \P \ z=b" abbreviation (input) @@ -272,9 +272,9 @@ (* binder syntax *) syntax - "_PROD" :: "[pttrn, i, i] \ i" (\(3\_\_./ _)\ 10) - "_SUM" :: "[pttrn, i, i] \ i" (\(3\_\_./ _)\ 10) - "_lam" :: "[pttrn, i, i] \ i" (\(3\_\_./ _)\ 10) + "_PROD" :: "[pttrn, i, i] \ i" (\(\indent=3 notation=\mixfix \\\\\_\_./ _)\ 10) + "_SUM" :: "[pttrn, i, i] \ i" (\(\indent=3 notation=\mixfix \\\\\_\_./ _)\ 10) + "_lam" :: "[pttrn, i, i] \ i" (\(\indent=3 notation=\mixfix \\\\\_\_./ _)\ 10) syntax_consts "_PROD" == Pi and "_SUM" == Sigma and @@ -297,16 +297,16 @@ not_mem (infixl \\:\ 50) syntax (ASCII) - "_Ball" :: "[pttrn, i, o] \ o" (\(3ALL _:_./ _)\ 10) - "_Bex" :: "[pttrn, i, o] \ o" (\(3EX _:_./ _)\ 10) - "_Collect" :: "[pttrn, i, o] \ i" (\(1{_: _ ./ _})\) - "_Replace" :: "[pttrn, pttrn, i, o] \ i" (\(1{_ ./ _: _, _})\) - "_RepFun" :: "[i, pttrn, i] \ i" (\(1{_ ./ _: _})\ [51,0,51]) - "_UNION" :: "[pttrn, i, i] \ i" (\(3UN _:_./ _)\ 10) - "_INTER" :: "[pttrn, i, i] \ i" (\(3INT _:_./ _)\ 10) - "_PROD" :: "[pttrn, i, i] \ i" (\(3PROD _:_./ _)\ 10) - "_SUM" :: "[pttrn, i, i] \ i" (\(3SUM _:_./ _)\ 10) - "_lam" :: "[pttrn, i, i] \ i" (\(3lam _:_./ _)\ 10) + "_Ball" :: "[pttrn, i, o] \ o" (\(\indent=3 notation=\binder ALL:\\ALL _:_./ _)\ 10) + "_Bex" :: "[pttrn, i, o] \ o" (\(\indent=3 notation=\binder EX:\\EX _:_./ _)\ 10) + "_Collect" :: "[pttrn, i, o] \ i" (\(\indent=1 notation=\mixfix Collect\\{_: _ ./ _})\) + "_Replace" :: "[pttrn, pttrn, i, o] \ i" (\(\indent=1 notation=\mixfix Replace\\{_ ./ _: _, _})\) + "_RepFun" :: "[i, pttrn, i] \ i" (\(\indent=1 notation=\mixfix RepFun\\{_ ./ _: _})\ [51,0,51]) + "_UNION" :: "[pttrn, i, i] \ i" (\(\indent=3 notation=\binder UN:\\UN _:_./ _)\ 10) + "_INTER" :: "[pttrn, i, i] \ i" (\(\indent=3 notation=\binder INT:\\INT _:_./ _)\ 10) + "_PROD" :: "[pttrn, i, i] \ i" (\(\indent=3 notation=\binder PROD:\\PROD _:_./ _)\ 10) + "_SUM" :: "[pttrn, i, i] \ i" (\(\indent=3 notation=\binder SUM:\\SUM _:_./ _)\ 10) + "_lam" :: "[pttrn, i, i] \ i" (\(\indent=3 notation=\binder lam:\\lam _:_./ _)\ 10) "_Tuple" :: "[i, tuple_args] \ i" (\<(_,/ _)>\) "_pattern" :: "patterns \ pttrn" (\<_>\) diff -r 01b8c8d17f13 -r 2a77bc3b4eac src/ZF/ex/Ring.thy --- a/src/ZF/ex/Ring.thy Fri Sep 20 23:36:33 2024 +0200 +++ b/src/ZF/ex/Ring.thy Fri Sep 20 23:37:00 2024 +0200 @@ -46,7 +46,7 @@ "a_inv(R) \ m_inv ()" definition - minus :: "[i,i,i] \ i" (\(_ \\ _)\ [65,66] 65) where + minus :: "[i,i,i] \ i" (\(\notation=\infix \\\_ \\ _)\ [65,66] 65) where "\x \ carrier(R); y \ carrier(R)\ \ x \\<^bsub>R\<^esub> y = x \\<^bsub>R\<^esub> (\\<^bsub>R\<^esub> y)" locale abelian_monoid = fixes G (structure) diff -r 01b8c8d17f13 -r 2a77bc3b4eac src/ZF/func.thy --- a/src/ZF/func.thy Fri Sep 20 23:36:33 2024 +0200 +++ b/src/ZF/func.thy Fri Sep 20 23:37:00 2024 +0200 @@ -448,7 +448,7 @@ nonterminal updbinds and updbind syntax - "_updbind" :: "[i, i] \ updbind" (\(2_ :=/ _)\) + "_updbind" :: "[i, i] \ updbind" (\(\indent=2 notation=\infix update\\_ :=/ _)\) "" :: "updbind \ updbinds" (\_\) "_updbinds" :: "[updbind, updbinds] \ updbinds" (\_,/ _\) "_Update" :: "[i, updbinds] \ i" (\_/'((_)')\ [900,0] 900)