Skip to content
GitLab
Projects
Groups
Snippets
Help
Loading...
Help
Help
Support
Community forum
Keyboard shortcuts
?
Submit feedback
Contribute to GitLab
Sign in / Register
Toggle navigation
I
iris-coq
Project overview
Project overview
Details
Activity
Releases
Repository
Repository
Files
Commits
Branches
Tags
Contributors
Graph
Compare
Issues
0
Issues
0
List
Boards
Labels
Service Desk
Milestones
Merge Requests
0
Merge Requests
0
CI / CD
CI / CD
Pipelines
Jobs
Schedules
Operations
Operations
Incidents
Environments
Analytics
Analytics
CI / CD
Repository
Value Stream
Wiki
Wiki
Snippets
Snippets
Members
Members
Collapse sidebar
Close sidebar
Activity
Graph
Create a new issue
Jobs
Commits
Issue Boards
Open sidebar
Janno
iris-coq
Commits
191a6f43
Commit
191a6f43
authored
Jun 28, 2018
by
Ralf Jung
Browse files
Options
Browse Files
Download
Email Patches
Plain Diff
fix nits
parent
6d15cf39
Changes
2
Show whitespace changes
Inline
Side-by-side
Showing
2 changed files
with
13 additions
and
14 deletions
+13
-14
tests/proofmode.v
tests/proofmode.v
+8
-9
theories/bi/telescopes.v
theories/bi/telescopes.v
+5
-5
No files found.
tests/proofmode.v
View file @
191a6f43
...
...
@@ -534,15 +534,14 @@ Proof.
Qed
.
Section
wandM
.
Import
proofmode
.
base
.
Lemma
test_wandM
mP
Q
R
:
Import
proofmode
.
base
.
Lemma
test_wandM
mP
Q
R
:
(
mP
-
∗
?
Q
)
-
∗
(
Q
-
∗
R
)
-
∗
(
mP
-
∗
?
R
).
Proof
.
Proof
.
iIntros
"HPQ HQR HP"
.
Show
.
iApply
"HQR"
.
iApply
"HPQ"
.
Show
.
done
.
Qed
.
Qed
.
End
wandM
.
End
tests
.
...
...
theories/bi/telescopes.v
View file @
191a6f43
...
...
@@ -23,8 +23,8 @@ Notation "'∀..' x .. y , P" := (bi_tforall (λ x, .. (bi_tforall (λ y, P)) ..
Section
telescope_quantifiers
.
Context
{
PROP
:
bi
}
{
TT
:
tele
}.
Lemma
bi_tforall_forall
(
Ψ
:
TT
->
PROP
)
:
(
bi_tforall
Ψ
)
⊣
⊢
(
bi_forall
Ψ
)
.
Lemma
bi_tforall_forall
(
Ψ
:
TT
→
PROP
)
:
bi_tforall
Ψ
⊣
⊢
bi_forall
Ψ
.
Proof
.
symmetry
.
unfold
bi_tforall
.
induction
TT
as
[|
X
ft
IH
].
-
simpl
.
apply
(
anti_symm
_
).
...
...
@@ -36,11 +36,11 @@ Section telescope_quantifiers.
by
rewrite
(
forall_elim
(
TargS
a
p
)).
+
move
/
tele_arg_inv
:
(
a
)
=>
[
x
[
pf
->]]
{
a
}
/=.
setoid_rewrite
<-
IH
.
do
2
rewrite
forall_elim
.
done
.
rewrite
2
!
forall_elim
.
done
.
Qed
.
Lemma
bi_texist_exist
(
Ψ
:
TT
->
PROP
)
:
(
bi_texist
Ψ
)
⊣
⊢
(
bi_exist
Ψ
)
.
Lemma
bi_texist_exist
(
Ψ
:
TT
→
PROP
)
:
bi_texist
Ψ
⊣
⊢
bi_exist
Ψ
.
Proof
.
symmetry
.
unfold
bi_texist
.
induction
TT
as
[|
X
ft
IH
].
-
simpl
.
apply
(
anti_symm
_
).
...
...
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