src/HOL/UNITY/Detects.thy
changeset 13798 4c1a53627500
parent 13785 e2fcd88be55d
child 13805 3786b2fd6808
equal deleted inserted replaced
13797:baefae13ad37 13798:4c1a53627500
     3     Author:     Tanja Vos, Cambridge University Computer Laboratory
     3     Author:     Tanja Vos, Cambridge University Computer Laboratory
     4     Copyright   2000  University of Cambridge
     4     Copyright   2000  University of Cambridge
     5 
     5 
     6 Detects definition (Section 3.8 of Chandy & Misra) using LeadsTo
     6 Detects definition (Section 3.8 of Chandy & Misra) using LeadsTo
     7 *)
     7 *)
       
     8 
       
     9 header{*The Detects Relation*}
     8 
    10 
     9 theory Detects = FP + SubstAx:
    11 theory Detects = FP + SubstAx:
    10 
    12 
    11 consts
    13 consts
    12    op_Detects  :: "['a set, 'a set] => 'a program set"  (infixl "Detects" 60)
    14    op_Detects  :: "['a set, 'a set] => 'a program set"  (infixl "Detects" 60)