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
Rodolphe Lepigre
Iris
Commits
1e579d55
Commit
1e579d55
authored
Dec 03, 2017
by
Robbert Krebbers
Browse files
One direction of wand_impl_persistently holds for non-affine BIs.
parent
35769f67
Changes
1
Show whitespace changes
Inline
Side-by-side
theories/bi/derived.v
View file @
1e579d55
...
@@ -1072,6 +1072,9 @@ Proof.
...
@@ -1072,6 +1072,9 @@ Proof.
by
rewrite
(
comm
bi_and
)
persistently_and_emp_elim
wand_elim_l
.
by
rewrite
(
comm
bi_and
)
persistently_and_emp_elim
wand_elim_l
.
Qed
.
Qed
.
Lemma
wand_impl_persistently_2
P
Q
:
(
bi_persistently
P
-
∗
Q
)
⊢
(
bi_persistently
P
→
Q
).
Proof
.
apply
impl_intro_l
.
by
rewrite
persistently_and_sep_l_1
wand_elim_r
.
Qed
.
Section
persistently_affinely_bi
.
Section
persistently_affinely_bi
.
Context
`
{
AffineBI
PROP
}.
Context
`
{
AffineBI
PROP
}.
...
@@ -1095,6 +1098,11 @@ Section persistently_affinely_bi.
...
@@ -1095,6 +1098,11 @@ Section persistently_affinely_bi.
by
rewrite
-
persistently_and_sep_r
persistently_elim
impl_elim_r
.
by
rewrite
-
persistently_and_sep_r
persistently_elim
impl_elim_r
.
Qed
.
Qed
.
Lemma
wand_impl_persistently
P
Q
:
(
bi_persistently
P
-
∗
Q
)
⊣
⊢
(
bi_persistently
P
→
Q
).
Proof
.
apply
(
anti_symm
(
⊢
)).
apply
wand_impl_persistently_2
.
by
rewrite
-
impl_wand_1
.
Qed
.
Lemma
wand_alt
P
Q
:
(
P
-
∗
Q
)
⊣
⊢
∃
R
,
R
∗
bi_persistently
(
P
∗
R
→
Q
).
Lemma
wand_alt
P
Q
:
(
P
-
∗
Q
)
⊣
⊢
∃
R
,
R
∗
bi_persistently
(
P
∗
R
→
Q
).
Proof
.
Proof
.
apply
(
anti_symm
(
⊢
)).
apply
(
anti_symm
(
⊢
)).
...
@@ -1259,6 +1267,9 @@ Proof.
...
@@ -1259,6 +1267,9 @@ Proof.
by
rewrite
(
comm
bi_and
)
plainly_and_emp_elim
wand_elim_l
.
by
rewrite
(
comm
bi_and
)
plainly_and_emp_elim
wand_elim_l
.
Qed
.
Qed
.
Lemma
wand_impl_plainly_2
P
Q
:
(
bi_plainly
P
-
∗
Q
)
⊢
(
bi_plainly
P
→
Q
).
Proof
.
apply
impl_intro_l
.
by
rewrite
plainly_and_sep_l_1
wand_elim_r
.
Qed
.
Section
plainly_affinely_bi
.
Section
plainly_affinely_bi
.
Context
`
{
AffineBI
PROP
}.
Context
`
{
AffineBI
PROP
}.
...
@@ -1280,16 +1291,9 @@ Section plainly_affinely_bi.
...
@@ -1280,16 +1291,9 @@ Section plainly_affinely_bi.
by
rewrite
-
plainly_and_sep_r
plainly_elim
impl_elim_r
.
by
rewrite
-
plainly_and_sep_r
plainly_elim
impl_elim_r
.
Qed
.
Qed
.
Lemma
wand_impl_persistently
P
Q
:
(
bi_persistently
P
-
∗
Q
)
⊣
⊢
(
bi_persistently
P
→
Q
).
Proof
.
apply
(
anti_symm
(
⊢
))
;
[|
by
rewrite
-
impl_wand_1
].
apply
impl_intro_l
.
by
rewrite
persistently_and_sep_l
wand_elim_r
.
Qed
.
Lemma
wand_impl_plainly
P
Q
:
(
bi_plainly
P
-
∗
Q
)
⊣
⊢
(
bi_plainly
P
→
Q
).
Lemma
wand_impl_plainly
P
Q
:
(
bi_plainly
P
-
∗
Q
)
⊣
⊢
(
bi_plainly
P
→
Q
).
Proof
.
Proof
.
apply
(
anti_symm
(
⊢
))
;
[|
by
rewrite
-
impl_wand_1
].
apply
(
anti_symm
(
⊢
)).
by
rewrite
wand_impl_plainly_2
.
by
rewrite
-
impl_wand_1
.
apply
impl_intro_l
.
by
rewrite
plainly_and_sep_l
wand_elim_r
.
Qed
.
Qed
.
End
plainly_affinely_bi
.
End
plainly_affinely_bi
.
...
...
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