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

heap_lang/proofmode: move pm_prettify to where we used to do lazy beta

parent 3d1e22c5
No related branches found
No related tags found
No related merge requests found
...@@ -27,8 +27,8 @@ Tactic Notation "wp_expr_eval" tactic(t) := ...@@ -27,8 +27,8 @@ Tactic Notation "wp_expr_eval" tactic(t) :=
| _ => fail "wp_expr_eval: not a 'wp'" | _ => fail "wp_expr_eval: not a 'wp'"
end. end.
Ltac wp_expr_simpl := (wp_expr_eval simpl); pm_prettify. Ltac wp_expr_simpl := wp_expr_eval simpl.
Ltac wp_expr_simpl_subst := (wp_expr_eval simpl_subst); pm_prettify. Ltac wp_expr_simpl_subst := wp_expr_eval simpl_subst.
Lemma tac_wp_pure `{heapG Σ} Δ Δ' s E e1 e2 φ Φ : Lemma tac_wp_pure `{heapG Σ} Δ Δ' s E e1 e2 φ Φ :
PureExec φ e1 e2 PureExec φ e1 e2
...@@ -61,7 +61,7 @@ Proof. rewrite envs_entails_eq=> ? ->. by apply twp_value. Qed. ...@@ -61,7 +61,7 @@ Proof. rewrite envs_entails_eq=> ? ->. by apply twp_value. Qed.
Ltac wp_value_head := Ltac wp_value_head :=
first [eapply tac_wp_value || eapply tac_twp_value]; first [eapply tac_wp_value || eapply tac_twp_value];
[iSolveTC [iSolveTC
|iEval (lazy beta; simpl of_val)]. |reduction.pm_prettify; iEval (simpl of_val)].
Tactic Notation "wp_pure" open_constr(efoc) := Tactic Notation "wp_pure" open_constr(efoc) :=
iStartProof; iStartProof;
...@@ -118,12 +118,12 @@ Proof. rewrite envs_entails_eq=> -> ->. by apply: twp_bind. Qed. ...@@ -118,12 +118,12 @@ Proof. rewrite envs_entails_eq=> -> ->. by apply: twp_bind. Qed.
Ltac wp_bind_core K := Ltac wp_bind_core K :=
lazymatch eval hnf in K with lazymatch eval hnf in K with
| [] => idtac | [] => idtac
| _ => eapply (tac_wp_bind K); [simpl; reflexivity|lazy beta] | _ => eapply (tac_wp_bind K); [simpl; reflexivity|reduction.pm_prettify]
end. end.
Ltac twp_bind_core K := Ltac twp_bind_core K :=
lazymatch eval hnf in K with lazymatch eval hnf in K with
| [] => idtac | [] => idtac
| _ => eapply (tac_twp_bind K); [simpl; reflexivity|lazy beta] | _ => eapply (tac_twp_bind K); [simpl; reflexivity|reduction.pm_prettify]
end. end.
Tactic Notation "wp_bind" open_constr(efoc) := Tactic Notation "wp_bind" open_constr(efoc) :=
......
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