Skip to content
GitLab
Menu
Projects
Groups
Snippets
Help
Help
Support
Community forum
Keyboard shortcuts
?
Submit feedback
Contribute to GitLab
Sign in / Register
Toggle navigation
Menu
Open sidebar
Pierre-Marie Pédrot
Iris
Commits
381e8509
Commit
381e8509
authored
Jun 13, 2017
by
Robbert Krebbers
Browse files
Let always_idemp be the rule `□ □ P ⊣⊢ □ P` in both ways.
parent
f72ccbec
Changes
2
Hide whitespace changes
Inline
Side-by-side
theories/base_logic/derived.v
View file @
381e8509
...
...
@@ -478,9 +478,9 @@ Global Instance always_flip_mono' :
Proof
.
intros
P
Q
;
apply
always_mono
.
Qed
.
Lemma
always_intro'
P
Q
:
(
□
P
⊢
Q
)
→
□
P
⊢
□
Q
.
Proof
.
intros
<-.
apply
always_idemp
.
Qed
.
Proof
.
intros
<-.
apply
always_idemp
_2
.
Qed
.
Lemma
always_idemp
P
:
□
□
P
⊣
⊢
□
P
.
Proof
.
apply
(
anti_symm
_
)
;
auto
using
always_idemp
.
Qed
.
Proof
.
apply
(
anti_symm
_
)
;
auto
using
always_idemp
_2
.
Qed
.
Lemma
always_pure
φ
:
□
⌜φ⌝
⊣
⊢
⌜φ⌝
.
Proof
.
apply
(
anti_symm
_
)
;
auto
using
always_pure_2
.
Qed
.
...
...
theories/base_logic/primitive.v
View file @
381e8509
...
...
@@ -427,7 +427,7 @@ Proof.
unseal
;
split
=>
n
x
?
/=.
eauto
using
uPred_mono
,
@
cmra_included_core
,
cmra_included_includedN
.
Qed
.
Lemma
always_idemp
P
:
□
P
⊢
□
□
P
.
Lemma
always_idemp
_2
P
:
□
P
⊢
□
□
P
.
Proof
.
unseal
;
split
=>
n
x
??
/=.
by
rewrite
cmra_core_idemp
.
Qed
.
Lemma
always_pure_2
φ
:
⌜φ⌝
⊢
□
⌜φ⌝
.
...
...
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