src/HOL/Auth/Guard/NS_Public.thy
changeset 16417 9bc16273c2d4
parent 13508 890d736b93a5
equal deleted inserted replaced
16416:6061ae1f90f2 16417:9bc16273c2d4
    11 Cambridge CB3 0FD, United Kingdom
    11 Cambridge CB3 0FD, United Kingdom
    12 ******************************************************************************)
    12 ******************************************************************************)
    13 
    13 
    14 header{*Needham-Schroeder-Lowe Public-Key Protocol*}
    14 header{*Needham-Schroeder-Lowe Public-Key Protocol*}
    15 
    15 
    16 theory NS_Public = Guard_Public:
    16 theory NS_Public imports Guard_Public begin
    17 
    17 
    18 subsection{*messages used in the protocol*}
    18 subsection{*messages used in the protocol*}
    19 
    19 
    20 syntax ns1 :: "agent => agent => nat => event"
    20 syntax ns1 :: "agent => agent => nat => event"
    21 
    21