diff -r 46f59511b7bb -r d97fdabd9e2b src/HOL/Codegenerator_Test/Code_Lazy_Test.thy --- a/src/HOL/Codegenerator_Test/Code_Lazy_Test.thy Fri Sep 20 19:07:10 2024 +0200 +++ b/src/HOL/Codegenerator_Test/Code_Lazy_Test.thy Fri Sep 20 19:51:08 2024 +0200 @@ -16,18 +16,18 @@ value [code] "cycle ''ab''" value [code] "let x = cycle ''ab''; y = snth x 10 in x" -datatype 'a llist = LNil ("\<^bold>[\<^bold>]") | LCons (lhd: 'a) (ltl: "'a llist") (infixr "\<^bold>#" 65) +datatype 'a llist = LNil (\\<^bold>[\<^bold>]\) | LCons (lhd: 'a) (ltl: "'a llist") (infixr \\<^bold>#\ 65) subsection \Finite lazy lists\ code_lazy_type llist -no_notation lazy_llist ("_") +no_notation lazy_llist (\_\) nonterminal llist_args syntax - "" :: "'a \ llist_args" ("_") - "_llist_args" :: "'a \ llist_args \ llist_args" ("_,/ _") - "_llist" :: "llist_args => 'a list" ("\<^bold>[(_)\<^bold>]") + "" :: "'a \ llist_args" (\_\) + "_llist_args" :: "'a \ llist_args \ llist_args" (\_,/ _\) + "_llist" :: "llist_args => 'a list" (\\<^bold>[(_)\<^bold>]\) syntax_consts "_llist_args" "_llist" == lazy_llist translations @@ -77,7 +77,7 @@ subsection \Branching codatatypes\ -codatatype tree = L | Node tree tree (infix "\" 900) +codatatype tree = L | Node tree tree (infix \\\ 900) code_lazy_type tree