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

Add test.

parent b3901a51
No related branches found
No related tags found
No related merge requests found
From iris.algebra Require Import gmap.
From iris.bi Require Import laterable. From iris.bi Require Import laterable.
From iris.proofmode Require Import tactics intro_patterns. From iris.proofmode Require Import tactics intro_patterns.
From iris.prelude Require Import options. From iris.prelude Require Import options.
...@@ -81,6 +82,11 @@ Proof. ...@@ -81,6 +82,11 @@ Proof.
auto. auto.
Qed. Qed.
Lemma test_iRewrite_dom `{!BiInternalEq PROP} {A : ofe} (m1 m2 : gmap nat A) :
m1 m2 ⊢@{PROP}
dom (gset nat) m1 = dom (gset nat) m2 ⌝.
Proof. iIntros "H". by iRewrite "H". Qed.
Check "test_iDestruct_and_emp". Check "test_iDestruct_and_emp".
Lemma test_iDestruct_and_emp P Q `{!Persistent P, !Persistent Q} : Lemma test_iDestruct_and_emp P Q `{!Persistent P, !Persistent Q} :
P emp -∗ emp Q -∗ <affine> (P Q). P emp -∗ emp Q -∗ <affine> (P Q).
......
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