more official task context via Task_Queue.enroll, which is required to participate in group cancellation (e.g. to terminate command exec);
tuned signature;
(* 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
begin
end