src/HOL/Auth/Guard/GuardK.thy
changeset 16417 9bc16273c2d4
parent 15236 f289e8ba2bb3
child 17087 0abf74bdf712
equal deleted inserted replaced
16416:6061ae1f90f2 16417:9bc16273c2d4
    14 Cambridge CB3 0FD, United Kingdom
    14 Cambridge CB3 0FD, United Kingdom
    15 ******************************************************************************)
    15 ******************************************************************************)
    16 
    16 
    17 header{*protocol-independent confidentiality theorem on keys*}
    17 header{*protocol-independent confidentiality theorem on keys*}
    18 
    18 
    19 theory GuardK = Analz + Extensions:
    19 theory GuardK imports Analz Extensions begin
    20 
    20 
    21 (******************************************************************************
    21 (******************************************************************************
    22 messages where all the occurrences of Key n are
    22 messages where all the occurrences of Key n are
    23 in a sub-message of the form Crypt (invKey K) X with K:Ks
    23 in a sub-message of the form Crypt (invKey K) X with K:Ks
    24 ******************************************************************************)
    24 ******************************************************************************)