discontinued somewhat pointless operation: Conjunction.intr_balanced / Conjunction.elim_balanced with single hyp performs better (e.g. see AFP/351b7b576892);
(* 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