| author | wenzelm |
| Sat, 18 Jan 2025 11:03:18 +0100 | |
| changeset 81904 | aa28d82d6b66 |
| parent 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>Smartcard protocols: rely on conventional Message and on new EventSC and Smartcard\<close> |
| 1944 | 6 |
|
| 32632 | 7 |
theory Auth_Smartcard |
8 |
imports |
|
| 65538 | 9 |
ShoupRubin |
10 |
ShoupRubinBella |
|
| 32632 | 11 |
begin |
|
14145
2e31b8cc8788
ZhouGollmann: new example (fair non-repudiation protocol)
paulson
parents:
13922
diff
changeset
|
12 |
|
| 32632 | 13 |
end |