src/HOL/Imperative_HOL/Imperative_HOL.thy
changeset 37772 026ed2fc15d4
parent 29822 c45845743f04
child 37776 df0350f1e7f2
--- a/src/HOL/Imperative_HOL/Imperative_HOL.thy	Mon Jul 12 16:05:08 2010 +0200
+++ b/src/HOL/Imperative_HOL/Imperative_HOL.thy	Mon Jul 12 16:19:15 2010 +0200
@@ -5,7 +5,7 @@
 header {* Entry point into monadic imperative HOL *}
 
 theory Imperative_HOL
-imports Array Ref Relational
+imports Array Ref Relational Mrec
 begin
 
 end