src/HOLCF/IOA/meta_theory/Deadlock.thy
author wenzelm
Mon, 02 Jan 2006 20:50:17 +0100
changeset 18539 35b9ed76b59a
parent 17233 41eee2e7b465
child 19741 f65265d71426
permissions -rw-r--r--
ISABELLE_USER for remote cvs access;

(*  Title:      HOLCF/IOA/meta_theory/Deadlock.thy
    ID:         $Id$
    Author:     Olaf Müller
*)

header {* Deadlock freedom of I/O Automata *}

theory Deadlock
imports RefCorrectness CompoScheds
begin

end