diff -r 83596aea48cb -r dd59daa3c37a src/HOL/ex/Code_Lazy_Demo.thy --- a/src/HOL/ex/Code_Lazy_Demo.thy Mon Sep 30 13:00:42 2024 +0200 +++ b/src/HOL/ex/Code_Lazy_Demo.thy Mon Sep 30 20:30:59 2024 +0200 @@ -39,13 +39,10 @@ = LNil (\\<^bold>\\<^bold>\\) | LCons (lhd: 'a) (ltl: "'a llist") (infixr \###\ 65) -nonterminal llist_args syntax - "" :: "'a \ llist_args" (\_\) - "_llist_args" :: "'a \ llist_args \ llist_args" (\_,/ _\) - "_llist" :: "llist_args => 'a list" (\\<^bold>\(_)\<^bold>\\) + "_llist" :: "args => 'a list" (\\<^bold>\(\notation=\mixfix lazy list enumeration\\_)\<^bold>\\) syntax_consts - "_llist_args" "_llist" == LCons + LCons translations "\<^bold>\x, xs\<^bold>\" == "x###\<^bold>\xs\<^bold>\" "\<^bold>\x\<^bold>\" == "x###\<^bold>\\<^bold>\"