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

Use uPred_pure for instead of uPred_forall in core.v.

parent 8e0effe3
No related branches found
No related tags found
No related merge requests found
......@@ -8,7 +8,7 @@ Import uPred.
in the shallow embedding. *)
Definition coreP {M : ucmraT} (P : uPred M) : uPred M :=
( `(!PersistentP Q, P Q), Q)%I.
( `(!PersistentP Q), P Q Q)%I.
Instance: Params (@coreP) 1.
Typeclasses Opaque coreP.
......@@ -25,7 +25,7 @@ Section core.
Global Instance coreP_mono : Proper (() ==> ()) (@coreP M).
Proof.
rewrite /coreP. iIntros (P P' ?) "H"; iIntros (Q ??).
unshelve iApply ("H" $! Q). by etrans.
iApply ("H" $! Q with "[%]"). by etrans.
Qed.
Global Instance coreP_proper : Proper ((⊣⊢) ==> (⊣⊢)) (@coreP M).
......
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