equal
deleted
inserted
replaced
450 |
450 |
451 text \<open> |
451 text \<open> |
452 \noindent |
452 \noindent |
453 Incidentally, this is how the traditional syntax can be set up: |
453 Incidentally, this is how the traditional syntax can be set up: |
454 \<close> |
454 \<close> |
455 |
455 (*<*) |
456 syntax "_list" :: "list_args \<Rightarrow> 'a list" (\<open>[(_)]\<close>) |
456 no_syntax |
|
457 "_list" :: "args => 'a list" (\<open>[(\<open>notation=\<open>mixfix list enumeration\<close>\<close>_)]\<close>) |
|
458 (*>*) |
|
459 syntax "_list" :: "args \<Rightarrow> 'a list" (\<open>[(_)]\<close>) |
457 |
460 |
458 text \<open>\blankline\<close> |
461 text \<open>\blankline\<close> |
459 |
462 |
460 translations |
463 translations |
461 "[x, xs]" == "x # [xs]" |
464 "[x, xs]" == "x # [xs]" |