src/HOL/Auth/Smartcard/EventSC.thy
changeset 21404 eb85850d3eb7
parent 20768 1d478c2d621f
child 26302 68b073052e8c
equal deleted inserted replaced
21403:dd58f13a8eb4 21404:eb85850d3eb7
    23  stolen    :: "card set" (* stolen smart cards *)
    23  stolen    :: "card set" (* stolen smart cards *)
    24  cloned  :: "card set"   (* cloned smart cards*)
    24  cloned  :: "card set"   (* cloned smart cards*)
    25  secureM :: "bool"(*assumption of secure means between agents and their cards*)
    25  secureM :: "bool"(*assumption of secure means between agents and their cards*)
    26 
    26 
    27 abbreviation
    27 abbreviation
    28   insecureM :: bool (*certain protocols make no assumption of secure means*)
    28   insecureM :: bool where (*certain protocols make no assumption of secure means*)
    29   "insecureM == \<not>secureM"
    29   "insecureM == \<not>secureM"
    30 
    30 
    31 
    31 
    32 text{*Spy has access to his own key for spoof messages, but Server is secure*}
    32 text{*Spy has access to his own key for spoof messages, but Server is secure*}
    33 specification (bad)
    33 specification (bad)