Skip to content
GitLab
Projects
Groups
Snippets
/
Help
Help
Support
Community forum
Keyboard shortcuts
?
Submit feedback
Contribute to GitLab
Sign in / Register
Toggle navigation
Menu
Open sidebar
Iris
Iris
Commits
5470da51
Commit
5470da51
authored
Feb 02, 2016
by
Ralf Jung
Browse files
less unnecessary importing
parent
531d88c1
Changes
1
Hide whitespace changes
Inline
Side-by-side
barrier/heap_lang.v
View file @
5470da51
...
...
@@ -309,7 +309,6 @@ Program Canonical Structure heap_lang : language := {|
|}.
Solve
Obligations
with
eauto
using
heap_lang
.
to_of_val
,
heap_lang
.
of_to_val
,
heap_lang
.
values_stuck
,
heap_lang
.
atomic_not_val
,
heap_lang
.
atomic_step
.
Import
heap_lang
.
Global
Instance
heap_lang_ctx
K
:
LanguageCtx
heap_lang
(
heap_lang
.
fill
K
).
...
...
@@ -322,6 +321,6 @@ Proof.
destruct
(
heap_lang
.
step_by_val
K
K''
e1
e1''
σ
1 e2
''
σ
2
ef
)
as
[
K'
->]
;
eauto
.
rewrite
heap_lang
.
fill_app
in
Heq1
;
apply
(
injective
_
)
in
Heq1
.
exists
(
fill
K'
e2''
)
;
rewrite
heap_lang
.
fill_app
;
split
;
auto
.
exists
(
heap_lang
.
fill
K'
e2''
)
;
rewrite
heap_lang
.
fill_app
;
split
;
auto
.
econstructor
;
eauto
.
Qed
.
Write
Preview
Supports
Markdown
0%
Try again
or
attach a new 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