src/HOL/HOLCF/IOA/meta_theory/IOA.thy
author wenzelm
Mon, 10 Feb 2014 22:22:06 +0100
changeset 55386 0c15ac6edcf7
parent 42151 4da4fc77664b
child 58880 0baae4311a9f
permissions -rw-r--r--
make triple-sure that the future scheduler is properly shutdown (see also 702278df3b57);

(*  Title:      HOL/HOLCF/IOA/meta_theory/IOA.thy
    Author:     Olaf Müller
*)

header {* The theory of I/O automata in HOLCF *}

theory IOA
imports SimCorrectness Compositionality Deadlock
begin

end