diff -r 46f59511b7bb -r d97fdabd9e2b src/HOL/HOLCF/IOA/Sequence.thy --- a/src/HOL/HOLCF/IOA/Sequence.thy Fri Sep 20 19:07:10 2024 +0200 +++ b/src/HOL/HOLCF/IOA/Sequence.thy Fri Sep 20 19:51:08 2024 +0200 @@ -63,7 +63,7 @@ UU \ UU | Def y \ (if P y then x ## (h \ xs) else h \ xs))))" -abbreviation Consq_syn ("(_/\_)" [66, 65] 65) +abbreviation Consq_syn (\(_/\_)\ [66, 65] 65) where "a \ s \ Consq a \ s" @@ -71,10 +71,10 @@ nonterminal llist_args syntax - "" :: "'a \ llist_args" ("_") - "_list_args" :: "'a \ llist_args \ llist_args" ("_,/ _") - "_totlist" :: "llist_args \ 'a Seq" ("[(_)!]") - "_partlist" :: "llist_args \ 'a Seq" ("[(_)?]") + "" :: "'a \ llist_args" (\_\) + "_list_args" :: "'a \ llist_args \ llist_args" (\_,/ _\) + "_totlist" :: "llist_args \ 'a Seq" (\[(_)!]\) + "_partlist" :: "llist_args \ 'a Seq" (\[(_)?]\) syntax_consts "_totlist" "_partlist" \ Consq translations