src/Doc/Datatypes/Datatypes.thy
changeset 81133 072cc2a92ba3
parent 81128 5b201b24d99b
child 81502 ed766dfdd2f1
--- a/src/Doc/Datatypes/Datatypes.thy	Tue Oct 08 16:15:31 2024 +0200
+++ b/src/Doc/Datatypes/Datatypes.thy	Tue Oct 08 17:26:31 2024 +0200
@@ -360,8 +360,7 @@
       "[x, xs]" == "x # [xs]"
       "[x]" == "x # []"
 
-    no_notation Nil  (\<open>[]\<close>) and Cons  (infixr \<open>#\<close> 65)
-
+    unbundle no list_syntax
     hide_type list
     hide_const Nil Cons case_list hd tl set map list_all2 rec_list size_list list_all
 
@@ -451,7 +450,7 @@
 Incidentally, this is how the traditional syntax can be set up:
 \<close>
 (*<*)
-unbundle no list_syntax
+unbundle no list_enumeration_syntax
 (*>*)
     syntax "_list" :: "args \<Rightarrow> 'a list" (\<open>[(_)]\<close>)