Theory Infrastructure
section ‹Infrastructures›
text ‹The Isabelle Infrastructure framework supports the representation of infrastructures
as graphs with actors and policies attached to nodes. These infrastructures
are the {\it states} of the Kripke structure.
The transition between states is triggered by non-parametrized
actions @{text ‹get, move, eval, put›} executed by actors.
Actors are given by an abstract type @{text ‹actor›} and a function
@{text ‹Actor›} that creates elements of that type from identities
(of type @{text ‹string›}). Policies are given by pairs of predicates
(conditions) and sets of (enabled) actions.›
subsection ‹Actors, actions, and data labels›
theory Infrastructure
imports AT
begin