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

Fix issue #181: let `wp_expr_eval` check that the goal is in fact a WP.

  Also, remove the inconsistency that `wp_expr_eval` succeeds on a goal
  that is not a WP.
parent be553c16
No related branches found
No related tags found
No related merge requests found
...@@ -15,11 +15,16 @@ Lemma tac_twp_expr_eval `{heapG Σ} Δ s E Φ e e' : ...@@ -15,11 +15,16 @@ Lemma tac_twp_expr_eval `{heapG Σ} Δ s E Φ e e' :
Proof. by intros ->. Qed. Proof. by intros ->. Qed.
Tactic Notation "wp_expr_eval" tactic(t) := Tactic Notation "wp_expr_eval" tactic(t) :=
try ( iStartProof;
iStartProof; lazymatch goal with
first [eapply tac_wp_expr_eval|eapply tac_twp_expr_eval]; | |- envs_entails _ (wp ?s ?E ?e ?Q) =>
[let x := fresh in intros x; t; unfold x; reflexivity eapply tac_wp_expr_eval;
|]). [let x := fresh in intros x; t; unfold x; reflexivity|]
| |- envs_entails _ (twp ?s ?E ?e ?Q) =>
eapply tac_twp_expr_eval;
[let x := fresh in intros x; t; unfold x; reflexivity|]
| _ => fail "wp_expr_eval: not a 'wp'"
end.
Ltac wp_expr_simpl := wp_expr_eval simpl. Ltac wp_expr_simpl := wp_expr_eval simpl.
Ltac wp_expr_simpl_subst := wp_expr_eval simpl_subst. Ltac wp_expr_simpl_subst := wp_expr_eval simpl_subst.
...@@ -293,13 +298,13 @@ Tactic Notation "wp_apply" open_constr(lem) := ...@@ -293,13 +298,13 @@ Tactic Notation "wp_apply" open_constr(lem) :=
lazymatch goal with lazymatch goal with
| |- envs_entails _ (wp ?s ?E ?e ?Q) => | |- envs_entails _ (wp ?s ?E ?e ?Q) =>
reshape_expr e ltac:(fun K e' => reshape_expr e ltac:(fun K e' =>
wp_bind_core K; iApplyHyp H; try iNext; wp_expr_simpl) || wp_bind_core K; iApplyHyp H; try iNext; try wp_expr_simpl) ||
lazymatch iTypeOf H with lazymatch iTypeOf H with
| Some (_,?P) => fail "wp_apply: cannot apply" P | Some (_,?P) => fail "wp_apply: cannot apply" P
end end
| |- envs_entails _ (twp ?s ?E ?e ?Q) => | |- envs_entails _ (twp ?s ?E ?e ?Q) =>
reshape_expr e ltac:(fun K e' => reshape_expr e ltac:(fun K e' =>
twp_bind_core K; iApplyHyp H; wp_expr_simpl) || twp_bind_core K; iApplyHyp H; try wp_expr_simpl) ||
lazymatch iTypeOf H with lazymatch iTypeOf H with
| Some (_,?P) => fail "wp_apply: cannot apply" P | Some (_,?P) => fail "wp_apply: cannot apply" P
end end
......
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