Skip to content
GitLab
Projects
Groups
Snippets
Help
Loading...
Help
What's new
10
Help
Support
Community forum
Keyboard shortcuts
?
Submit feedback
Contribute to GitLab
Sign in / Register
Toggle navigation
Open sidebar
Joshua Yanovski
iris-coq
Commits
65171af2
Commit
65171af2
authored
Sep 23, 2016
by
Robbert Krebbers
Browse files
Options
Browse Files
Download
Email Patches
Plain Diff
Alternative version of ownM_empty.
parent
1aac61c4
Changes
1
Hide whitespace changes
Inline
Side-by-side
Showing
1 changed file
with
2 additions
and
0 deletions
+2
-0
algebra/upred.v
algebra/upred.v
+2
-0
No files found.
algebra/upred.v
View file @
65171af2
...
...
@@ -1257,6 +1257,8 @@ Lemma ownM_invalid (a : M) : ¬ ✓{0} a → uPred_ownM a ⊢ False.
Proof
.
by
intros
;
rewrite
ownM_valid
valid_elim
.
Qed
.
Global
Instance
ownM_mono
:
Proper
(
flip
(
≼
)
==>
(
⊢
))
(
@
uPred_ownM
M
).
Proof
.
intros
a
b
[
b
'
->
].
rewrite
ownM_op
.
eauto
.
Qed
.
Lemma
ownM_empty
'
:
uPred_ownM
∅
⊣⊢
True
.
Proof
.
apply
(
anti_symm
_
);
auto
using
ownM_empty
.
Qed
.
(
*
Viewshifts
*
)
Lemma
rvs_intro
P
:
P
=
r
=>
P
.
...
...
Write
Preview
Markdown
is supported
0%
Try again
or
attach a new file
.
Attach a file
Cancel
You are about to add
0
people
to the discussion. Proceed with caution.
Finish editing this message first!
Cancel
Please
register
or
sign in
to comment