recoded latin1 as utf8;
use textcomp for some text symbols where it appears appropriate;
(* Title: HOL/Imperative_HOL/Imperative_HOL.thy
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 Mrec
begin
end