--- 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" (\<open>(\<open>indent=1 notation=\<open>mixfix list enumeration\<close>\<close>[_])\<close>)
-syntax_consts
- Cons
translations
"[x, xs]" == "x#[xs]"
"[x]" == "x#[]"
@@ -137,9 +135,6 @@
"_lupdbinds" :: "[lupdbind, lupdbinds] => lupdbinds" (\<open>_,/ _\<close>)
"_LUpdate" :: "['a, lupdbinds] => 'a" (\<open>_/[(_)]\<close> [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"