Skip to content
Snippets Groups Projects
Commit 78d3d724 authored by Robbert Krebbers's avatar Robbert Krebbers
Browse files

Merge branch 'robbert/adequacy' into 'master'

A strong adequacy statement to rule them all

See merge request iris/iris!258
parents 243d8707 d857cb91
No related branches found
No related tags found
No related merge requests found
...@@ -14,8 +14,6 @@ Changes in the theory of Iris itself: ...@@ -14,8 +14,6 @@ Changes in the theory of Iris itself:
* Add weakest preconditions for total program correctness. * Add weakest preconditions for total program correctness.
* "(Potentially) stuck" weakest preconditions and the "plainly modality" are no * "(Potentially) stuck" weakest preconditions and the "plainly modality" are no
longer considered experimental. longer considered experimental.
* The adequacy statement for weakest preconditions now also involves the
final state.
* Add the notion of an "observation" to the language interface, so that * Add the notion of an "observation" to the language interface, so that
every reduction step can optionally be marked with an event, and an execution every reduction step can optionally be marked with an event, and an execution
trace has a matching list of events. Change WP so that it is told the entire trace has a matching list of events. Change WP so that it is told the entire
...@@ -28,8 +26,10 @@ Changes in the theory of Iris itself: ...@@ -28,8 +26,10 @@ Changes in the theory of Iris itself:
* Extend the state interpretation with a natural number that keeps track of * Extend the state interpretation with a natural number that keeps track of
the number of forked-off threads, and have a global fixed proposition that the number of forked-off threads, and have a global fixed proposition that
describes the postcondition of each forked-off thread (instead of it being describes the postcondition of each forked-off thread (instead of it being
`True`). Additionally, there is a stronger variant of the adequacy theorem `True`).
that allows to make use of the postconditions of the forked-off threads. * A stronger adequacy statement for weakest preconditions that involves
the final state, the post-condition of forked-off threads, and also applies if
the main-thread has not terminated.
* The user-chosen functor used to instantiate the Iris logic now goes from * The user-chosen functor used to instantiate the Iris logic now goes from
COFEs to Cameras (it was OFEs to Cameras). COFEs to Cameras (it was OFEs to Cameras).
......
...@@ -250,48 +250,77 @@ This basically just copies the second branch (the non-value case) of the definit ...@@ -250,48 +250,77 @@ This basically just copies the second branch (the non-value case) of the definit
\paragraph{Adequacy of weakest precondition.} \paragraph{Adequacy of weakest precondition.}
\newcommand\traceprop{\Sigma}
The purpose of the adequacy statement is to show that our notion of weakest preconditions is \emph{realistic} in the sense that it actually has anything to do with the actual behavior of the program. The purpose of the adequacy statement is to show that our notion of weakest preconditions is \emph{realistic} in the sense that it actually has anything to do with the actual behavior of the program.
There are two properties we are looking for: First of all, the postcondition should reflect actual properties of the values the program can terminate with. The most general form of the adequacy statement is about proving properties of arbitrary program executions.
Second, a proof of a weakest precondition with any postcondition should imply that the program is \emph{safe}, \ie that it does not get stuck. That is, the goal is to prove a statement of the form
\[
\begin{defn}[Adequacy] \All \expr_0, \state_0, \vec\obs, \tpool_1, \state_1. ([\expr_0], \state_0) \tpsteps[\vec\obs] (\tpool_1, \state_1) \Ra (\expr_0, \state_0, \vec\obs, \tpool_1, \state_1) \in \traceprop
A program $\expr$ in some initial state $\state$ is \emph{adequate} for stuckness $\stuckness$ and a set $V \subseteq \Val \times \State$ of legal return-value-final-state combinations (written $\expr, \state \vDash_\stuckness V$) if for all $\tpool', \state'$ such that $([\expr], \state) \tpsteps[\vec\obs] (\tpool', \state')$ we have \]
\begin{enumerate} for some \emph{meta-level} relation $\traceprop$ characterizing the ``trace property'' we are interested in.
\item Safety: If $\stuckness = \NotStuck$, then for any $\expr' \in \tpool'$ we have that either $\expr'$ is a
value, or \(\red(\expr'_i,\state')\): To state the adequacy theorem, we need a way to talk about $\traceprop$ inside Iris.
\[ \stuckness = \NotStuck \Ra \All\expr'\in\tpool'. \toval(\expr') \neq \bot \lor \red(\expr', \state') \] To this end, we assume that the signature $\Sig$ contains some predicate $\hat{\traceprop}$:
Notice that this is stronger than saying that the thread pool can reduce; we actually assert that \emph{every} non-finished thread can take a step. \[ \hat{\traceprop} : \Expr \times \State \times \List(\Obs) \times \List(\Expr) \times \State \to \Prop \in \SigFn \]
\item Legal return value: If $\tpool'_1$ (the main thread) is a value $\val'$, then $\val' \in V$: Furthermore, we assume that the \emph{interpretation} $\Sem{\hat{\traceprop}}$ of $\hat{\traceprop}$ reflects $\traceprop$ (also see \Sref{sec:model}):
\[ \All \val',\tpool''. \tpool' = [\val'] \dplus \tpool'' \Ra (\val',\state') \in V \]
\end{enumerate}
\end{defn}
To express the adequacy statement for functional correctness, we assume that the signature $\Sig$ adds a predicate $\pred$ to the logic:
\[ \pred : \Val \times \State \to \Prop \in \SigFn \]
Furthermore, we assume that the \emph{interpretation} $\Sem\pred$ of $\pred$ reflects some set $V$ of legal return values and final states into the logic (also see \Sref{sec:model}):
\[\begin{array}{rMcMl} \[\begin{array}{rMcMl}
\Sem\pred &:& \Sem{\Val\times\State\,} \nfn \Sem\Prop \\ \Sem{\hat{\traceprop}} &:& \Sem{\Expr \times \State \times \List(\Obs) \times \List(\Expr) \times \State\,} \nfn \Sem\Prop \\
\Sem\pred &\eqdef& \Lam (\val,\state). \Lam \any. \setComp{n}{(v,\state) \in V} \Sem{\hat{\traceprop}} &\eqdef& \Lam (\expr_0, \state_0, \vec\obs, \tpool_1, \state_1). \Lam \any. \setComp{n}{(\expr_0, \state_0, \vec\obs, \tpool_1, \state_1) \in \traceprop}
\end{array}\] \end{array}\]
The signature can of course state arbitrary additional properties of $\pred$, as long as they are proven sound. The signature can of course state arbitrary additional properties of $\hat{\traceprop}$, as long as they are proven sound.
The adequacy statement now reads as follows: The adequacy statement now reads as follows:
\begin{align*} \begin{align*}
&\All \mask, \expr, \state. &\All \expr_0, \state_0, \vec\obs, \tpool_1, \state_1.\\
\\&( \TRUE \proves \All\vec\obs. \pvs[\mask] \Exists \stateinterp, \pred_F. \stateinterp(\state,\vec\obs,0) * \wpre[\stateinterp;\pred_F]{\expr}[\stuckness;\mask]{x.\; \All \state, m. \stateinterp(\state', (), m) \vsW[\top][\emptyset] \pred(x,\state')}) \Ra &( \TRUE \proves \pvs[\top] \Exists \stuckness, \stateinterp, \pred_F, \pred. {}\\
\\&\expr, \state \vDash_\stuckness V &\quad\stateinterp(\state_0,\vec\obs,0) * \wpre[\stateinterp;\pred_F]{\expr_0}[\stuckness;\top]{x.\; \pred(x)} * {}\\
&\quad(\All \expr_1, \tpool_1'. \tpool_1 = [\expr_1] \dplus \tpool_1' \wand {}\\
&\quad\quad (s = \NotStuck \Ra \All \expr \in \tpool_1. \toval(\expr) \neq \bot \lor \red(\expr, \state_1) ) \wand {}\\
&\quad\quad \stateinterp(\state_1, (), |\tpool_1'|) \wand{}\\
&\quad\quad (\toval(\expr_1) \ne \bot \wand \pred(\toval(\expr_1))) \wand{}\\
&\quad\quad (\Sep[\expr \in \tpool_1'] \toval(\expr) \ne \bot \wand \pred_F(\toval(\expr))) \wand{}\\
&\quad\quad \pvs[\top,\emptyset] \hat{\traceprop}(\expr_0, \state_0, \vec\obs, \tpool_1, \state_1) \\
&\quad ) \Ra{}\\
&([\expr_0], \state_0) \tpsteps[\vec\obs] (\tpool_1, \state_1) \Ra (\expr_0, \state_0, \vec\obs, \tpool_1, \state_1) \in \traceprop
\end{align*} \end{align*}
Notice that the state invariant $S$ used by the weakest precondition is chosen \emph{after} doing a fancy update, which allows it to depend on the names of ghost variables that are picked in that initial fancy update. In other words, to show that $\traceprop$ holds for all possible executions of the program, we have to prove an entailment in Iris that, starting from the empty context, proves that the initial state interpretation holds, proves a weakest precondition, \emph{and} proves that $\hat{\traceprop}$ holds under the following assumptions:
Also, notice that the proof of $\expr$ must be performed with a universally quantified list of observations $\vec\obs$, but the \emph{entire} list is known to the proof from the beginning. \begin{itemize}
\item The final thread-pool $\tpool_1$ contains the final state of the main thread $\expr_1$, and any number of additional threads in $\tpool_1'$.
\item If this is a stuck-free weakest precondition, then all threads in the final thread-pool are either values or are reducible in the final state $\state_1$.
\item The state interpretation holds for the final state.
\item If the main thread reduced to a value, the post-condition $\pred$ of the weakest precondition holds for that value.
\item If any other thread reduced to a value, the forked-thread post-condition $\pred_F$ holds for that value.
\end{itemize}
Notice also that the adequacy statement quantifies over the program trace only once, so it can be easily specialized to, say, some particular initial state $\state_0$.
This lets us show properties that only hold for some executions.
Furthermore, the state invariant $S$ used by the weakest precondition is chosen \emph{after} doing a fancy update, which allows it to depend on the names of ghost variables that are picked in that initial fancy update.
As an example for how to use this adequacy theorem, let us say we wanted to prove that a program $\expr_0$ for which we derived a $\NotStuck$ weakest-precondition cannot get stuck.
We would pick
\[
\traceprop(\expr_0, \state_0, \vec\obs, \tpool_1, \state_1) \eqdef \All \expr \in \tpool_1. \toval(\expr) \neq \bot \lor \red(\expr, \state_1)
\]
and we would show the following in Iris:
\[
\TRUE \proves \All \state_0, \vec\obs. \pvs[\top] \Exists \stateinterp, \pred_F, \pred. \stateinterp(\state_0,\vec\obs,0) * \wpre[\stateinterp;\pred_F]{\expr_0}[\NotStuck;\top]{x.\; \pred(x)}
\]
The adequacy theorem would then give us:
\[
\All \state_0, \vec\obs, \tpool_1, \state_1. ([\expr_0], \state_0) \tpsteps[\vec\obs] (\tpool_1, \state_1) \Ra \All \expr \in \tpool_1. \toval(\expr) \neq \bot \lor \red(\expr, \state_1)
\]
The following variant of adequacy also allows exploiting the second parameter of $\stateinterp$, the number of threads, but only applies when \emph{all} threads have reduced to a value: Similarly, if we wanted to show that the final value of the main thread is always in some set $V \subseteq \Val$, we could pick
\[
\traceprop(\expr_0, \state_0, \vec\obs, \tpool_1, \state_1) \eqdef \All\val_1, \tpool_1'. \tpool_1 = [\ofval(\val_1)] \dplus \tpool_1' \Ra \val_1 \in \Val
\]
and then we could derive the following from the main adequacy theorem:
\begin{align*} \begin{align*}
&\All \mask, \expr, \state, \vec\obs, \val, \vec\val, \state'. &(\TRUE \proves \All\state_0, \vec\obs. \pvs[\top] \Exists \stuckness, \stateinterp, \pred_F. \stateinterp(\state_0,\vec\obs,0) * \wpre[\stateinterp;\pred_F]{\expr_0}[\stuckness;\top]{x.\; x \in V}) \Ra{}\\
\\&( \TRUE \proves \pvs[\mask] \Exists \stateinterp, \pred_F. \stateinterp(\state,\vec\obs,0) * \wpre[\stateinterp;\pred_F]{\expr}[\stuckness;\mask]% &\All \state_0, \vec\obs, \val_1, \tpool_1, \state_1. ([\expr_0], \state_0) \tpsteps[\vec\obs] ([\ofval(\val_1)] \dplus \tpool_1, \state_1) \Ra \val_1 \in V
{x.\; \stateinterp(\state',(),|\vec\val|) * \Sep_{y \in \vec\val} \pred_F(y) \vsW[\top][\emptyset] \pred(x,\state')}) \Ra
\\&([\expr], \state) \tpsteps[\vec\obs] (\val :: \vec\val, \state') \Ra
\\&(\val,\state') \in V
\end{align*} \end{align*}
\paragraph{Hoare triples.} \paragraph{Hoare triples.}
It turns out that weakest precondition is actually quite convenient to work with, in particular when performing these proofs in Coq. It turns out that weakest precondition is actually quite convenient to work with, in particular when performing these proofs in Coq.
Still, for a more traditional presentation, we can easily derive the notion of a Hoare triple: Still, for a more traditional presentation, we can easily derive the notion of a Hoare triple:
......
...@@ -22,7 +22,8 @@ Proof. ...@@ -22,7 +22,8 @@ Proof.
intros Hwp; eapply (wp_adequacy _ _); iIntros (??) "". intros Hwp; eapply (wp_adequacy _ _); iIntros (??) "".
iMod (gen_heap_init σ.(heap)) as (?) "Hh". iMod (gen_heap_init σ.(heap)) as (?) "Hh".
iMod (proph_map_init κs σ.(used_proph_id)) as (?) "Hp". iMod (proph_map_init κs σ.(used_proph_id)) as (?) "Hp".
iModIntro. iModIntro. iExists
iExists (λ σ κs, (gen_heap_ctx σ.(heap) proph_map_ctx κs σ.(used_proph_id))%I). iFrame. (λ σ κs, (gen_heap_ctx σ.(heap) proph_map_ctx κs σ.(used_proph_id))%I),
iApply (Hwp (HeapG _ _ _ _)). (λ _, True%I).
iFrame. iApply (Hwp (HeapG _ _ _ _)).
Qed. Qed.
From stdpp Require Import namespaces.
From iris.program_logic Require Export weakestpre. From iris.program_logic Require Export weakestpre.
From iris.algebra Require Import gmap auth agree gset coPset. From iris.algebra Require Import gmap auth agree gset coPset.
From iris.base_logic.lib Require Import wsat. From iris.base_logic.lib Require Import wsat.
...@@ -6,32 +5,8 @@ From iris.proofmode Require Import tactics. ...@@ -6,32 +5,8 @@ From iris.proofmode Require Import tactics.
Set Default Proof Using "Type". Set Default Proof Using "Type".
Import uPred. Import uPred.
(* Program logic adequacy *) (** This file contains the adequacy statements of the Iris program logic. First
Record adequate {Λ} (s : stuckness) (e1 : expr Λ) (σ1 : state Λ) we prove a number of auxilary results. *)
(φ : val Λ state Λ Prop) := {
adequate_result t2 σ2 v2 :
rtc erased_step ([e1], σ1) (of_val v2 :: t2, σ2) φ v2 σ2;
adequate_not_stuck t2 σ2 e2 :
s = NotStuck
rtc erased_step ([e1], σ1) (t2, σ2)
e2 t2 (is_Some (to_val e2) reducible e2 σ2)
}.
Theorem adequate_tp_safe {Λ} (e1 : expr Λ) t2 σ1 σ2 φ :
adequate NotStuck e1 σ1 φ
rtc erased_step ([e1], σ1) (t2, σ2)
Forall (λ e, is_Some (to_val e)) t2 κ t3 σ3, step (t2, σ2) κ (t3, σ3).
Proof.
intros Had ?.
destruct (decide (Forall (λ e, is_Some (to_val e)) t2)) as [|Ht2]; [by left|].
apply (not_Forall_Exists _), Exists_exists in Ht2; destruct Ht2 as (e2&?&He2).
destruct (adequate_not_stuck NotStuck e1 σ1 φ Had t2 σ2 e2) as [?|(κ&e3&σ3&efs&?)];
rewrite ?eq_None_not_Some; auto.
{ exfalso. eauto. }
destruct (elem_of_list_split t2 e2) as (t2'&t2''&->); auto.
right; exists κ, (t2' ++ e3 :: t2'' ++ efs), σ3; econstructor; eauto.
Qed.
Section adequacy. Section adequacy.
Context `{!irisG Λ Σ}. Context `{!irisG Λ Σ}.
Implicit Types e : expr Λ. Implicit Types e : expr Λ.
...@@ -92,184 +67,163 @@ Proof. ...@@ -92,184 +67,163 @@ Proof.
by iApply (IH with "Hσ He Ht"). by iApply (IH with "Hσ He Ht").
Qed. Qed.
Lemma wptp_result φ κs' s n e1 t1 κs v2 t2 σ1 σ2 :
nsteps n (e1 :: t1, σ1) κs (of_val v2 :: t2, σ2)
state_interp σ1 (κs ++ κs') (length t1) -∗
WP e1 @ s; {{ v, σ, state_interp σ κs' (length t2) ={,}=∗ φ v σ }} -∗
wptp s t1 ={,}▷=∗^(S n) φ v2 σ2⌝.
Proof.
iIntros (?) "Hσ He Ht". rewrite Nat_iter_S_r.
iDestruct (wptp_steps with "Hσ He Ht") as "H"; first done.
iApply (step_fupdN_wand with "H").
iDestruct 1 as (e2 t2' ?) "(Hσ & H & _)"; simplify_eq.
iMod (wp_value_inv' with "H") as "H".
iMod (fupd_plain_mask_empty _ φ v2 σ2⌝%I with "[H Hσ]") as %?.
{ by iMod ("H" with "Hσ") as "$". }
by iApply step_fupd_intro.
Qed.
Lemma wptp_all_result φ κs' s n e1 t1 κs v2 vs2 σ1 σ2 :
nsteps n (e1 :: t1, σ1) κs (of_val <$> v2 :: vs2, σ2)
state_interp σ1 (κs ++ κs') (length t1) -∗
WP e1 @ s; {{ v,
state_interp σ2 κs' (length vs2) -∗
([ list] v vs2, fork_post v) ={,}=∗ φ v }} -∗
wptp s t1
={,}▷=∗^(S n) φ v2 ⌝.
Proof.
iIntros (Hstep) "Hσ He Ht". rewrite Nat_iter_S_r.
iDestruct (wptp_steps with "Hσ He Ht") as "H"; first done.
iApply (step_fupdN_wand with "H").
iDestruct 1 as (e2 t2' ?) "(Hσ & H & Hvs)"; simplify_eq/=.
rewrite fmap_length. iMod (wp_value_inv' with "H") as "H".
iAssert ([ list] v vs2, fork_post v)%I with "[> Hvs]" as "Hm".
{ clear Hstep. iInduction vs2 as [|v vs] "IH"; csimpl; first by iFrame.
iDestruct "Hvs" as "[Hv Hvs]".
iMod (wp_value_inv' with "Hv") as "$". by iApply "IH". }
iMod (fupd_plain_mask_empty _ φ v2⌝%I with "[H Hm Hσ]") as %?.
{ iApply ("H" with "Hσ Hm"). }
by iApply step_fupd_intro.
Qed.
Lemma wp_safe κs m e σ Φ : Lemma wp_safe κs m e σ Φ :
state_interp σ κs m -∗ state_interp σ κs m -∗
WP e {{ Φ }} ={,}=∗ is_Some (to_val e) reducible e σ⌝. WP e {{ Φ }} ={}=∗ is_Some (to_val e) reducible e σ⌝.
Proof. Proof.
rewrite wp_unfold /wp_pre. iIntros "Hσ H". rewrite wp_unfold /wp_pre. iIntros "Hσ H".
destruct (to_val e) as [v|] eqn:?. destruct (to_val e) as [v|] eqn:?; first by eauto.
{ iApply step_fupd_intro. set_solver. eauto. } iSpecialize ("H" $! σ [] κs with "Hσ"). rewrite sep_elim_l.
iMod (fupd_plain_mask_empty _ reducible e σ⌝%I with "[H Hσ]") as %?. iMod (fupd_plain_mask with "H") as %?; eauto.
{ by iMod ("H" $! σ [] κs with "Hσ") as "[$ H]". }
iApply step_fupd_intro; first by set_solver+.
iIntros "!> !%". by right.
Qed. Qed.
Lemma wptp_safe κs' n e1 κs e2 t1 t2 σ1 σ2 Φ : Lemma wptp_strong_adequacy Φ κs' s n e1 t1 κs e2 t2 σ1 σ2 :
nsteps n (e1 :: t1, σ1) κs (t2, σ2) e2 t2
state_interp σ1 (κs ++ κs') (length t1) -∗ WP e1 {{ Φ }} -∗ wptp NotStuck t1
={,}▷=∗^(S n) is_Some (to_val e2) reducible e2 σ2⌝.
Proof.
iIntros (? He2) "Hσ He Ht". rewrite Nat_iter_S_r.
iDestruct (wptp_steps with "Hσ He Ht") as "H"; first done.
iApply (step_fupdN_wand with "H").
iDestruct 1 as (e2' t2' ?) "(Hσ & H & Ht)"; simplify_eq.
apply elem_of_cons in He2 as [<-|(t1''&t2''&->)%elem_of_list_split].
- iMod (wp_safe with "Hσ H") as "$"; auto.
- iDestruct "Ht" as "(_ & He2 & _)". by iMod (wp_safe with "Hσ He2").
Qed.
Lemma wptp_invariance φ s n e1 κs κs' t1 t2 σ1 σ2 Φ :
nsteps n (e1 :: t1, σ1) κs (t2, σ2) nsteps n (e1 :: t1, σ1) κs (t2, σ2)
(state_interp σ2 κs' (pred (length t2)) ={,}=∗ φ) -∗
state_interp σ1 (κs ++ κs') (length t1) -∗ state_interp σ1 (κs ++ κs') (length t1) -∗
WP e1 @ s; {{ Φ }} -∗ wptp s t1 WP e1 @ s; {{ Φ }} -∗
={,}▷=∗^(S n) φ⌝. wptp s t1 ={,}▷=∗^(S n) e2 t2',
t2 = e2 :: t2'
e2, s = NotStuck e2 t2 (is_Some (to_val e2) reducible e2 σ2)
state_interp σ2 κs' (length t2')
from_option Φ True (to_val e2)
([ list] v omap to_val t2', fork_post v).
Proof. Proof.
iIntros (?) "Hφ Hσ He Ht". rewrite Nat_iter_S_r. iIntros (Hstep) "Hσ He Ht". rewrite Nat_iter_S_r.
iDestruct (wptp_steps _ n with "Hσ He Ht") as "H"; first done. iDestruct (wptp_steps with "Hσ He Ht") as "Hwp"; first done.
iApply (step_fupdN_wand with "H"). iDestruct 1 as (e2' t2' ->) "[Hσ _]". iApply (step_fupdN_wand with "Hwp").
iMod (fupd_plain_mask_empty _ φ⌝%I with "(Hφ Hσ)") as %?. iDestruct 1 as (e2' t2' ?) "(Hσ & Hwp & Ht)"; simplify_eq/=.
by iApply step_fupd_intro. iMod (fupd_plain_keep_l
e2, s = NotStuck e2 (e2' :: t2') (is_Some (to_val e2) reducible e2 σ2) ⌝%I
(state_interp σ2 κs' (length t2') WP e2' @ s; {{ v, Φ v }} wptp s t2')%I
with "[$Hσ $Hwp $Ht]") as "(Hsafe&Hσ&Hwp&Hvs)".
{ iIntros "(Hσ & Hwp & Ht)" (e' -> He').
apply elem_of_cons in He' as [<-|(t1''&t2''&->)%elem_of_list_split].
- iMod (wp_safe with "Hσ Hwp") as "$"; auto.
- iDestruct "Ht" as "(_ & He' & _)". by iMod (wp_safe with "Hσ He'"). }
iApply step_fupd_fupd. iApply step_fupd_intro; first done. iNext.
iExists _, _. iSplitL ""; first done. iFrame "Hsafe Hσ".
iSplitL "Hwp".
- destruct (to_val e2') as [v2|] eqn:He2'; last done.
apply of_to_val in He2' as <-. iApply (wp_value_inv' with "Hwp").
- clear Hstep. iInduction t2' as [|e t2'] "IH"; csimpl; first by iFrame.
iDestruct "Hvs" as "[Hv Hvs]". destruct (to_val e) as [v|] eqn:He.
+ apply of_to_val in He as <-. iMod (wp_value_inv' with "Hv") as "$".
by iApply "IH".
+ by iApply "IH".
Qed. Qed.
End adequacy. End adequacy.
Theorem wp_strong_adequacy Σ Λ `{!invPreG Σ} s e σ φ : (** Iris's generic adequacy result *)
( `{Hinv : !invG Σ} κs, Theorem wp_strong_adequacy Σ Λ `{!invPreG Σ} s e σ1 n κs t2 σ2 φ :
( `{Hinv : !invG Σ},
(|={}=> (|={}=>
(stateI : state Λ list (observation Λ) nat iProp Σ) (stateI : state Λ list (observation Λ) nat iProp Σ)
(fork_post : val Λ iProp Σ), (Φ fork_post : val Λ iProp Σ),
let _ : irisG Λ Σ := IrisG _ _ Hinv stateI fork_post in let _ : irisG Λ Σ := IrisG _ _ Hinv stateI fork_post in
(* This could be strengthened so that φ also talks about the number stateI σ1 κs 0
of forked-off threads *) WP e @ s; {{ Φ }}
stateI σ κs 0 WP e @ s; {{ v, σ m, stateI σ [] m ={,}=∗ φ v σ }})%I) ( e2 t2',
adequate s e σ φ. (* e2 is the final state of the main thread, t2' the rest *)
t2 = e2 :: t2' -∗
(* If this is a stuck-free triple (i.e. [s = NotStuck]), then all
threads in [t2] are either done (a value) or reducible *)
e2, s = NotStuck e2 t2 (is_Some (to_val e2) reducible e2 σ2) -∗
(* The state interpretation holds for [σ2] *)
stateI σ2 [] (length t2') -∗
(* If the main thread is done, its post-condition [Φ] holds *)
from_option Φ True (to_val e2) -∗
(* For all threads that are done, their postcondition [fork_post] holds. *)
([ list] v omap to_val t2', fork_post v) -∗
(* Under all these assumptions, and while opening all invariants, we
can conclude [φ] in the logic. After opening all required invariants,
one can use [fupd_intro_mask'] or [fupd_mask_weaken] to introduce the
fancy update. *)
|={,}=> φ ))%I)
nsteps n ([e], σ1) κs (t2, σ2)
(* Then we can conclude [φ] at the meta-level. *)
φ.
Proof. Proof.
intros Hwp; split. intros Hwp ?.
- intros t2 σ2 v2 [n [κs ?]]%erased_steps_nsteps. eapply (step_fupdN_soundness' _ (S (S n)))=> Hinv. rewrite Nat_iter_S.
eapply (step_fupdN_soundness' _ (S (S n)))=> Hinv. rewrite Nat_iter_S. iMod Hwp as (stateI Φ fork_post) "(Hσ & Hwp & Hφ)".
iMod (Hwp _ (κs ++ [])) as (stateI fork_post) "[Hσ Hwp]". iApply step_fupd_intro; [done|]; iModIntro.
iApply step_fupd_intro; first done. iModIntro. iApply step_fupdN_S_fupd. iApply (step_fupdN_wand with "[-Hφ]").
iApply (@wptp_result _ _ (IrisG _ _ Hinv stateI fork_post) with "[Hσ] [Hwp]"); eauto. { iApply (@wptp_strong_adequacy _ _ (IrisG _ _ Hinv stateI fork_post) _ []
iApply (wp_wand with "Hwp"). iIntros (v) "H"; iIntros (σ'). iApply "H". with "[Hσ] Hwp"); eauto; by rewrite right_id_L. }
- destruct s; last done. intros t2 σ2 e2 _ [n [κs ?]]%erased_steps_nsteps ?. iIntros "Hpost". iDestruct "Hpost" as (e2 t2' ->) "(? & ? & ? & ?)".
eapply (step_fupdN_soundness' _ (S (S n)))=> Hinv. rewrite Nat_iter_S. iApply fupd_plain_mask_empty.
iMod (Hwp _ (κs ++ [])) as (stateI fork_post) "[Hσ Hwp]". iMod ("Hφ" with "[% //] [$] [$] [$] [$]"). done.
iApply step_fupd_intro; first done. iModIntro.
iApply (@wptp_safe _ _ (IrisG _ _ Hinv stateI fork_post) with "[Hσ] Hwp"); eauto.
Qed. Qed.
Theorem wp_adequacy Σ Λ `{!invPreG Σ} s e σ φ : (** Since the full adequacy statement is quite a mouthful, we prove some more
( `{Hinv : !invG Σ} κs, intuitive and simpler corollaries. These lemmas are morover stated in terms of
(|={}=> stateI : state Λ list (observation Λ) iProp Σ, [rtc erased_step] so one does not have to provide the trace. *)
let _ : irisG Λ Σ := IrisG _ _ Hinv (λ σ κs _, stateI σ κs) (λ _, True%I) in Record adequate {Λ} (s : stuckness) (e1 : expr Λ) (σ1 : state Λ)
stateI σ κs WP e @ s; {{ v, φ v }})%I) (φ : val Λ state Λ Prop) := {
adequate s e σ (λ v _, φ v). adequate_result t2 σ2 v2 :
Proof. rtc erased_step ([e1], σ1) (of_val v2 :: t2, σ2) φ v2 σ2;
intros Hwp. apply (wp_strong_adequacy Σ _)=> Hinv κs. adequate_not_stuck t2 σ2 e2 :
iMod Hwp as (stateI) "[Hσ H]". iExists (λ σ κs _, stateI σ κs), (λ _, True%I). s = NotStuck
iIntros "{$Hσ} !>". rtc erased_step ([e1], σ1) (t2, σ2)
iApply (wp_wand with "H"). iIntros (v ? σ') "_". e2 t2 (is_Some (to_val e2) reducible e2 σ2)
iIntros "_". by iApply fupd_mask_weaken. }.
Qed.
(* Special adequacy for when *all threads* evaluate to a value. Here we let the Lemma adequate_alt {Λ} s e1 σ1 (φ : val Λ state Λ Prop) :
user pick the one list of observations for which the proof needs to apply. If adequate s e1 σ1 φ t2 σ2,
you just got an [rtc erased_step], use [erased_steps_nsteps]. *) rtc erased_step ([e1], σ1) (t2, σ2)
Theorem wp_strong_all_adequacy Σ Λ `{!invPreG Σ} s e σ1 n κs v vs σ2 φ : ( v2 t2', t2 = of_val v2 :: t2' φ v2 σ2)
( `{Hinv : !invG Σ}, ( e2, s = NotStuck e2 t2 (is_Some (to_val e2) reducible e2 σ2)).
(|={}=> Proof. split. intros []; naive_solver. constructor; naive_solver. Qed.
(stateI : state Λ list (observation Λ) nat iProp Σ)
(fork_post : val Λ iProp Σ), Theorem adequate_tp_safe {Λ} (e1 : expr Λ) t2 σ1 σ2 φ :
let _ : irisG Λ Σ := IrisG _ _ Hinv stateI fork_post in adequate NotStuck e1 σ1 φ
stateI σ1 κs 0 WP e @ s; {{ v, rtc erased_step ([e1], σ1) (t2, σ2)
stateI σ2 [] (length vs) -∗ Forall (λ e, is_Some (to_val e)) t2 t3 σ3, erased_step (t2, σ2) (t3, σ3).
([ list] v vs, fork_post v) ={,}=∗ φ v }})%I)
nsteps n ([e], σ1) κs (of_val <$> v :: vs, σ2)
φ v.
Proof. Proof.
intros Hwp ?. intros Had ?.
eapply (step_fupdN_soundness' _ (S (S n)))=> Hinv. rewrite Nat_iter_S. destruct (decide (Forall (λ e, is_Some (to_val e)) t2)) as [|Ht2]; [by left|].
iMod Hwp as (stateI fork_post) "[Hσ Hwp]". apply (not_Forall_Exists _), Exists_exists in Ht2; destruct Ht2 as (e2&?&He2).
iApply step_fupd_intro; first done. iModIntro. destruct (adequate_not_stuck NotStuck e1 σ1 φ Had t2 σ2 e2) as [?|(κ&e3&σ3&efs&?)];
iApply (@wptp_all_result _ _ (IrisG _ _ Hinv stateI fork_post) rewrite ?eq_None_not_Some; auto.
with "[Hσ] [Hwp]"); eauto. by rewrite right_id_L. { exfalso. eauto. }
destruct (elem_of_list_split t2 e2) as (t2'&t2''&->); auto.
right; exists (t2' ++ e3 :: t2'' ++ efs), σ3, κ; econstructor; eauto.
Qed. Qed.
Theorem wp_invariance Σ Λ `{!invPreG Σ} s e σ1 t2 σ2 φ : Corollary wp_adequacy Σ Λ `{!invPreG Σ} s e σ φ :
( `{Hinv : !invG Σ} κs κs', ( `{Hinv : !invG Σ} κs,
(|={}=> (|={}=>
(stateI : state Λ list (observation Λ) nat iProp Σ) (stateI : state Λ list (observation Λ) iProp Σ)
(fork_post : val Λ iProp Σ), (fork_post : val Λ iProp Σ),
let _ : irisG Λ Σ := IrisG _ _ Hinv stateI fork_post in let _ : irisG Λ Σ := IrisG _ _ Hinv (λ σ κs _, stateI σ κs) fork_post in
stateI σ1 (κs ++ κs') 0 WP e @ s; {{ _, True }} stateI σ κs WP e @ s; {{ v, φ v }})%I)
(stateI σ2 κs' (pred (length t2)) ={,}=∗ φ))%I) adequate s e σ (λ v _, φ v).
rtc erased_step ([e], σ1) (t2, σ2)
φ.
Proof. Proof.
intros Hwp [n [κs ?]]%erased_steps_nsteps. intros Hwp. apply adequate_alt; intros t2 σ2 [n [κs ?]]%erased_steps_nsteps.
apply (step_fupdN_soundness' _ (S (S n)))=> Hinv. rewrite Nat_iter_S. eapply (wp_strong_adequacy Σ _); [|done]=> ?.
iMod (Hwp Hinv κs []) as (Istate fork_post) "(Hσ & Hwp & Hclose)". iMod Hwp as (stateI fork_post) "[Hσ Hwp]".
iApply step_fupd_intro; first done. iExists (λ σ κs _, stateI σ κs), (λ v, φ v⌝%I), fork_post.
iApply (@wptp_invariance _ _ (IrisG _ _ Hinv Istate fork_post) iIntros "{$Hσ $Hwp} !>" (e2 t2' -> ?) "_ H _".
with "Hclose [Hσ] [Hwp]"); eauto. iApply fupd_mask_weaken; [done|]. iSplit; [|done].
iIntros (v2 t2'' [= -> <-]). by rewrite to_of_val.
Qed. Qed.
(* An equivalent version that does not require finding [fupd_intro_mask'], but Corollary wp_invariance Σ Λ `{!invPreG Σ} s e σ1 t2 σ2 φ :
can be confusing to use. *) ( `{Hinv : !invG Σ} κs,
Corollary wp_invariance' Σ Λ `{!invPreG Σ} s e σ1 t2 σ2 φ :
( `{Hinv : !invG Σ} κs κs',
(|={}=> (|={}=>
(stateI : state Λ list (observation Λ) nat iProp Σ) (stateI : state Λ list (observation Λ) nat iProp Σ)
(fork_post : val Λ iProp Σ), (fork_post : val Λ iProp Σ),
let _ : irisG Λ Σ := IrisG _ _ Hinv stateI fork_post in let _ : irisG Λ Σ := IrisG _ _ Hinv stateI fork_post in
stateI σ1 κs 0 WP e @ s; {{ _, True }} stateI σ1 κs 0 WP e @ s; {{ _, True }}
(stateI σ2 κs' (pred (length t2)) -∗ E, |={,E}=> φ))%I) (stateI σ2 [] (pred (length t2)) -∗ E, |={,E}=> φ))%I)
rtc erased_step ([e], σ1) (t2, σ2) rtc erased_step ([e], σ1) (t2, σ2)
φ. φ.
Proof. Proof.
intros Hwp. eapply wp_invariance; first done. intros Hwp [n [κs ?]]%erased_steps_nsteps.
intros Hinv κs κs'. iMod (Hwp Hinv) as (stateI fork_post) "(? & ? & Hφ)". eapply (wp_strong_adequacy Σ _); [|done]=> ?.
iModIntro. iExists stateI, fork_post. iFrame. iIntros "Hσ". iMod (Hwp _ κs) as (stateI fork_post) "(Hσ & Hwp & Hφ)".
iExists stateI, (λ _, True)%I, fork_post.
iIntros "{$Hσ $Hwp} !>" (e2 t2' -> _) "Hσ _ _ /=".
iDestruct ("Hφ" with "Hσ") as (E) ">Hφ". iDestruct ("Hφ" with "Hσ") as (E) ">Hφ".
by iApply fupd_mask_weaken; first set_solver. by iApply fupd_mask_weaken; first set_solver.
Qed. Qed.
...@@ -55,7 +55,7 @@ Proof. ...@@ -55,7 +55,7 @@ Proof.
iIntros (? κs). iIntros (? κs).
iMod (own_alloc ( (Excl' σ) (Excl' σ))) as (γσ) "[Hσ Hσf]"; iMod (own_alloc ( (Excl' σ) (Excl' σ))) as (γσ) "[Hσ Hσf]";
first by apply auth_both_valid. first by apply auth_both_valid.
iModIntro. iExists (λ σ κs, own γσ ( (Excl' σ)))%I. iModIntro. iExists (λ σ κs, own γσ ( (Excl' σ)))%I, (λ _, True%I).
iFrame "Hσ". iFrame "Hσ".
iApply (Hwp (OwnPG _ _ _ _ γσ)). rewrite /ownP. iFrame. iApply (Hwp (OwnPG _ _ _ _ γσ)). rewrite /ownP. iFrame.
Qed. Qed.
...@@ -68,14 +68,14 @@ Theorem ownP_invariance Σ `{!ownPPreG Λ Σ} s e σ1 t2 σ2 φ : ...@@ -68,14 +68,14 @@ Theorem ownP_invariance Σ `{!ownPPreG Λ Σ} s e σ1 t2 σ2 φ :
φ σ2. φ σ2.
Proof. Proof.
intros Hwp Hsteps. eapply (wp_invariance Σ Λ s e σ1 t2 σ2 _)=> //. intros Hwp Hsteps. eapply (wp_invariance Σ Λ s e σ1 t2 σ2 _)=> //.
iIntros (? κs κs'). iIntros (? κs).
iMod (own_alloc ( (Excl' σ1) (Excl' σ1))) as (γσ) "[Hσ Hσf]"; iMod (own_alloc ( (Excl' σ1) (Excl' σ1))) as (γσ) "[Hσ Hσf]";
first by apply auth_both_valid. first by apply auth_both_valid.
iExists (λ σ κs' _, own γσ ( (Excl' σ)))%I, (λ _, True%I). iExists (λ σ κs' _, own γσ ( (Excl' σ)))%I, (λ _, True%I).
iFrame "Hσ". iFrame "Hσ".
iMod (Hwp (OwnPG _ _ _ _ γσ) with "[Hσf]") as "[$ H]"; iMod (Hwp (OwnPG _ _ _ _ γσ) with "[Hσf]") as "[$ H]";
first by rewrite /ownP; iFrame. first by rewrite /ownP; iFrame.
iIntros "!> Hσ". iMod "H" as (σ2') "[Hσf %]". rewrite /ownP. iIntros "!> Hσ". iExists ∅. iMod "H" as (σ2') "[Hσf %]". rewrite /ownP.
iDestruct (own_valid_2 with "Hσ Hσf") iDestruct (own_valid_2 with "Hσ Hσf")
as %[Hp%Excl_included _]%auth_both_valid; simplify_eq; auto. as %[Hp%Excl_included _]%auth_both_valid; simplify_eq; auto.
Qed. Qed.
......
0% Loading or .
You are about to add 0 people to the discussion. Proceed with caution.
Finish editing this message first!
Please register or to comment