src/HOL/Auth/TLS.thy
changeset 37936 1e4c5015a72e
parent 35702 fb7a386a15cb
child 41413 64cd30d6b0b8
equal deleted inserted replaced
37935:7551769de556 37936:1e4c5015a72e
     1 (*  Title:      HOL/Auth/TLS
     1 (*  Title:      HOL/Auth/TLS.thy
     2     ID:         $Id$
       
     3     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     2     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     4     Copyright   1997  University of Cambridge
     3     Copyright   1997  University of Cambridge
     5 
     4 
     6 Inductive relation "tls" for the TLS (Transport Layer Security) protocol.
     5 Inductive relation "tls" for the TLS (Transport Layer Security) protocol.
     7 This protocol is essentially the same as SSL 3.0.
     6 This protocol is essentially the same as SSL 3.0.