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

Tests for type-directed unsealing of `monPred` and `uPred`.

parent bab52efb
No related branches found
No related tags found
No related merge requests found
"monPred_unseal_test_1"
: string
1 goal
I : biIndex
M : ucmra
P, Q : uPredI M
R : monPred
i : I
============================
(P ∗ Q) ∗ R i ⊣⊢ False
"monPred_unseal_test_2"
: string
1 goal
I : biIndex
M : ucmra
P, Q : uPredI M
R : monPred
============================
⎡ upred.uPred_sep_def P Q ⎤ ∗ R ⊣⊢ False
From stdpp Require Import strings.
From iris.base_logic Require Import bi.
From iris.bi Require Import embedding monpred.
Section tests_unseal.
Context {I : biIndex} (M : ucmra).
Local Notation monPred := (monPred I (uPredI M)).
Check "monPred_unseal_test_1".
Lemma monPred_unseal_test_1 P Q (R : monPred) :
P Q R ⊣⊢ False.
Proof.
intros. split=> i. monPred.unseal.
(** Make sure [∗] on uPred is not unfolded *)
Show.
Abort.
Check "monPred_unseal_test_2".
Lemma monPred_unseal_test_2 P Q (R : monPred) :
P Q R ⊣⊢ False.
Restart.
uPred.unseal.
(** Make sure [∗] on monPred is not unfolded *)
Show.
Abort.
End tests_unseal.
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