src/HOL/Imperative_HOL/Imperative_HOL.thy
author wenzelm
Thu, 15 Oct 2015 22:25:57 +0200
changeset 61456 b521b8b400f7
parent 58889 5b7a9633cfa8
child 63167 0909deb8059b
permissions -rw-r--r--
trim_blanks after read, before eval; clarified Raw_Token: uniform output_text; tuned signature;

(*  Title:      HOL/Imperative_HOL/Imperative_HOL.thy
    Author:     John Matthews, Galois Connections; Alexander Krauss, Lukas Bulwahn & Florian Haftmann, TU Muenchen
*)

section {* Entry point into monadic imperative HOL *}

theory Imperative_HOL
imports Array Ref
begin

end