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
c78daf89
Commit
c78daf89
authored
Feb 13, 2016
by
Ralf Jung
Browse files
Options
Browse Files
Download
Email Patches
Plain Diff
try to rely more on eauto - and fail and leave some FIXMEs
parent
ef3214e0
Changes
1
Hide whitespace changes
Inline
Side-by-side
Showing
1 changed file
with
6 additions
and
1 deletion
+6
-1
program_logic/viewshifts.v
program_logic/viewshifts.v
+6
-1
No files found.
program_logic/viewshifts.v
View file @
c78daf89
...
...
@@ -86,13 +86,18 @@ Qed.
Lemma
vs_mask_frame
'
E
Ef
P
Q
:
Ef
∩
E
=
∅
→
(
P
={
E
}=>
Q
)
⊑
(
P
={
E
∪
Ef
}=>
Q
).
Proof
.
intros
;
apply
vs_mask_frame
;
solve_elem_of
.
Qed
.
(
*
FIXME
:
This
is
needed
to
make
eauto
solve
[
inv
N
R
⊑
inv
N
?
c
].
*
)
Local
Hint
Extern
100
(
_
⊑
_
)
=>
reflexivity
.
Lemma
vs_open_close
N
E
P
Q
R
:
nclose
N
⊆
E
→
(
inv
N
R
★
(
▷
R
★
P
={
E
∖
nclose
N
}=>
▷
R
★
Q
))
⊑
(
P
={
E
}=>
Q
).
Proof
.
intros
;
apply
(
always_intro
_
_
),
impl_intro_l
.
rewrite
always_and_sep_r
assoc
[(
P
★
_
)
%
I
]
comm
-
assoc
.
apply:
(
pvs_open_close
E
N
);
[
by
eauto
using
sep_elim_l
..
|
].
(
*
FIXME
sep_elim_l
'
is
already
added
to
the
DB
in
upred
.
v
.
Why
do
I
have
to
mention
it
here
again
?
*
)
apply:
(
pvs_open_close
E
N
);
[
by
eauto
using
sep_elim_l
'
..
|
].
rewrite
sep_elim_r
.
apply
wand_intro_l
.
(
*
Oh
wow
,
this
is
annyoing
...
*
)
rewrite
assoc
-
always_and_sep_r
'
.
...
...
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