--- a/src/HOL/Library/IArray.thy Thu Jan 02 08:37:52 2025 +0100
+++ b/src/HOL/Library/IArray.thy Thu Jan 02 08:37:55 2025 +0100
@@ -177,7 +177,7 @@
lists first. Arrays could be converted back into lists for printing if they
were wrapped up in an additional constructor.\<close>
-code_reserved SML Vector
+code_reserved (SML) Vector
code_printing
type_constructor iarray \<rightharpoonup> (SML) "_ Vector.vector"
@@ -222,7 +222,7 @@
}\<close> for type_constructor iarray constant IArray IArray.tabulate IArray.sub' IArray.length'
-code_reserved Haskell IArray_Impl
+code_reserved (Haskell) IArray_Impl
code_printing
type_constructor iarray \<rightharpoonup> (Haskell) "IArray.IArray _"