src/HOL/Auth/TLS.thy
changeset 16417 9bc16273c2d4
parent 14126 28824746d046
child 20768 1d478c2d621f
     1.1 --- a/src/HOL/Auth/TLS.thy	Fri Jun 17 11:35:35 2005 +0200
     1.2 +++ b/src/HOL/Auth/TLS.thy	Fri Jun 17 16:12:49 2005 +0200
     1.3 @@ -41,7 +41,7 @@
     1.4  
     1.5  header{*The TLS Protocol: Transport Layer Security*}
     1.6  
     1.7 -theory TLS = Public + NatPair:
     1.8 +theory TLS imports Public NatPair begin
     1.9  
    1.10  constdefs
    1.11    certificate      :: "[agent,key] => msg"