src/HOL/Codegenerator_Test/Candidates.thy
changeset 81706 7beb0cf38292
parent 75955 5305c65dcbb2
child 82516 88f101c3cfe2
--- a/src/HOL/Codegenerator_Test/Candidates.thy	Thu Jan 02 08:37:52 2025 +0100
+++ b/src/HOL/Codegenerator_Test/Candidates.thy	Thu Jan 02 08:37:55 2025 +0100
@@ -42,7 +42,7 @@
 
 text \<open>Avoid popular infix.\<close>
 
-code_reserved SML upto
+code_reserved (SML) upto
 
 text \<open>Explicit check in \<open>OCaml\<close> for correct precedence of let expressions in list expressions\<close>