author | wenzelm |
Sun, 30 Jan 2011 13:02:18 +0100 | |
changeset 41648 | 6d736d983d5c |
parent 32632 | 8ae912371831 |
child 58889 | 5b7a9633cfa8 |
permissions | -rw-r--r-- |
32632 | 1 |
(* Author: Lawrence C Paulson, Cambridge University Computer Laboratory |
1944 | 2 |
Copyright 1996 University of Cambridge |
3 |
*) |
|
4 |
||
32632 | 5 |
header {* Smartcard protocols: rely on conventional Message and on new EventSC and Smartcard *} |
1944 | 6 |
|
32632 | 7 |
theory Auth_Smartcard |
8 |
imports |
|
9 |
"ShoupRubin" |
|
10 |
"ShoupRubinBella" |
|
11 |
begin |
|
14145
2e31b8cc8788
ZhouGollmann: new example (fair non-repudiation protocol)
paulson
parents:
13922
diff
changeset
|
12 |
|
32632 | 13 |
end |