Theory System_Specification
section ‹The CoSMeDis single node specification›
text ‹This is the specification of a CoSMeDis node, as described
in Sections II and IV.B of \<^cite>‹"cosmedis-SandP2017"›.
NB: What that paper refers to as "nodes" are referred in this formalization
as "APIs".
A CoSMeDis node extends CoSMed \<^cite>‹"cosmed-itp2016" and "cosmed-jar2018" and "cosmed-AFP"›
with inter-node communication actions.
›
theory System_Specification
imports
Prelim
"Bounded_Deducibility_Security.IO_Automaton"
begin
text ‹An aspect not handled in this specification is the uniqueness of the node IDs. These
are assumed to be handled externally as follows: a node ID is an URI, and therefore is unique.›
declare List.insert[simp]
subsection ‹The state›