src/HOL/List.thy
changeset 81019 dd59daa3c37a
parent 81018 83596aea48cb
child 81090 843dba3d307a
--- a/src/HOL/List.thy	Mon Sep 30 13:00:42 2024 +0200
+++ b/src/HOL/List.thy	Mon Sep 30 20:30:59 2024 +0200
@@ -45,13 +45,10 @@
 
 text \<open>List enumeration\<close>
 
-nonterminal list_args
 syntax
-  "" :: "'a \<Rightarrow> list_args"  (\<open>_\<close>)
-  "_list_args" :: "'a \<Rightarrow> list_args \<Rightarrow> list_args"  (\<open>_,/ _\<close>)
-  "_list" :: "list_args => 'a list"    (\<open>[(_)]\<close>)
+  "_list" :: "args => 'a list"    (\<open>[(\<open>notation=\<open>mixfix list enumeration\<close>\<close>_)]\<close>)
 syntax_consts
-  "_list_args" "_list" == Cons
+  Cons
 translations
   "[x, xs]" == "x#[xs]"
   "[x]" == "x#[]"