src/HOLCF/IOA/meta_theory/Deadlock.thy
author wenzelm
Fri, 02 Sep 2005 17:23:59 +0200
changeset 17233 41eee2e7b465
parent 14981 e73f8140af78
child 19741 f65265d71426
permissions -rw-r--r--
converted specifications to Isar theories;

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