Theory Paper_Aut
theory Paper_Aut
imports "../Observation_Setup" Paper_Value_Setup "Bounded_Deducibility_Security.Compositional_Reasoning"
begin
subsection ‹Confidentiality protection from non-authors›
text ‹We verify the following property:
\ \\
A group of users UIDs
learns nothing about the various uploads of a paper PID
except for the last (most recent) upload
unless/until a user in UIDs becomes an author of the paper.
\ \\
›
fun T :: "(state,act,out) trans ⇒ bool" where
"T (Trans _ _ ou s') = (∃ uid ∈ UIDs. isAUT s' uid PID)"
declare T.simps [simp del]
definition B :: "value list ⇒ value list ⇒ bool" where
"B vl vl1 ≡ vl ≠ [] ∧ vl1 ≠ [] ∧ last vl = last vl1"