src/ZF/UNITY/SubstAx.thy
changeset 69587 53982d5ec0bb
parent 63120 629a4c5e953e
child 69593 3dda49e08b9d
equal deleted inserted replaced
69586:9171d1ce5a35 69587:53982d5ec0bb
    11 imports WFair Constrains
    11 imports WFair Constrains
    12 begin
    12 begin
    13 
    13 
    14 definition
    14 definition
    15   (* The definitions below are not `conventional', but yield simpler rules *)
    15   (* The definitions below are not `conventional', but yield simpler rules *)
    16   Ensures :: "[i,i] => i"            (infixl "Ensures" 60)  where
    16   Ensures :: "[i,i] => i"            (infixl \<open>Ensures\<close> 60)  where
    17   "A Ensures B == {F \<in> program. F \<in> (reachable(F) \<inter> A) ensures (reachable(F) \<inter> B) }"
    17   "A Ensures B == {F \<in> program. F \<in> (reachable(F) \<inter> A) ensures (reachable(F) \<inter> B) }"
    18 
    18 
    19 definition
    19 definition
    20   LeadsTo :: "[i, i] => i"            (infixl "\<longmapsto>w" 60)  where
    20   LeadsTo :: "[i, i] => i"            (infixl \<open>\<longmapsto>w\<close> 60)  where
    21   "A \<longmapsto>w B == {F \<in> program. F:(reachable(F) \<inter> A) \<longmapsto> (reachable(F) \<inter> B)}"
    21   "A \<longmapsto>w B == {F \<in> program. F:(reachable(F) \<inter> A) \<longmapsto> (reachable(F) \<inter> B)}"
    22 
    22 
    23 
    23 
    24 (*Resembles the previous definition of LeadsTo*)
    24 (*Resembles the previous definition of LeadsTo*)
    25 
    25