Theory SecureSystems
theory SecureSystems
imports "../../SystemSpecification/StateEventSystems"
"../../SecuritySpecification/InformationFlowProperties"
begin
locale SecureESIFP =
fixes ES :: "'e ES_rec"
and IFP :: "'e IFP_type"
assumes validES: "ES_valid ES"
and validIFPES: "IFP_valid E⇘ES⇙ IFP"
context SecureESIFP
begin
definition ES_sat_IFP :: "bool"
where
"ES_sat_IFP ≡ IFPIsSatisfied IFP Tr⇘ES⇙"
end
locale SecureSESIFP =
fixes SES :: "('s, 'e) SES_rec"
and IFP :: "'e IFP_type"
assumes validSES: "SES_valid SES"
and validIFPSES: "IFP_valid E⇘SES⇙ IFP"
sublocale SecureSESIFP ⊆ SecureESIFP "induceES SES" "IFP"
by (unfold_locales, rule induceES_yields_ES, rule validSES,
simp add: induceES_def, rule validIFPSES)
context SecureSESIFP
begin
abbreviation SES_sat_IFP
where
"SES_sat_IFP ≡ ES_sat_IFP"
end
end