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

add a version of [cancel] that works with goals of the form [_ |- pvs _]; and...

add a version of [cancel] that works with goals of the form [_ |- pvs _]; and use that for the barrier proof
parent 7884512b
No related branches found
No related tags found
No related merge requests found
...@@ -74,6 +74,7 @@ program_logic/saved_prop.v ...@@ -74,6 +74,7 @@ program_logic/saved_prop.v
program_logic/auth.v program_logic/auth.v
program_logic/sts.v program_logic/sts.v
program_logic/namespaces.v program_logic/namespaces.v
program_logic/tactics.v
heap_lang/lang.v heap_lang/lang.v
heap_lang/tactics.v heap_lang/tactics.v
heap_lang/wp_tactics.v heap_lang/wp_tactics.v
......
From prelude Require Import functions. From prelude Require Import functions.
From algebra Require Import upred_big_op upred_tactics. From algebra Require Import upred_big_op.
From program_logic Require Import sts saved_prop. From program_logic Require Import sts saved_prop tactics.
From heap_lang Require Export heap wp_tactics. From heap_lang Require Export heap wp_tactics.
From barrier Require Export barrier. From barrier Require Export barrier.
From barrier Require Import protocol. From barrier Require Import protocol.
...@@ -50,6 +50,14 @@ Definition recv (l : loc) (R : iProp) : iProp := ...@@ -50,6 +50,14 @@ Definition recv (l : loc) (R : iProp) : iProp :=
barrier_ctx γ l P sts_ownS γ (i_states i) {[ Change i ]} barrier_ctx γ l P sts_ownS γ (i_states i) {[ Change i ]}
saved_prop_own i (Next Q) (Q -★ R))%I. saved_prop_own i (Next Q) (Q -★ R))%I.
Global Instance barrier_ctx_always_stable (γ : gname) (l : loc) (P : iProp) :
AlwaysStable (barrier_ctx γ l P).
Proof. apply _. Qed.
(* TODO: Figure out if this has a "Global" or "Local" effect.
We want it to be Global. *)
Typeclasses Opaque barrier_ctx send recv.
Implicit Types I : gset gname. Implicit Types I : gset gname.
(** Setoids *) (** Setoids *)
...@@ -62,7 +70,7 @@ Global Instance barrier_inv_ne n l : ...@@ -62,7 +70,7 @@ Global Instance barrier_inv_ne n l :
Proper (dist n ==> eq ==> dist n) (barrier_inv l). Proper (dist n ==> eq ==> dist n) (barrier_inv l).
Proof. solve_proper. Qed. Proof. solve_proper. Qed.
Global Instance barrier_ctx_ne n γ l : Proper (dist n ==> dist n) (barrier_ctx γ l). Global Instance barrier_ctx_ne n γ l : Proper (dist n ==> dist n) (barrier_ctx γ l).
Proof. solve_proper. Qed. Proof. solve_proper. Qed.
Global Instance send_ne n l : Proper (dist n ==> dist n) (send l). Global Instance send_ne n l : Proper (dist n ==> dist n) (send l).
Proof. solve_proper. Qed. Proof. solve_proper. Qed.
Global Instance recv_ne n l : Proper (dist n ==> dist n) (recv l). Global Instance recv_ne n l : Proper (dist n ==> dist n) (recv l).
...@@ -127,18 +135,11 @@ Proof. ...@@ -127,18 +135,11 @@ Proof.
apply exist_elim=>γ. apply exist_elim=>γ.
rewrite /recv /send. rewrite -(exist_intro γ) -(exist_intro P). rewrite /recv /send. rewrite -(exist_intro γ) -(exist_intro P).
rewrite -(exist_intro P) -(exist_intro i) -(exist_intro γ). rewrite -(exist_intro P) -(exist_intro i) -(exist_intro γ).
(* This is even more annoying than usually, since rewrite sometimes unfolds stuff... *) rewrite always_and_sep_l wand_diag later_True right_id.
rewrite [barrier_ctx _ _ _]lock !assoc rewrite [heap_ctx _]always_sep_dup [sts_ctx _ _ _]always_sep_dup.
[(_ locked (barrier_ctx _ _ _))%I]comm !assoc -lock. rewrite /barrier_ctx const_equiv // left_id.
rewrite -always_sep_dup. ecancel_pvs [saved_prop_own i _; heap_ctx _; heap_ctx _;
(* TODO: This is cancelling below a pvs. *) sts_ctx _ _ _; sts_ctx _ _ _].
rewrite [barrier_ctx _ _ _]lock always_and_sep_l -!assoc assoc -lock.
rewrite -pvs_frame_l. rewrite /barrier_ctx const_equiv // left_id. apply sep_mono_r.
rewrite [(saved_prop_own _ _ _)%I]comm !assoc. rewrite -pvs_frame_r.
apply sep_mono_l.
rewrite -assoc [( _ _)%I]comm assoc -pvs_frame_r.
eapply sep_elim_True_r; last eapply sep_mono_l.
{ rewrite -later_intro. apply wand_intro_l. by rewrite right_id. }
rewrite (sts_own_weaken _ _ (i_states i low_states) _ rewrite (sts_own_weaken _ _ (i_states i low_states) _
({[ Change i ]} {[ Send ]})). ({[ Change i ]} {[ Send ]})).
+ apply pvs_mono. + apply pvs_mono.
...@@ -157,7 +158,7 @@ Proof. ...@@ -157,7 +158,7 @@ Proof.
(* I think some evars here are better than repeating *everything* *) (* I think some evars here are better than repeating *everything* *)
eapply (sts_fsaS _ (wp_fsa _)) with (N0:=N) (γ0:=γ); simpl; eapply (sts_fsaS _ (wp_fsa _)) with (N0:=N) (γ0:=γ); simpl;
eauto with I ndisj. eauto with I ndisj.
rewrite !assoc [(_ sts_ownS _ _ _)%I]comm -!assoc. apply sep_mono_r. ecancel [sts_ownS γ _ _].
apply forall_intro=>-[p I]. apply wand_intro_l. rewrite -!assoc. apply forall_intro=>-[p I]. apply wand_intro_l. rewrite -!assoc.
apply const_elim_sep_l=>Hs. destruct p; last done. apply const_elim_sep_l=>Hs. destruct p; last done.
rewrite {1}/barrier_inv =>/={Hs}. rewrite later_sep. rewrite {1}/barrier_inv =>/={Hs}. rewrite later_sep.
...@@ -166,12 +167,12 @@ Proof. ...@@ -166,12 +167,12 @@ Proof.
apply wand_intro_l. rewrite -(exist_intro (State High I)). apply wand_intro_l. rewrite -(exist_intro (State High I)).
rewrite -(exist_intro ). rewrite const_equiv /=; last by eauto using signal_step. rewrite -(exist_intro ). rewrite const_equiv /=; last by eauto using signal_step.
rewrite left_id -later_intro {2}/barrier_inv -!assoc. apply sep_mono_r. rewrite left_id -later_intro {2}/barrier_inv -!assoc. apply sep_mono_r.
rewrite !assoc [(_ P)%I]comm !assoc -2!assoc. sep_split right: [Φ _]; last first.
apply sep_mono; last first.
{ apply wand_intro_l. eauto with I. } { apply wand_intro_l. eauto with I. }
(* Now we come to the core of the proof: Updating from waiting to ress. *) (* Now we come to the core of the proof: Updating from waiting to ress. *)
rewrite /ress sep_exist_l. apply exist_mono=>{Φ} Φ. rewrite /ress sep_exist_r. apply exist_mono=>{Φ} Φ.
rewrite later_wand {1}(later_intro P) !assoc wand_elim_r /= wand_True //. ecancel [Π{set I} (λ _, saved_prop_own _ _)]%I. strip_later.
rewrite wand_True. eapply wand_apply_l'; eauto with I.
Qed. Qed.
Lemma wait_spec l P (Φ : val iProp) : Lemma wait_spec l P (Φ : val iProp) :
...@@ -186,12 +187,12 @@ Proof. ...@@ -186,12 +187,12 @@ Proof.
(* I think some evars here are better than repeating *everything* *) (* I think some evars here are better than repeating *everything* *)
eapply (sts_fsaS _ (wp_fsa _)) with (N0:=N) (γ0:=γ); simpl; eapply (sts_fsaS _ (wp_fsa _)) with (N0:=N) (γ0:=γ); simpl;
eauto with I ndisj. eauto with I ndisj.
rewrite !assoc [(_ sts_ownS _ _ _)%I]comm -!assoc. apply sep_mono_r. ecancel [sts_ownS γ _ _].
apply forall_intro=>-[p I]. apply wand_intro_l. rewrite -!assoc. apply forall_intro=>-[p I]. apply wand_intro_l. rewrite -!assoc.
apply const_elim_sep_l=>Hs. apply const_elim_sep_l=>Hs.
rewrite {1}/barrier_inv =>/=. rewrite later_sep. rewrite {1}/barrier_inv =>/=. rewrite later_sep.
eapply wp_load; eauto with I ndisj. eapply wp_load; eauto with I ndisj.
rewrite -!assoc. apply sep_mono_r. strip_later. ecancel [ l {_} _]%I. strip_later.
apply wand_intro_l. destruct p. apply wand_intro_l. destruct p.
{ (* a Low state. The comparison fails, and we recurse. *) { (* a Low state. The comparison fails, and we recurse. *)
rewrite -(exist_intro (State Low I)) -(exist_intro {[ Change i ]}). rewrite -(exist_intro (State Low I)) -(exist_intro {[ Change i ]}).
...@@ -202,11 +203,8 @@ Proof. ...@@ -202,11 +203,8 @@ Proof.
rewrite -always_wand_impl always_elim. rewrite -always_wand_impl always_elim.
rewrite -{2}pvs_wp. apply pvs_wand_r. rewrite -{2}pvs_wp. apply pvs_wand_r.
rewrite -(exist_intro γ) -(exist_intro P) -(exist_intro Q) -(exist_intro i). rewrite -(exist_intro γ) -(exist_intro P) -(exist_intro Q) -(exist_intro i).
rewrite !assoc. rewrite const_equiv // left_id -later_intro.
do 3 (rewrite -pvs_frame_r; apply sep_mono; last (try apply later_intro; reflexivity)). ecancel_pvs [heap_ctx _; saved_prop_own _ _; Q -★ _; R -★ _; sts_ctx _ _ _]%I.
rewrite [(_ heap_ctx _)%I]comm -!assoc.
rewrite const_equiv // left_id -pvs_frame_l. apply sep_mono_r.
rewrite comm -pvs_frame_l. apply sep_mono_r.
apply sts_own_weaken; eauto using i_states_closed. } apply sts_own_weaken; eauto using i_states_closed. }
(* a High state: the comparison succeeds, and we perform a transition and (* a High state: the comparison succeeds, and we perform a transition and
return to the client *) return to the client *)
...@@ -217,15 +215,12 @@ Proof. ...@@ -217,15 +215,12 @@ Proof.
rewrite left_id -[( barrier_inv _ _ _)%I]later_intro {2}/barrier_inv. rewrite left_id -[( barrier_inv _ _ _)%I]later_intro {2}/barrier_inv.
rewrite -!assoc. apply sep_mono_r. rewrite /ress. rewrite -!assoc. apply sep_mono_r. rewrite /ress.
rewrite !sep_exist_r. apply exist_mono=>Ψ. rewrite !sep_exist_r. apply exist_mono=>Ψ.
rewrite !(big_sepS_delete _ I i) // [(_ Π{set _} _)%I]comm -!assoc. rewrite !(big_sepS_delete _ I i) //= !wand_True later_sep.
rewrite /= !wand_True later_sep. ecancel [ Π{set _} Ψ; Π{set _} (λ _, saved_prop_own _ _)]%I.
ecancel [ Π{set _} _; Π{set _} (λ _, saved_prop_own _ _)]%I. apply wand_intro_l. set savedΨ := _ i _. set savedQ := _ i _.
apply wand_intro_l. rewrite [(heap_ctx _ _)%I]sep_elim_r. to_front [savedΨ; savedQ]. rewrite saved_prop_agree later_equivI /=.
rewrite [(sts_own _ _ _ _)%I]sep_elim_r [(sts_ctx _ _ _ _)%I]sep_elim_r. wp_op; [|done]=> _. wp_if. rewrite !assoc. eapply wand_apply_r'; first done.
rewrite [(saved_prop_own _ _ _ _)%I]assoc. eapply wand_apply_r'; first done.
rewrite saved_prop_agree later_equivI /=.
wp_op; [|done]=> _. wp_if. rewrite !assoc.
eapply wand_apply_r; [done..|]. eapply wand_apply_r; [done..|].
apply: (eq_rewrite (Ψ i) Q (λ x, x)%I); by eauto with I. apply: (eq_rewrite (Ψ i) Q (λ x, x)%I); by eauto with I.
Qed. Qed.
...@@ -241,7 +236,7 @@ Proof. ...@@ -241,7 +236,7 @@ Proof.
(* I think some evars here are better than repeating *everything* *) (* I think some evars here are better than repeating *everything* *)
eapply pvs_mk_fsa, (sts_fsaS _ pvs_fsa) with (N0:=N) (γ0:=γ); simpl; eapply pvs_mk_fsa, (sts_fsaS _ pvs_fsa) with (N0:=N) (γ0:=γ); simpl;
eauto with I ndisj. eauto with I ndisj.
rewrite !assoc [(_ sts_ownS _ _ _)%I]comm -!assoc. apply sep_mono_r. ecancel [sts_ownS γ _ _].
apply forall_intro=>-[p I]. apply wand_intro_l. rewrite -!assoc. apply forall_intro=>-[p I]. apply wand_intro_l. rewrite -!assoc.
apply const_elim_sep_l=>Hs. rewrite /pvs_fsa. apply const_elim_sep_l=>Hs. rewrite /pvs_fsa.
eapply sep_elim_True_l. eapply sep_elim_True_l.
...@@ -270,16 +265,15 @@ Proof. ...@@ -270,16 +265,15 @@ Proof.
apply wand_intro_l. rewrite !assoc. rewrite /recv. apply wand_intro_l. rewrite !assoc. rewrite /recv.
rewrite -(exist_intro γ) -(exist_intro P) -(exist_intro R1) -(exist_intro i1). rewrite -(exist_intro γ) -(exist_intro P) -(exist_intro R1) -(exist_intro i1).
rewrite -(exist_intro γ) -(exist_intro P) -(exist_intro R2) -(exist_intro i2). rewrite -(exist_intro γ) -(exist_intro P) -(exist_intro R2) -(exist_intro i2).
do 2 rewrite !(assoc ()%I) [(_ sts_ownS _ _ _)%I]comm. rewrite [heap_ctx _]always_sep_dup [sts_ctx _ _ _]always_sep_dup.
rewrite -!assoc. rewrite [(sts_ownS _ _ _ _ _)%I]assoc. rewrite /barrier_ctx const_equiv // left_id.
rewrite -pvs_frame_r. apply sep_mono. ecancel_pvs [saved_prop_own i1 _; saved_prop_own i2 _; heap_ctx _; heap_ctx _;
- rewrite -sts_ownS_op; eauto using i_states_closed. sts_ctx _ _ _; sts_ctx _ _ _].
+ apply sts_own_weaken; rewrite !wand_diag later_True !right_id.
eauto using sts.closed_op, i_states_closed. set_solver. rewrite -sts_ownS_op; eauto using i_states_closed.
+ set_solver. - apply sts_own_weaken;
- rewrite const_equiv // !left_id. eauto using sts.closed_op, i_states_closed. set_solver.
rewrite {1}[heap_ctx _]always_sep_dup {1}[sts_ctx _ _ _]always_sep_dup. - set_solver.
rewrite !wand_diag -!later_intro. solve_sep_entails.
Qed. Qed.
Lemma recv_weaken l P1 P2 : Lemma recv_weaken l P1 P2 :
...@@ -288,9 +282,8 @@ Proof. ...@@ -288,9 +282,8 @@ Proof.
apply wand_intro_l. rewrite /recv. rewrite sep_exist_r. apply exist_mono=>γ. apply wand_intro_l. rewrite /recv. rewrite sep_exist_r. apply exist_mono=>γ.
rewrite sep_exist_r. apply exist_mono=>P. rewrite sep_exist_r. rewrite sep_exist_r. apply exist_mono=>P. rewrite sep_exist_r.
apply exist_mono=>Q. rewrite sep_exist_r. apply exist_mono=>i. apply exist_mono=>Q. rewrite sep_exist_r. apply exist_mono=>i.
rewrite -!assoc. apply sep_mono_r, sep_mono_r, sep_mono_r, sep_mono_r, sep_mono_r. ecancel [barrier_ctx _ _ _; sts_ownS _ _ _; saved_prop_own _ _].
rewrite (later_intro (P1 -★ _)%I) -later_sep. apply later_mono. strip_later. apply wand_intro_l. by rewrite !assoc wand_elim_r wand_elim_r.
apply wand_intro_l. by rewrite !assoc wand_elim_r wand_elim_r.
Qed. Qed.
Lemma recv_mono l P1 P2 : Lemma recv_mono l P1 P2 :
......
From algebra Require Export upred_tactics.
From program_logic Require Export pviewshifts.
Import uPred.
Module uPred_reflection_pvs.
Import uPred_reflection.
Section uPred_reflection_pvs.
Context {Λ : language} {Σ : rFunctor}.
Local Notation iProp := (iProp Λ Σ).
Lemma cancel_entails_pvs Σ' E1 E2 e1 e2 e1' e2' ns :
cancel ns e1 = Some e1' cancel ns e2 = Some e2'
eval Σ' e1' pvs E1 E2 (eval Σ' e2' : iProp) eval Σ' e1 pvs E1 E2 (eval Σ' e2).
Proof.
intros ??. rewrite !eval_flatten.
rewrite (flatten_cancel e1 e1' ns) // (flatten_cancel e2 e2' ns) //; csimpl.
rewrite !fmap_app !big_sep_app. rewrite -pvs_frame_l. apply sep_mono_r.
Qed.
End uPred_reflection_pvs.
Ltac quote_pvs :=
match goal with
| |- ?P1 pvs ?E1 ?E2 ?P2 =>
lazymatch type of (_ : Quote [] _ P1 _) with Quote _ ?Σ2 _ ?e1 =>
lazymatch type of (_ : Quote Σ2 _ P2 _) with Quote _ ?Σ3 _ ?e2 =>
change (eval Σ3 e1 pvs E1 E2 (eval Σ3 e2)) end end
end.
End uPred_reflection_pvs.
Tactic Notation "cancel_pvs" constr(Ps) :=
uPred_reflection_pvs.quote_pvs;
let Σ := match goal with |- uPred_reflection.eval _ _ => Σ end in
let ns' := lazymatch type of (_ : uPred_reflection.QuoteArgs Σ Ps _) with
| uPred_reflection.QuoteArgs _ _ ?ns' => ns'
end in
eapply uPred_reflection_pvs.cancel_entails_pvs with (ns:=ns');
[cbv; reflexivity|cbv; reflexivity|simpl].
Tactic Notation "ecancel_pvs" open_constr(Ps) :=
close_uPreds Ps ltac:(fun Qs => cancel_pvs Qs).
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