diff -r be8c0e039a5e -r bc936d3d8b45 src/CCL/Type.thy --- a/src/CCL/Type.thy Sun Aug 25 15:02:19 2024 +0200 +++ b/src/CCL/Type.thy Sun Aug 25 15:07:22 2024 +0200 @@ -14,10 +14,10 @@ syntax "_Subtype" :: "[idt, 'a set, o] \ 'a set" ("(1{_: _ ./ _})") +syntax_consts + "_Subtype" == Subtype translations "{x: A. B}" == "CONST Subtype(A, \x. B)" -syntax_consts - "_Subtype" == Subtype definition Unit :: "i set" where "Unit == {x. x=one}" @@ -39,6 +39,9 @@ "_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) +syntax_consts + "_Pi" "_arrow" \ Pi and + "_Sigma" "_star" \ Sigma translations "PROD x:A. B" \ "CONST Pi(A, \x. B)" "A -> B" \ "CONST Pi(A, \_. B)" @@ -50,9 +53,6 @@ (\<^const_syntax>\Sigma\, fn _ => Syntax_Trans.dependent_tr' (\<^syntax_const>\_Sigma\, \<^syntax_const>\_star\))] \ -syntax_consts - "_Pi" "_arrow" \ Pi and - "_Sigma" "_star" \ Sigma definition Nat :: "i set" where "Nat == lfp(\X. Unit + X)"