src/Pure/Pure.thy
changeset 80752 2c9b5288eb84
parent 80750 1319c729c65d
child 81010 5ea48342e0ae
--- a/src/Pure/Pure.thy	Fri Aug 23 21:32:09 2024 +0200
+++ b/src/Pure/Pure.thy	Fri Aug 23 22:45:18 2024 +0200
@@ -404,7 +404,7 @@
 
 val syntax_consts =
   Parse.and_list1
-    ((Parse.name_position --| (\<^keyword>\<open>\<rightleftharpoons>\<close> || \<^keyword>\<open>==\<close>)) --
+    ((Scan.repeat1 Parse.name_position --| (\<^keyword>\<open>\<rightleftharpoons>\<close> || \<^keyword>\<open>==\<close>)) --
       Parse.!!! (Scan.repeat1 Parse.name_position));
 
 val _ =