Skip to content
GitLab
Explore
Sign in
Primary navigation
Search or go to…
Project
ReLoC
Manage
Activity
Members
Labels
Plan
Issues
Issue boards
Milestones
Code
Merge requests
Repository
Branches
Commits
Tags
Repository graph
Compare revisions
Snippets
Build
Pipelines
Jobs
Pipeline schedules
Artifacts
Deploy
Releases
Model registry
Operate
Environments
Monitor
Incidents
Service Desk
Analyze
Value stream analytics
Contributor analytics
CI/CD analytics
Repository analytics
Model experiments
Help
Help
Support
GitLab documentation
Compare GitLab plans
Community forum
Contribute to GitLab
Provide feedback
Terms and privacy
Keyboard shortcuts
?
Snippets
Groups
Projects
Show more breadcrumbs
Iris
ReLoC
Commits
b7ca3e83
Commit
b7ca3e83
authored
6 years ago
by
Dan Frumin
Browse files
Options
Downloads
Patches
Plain Diff
Renamings
parent
94d94ab2
No related branches found
Branches containing commit
No related tags found
No related merge requests found
Changes
3
Hide whitespace changes
Inline
Side-by-side
Showing
3 changed files
theories/logic/model.v
+33
-24
33 additions, 24 deletions
theories/logic/model.v
theories/logic/spec_ra.v
+3
-3
3 additions, 3 deletions
theories/logic/spec_ra.v
theories/logic/spec_rules.v
+1
-1
1 addition, 1 deletion
theories/logic/spec_rules.v
with
37 additions
and
28 deletions
theories/logic/model.v
+
33
−
24
View file @
b7ca3e83
...
@@ -10,7 +10,7 @@ From iris.heap_lang Require Import notation proofmode.
...
@@ -10,7 +10,7 @@ From iris.heap_lang Require Import notation proofmode.
From
reloc
Require
Import
logic
.
spec_rules
prelude
.
ctx_subst
.
From
reloc
Require
Import
logic
.
spec_rules
prelude
.
ctx_subst
.
(** Semantic intepretation of types *)
(** Semantic intepretation of types *)
Record
lty2
`{
log
relG
Σ
}
:=
Lty2
{
Record
lty2
`{
rel
oc
G
Σ
}
:=
Lty2
{
lty2_car
:>
val
→
val
→
iProp
Σ
;
lty2_car
:>
val
→
val
→
iProp
Σ
;
lty2_persistent
v1
v2
:
Persistent
(
lty2_car
v1
v2
)
lty2_persistent
v1
v2
:
Persistent
(
lty2_car
v1
v2
)
}
.
}
.
...
@@ -22,7 +22,7 @@ Existing Instance lty2_persistent.
...
@@ -22,7 +22,7 @@ Existing Instance lty2_persistent.
(* The COFE structure on semantic types *)
(* The COFE structure on semantic types *)
Section
lty2_ofe
.
Section
lty2_ofe
.
Context
`{
log
relG
Σ
}
.
Context
`{
rel
oc
G
Σ
}
.
Instance
lty2_equiv
:
Equiv
lty2
:=
λ
A
B
,
∀
w1
w2
,
A
w1
w2
≡
B
w1
w2
.
Instance
lty2_equiv
:
Equiv
lty2
:=
λ
A
B
,
∀
w1
w2
,
A
w1
w2
≡
B
w1
w2
.
Instance
lty2_dist
:
Dist
lty2
:=
λ
n
A
B
,
∀
w1
w2
,
A
w1
w2
≡
{
n
}
≡
B
w1
w2
.
Instance
lty2_dist
:
Dist
lty2
:=
λ
n
A
B
,
∀
w1
w2
,
A
w1
w2
≡
{
n
}
≡
B
w1
w2
.
...
@@ -47,7 +47,7 @@ Section lty2_ofe.
...
@@ -47,7 +47,7 @@ Section lty2_ofe.
End
lty2_ofe
.
End
lty2_ofe
.
Section
semtypes
.
Section
semtypes
.
Context
`{
log
relG
Σ
}
.
Context
`{
rel
oc
G
Σ
}
.
Implicit
Types
A
B
:
lty2
.
Implicit
Types
A
B
:
lty2
.
...
@@ -79,13 +79,13 @@ Infix "→" := lty2_arr : lty_scope.
...
@@ -79,13 +79,13 @@ Infix "→" := lty2_arr : lty_scope.
Notation
"'ref' A"
:=
(
lty2_ref
A
)
:
lty_scope
.
Notation
"'ref' A"
:=
(
lty2_ref
A
)
:
lty_scope
.
(* The semantic typing judgment *)
(* The semantic typing judgment *)
Definition
env_ltyped2
`{
log
relG
Σ
}
(
Γ
:
gmap
string
lty2
)
Definition
env_ltyped2
`{
rel
oc
G
Σ
}
(
Γ
:
gmap
string
lty2
)
(
vs
:
gmap
string
(
val
*
val
))
:
iProp
Σ
:=
(
vs
:
gmap
string
(
val
*
val
))
:
iProp
Σ
:=
(
⌜
∀
x
,
is_Some
(
Γ
!!
x
)
↔
is_Some
(
vs
!!
x
)
⌝
∧
(
⌜
∀
x
,
is_Some
(
Γ
!!
x
)
↔
is_Some
(
vs
!!
x
)
⌝
∧
[
∗
map
]
i
↦
Avv
∈
map_zip
Γ
vs
,
lty2_car
Avv
.
1
Avv
.
2
.
1
Avv
.
2
.
2
)
%
I
.
[
∗
map
]
i
↦
Avv
∈
map_zip
Γ
vs
,
lty2_car
Avv
.
1
Avv
.
2
.
1
Avv
.
2
.
2
)
%
I
.
Section
refinement
.
Section
refinement
.
Context
`{
log
relG
Σ
}
.
Context
`{
rel
oc
G
Σ
}
.
Definition
refines_def
(
E
:
coPset
)
Definition
refines_def
(
E
:
coPset
)
(
Γ
:
gmap
string
lty2
)
(
Γ
:
gmap
string
lty2
)
...
@@ -106,7 +106,7 @@ Notation "⟦ A ⟧ₑ" := (λ e e', interp_expr ⊤ e e' A).
...
@@ -106,7 +106,7 @@ Notation "⟦ A ⟧ₑ" := (λ e e', interp_expr ⊤ e e' A).
Notation
"⟦ Γ ⟧*"
:=
(
env_ltyped2
Γ
)
.
Notation
"⟦ Γ ⟧*"
:=
(
env_ltyped2
Γ
)
.
Section
semtypes_properties
.
Section
semtypes_properties
.
Context
`{
log
relG
Σ
}
.
Context
`{
rel
oc
G
Σ
}
.
(* The reference type relation is functional and injective.
(* The reference type relation is functional and injective.
Thanks to Amin. *)
Thanks to Amin. *)
...
@@ -154,7 +154,7 @@ Section semtypes_properties.
...
@@ -154,7 +154,7 @@ Section semtypes_properties.
End
semtypes_properties
.
End
semtypes_properties
.
Section
environment_properties
.
Section
environment_properties
.
Context
`{
log
relG
Σ
}
.
Context
`{
rel
oc
G
Σ
}
.
Implicit
Types
A
B
:
lty2
.
Implicit
Types
A
B
:
lty2
.
Implicit
Types
Γ
:
gmap
string
lty2
.
Implicit
Types
Γ
:
gmap
string
lty2
.
...
@@ -168,6 +168,7 @@ Section environment_properties.
...
@@ -168,6 +168,7 @@ Section environment_properties.
iApply
(
big_sepM_lookup
_
_
x
(
A
,
v
)
with
"HΓ"
)
.
iApply
(
big_sepM_lookup
_
_
x
(
A
,
v
)
with
"HΓ"
)
.
by
rewrite
map_lookup_zip_with
HΓx
/=
Hx
.
by
rewrite
map_lookup_zip_with
HΓx
/=
Hx
.
Qed
.
Qed
.
Lemma
env_ltyped2_insert
Γ
vs
x
A
v1
v2
:
Lemma
env_ltyped2_insert
Γ
vs
x
A
v1
v2
:
A
v1
v2
-∗
⟦
Γ
⟧
*
vs
-∗
A
v1
v2
-∗
⟦
Γ
⟧
*
vs
-∗
⟦
(
binder_insert
x
A
Γ
)
⟧
*
(
binder_insert
x
(
v1
,
v2
)
vs
)
.
⟦
(
binder_insert
x
A
Γ
)
⟧
*
(
binder_insert
x
(
v1
,
v2
)
vs
)
.
...
@@ -178,27 +179,35 @@ Section environment_properties.
...
@@ -178,27 +179,35 @@ Section environment_properties.
-
rewrite
-
map_insert_zip_with
.
by
iApply
big_sepM_insert_2
.
-
rewrite
-
map_insert_zip_with
.
by
iApply
big_sepM_insert_2
.
Qed
.
Qed
.
Lemma
env_ltyped2_empty
:
⟦
∅
⟧
*
∅.
Proof
.
iSplit
.
-
iPureIntro
=>
y
.
rewrite
!
lookup_empty
-!
not_eq_None_Some
.
by
naive_solver
.
-
by
rewrite
map_zip_with_empty
.
Qed
.
End
environment_properties
.
End
environment_properties
.
Notation
"'{' E ';' Γ '}' ⊨ e1 '
≼
' e2 : A"
:=
Notation
"'{' E ';' Γ '}' ⊨ e1 '
<<
' e2 : A"
:=
(
refines
E
Γ
e1
%
E
e2
%
E
(
A
)
%
lty2
)
(
refines
E
Γ
e1
%
E
e2
%
E
(
A
)
%
lty2
)
(
at
level
68
,
E
at
level
50
,
Γ
at
next
level
,
e1
,
e2
at
level
69
,
(
at
level
100
,
E
at
level
50
,
Γ
at
next
level
,
e1
,
e2
at
next
level
,
A
at
level
200
,
A
at
level
200
,
format
"'[hv' '{' E ';' Γ '}' ⊨ '/ ' e1 '/' '
≼
' '/ ' e2 : A ']'"
)
.
format
"'[hv' '{' E ';' Γ '}' ⊨ '/ ' e1 '/' '
<<
' '/ ' e2 : A ']'"
)
.
Notation
"Γ ⊨ e1 '
≼
' e2 : A"
:=
Notation
"Γ ⊨ e1 '
<<
' e2 : A"
:=
(
refines
⊤
Γ
e1
%
E
e2
%
E
(
A
)
%
lty2
)
%
I
(
refines
⊤
Γ
e1
%
E
e2
%
E
(
A
)
%
lty2
)
%
I
(
at
level
68
,
e1
,
e2
at
level
69
,
(
at
level
100
,
e1
,
e2
at
next
level
,
A
at
level
200
,
A
at
level
200
,
format
"'[hv' Γ ⊨ '/ ' e1 '/' '
≼
' '/ ' e2 : A ']'"
)
.
format
"'[hv' Γ ⊨ '/ ' e1 '/' '
<<
' '/ ' e2 : A ']'"
)
.
(** Properties of the relational interpretation *)
(** Properties of the relational interpretation *)
Section
related_facts
.
Section
related_facts
.
Context
`{
log
relG
Σ
}
.
Context
`{
rel
oc
G
Σ
}
.
(* We need this to be able to open and closed invariants in front of logrels *)
(* We need this to be able to open and closed invariants in front of logrels *)
Lemma
fupd_logrel
E1
E2
Γ
e
e'
A
:
Lemma
fupd_logrel
E1
E2
Γ
e
e'
A
:
((|
=
{
E1
,
E2
}=>
{
E2
;
Γ
}
⊨
e
≼
e'
:
A
)
((|
=
{
E1
,
E2
}=>
{
E2
;
Γ
}
⊨
e
<<
e'
:
A
)
-∗
({
E1
;
Γ
}
⊨
e
≼
e'
:
A
))
%
I
.
-∗
({
E1
;
Γ
}
⊨
e
<<
e'
:
A
))
%
I
.
Proof
.
Proof
.
rewrite
refines_eq
/
refines_def
.
rewrite
refines_eq
/
refines_def
.
iIntros
"H"
.
iIntros
"H"
.
...
@@ -210,7 +219,7 @@ Section related_facts.
...
@@ -210,7 +219,7 @@ Section related_facts.
Global
Instance
elim_fupd_logrel
p
E1
E2
Γ
e
e'
P
A
:
Global
Instance
elim_fupd_logrel
p
E1
E2
Γ
e
e'
P
A
:
(* TODO: DF: look at the booleans here *)
(* TODO: DF: look at the booleans here *)
ElimModal
True
p
false
(|
=
{
E1
,
E2
}=>
P
)
P
ElimModal
True
p
false
(|
=
{
E1
,
E2
}=>
P
)
P
({
E1
;
Γ
}
⊨
e
≼
e'
:
A
)
({
E2
;
Γ
}
⊨
e
≼
e'
:
A
)
.
({
E1
;
Γ
}
⊨
e
<<
e'
:
A
)
({
E2
;
Γ
}
⊨
e
<<
e'
:
A
)
.
Proof
.
Proof
.
rewrite
/
ElimModal
.
intros
_
.
rewrite
/
ElimModal
.
intros
_
.
iIntros
"[HP HI]"
.
iApply
fupd_logrel
.
iIntros
"[HP HI]"
.
iApply
fupd_logrel
.
...
@@ -220,7 +229,7 @@ Section related_facts.
...
@@ -220,7 +229,7 @@ Section related_facts.
Global
Instance
elim_bupd_logrel
p
E
Γ
e
e'
P
A
:
Global
Instance
elim_bupd_logrel
p
E
Γ
e
e'
P
A
:
ElimModal
True
p
false
(|
==>
P
)
P
ElimModal
True
p
false
(|
==>
P
)
P
({
E
;
Γ
}
⊨
e
≼
e'
:
A
)
({
E
;
Γ
}
⊨
e
≼
e'
:
A
)
.
({
E
;
Γ
}
⊨
e
<<
e'
:
A
)
({
E
;
Γ
}
⊨
e
<<
e'
:
A
)
.
Proof
.
Proof
.
rewrite
/
ElimModal
(
bupd_fupd
E
)
.
rewrite
/
ElimModal
(
bupd_fupd
E
)
.
apply
:
elim_fupd_logrel
.
apply
:
elim_fupd_logrel
.
...
@@ -228,7 +237,7 @@ Section related_facts.
...
@@ -228,7 +237,7 @@ Section related_facts.
(* This + elim_modal_timless_bupd' is useful for stripping off laters of timeless propositions. *)
(* This + elim_modal_timless_bupd' is useful for stripping off laters of timeless propositions. *)
Global
Instance
is_except_0_logrel
E
Γ
e
e'
A
:
Global
Instance
is_except_0_logrel
E
Γ
e
e'
A
:
IsExcept0
({
E
;
Γ
}
⊨
e
≼
e'
:
A
)
.
IsExcept0
({
E
;
Γ
}
⊨
e
<<
e'
:
A
)
.
Proof
.
Proof
.
rewrite
/
IsExcept0
.
rewrite
/
IsExcept0
.
iIntros
"HL"
.
iIntros
"HL"
.
...
@@ -239,12 +248,12 @@ Section related_facts.
...
@@ -239,12 +248,12 @@ Section related_facts.
End
related_facts
.
End
related_facts
.
Section
monadic
.
Section
monadic
.
Context
`{
log
relG
Σ
}
.
Context
`{
rel
oc
G
Σ
}
.
Lemma
refines_ret
E
Γ
e1
e2
A
:
Lemma
refines_ret
E
Γ
e1
e2
A
:
is_closed_expr
[]
e1
→
is_closed_expr
[]
e1
→
is_closed_expr
[]
e2
→
is_closed_expr
[]
e2
→
interp_expr
E
e1
e2
A
-∗
{
E
;
Γ
}
⊨
e1
≼
e2
:
A
.
interp_expr
E
e1
e2
A
-∗
{
E
;
Γ
}
⊨
e1
<<
e2
:
A
.
Proof
.
Proof
.
iIntros
(??)
"HA"
.
iIntros
(??)
"HA"
.
rewrite
refines_eq
/
refines_def
.
rewrite
refines_eq
/
refines_def
.
...
@@ -253,10 +262,10 @@ Section monadic.
...
@@ -253,10 +262,10 @@ Section monadic.
Qed
.
Qed
.
Lemma
refines_bind
A
E
Γ
A'
e
e'
K
K'
:
Lemma
refines_bind
A
E
Γ
A'
e
e'
K
K'
:
({
E
;
Γ
}
⊨
e
≼
e'
:
A
)
-∗
({
E
;
Γ
}
⊨
e
<<
e'
:
A
)
-∗
(
∀
v
v'
,
A
v
v'
-∗
(
∀
v
v'
,
A
v
v'
-∗
({
⊤
;
Γ
}
⊨
fill
K
(
of_val
v
)
≼
fill
K'
(
of_val
v'
)
:
A'
))
-∗
({
⊤
;
Γ
}
⊨
fill
K
(
of_val
v
)
<<
fill
K'
(
of_val
v'
)
:
A'
))
-∗
({
E
;
Γ
}
⊨
fill
K
e
≼
fill
K'
e'
:
A'
)
.
({
E
;
Γ
}
⊨
fill
K
e
<<
fill
K'
e'
:
A'
)
.
Proof
.
Proof
.
iIntros
"Hm Hf"
.
iIntros
"Hm Hf"
.
rewrite
refines_eq
/
refines_def
.
rewrite
refines_eq
/
refines_def
.
...
...
This diff is collapsed.
Click to expand it.
theories/logic/spec_ra.v
+
3
−
3
View file @
b7ca3e83
...
@@ -16,9 +16,9 @@ Definition cfgUR := prodUR tpoolUR (gen_heapUR loc val).
...
@@ -16,9 +16,9 @@ Definition cfgUR := prodUR tpoolUR (gen_heapUR loc val).
(** The CMRA for the thread pool. *)
(** The CMRA for the thread pool. *)
Class
cfgSG
Σ
:=
CFGSG
{
cfg_inG
:>
inG
Σ
(
authR
cfgUR
);
cfg_name
:
gname
}
.
Class
cfgSG
Σ
:=
CFGSG
{
cfg_inG
:>
inG
Σ
(
authR
cfgUR
);
cfg_name
:
gname
}
.
Class
log
relG
Σ
:=
Logrel
G
{
Class
rel
oc
G
Σ
:=
Reloc
G
{
log
relG_heapG
:>
heapG
Σ
;
rel
oc
G_heapG
:>
heapG
Σ
;
log
relG_cfgG
:>
cfgSG
Σ
;
rel
oc
G_cfgG
:>
cfgSG
Σ
;
}
.
}
.
Fixpoint
to_tpool_go
(
i
:
nat
)
(
tp
:
list
expr
)
:
tpoolUR
:=
Fixpoint
to_tpool_go
(
i
:
nat
)
(
tp
:
list
expr
)
:
tpoolUR
:=
...
...
This diff is collapsed.
Click to expand it.
theories/logic/spec_rules.v
+
1
−
1
View file @
b7ca3e83
...
@@ -6,7 +6,7 @@ From iris.heap_lang Require Export lang notation.
...
@@ -6,7 +6,7 @@ From iris.heap_lang Require Export lang notation.
From
reloc
.
logic
Require
Export
spec_ra
.
From
reloc
.
logic
Require
Export
spec_ra
.
Import
uPred
.
Import
uPred
.
Section
rules
.
Section
rules
.
Context
`{
log
relG
Σ
}
.
Context
`{
rel
oc
G
Σ
}
.
Implicit
Types
P
Q
:
iProp
Σ
.
Implicit
Types
P
Q
:
iProp
Σ
.
Implicit
Types
Φ
:
val
→
iProp
Σ
.
Implicit
Types
Φ
:
val
→
iProp
Σ
.
Implicit
Types
σ
:
state
.
Implicit
Types
σ
:
state
.
...
...
This diff is collapsed.
Click to expand it.
Preview
0%
Loading
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!
Save comment
Cancel
Please
register
or
sign in
to comment