Theory Decision_NCPC_Aut
theory Decision_NCPC_Aut
imports "../Observation_Setup" Decision_Value_Setup "Bounded_Deducibility_Security.Compositional_Reasoning"
begin
subsection ‹Confidentiality protection from users who are not PC members or authors of the paper›
text ‹We verify the following property:
A group of users UIDs learn
nothing about the various updates of a paper's decision
(save for the non-existence of any update)
unless/until one of the following happens:
\begin{itemize}
\item a user in UIDs becomes a PC member in the paper's conference having no conflict with that paper
and the conference moves to the discussion phase,
or
\item a user in UIDs becomes a PC member in the paper's conference or an author of the paper,
and the conference moves to the notification phase
\end{itemize}
›
fun T :: "(state,act,out) trans ⇒ bool" where
"T (Trans _ _ ou s') =
(∃ uid ∈ UIDs.
(∃ cid. PID ∈∈ paperIDs s' cid ∧ isPC s' cid uid ∧
pref s' uid PID ≠ Conflict ∧ phase s' cid ≥ disPH)
∨
(∃ cid. PID ∈∈ paperIDs s' cid ∧ isPC s' cid uid ∧ phase s' cid ≥ notifPH)
∨
isAUT s' uid PID ∧ (∃ cid. PID ∈∈ paperIDs s' cid ∧ phase s' cid ≥ notifPH)
)"
declare T.simps [simp del]
definition B :: "value list ⇒ value list ⇒ bool" where
"B vl vl1 ≡ vl ≠ []"