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
Simon Spies
Iris
Commits
cbf274c0
Commit
cbf274c0
authored
Nov 17, 2016
by
Robbert Krebbers
Browse files
Existentials commute with disjunction.
parent
4ecb139a
Changes
1
Show whitespace changes
Inline
Side-by-side
base_logic/derived.v
View file @
cbf274c0
...
...
@@ -199,6 +199,13 @@ Lemma and_exist_r {A} P (Φ: A → uPred M) : (∃ a, Φ a) ∧ P ⊣⊢ ∃ a,
Proof
.
rewrite
-(
comm
_
P
)
and_exist_l
.
apply
exist_proper
=>
a
.
by
rewrite
comm
.
Qed
.
Lemma
or_exist
{
A
}
(
Φ
Ψ
:
A
→
uPred
M
)
:
(
∃
a
,
Φ
a
∨
Ψ
a
)
⊣
⊢
(
∃
a
,
Φ
a
)
∨
(
∃
a
,
Ψ
a
).
Proof
.
apply
(
anti_symm
(
⊢
)).
-
apply
exist_elim
=>
a
.
by
rewrite
-!(
exist_intro
a
).
-
apply
or_elim
;
apply
exist_elim
=>
a
;
rewrite
-(
exist_intro
a
)
;
auto
.
Qed
.
Lemma
pure_mono
φ
1
φ
2
:
(
φ
1
→
φ
2
)
→
■
φ
1
⊢
■
φ
2
.
Proof
.
intros
;
apply
pure_elim
with
φ
1
;
eauto
.
Qed
.
...
...
Write
Preview
Supports
Markdown
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