equal
deleted
inserted
replaced
1 (* Title: HOL/Auth/Yahalom2.thy |
1 (* Title: HOL/Auth/Yahalom2.thy |
2 Author: Lawrence C Paulson, Cambridge University Computer Laboratory |
2 Author: Lawrence C Paulson, Cambridge University Computer Laboratory |
3 Copyright 1996 University of Cambridge |
3 Copyright 1996 University of Cambridge |
4 *) |
4 *) |
5 |
5 |
6 header{*The Yahalom Protocol, Variant 2*} |
6 section{*The Yahalom Protocol, Variant 2*} |
7 |
7 |
8 theory Yahalom2 imports Public begin |
8 theory Yahalom2 imports Public begin |
9 |
9 |
10 text{* |
10 text{* |
11 This version trades encryption of NB for additional explicitness in YM3. |
11 This version trades encryption of NB for additional explicitness in YM3. |