diff -r aab26a65e80f -r ebcd69a00872 src/HOL/Imperative_HOL/Imperative_HOL.thy --- /dev/null Thu Jan 01 00:00:00 1970 +0000 +++ b/src/HOL/Imperative_HOL/Imperative_HOL.thy Thu Jan 08 17:10:41 2009 +0100 @@ -0,0 +1,12 @@ +(* Title: HOL/Library/Imperative_HOL.thy + ID: $Id$ + Author: John Matthews, Galois Connections; Alexander Krauss, Lukas Bulwahn & Florian Haftmann, TU Muenchen +*) + +header {* Entry point into monadic imperative HOL *} + +theory Imperative_HOL +imports Array Ref Relational +begin + +end