Skip to content
Snippets Groups Projects
Commit c1449e94 authored by Ralf Jung's avatar Ralf Jung
Browse files

make wp_par usable

parent 6d15d440
No related branches found
No related tags found
No related merge requests found
......@@ -155,7 +155,7 @@ Section increment_client.
(* The continuation: From after the atomic triple to the postcondition of the WP *)
done.
}
wp_apply par_spec; wp_pures.
wp_apply wp_par.
- iAssumption.
- iAssumption.
- iIntros (??) "_ !>". done.
......
......@@ -12,6 +12,8 @@ Definition par : val :=
let: "v1" := join "handle" in
("v1", "v2").
Notation "e1 ||| e2" := (par (λ: <>, e1)%E (λ: <>, e2)%E) : expr_scope.
(* Not a value itself, but with *unlocked* value lambdas. *)
Local Notation "e1 ||| e2" := (par (LamV BAnon e1%E) (LamV BAnon e2%E)) : val_scope.
Section proof.
Local Set Default Proof Using "Type*".
......@@ -37,7 +39,7 @@ Qed.
Lemma wp_par (Ψ1 Ψ2 : val iProp Σ) (e1 e2 : expr) (Φ : val iProp Σ) :
WP e1 {{ Ψ1 }} -∗ WP e2 {{ Ψ2 }} -∗
( v1 v2, Ψ1 v1 Ψ2 v2 -∗ Φ (v1,v2)%V) -∗
WP e1 ||| e2 {{ Φ }}.
WP (e1 ||| e2)%V {{ Φ }}.
Proof.
iIntros "H1 H2 H".
wp_apply (par_spec Ψ1 Ψ2 with "[H1] [H2] [H]"); [by wp_lam..|auto].
......
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