src/HOL/Imperative_HOL/Heap_Monad.thy
changeset 81706 7beb0cf38292
parent 77703 0262155d2743
child 81995 d67dadd69d07
--- a/src/HOL/Imperative_HOL/Heap_Monad.thy	Thu Jan 02 08:37:52 2025 +0100
+++ b/src/HOL/Imperative_HOL/Heap_Monad.thy	Thu Jan 02 08:37:55 2025 +0100
@@ -565,7 +565,7 @@
 writeArray :: STArray s a -> Integer -> a -> ST s ()
 writeArray = Data.Array.ST.writeArray\<close>
 
-code_reserved Haskell Heap
+code_reserved (Haskell) Heap
 
 text \<open>Monad\<close>
 
@@ -620,7 +620,7 @@
 
 \<close>
 
-code_reserved Scala Heap Ref Array
+code_reserved (Scala) Heap Ref Array
 
 code_printing type_constructor Heap \<rightharpoonup> (Scala) "(Unit/ =>/ _)"
 code_printing constant bind \<rightharpoonup> (Scala) "Heap.bind"