src/HOL/Library/Imperative_HOL.thy
changeset 29399 ebcd69a00872
parent 29397 aab26a65e80f
child 29400 a462459fb5ce
--- a/src/HOL/Library/Imperative_HOL.thy	Thu Jan 08 10:53:48 2009 +0100
+++ /dev/null	Thu Jan 01 00:00:00 1970 +0000
@@ -1,12 +0,0 @@
-(*  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