src/HOL/Imperative_HOL/Heap_Monad.thy
changeset 41413 64cd30d6b0b8
parent 40671 5e46057ba8e0
child 42949 618adb3584e5
--- a/src/HOL/Imperative_HOL/Heap_Monad.thy	Wed Dec 29 13:51:17 2010 +0100
+++ b/src/HOL/Imperative_HOL/Heap_Monad.thy	Wed Dec 29 17:34:41 2010 +0100
@@ -5,7 +5,10 @@
 header {* A monad with a polymorphic heap and primitive reasoning infrastructure *}
 
 theory Heap_Monad
-imports Heap Monad_Syntax Code_Natural
+imports
+  Heap
+  "~~/src/HOL/Library/Monad_Syntax"
+  "~~/src/HOL/Library/Code_Natural"
 begin
 
 subsection {* The monad *}