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"