src/HOL/Imperative_HOL/Heap_Monad.thy
changeset 55372 3662c44d018c
parent 55147 bce3dbc11f95
child 57437 0baf08c075b9
--- a/src/HOL/Imperative_HOL/Heap_Monad.thy	Sun Feb 09 19:10:12 2014 +0000
+++ b/src/HOL/Imperative_HOL/Heap_Monad.thy	Sun Feb 09 21:37:27 2014 +0100
@@ -575,7 +575,7 @@
 
 text {* Adaption layer *}
 
-code_include Haskell "Heap"
+code_printing code_module "Heap" \<rightharpoonup> (Haskell)
 {*import qualified Control.Monad;
 import qualified Control.Monad.ST;
 import qualified Data.STRef;
@@ -620,7 +620,7 @@
 
 subsubsection {* Scala *}
 
-code_include Scala "Heap"
+code_printing code_module "Heap" \<rightharpoonup> (Scala)
 {*object Heap {
   def bind[A, B](f: Unit => A, g: A => Unit => B): Unit => B = (_: Unit) => g (f ()) ()
 }