src/HOL/Library/Imperative_HOL.thy
changeset 29400 a462459fb5ce
parent 29398 89813bbf0f3e
parent 29399 ebcd69a00872
child 29413 43a12fc76f48
child 29439 83601bdadae8
child 29682 7bae3abff5d7
--- a/src/HOL/Library/Imperative_HOL.thy	Thu Jan 08 17:25:06 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