| author | wenzelm | 
| Fri, 08 Apr 2016 20:52:40 +0200 | |
| changeset 62914 | 930a30c1a9af | 
| parent 61830 | 4f5ab843cf5b | 
| child 65538 | a39ef48fbee0 | 
| permissions | -rw-r--r-- | 
| 32632 | 1  | 
(* Author: Lawrence C Paulson, Cambridge University Computer Laboratory  | 
| 1944 | 2  | 
Copyright 1996 University of Cambridge  | 
3  | 
*)  | 
|
4  | 
||
| 61830 | 5  | 
section \<open>Blanqui's "guard" concept: protocol-independent secrecy\<close>  | 
| 1944 | 6  | 
|
| 32632 | 7  | 
theory Auth_Guard_Shared  | 
8  | 
imports  | 
|
9  | 
"Guard_OtwayRees"  | 
|
10  | 
"Guard_Yahalom"  | 
|
11  | 
begin  | 
|
| 
14145
 
2e31b8cc8788
ZhouGollmann: new example (fair non-repudiation protocol)
 
paulson 
parents: 
13922 
diff
changeset
 | 
12  | 
|
| 32632 | 13  | 
end  |