equal
deleted
inserted
replaced
358 (*<*) |
358 (*<*) |
359 no_translations |
359 no_translations |
360 "[x, xs]" == "x # [xs]" |
360 "[x, xs]" == "x # [xs]" |
361 "[x]" == "x # []" |
361 "[x]" == "x # []" |
362 |
362 |
363 no_notation Nil (\<open>[]\<close>) and Cons (infixr \<open>#\<close> 65) |
363 unbundle no list_syntax |
364 |
|
365 hide_type list |
364 hide_type list |
366 hide_const Nil Cons case_list hd tl set map list_all2 rec_list size_list list_all |
365 hide_const Nil Cons case_list hd tl set map list_all2 rec_list size_list list_all |
367 |
366 |
368 context early |
367 context early |
369 begin |
368 begin |
449 text \<open> |
448 text \<open> |
450 \noindent |
449 \noindent |
451 Incidentally, this is how the traditional syntax can be set up: |
450 Incidentally, this is how the traditional syntax can be set up: |
452 \<close> |
451 \<close> |
453 (*<*) |
452 (*<*) |
454 unbundle no list_syntax |
453 unbundle no list_enumeration_syntax |
455 (*>*) |
454 (*>*) |
456 syntax "_list" :: "args \<Rightarrow> 'a list" (\<open>[(_)]\<close>) |
455 syntax "_list" :: "args \<Rightarrow> 'a list" (\<open>[(_)]\<close>) |
457 |
456 |
458 text \<open>\blankline\<close> |
457 text \<open>\blankline\<close> |
459 |
458 |