tuned target inheritance bookkeeping: ancestry is always fully maintained at current entry using canonical merge;
n. b. merging of bidirectional dependencies results in effective join of involved nodes: no termination problem since ancestry is always kept explicitly normalized
(* 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