Theory SINVAR_CommunicationPartners
theory SINVAR_CommunicationPartners
imports "../TopoS_Helper"
begin
subsection ‹SecurityInvariant CommunicationPartners›
text‹
Idea of this securityinvariant:
Only some nodes can communicate with Master nodes.
It constrains who may access master nodes, Master nodes can access the world (except other prohibited master nodes).
A node configured as Master has a list of nodes that can access it.
Also, in order to be able to access a Master node, the sender must be denoted as a node we Care about.
By default, all nodes are set to DontCare, thus they cannot access Master nodes. But they can access
all other DontCare nodes and Care nodes.
TL;DR: An access control list determines who can access a master node.
›