diff -r ff2a637a449e -r fc5066122e68 src/HOL/List.thy --- a/src/HOL/List.thy Fri Oct 18 11:44:05 2024 +0200 +++ b/src/HOL/List.thy Fri Oct 18 14:20:09 2024 +0200 @@ -56,6 +56,8 @@ syntax "_list" :: "args \ 'a list" (\(\indent=1 notation=\mixfix list enumeration\\[_])\) end +syntax_consts + "_list" \ Cons translations "[x, xs]" \ "x#[xs]" "[x]" \ "x#[]" @@ -144,7 +146,8 @@ "_lupdbinds" :: "[lupdbind, lupdbinds] => lupdbinds" (\_,/ _\) "_LUpdate" :: "['a, lupdbinds] => 'a" (\(\open_block notation=\mixfix list update\\_/[(_)])\ [1000,0] 900) - +syntax_consts + "_LUpdate" \ list_update translations "_LUpdate xs (_lupdbinds b bs)" == "_LUpdate (_LUpdate xs b) bs" "xs[i:=x]" == "CONST list_update xs i x"