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

add more tests

parent 260e0593
No related branches found
No related tags found
No related merge requests found
...@@ -457,17 +457,17 @@ Proof. iIntros (?) "HP #HQ HR". iPureIntro; eauto. Qed. ...@@ -457,17 +457,17 @@ Proof. iIntros (?) "HP #HQ HR". iPureIntro; eauto. Qed.
(* Ensure that [% ...] works as a pattern when the left-hand side of and/sep is (* Ensure that [% ...] works as a pattern when the left-hand side of and/sep is
pure. *) pure. *)
Lemma test_pure_and_sep_destruct_affine `{!BiAffine PROP} (φ : Prop) (P : PROP) : Lemma test_pure_and_sep_destruct_affine `{!BiAffine PROP} (φ : Prop) P :
φ (φ P) -∗ P. φ (φ P) -∗ P.
Proof. Proof.
iIntros "[% [% $]]". iIntros "[% [% $]]".
Qed. Qed.
Lemma test_pure_and_sep_destruct_1 (φ : Prop) (P : PROP) : Lemma test_pure_and_sep_destruct_1 (φ : Prop) P :
φ (<affine> φ P) -∗ P. φ (<affine> φ P) -∗ P.
Proof. Proof.
iIntros "[% [% $]]". iIntros "[% [% $]]".
Qed. Qed.
Lemma test_pure_and_sep_destruct_2 (φ : Prop) (P : PROP) : Lemma test_pure_and_sep_destruct_2 (φ : Prop) P :
φ (φ <absorb> P) -∗ <absorb> P. φ (φ <absorb> P) -∗ <absorb> P.
Proof. Proof.
iIntros "[% [% $]]". iIntros "[% [% $]]".
......
...@@ -103,6 +103,17 @@ Section tests. ...@@ -103,6 +103,17 @@ Section tests.
iAssumption. iAssumption.
Qed. Qed.
Lemma test_monPred_at_and_pure P i j :
(monPred_in j P) i j i P i.
Proof.
iDestruct 1 as "[% $]". done.
Qed.
Lemma test_monPred_at_sep_pure P i j :
(monPred_in j <absorb> P) i j i <absorb> P i.
Proof.
iDestruct 1 as "[% ?]". auto.
Qed.
Context (FU : BiFUpd PROP). Context (FU : BiFUpd PROP).
Lemma test_apply_fupd_intro_mask_subseteq E1 E2 P : Lemma test_apply_fupd_intro_mask_subseteq E1 E2 P :
......
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