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
Jonas Kastberg
iris
Commits
c5fa01fe
Commit
c5fa01fe
authored
Dec 07, 2017
by
Ralf Jung
Browse files
Options
Browse Files
Download
Email Patches
Plain Diff
rename adequate_safe -> adequate_not_stuck
parent
f8890ff9
Changes
2
Hide whitespace changes
Inline
Side-by-side
Showing
2 changed files
with
3 additions
and
2 deletions
+3
-2
CHANGELOG.md
CHANGELOG.md
+1
-0
theories/program_logic/adequacy.v
theories/program_logic/adequacy.v
+2
-2
No files found.
CHANGELOG.md
View file @
c5fa01fe
...
...
@@ -34,6 +34,7 @@ Changes in Coq:
-
Camera elements such that
`core x = x`
:
`Persistent`
->
`CoreId`
-
Persistent propositions:
`PersistentP`
->
`Persistent`
-
The persistent modality:
`always`
->
`persistently`
-
Adequacy for non-stuck weakestpre:
`adequate_safe`
->
`adequate_not_stuck`
-
Consistently SnakeCase identifiers:
+
`CMRAMixin`
->
`CmraMixin`
+
`CMRAT`
->
`CmraT`
...
...
theories/program_logic/adequacy.v
View file @
c5fa01fe
...
...
@@ -37,7 +37,7 @@ Qed.
Record
adequate
{
Λ
}
(
s
:
stuckness
)
(
e1
:
expr
Λ
)
(
σ
1
:
state
Λ
)
(
φ
:
val
Λ
→
Prop
)
:
=
{
adequate_result
t2
σ
2
v2
:
rtc
step
([
e1
],
σ
1
)
(
of_val
v2
::
t2
,
σ
2
)
→
φ
v2
;
adequate_
safe
t2
σ
2 e2
:
adequate_
not_stuck
t2
σ
2 e2
:
s
=
NotStuck
→
rtc
step
([
e1
],
σ
1
)
(
t2
,
σ
2
)
→
e2
∈
t2
→
(
is_Some
(
to_val
e2
)
∨
reducible
e2
σ
2
)
...
...
@@ -51,7 +51,7 @@ Proof.
intros
Had
?.
destruct
(
decide
(
Forall
(
λ
e
,
is_Some
(
to_val
e
))
t2
))
as
[|
Ht2
]
;
[
by
left
|].
apply
(
not_Forall_Exists
_
),
Exists_exists
in
Ht2
;
destruct
Ht2
as
(
e2
&?&
He2
).
destruct
(
adequate_
safe
NotStuck
e1
σ
1
φ
Had
t2
σ
2 e2
)
as
[?|(
e3
&
σ
3
&
efs
&?)]
;
destruct
(
adequate_
not_stuck
NotStuck
e1
σ
1
φ
Had
t2
σ
2 e2
)
as
[?|(
e3
&
σ
3
&
efs
&?)]
;
rewrite
?eq_None_not_Some
;
auto
.
{
exfalso
.
eauto
.
}
destruct
(
elem_of_list_split
t2
e2
)
as
(
t2'
&
t2''
&->)
;
auto
.
...
...
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