File: monpred.v

package info (click to toggle)
coq-iris 4.3.0-1
  • links: PTS, VCS
  • area: main
  • in suites: forky, sid, trixie
  • size: 4,116 kB
  • sloc: python: 130; makefile: 61; sh: 28; sed: 2
file content (27 lines) | stat: -rw-r--r-- 720 bytes parent folder | download
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
22
23
24
25
26
27
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.
  Proof.
    uPred.unseal.
    (** Make sure [∗] on monPred is not unfolded *)
    Show.
  Abort.
End tests_unseal.