| author | wenzelm | 
| Fri, 23 Nov 2018 21:47:35 +0100 | |
| changeset 69335 | 76c8beaf3bab | 
| parent 39769 | 5bcf4253d579 | 
| permissions | -rw-r--r-- | 
| 39769 | 1 | (* Title: HOL/SET_Protocol/SET_Protocol.thy | 
| 2 | Author: Lawrence C Paulson, Cambridge University Computer Laboratory | |
| 3 | Copyright 2003 University of Cambridge | |
| 4 | ||
| 5 | Root file for the SET protocol proofs. | |
| 6 | *) | |
| 7 | ||
| 8 | theory SET_Protocol | |
| 9 | imports Cardholder_Registration Merchant_Registration Purchase | |
| 10 | begin | |
| 11 | ||
| 12 | end |