diff -r 843dba3d307a -r c007e6d9941d src/ZF/ZF_Base.thy --- a/src/ZF/ZF_Base.thy Mon Sep 30 23:32:26 2024 +0200 +++ b/src/ZF/ZF_Base.thy Tue Oct 01 20:39:16 2024 +0200 @@ -56,8 +56,6 @@ syntax "_Replace" :: "[pttrn, pttrn, i, o] \ i" (\(\indent=1 notation=\mixfix relational replacement\\{_ ./ _ \ _, _})\) -syntax_consts - Replace translations "{y. x\A, Q}" \ "CONST Replace(A, \x y. Q)" @@ -69,8 +67,6 @@ syntax "_RepFun" :: "[i, pttrn, i] \ i" (\(\indent=1 notation=\mixfix functional replacement\\{_ ./ _ \ _})\ [51,0,51]) -syntax_consts - RepFun translations "{b. x\A}" \ "CONST RepFun(A, \x. b)" @@ -81,8 +77,6 @@ syntax "_Collect" :: "[pttrn, i, o] \ i" (\(\indent=1 notation=\mixfix set comprehension\\{_ \ _ ./ _})\) -syntax_consts - Collect translations "{x\A. P}" \ "CONST Collect(A, \x. P)" @@ -134,8 +128,6 @@ "" :: "i \ is" (\_\) "_Enum" :: "[i, is] \ is" (\_,/ _\) "_Finset" :: "is \ i" (\(\indent=1 notation=\mixfix set enumeration\\{_})\) -syntax_consts - cons translations "{x, xs}" == "CONST cons(x, {xs})" "{x}" == "CONST cons(x, 0)" @@ -197,8 +189,6 @@ "" :: "i \ tuple_args" (\_\) "_Tuple_args" :: "[i, tuple_args] \ tuple_args" (\_,/ _\) "_Tuple" :: "[i, tuple_args] \ i" (\(\indent=1 notation=\mixfix tuple enumeration\\\_,/ _\)\) -syntax_consts - Pair translations "\x, y, z\" == "\x, \y, z\\" "\x, y\" == "CONST Pair(x, y)"