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
Iris
c
Commits
225b639d
Commit
225b639d
authored
Jan 25, 2019
by
Robbert Krebbers
Browse files
Options
Browse Files
Download
Email Patches
Plain Diff
Remove useless eta expansion.
parent
845d6b1d
Changes
1
Hide whitespace changes
Inline
Side-by-side
Showing
1 changed file
with
2 additions
and
2 deletions
+2
-2
theories/c_translation/translation.v
theories/c_translation/translation.v
+2
-2
No files found.
theories/c_translation/translation.v
View file @
225b639d
...
...
@@ -90,7 +90,7 @@ Notation "'skipᶜ'" := (c_ret #()).
Definition
c_seq_bind
:
val
:
=
λ
:
"x"
"f"
,
"a"
←ᶜ
"x"
;;
ᶜ
c_atomic_env
(
λ
:
"env"
,
mset_clear
"env"
)
;;
ᶜ
c_atomic_env
mset_clear
;;
ᶜ
"f"
"a"
.
Notation
"x ←ᶜ e1 ;ᶜ e2"
:
=
(
c_seq_bind
e1
%
E
(
λ
:
x
,
e2
)%
E
)%
E
...
...
@@ -393,7 +393,7 @@ Section proofs.
cwp_pures
.
iApply
cwp_bind
.
iApply
cwp_atomic_env
.
iIntros
(
env
)
"Henv $"
.
iApply
wp_fupd
.
iDestruct
"Henv"
as
(
X
σ
_
)
"[Hlocks Hσ]"
.
wp_lam
.
wp_apply
(
mset_clear_spec
with
"Hlocks"
)
;
iIntros
"Hlocks"
.
wp_apply
(
mset_clear_spec
with
"Hlocks"
)
;
iIntros
"Hlocks"
.
rewrite
U_eq
.
iDestruct
"H"
as
(
us
)
"[Hus H]"
.
iInduction
us
as
[|[
ul
[
uq
uv
]]
us
]
"IH"
forall
(
σ
)
;
simpl
.
-
iModIntro
.
iSplitR
"H"
.
...
...
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