proper support for "isabelle update -D DIR": avoid accidental exclusion of select_dirs (amending e5dafe9e120f);
(* Title: HOL/SET_Protocol/SET_Protocol.thy
Author: Lawrence C Paulson, Cambridge University Computer Laboratory
Copyright 2003 University of Cambridge
Root file for the SET protocol proofs.
*)
theory SET_Protocol
imports Cardholder_Registration Merchant_Registration Purchase
begin
end