proper support for "isabelle update -D DIR": avoid accidental exclusion of select_dirs (amending e5dafe9e120f);
(* Title: HOL/HOLCF/IOA/IOA.thy
Author: Olaf Müller
*)
section \<open>The theory of I/O automata in HOLCF\<close>
theory IOA
imports SimCorrectness Compositionality Deadlock
begin
end