Theory SINVAR_SecGwExt
theory SINVAR_SecGwExt
imports "../TopoS_Helper"
begin
subsection ‹SecurityInvariant PolEnforcePointExtended›
text ‹A PolEnforcePoint is an application-level central policy enforcement point.
Legacy note: The old verions called it a SecurityGateway.
Hosts may belong to a certain domain.
Sometimes, a pattern where intra-domain communication between domain members must be approved by a central instance is required.
We call such a central instance PolEnforcePoint and present a template for this architecture.
Five host roles are distinguished:.
A PolEnforcePoint, aPolEnforcePointIN which accessible from the outside, a DomainMember,
a less-restricted AccessibleMember which is accessible from the outside world,
and a default value Unassigned that reflects none of these roles.›