Theory Aczel_Sequences
theory Aczel_Sequences
imports
HOL_Basis
begin
section‹ Terminated Aczel sequences\label{sec:aczel_sequences} ›
text‹
We model a ∗‹behavior› of a system as a non-empty finite or infinite sequence of the form
‹s⇩0 -a⇩1→ s⇩1 -a⇩2→ … (→ v)?› where ‹s⇩i› is a state, ‹a⇩i› an agent and ‹v› a return value for
finite sequences (see \S\ref{sec:tls}). A ∗‹trace› is a finite sequence
‹s⇩0 -a⇩1→ s⇩1 -a⇩2→ … -a⇩n→ s⇩n → v› for ‹n ≥ 0› with optional return value ‹v› (see
\S\ref{sec:safety_logic}). States, agents and return values are of arbitrary type.
›
subsection‹ Traces\label{sec:aczel_sequences-traces} ›
setup ‹Sign.mandatory_path "trace"›