Theory Trace
theory Trace
imports Basis
begin
declare Let_def[simp] if_split_asm[split]
section‹A trace based model›
text‹The only clumsy aspect of the state based model is ‹safe›: we use a state component to record if the sequence of events
that lead to a state satisfies some property. That is, we simulate a
condition on traces via the state. Unsurprisingly, it is not trivial
to convince oneself that ‹safe› really has the informal meaning
set out at the beginning of subsection~\ref{sec:formalizing-safety}.
Hence we now describe an alternative, purely trace based model,
similar to Paulson's inductive protocol model~\<^cite>‹"Paulson-JCS98"›.
The events are:
›