src/HOL/UNITY/UNITY.thy
author paulson
Mon, 13 Jul 1998 16:41:30 +0200
changeset 5135 c12a6eb09574
parent 4776 1f9362e769c1
child 5253 82a5ca6290aa
permissions -rw-r--r--
renamed mutex to Acts

(*  Title:      HOL/UNITY/UNITY
    ID:         $Id$
    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
    Copyright   1998  University of Cambridge

The basic UNITY theory (revised version, based upon the "co" operator)

From Misra, "A Logic for Concurrent Programming", 1994
*)

UNITY = LessThan +

constdefs

  constrains :: "[('a * 'a)set set, 'a set, 'a set] => bool"
    "constrains Acts A B == ALL act:Acts. act^^A <= B"

  stable     :: "('a * 'a)set set => 'a set => bool"
    "stable Acts A == constrains Acts A A"

  strongest_rhs :: "[('a * 'a)set set, 'a set] => 'a set"
    "strongest_rhs Acts A == Inter {B. constrains Acts A B}"

  unless :: "[('a * 'a)set set, 'a set, 'a set] => bool"
    "unless Acts A B == constrains Acts (A-B) (A Un B)"

end