src/HOL/List.thy
changeset 81182 fc5066122e68
parent 81133 072cc2a92ba3
child 81282 fa3d678ea1f4
--- 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 \<Rightarrow> 'a list"  (\<open>(\<open>indent=1 notation=\<open>mixfix list enumeration\<close>\<close>[_])\<close>)
 end
+syntax_consts
+  "_list" \<rightleftharpoons> Cons
 translations
   "[x, xs]" \<rightleftharpoons> "x#[xs]"
   "[x]" \<rightleftharpoons> "x#[]"
@@ -144,7 +146,8 @@
   "_lupdbinds" :: "[lupdbind, lupdbinds] => lupdbinds"    (\<open>_,/ _\<close>)
   "_LUpdate" :: "['a, lupdbinds] => 'a"
     (\<open>(\<open>open_block notation=\<open>mixfix list update\<close>\<close>_/[(_)])\<close> [1000,0] 900)
-
+syntax_consts
+  "_LUpdate" \<rightleftharpoons> list_update
 translations
   "_LUpdate xs (_lupdbinds b bs)" == "_LUpdate (_LUpdate xs b) bs"
   "xs[i:=x]" == "CONST list_update xs i x"