src/HOL/SET-Protocol/EventSET.thy
changeset 16417 9bc16273c2d4
parent 14218 db95d1c2f51b
child 21588 cd0dc678a205
equal deleted inserted replaced
16416:6061ae1f90f2 16417:9bc16273c2d4
     3     Authors:     Giampaolo Bella, Fabio Massacci, Lawrence C Paulson
     3     Authors:     Giampaolo Bella, Fabio Massacci, Lawrence C Paulson
     4 *)
     4 *)
     5 
     5 
     6 header{*Theory of Events for SET*}
     6 header{*Theory of Events for SET*}
     7 
     7 
     8 theory EventSET = MessageSET:
     8 theory EventSET imports MessageSET begin
     9 
     9 
    10 text{*The Root Certification Authority*}
    10 text{*The Root Certification Authority*}
    11 syntax        RCA :: agent
    11 syntax        RCA :: agent
    12 translations "RCA" == "CA 0"
    12 translations "RCA" == "CA 0"
    13 
    13