src/ZF/UNITY/SubstAx.thy
author kleing
Tue, 13 May 2003 08:59:21 +0200
changeset 14024 213dcc39358f
parent 12195 ed2893765a08
child 15634 bca33c49b083
permissions -rw-r--r--
HOL-Real -> HOL-Complex

(*  Title:      ZF/UNITY/SubstAx.thy
    ID:         $Id$
    Author:     Sidi O Ehmety, Computer Laboratory
    Copyright   2001  University of Cambridge

Weak LeadsTo relation (restricted to the set of reachable states)

Theory ported from HOL.
*)

SubstAx = WFair + Constrains + 

constdefs
  (* The definitions below are not `conventional', but yields simpler rules *)
   Ensures :: "[i,i] => i"            (infixl 60)
    "A Ensures B == {F:program. F : (reachable(F) Int A) ensures (reachable(F) Int B) }"

  LeadsTo :: "[i, i] => i"            (infixl 60)
    "A LeadsTo B == {F:program. F:(reachable(F) Int A) leadsTo (reachable(F) Int B)}"

syntax (xsymbols)
  "op LeadsTo" :: "[i, i] => i" (infixl " \\<longmapsto>w " 60)

end