src/HOL/Imperative_HOL/Heap_Monad.thy
changeset 66453 cc19f7ca2ed6
parent 66148 5e60c2d0a1f1
child 67399 eab6ce8368fa
--- a/src/HOL/Imperative_HOL/Heap_Monad.thy	Fri Aug 18 13:55:05 2017 +0200
+++ b/src/HOL/Imperative_HOL/Heap_Monad.thy	Fri Aug 18 20:47:47 2017 +0200
@@ -7,7 +7,7 @@
 theory Heap_Monad
 imports
   Heap
-  "~~/src/HOL/Library/Monad_Syntax"
+  "HOL-Library.Monad_Syntax"
 begin
 
 subsection \<open>The monad\<close>