diff -r 5ea48342e0ae -r 6d34c2bedaa3 src/ZF/List.thy --- a/src/ZF/List.thy Sun Sep 29 21:40:37 2024 +0200 +++ b/src/ZF/List.thy Sun Sep 29 21:57:47 2024 +0200 @@ -19,9 +19,9 @@ syntax "" :: "i \ list_args" (\_\) "_List_args" :: "[i, list_args] \ list_args" (\_,/ _\) - "_List" :: "list_args \ i" (\[(_)]\) + "_List" :: "list_args \ i" (\[(\notation=\mixfix list enumeration\\_)]\) syntax_consts - "_List_args" "_List" \ Cons + Cons translations "[x, xs]" == "CONST Cons(x, [xs])" "[x]" == "CONST Cons(x, [])"