diff -r 843dba3d307a -r c007e6d9941d src/HOL/List.thy --- a/src/HOL/List.thy Mon Sep 30 23:32:26 2024 +0200 +++ b/src/HOL/List.thy Tue Oct 01 20:39:16 2024 +0200 @@ -47,8 +47,6 @@ syntax "_list" :: "args => 'a list" (\(\indent=1 notation=\mixfix list enumeration\\[_])\) -syntax_consts - Cons translations "[x, xs]" == "x#[xs]" "[x]" == "x#[]" @@ -137,9 +135,6 @@ "_lupdbinds" :: "[lupdbind, lupdbinds] => lupdbinds" (\_,/ _\) "_LUpdate" :: "['a, lupdbinds] => 'a" (\_/[(_)]\ [1000,0] 900) -syntax_consts - list_update - translations "_LUpdate xs (_lupdbinds b bs)" == "_LUpdate (_LUpdate xs b) bs" "xs[i:=x]" == "CONST list_update xs i x"