clarified NEWS: document_files are officially required since Isabelle2014, but the absence was tolerated as legacy feature;
(* 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