src/ZF/UNITY/SubstAx.thy
changeset 11479 697dcaaf478f
child 12195 ed2893765a08
equal deleted inserted replaced
11478:0f57375aafce 11479:697dcaaf478f
       
     1 (*  Title:      ZF/UNITY/SubstAx.thy
       
     2     ID:         $Id$
       
     3     Author:     Sidi O Ehmety, Computer Laboratory
       
     4     Copyright   2001  University of Cambridge
       
     5 
       
     6 Weak LeadsTo relation (restricted to the set of reachable states)
       
     7 
       
     8 Theory ported from HOL.
       
     9 *)
       
    10 
       
    11 SubstAx = WFair + Constrains + 
       
    12 
       
    13 constdefs
       
    14    Ensures :: "[i,i] => i"            (infixl 60)
       
    15     "A Ensures B == {F:program. F : (reachable(F) Int A) ensures B &
       
    16 		                A:condition & B:condition}"
       
    17 
       
    18    LeadsTo :: "[i, i] => i"            (infixl 60)
       
    19     "A LeadsTo B == {F:program. F:(reachable(F) Int A) leadsTo B &
       
    20 		                A:condition & B:condition}"
       
    21 
       
    22 syntax (xsymbols)
       
    23   "op LeadsTo" :: "[i, i] => i" (infixl " \\<longmapsto>w " 60)
       
    24 
       
    25 end