src/HOL/Library/Imperative_HOL.thy
changeset 29413 43a12fc76f48
parent 29412 4085a531153d
parent 29400 a462459fb5ce
child 29414 747c95f7bb7e
child 29424 948d616959e4
--- a/src/HOL/Library/Imperative_HOL.thy	Fri Jan 09 09:34:49 2009 -0800
+++ /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