src/ZF/UNITY/Constrains.thy
changeset 69587 53982d5ec0bb
parent 68233 5e0e9376b2b0
child 69593 3dda49e08b9d
equal deleted inserted replaced
69586:9171d1ce5a35 69587:53982d5ec0bb
    38 
    38 
    39   type_intros UnI1 UnI2 fieldI2 UN_I
    39   type_intros UnI1 UnI2 fieldI2 UN_I
    40 
    40 
    41   
    41   
    42 definition
    42 definition
    43   Constrains :: "[i,i] => i"  (infixl "Co" 60)  where
    43   Constrains :: "[i,i] => i"  (infixl \<open>Co\<close> 60)  where
    44   "A Co B == {F:program. F:(reachable(F) \<inter> A) co B}"
    44   "A Co B == {F:program. F:(reachable(F) \<inter> A) co B}"
    45 
    45 
    46 definition
    46 definition
    47   op_Unless  :: "[i, i] => i"  (infixl "Unless" 60)  where
    47   op_Unless  :: "[i, i] => i"  (infixl \<open>Unless\<close> 60)  where
    48   "A Unless B == (A-B) Co (A \<union> B)"
    48   "A Unless B == (A-B) Co (A \<union> B)"
    49 
    49 
    50 definition
    50 definition
    51   Stable     :: "i => i"  where
    51   Stable     :: "i => i"  where
    52   "Stable(A) == A Co A"
    52   "Stable(A) == A Co A"