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

Use ;; for seq, ; conflicts with lists.

parent 8c96ad4e
No related branches found
No related tags found
No related merge requests found
...@@ -50,5 +50,5 @@ Notation "λ: x , e" := (LamV x e%L) ...@@ -50,5 +50,5 @@ Notation "λ: x , e" := (LamV x e%L)
(at level 102, x at level 1, e at level 200) : lang_scope. (at level 102, x at level 1, e at level 200) : lang_scope.
Notation "'let:' x := e1 'in' e2" := (Lam x e2%L e1%L) Notation "'let:' x := e1 'in' e2" := (Lam x e2%L e1%L)
(at level 102, x at level 1, e1, e2 at level 200) : lang_scope. (at level 102, x at level 1, e1, e2 at level 200) : lang_scope.
Notation "e1 ; e2" := (Lam "" e2%L e1%L) Notation "e1 ;; e2" := (Lam "" e2%L e1%L)
(at level 100, e2 at level 200) : lang_scope. (at level 100, e2 at level 200) : lang_scope.
...@@ -27,7 +27,7 @@ Module LiftingTests. ...@@ -27,7 +27,7 @@ Module LiftingTests.
Implicit Types Q : val iProp heap_lang Σ. Implicit Types Q : val iProp heap_lang Σ.
Definition e : expr := Definition e : expr :=
let: "x" := ref '1 in "x" <- !"x" + '1; !"x". let: "x" := ref '1 in "x" <- !"x" + '1;; !"x".
Goal σ E, ownP (Σ:=Σ) σ wp E e (λ v, v = ('2)%L). Goal σ E, ownP (Σ:=Σ) σ wp E e (λ v, v = ('2)%L).
Proof. Proof.
move=> σ E. rewrite /e. move=> σ E. rewrite /e.
...@@ -86,10 +86,6 @@ Module LiftingTests. ...@@ -86,10 +86,6 @@ Module LiftingTests.
by rewrite -!later_intro -wp_value' // and_elim_r. by rewrite -!later_intro -wp_value' // and_elim_r.
Qed. Qed.
(* FIXME : For now apparent reason, I cannot prove this inline. *)
Lemma Pred_sub_helper n : n - 1 = - (- n + 2 - 1).
Proof. intros. omega. Qed.
Lemma Pred_spec n E Q : Q (LitV (n - 1)) wp E (Pred 'n)%L Q. Lemma Pred_spec n E Q : Q (LitV (n - 1)) wp E (Pred 'n)%L Q.
Proof. Proof.
rewrite -wp_lam //=. rewrite -wp_lam //=.
...@@ -97,8 +93,7 @@ Module LiftingTests. ...@@ -97,8 +93,7 @@ Module LiftingTests.
apply later_mono, wp_le=> Hn. apply later_mono, wp_le=> Hn.
- rewrite -wp_if_true. - rewrite -wp_if_true.
rewrite -(wp_bindi (UnOpCtx _)). rewrite -(wp_bindi (UnOpCtx _)).
(* FIXME use list notation. *) rewrite -(wp_bind [AppLCtx _; AppRCtx FindPred]).
rewrite -(wp_bind ((AppLCtx _)::(AppRCtx FindPred)::nil)).
rewrite -(wp_bindi (BinOpLCtx _ _)). rewrite -(wp_bindi (BinOpLCtx _ _)).
rewrite -wp_un_op //=. rewrite -wp_un_op //=.
rewrite -wp_bin_op //= -!later_intro. rewrite -wp_bin_op //= -!later_intro.
......
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