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