src/HOL/HOLCF/IOA/IOA.thy
author paulson <lp15@cam.ac.uk>
Thu, 24 Aug 2023 21:40:24 +0100
changeset 78522 918a9ed06898
parent 62008 cbedaddc9351
permissions -rw-r--r--
some refinements in Algebra and Number_Theory

(*  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