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
Actris
Commits
31346e33
Commit
31346e33
authored
Jun 11, 2019
by
Jonas Kastberg Hinrichsen
Browse files
Refactoring: encodings -> proto
parent
03de6315
Changes
16
Hide whitespace changes
Inline
Side-by-side
_CoqProject
View file @
31346e33
-Q theories osiris
-arg -w -arg -notation-overridden,-redundant-canonical-projection,-several-object-files
theories/base_logic/auth_excl.v
theories/
encodings/involutiv
e.v
theories/
encodings/side
.v
theories/
encodings/stype_def
.v
theories/
encodings/encodabl
e.v
theories/
encodings/list
.v
theories/
encodings/channel
.v
theories/
encodings
/stype.v
theories/
encodings
/stype_enc.v
theories/
encodings
/branching.v
theories/
proto/encodabl
e.v
theories/
proto/list
.v
theories/
proto/channel
.v
theories/
proto/involutiv
e.v
theories/
proto/side
.v
theories/
proto/stype_def
.v
theories/
proto
/stype.v
theories/
proto
/stype_enc.v
theories/
proto
/branching.v
theories/examples/examples.v
theories/examples/proofs.v
theories/examples/proofs_enc.v
...
...
theories/examples/branching_examples.v
View file @
31346e33
From
iris
.
proofmode
Require
Import
tactics
.
From
iris
.
program_logic
Require
Export
weakestpre
.
From
iris
.
heap_lang
Require
Import
proofmode
notation
.
From
osiris
.
encodings
Require
Import
channel
branching
.
From
iris
.
base_logic
Require
Import
invariants
.
From
osiris
.
proto
Require
Import
channel
branching
.
Section
BranchingExamples
.
Context
`
{!
heapG
Σ
}
(
N
:
namespace
).
...
...
theories/examples/branching_proofs.v
View file @
31346e33
...
...
@@ -2,7 +2,7 @@ From iris.proofmode Require Import tactics.
From
iris
.
program_logic
Require
Export
weakestpre
.
From
iris
.
heap_lang
Require
Import
proofmode
notation
.
From
iris
.
base_logic
Require
Import
invariants
.
From
osiris
.
encodings
Require
Import
branching
.
From
osiris
.
proto
Require
Import
branching
.
From
osiris
.
examples
Require
Import
branching_examples
.
Section
BranchingExampleProofs
.
...
...
theories/examples/examples.v
View file @
31346e33
From
iris
.
proofmode
Require
Import
tactics
.
From
iris
.
program_logic
Require
Export
weakestpre
.
From
iris
.
heap_lang
Require
Import
proofmode
notation
.
From
osiris
.
encodings
Require
Import
stype
.
From
iris
.
base_logic
Require
Import
invariants
.
From
osiris
.
proto
Require
Import
stype
.
Section
Examples
.
Context
`
{!
heapG
Σ
}
(
N
:
namespace
).
...
...
theories/examples/list_sort.v
View file @
31346e33
From
stdpp
Require
Import
sorting
.
Require
Import
Coq
.
Lists
.
List
.
Require
Import
Omega
.
From
iris
.
proofmode
Require
Import
tactics
.
From
iris
.
program_logic
Require
Export
weakestpre
.
From
iris
.
heap_lang
Require
Import
proofmode
notation
.
From
osiris
.
encodings
Require
Import
list
channel
stype_enc
.
From
osiris
.
proto
Require
Import
list
channel
stype_enc
.
From
iris
.
base_logic
Require
Import
invariants
.
From
stdpp
Require
Import
sorting
.
Require
Import
Coq
.
Lists
.
List
.
Require
Import
Omega
.
Section
ListSortExample
.
Context
`
{!
heapG
Σ
}
`
{
logrelG
val
Σ
}
(
N
:
namespace
).
...
...
theories/examples/proofs.v
View file @
31346e33
...
...
@@ -2,7 +2,7 @@ From iris.proofmode Require Import tactics.
From
iris
.
program_logic
Require
Export
weakestpre
.
From
iris
.
heap_lang
Require
Import
proofmode
notation
.
From
iris
.
base_logic
Require
Import
invariants
.
From
osiris
.
encodings
Require
Import
stype
.
From
osiris
.
proto
Require
Import
stype
.
From
osiris
.
examples
Require
Import
examples
.
Section
ExampleProofs
.
...
...
theories/examples/proofs_enc.v
View file @
31346e33
...
...
@@ -3,7 +3,7 @@ From iris.program_logic Require Export weakestpre.
From
iris
.
heap_lang
Require
Import
proofmode
notation
.
From
iris
.
algebra
Require
Import
list
auth
excl
.
From
iris
.
base_logic
Require
Import
invariants
.
From
osiris
.
encodings
Require
Import
stype_enc
.
From
osiris
.
proto
Require
Import
stype_enc
.
From
osiris
.
examples
Require
Import
examples
.
Section
ExampleProofsEnc
.
...
...
theories/
encodings
/branching.v
→
theories/
proto
/branching.v
View file @
31346e33
...
...
@@ -3,7 +3,7 @@ From iris.program_logic Require Export weakestpre.
From
iris
.
heap_lang
Require
Import
proofmode
notation
.
From
iris
.
algebra
Require
Import
list
auth
excl
.
From
iris
.
base_logic
Require
Import
invariants
.
From
osiris
.
encodings
Require
Export
stype_enc
.
From
osiris
.
proto
Require
Export
stype_enc
.
Section
DualBranch
.
Context
`
{
PROP
:
bi
}.
...
...
theories/
encodings
/channel.v
→
theories/
proto
/channel.v
View file @
31346e33
...
...
@@ -6,8 +6,8 @@ From iris.algebra Require Import excl auth list.
From
iris
.
base_logic
.
lib
Require
Import
auth
.
From
iris
.
heap_lang
.
lib
Require
Import
spin_lock
.
From
osiris
.
base_logic
Require
Import
auth_excl
.
From
osiris
.
encodings
Require
Export
side
.
From
osiris
.
encodings
Require
Import
list
.
From
osiris
.
proto
Require
Export
side
.
From
osiris
.
proto
Require
Import
list
.
Set
Default
Proof
Using
"Type"
.
Import
uPred
.
...
...
theories/
encodings
/encodable.v
→
theories/
proto
/encodable.v
View file @
31346e33
File moved
theories/proto/involutive.v
0 → 100644
View file @
31346e33
From
iris
.
heap_lang
Require
Import
proofmode
notation
.
Class
Involutive
{
A
}
(
R
:
relation
A
)
(
f
:
A
→
A
)
:
=
involutive
x
:
R
(
f
(
f
x
))
x
.
theories/
encodings
/list.v
→
theories/
proto
/list.v
View file @
31346e33
File moved
theories/
encodings
/side.v
→
theories/
proto
/side.v
View file @
31346e33
From
iris
.
heap_lang
Require
Import
proofmode
notation
.
From
osiris
.
encodings
Require
Export
involutive
.
From
osiris
.
proto
Require
Export
involutive
.
Inductive
side
:
=
Left
|
Right
.
Instance
side_inhabited
:
Inhabited
side
:
=
populate
Left
.
...
...
theories/
encodings
/stype.v
→
theories/
proto
/stype.v
View file @
31346e33
...
...
@@ -6,8 +6,8 @@ From iris.heap_lang.lib Require Import spin_lock.
From
iris
.
algebra
Require
Import
list
auth
excl
.
From
iris
.
base_logic
Require
Import
invariants
.
From
osiris
.
base_logic
Require
Import
auth_excl
.
From
osiris
.
encodings
Require
Export
stype_def
.
From
osiris
.
encodings
Require
Export
channel
.
From
osiris
.
proto
Require
Export
stype_def
.
From
osiris
.
proto
Require
Export
channel
.
Class
logrelG
A
Σ
:
=
{
logrelG_channelG
:
>
chanG
Σ
;
...
...
theories/
encodings
/stype_def.v
→
theories/
proto
/stype_def.v
View file @
31346e33
...
...
@@ -4,7 +4,7 @@ From stdpp Require Export list.
From
iris
.
base_logic
Require
Import
base_logic
.
From
iris
.
algebra
Require
Import
updates
local_updates
.
From
iris
.
heap_lang
Require
Import
proofmode
notation
.
From
osiris
.
encodings
Require
Import
involutive
.
From
osiris
.
proto
Require
Import
involutive
.
Set
Default
Proof
Using
"Type"
.
Inductive
action
:
=
Send
|
Receive
.
...
...
theories/
encodings
/stype_enc.v
→
theories/
proto
/stype_enc.v
View file @
31346e33
...
...
@@ -3,7 +3,7 @@ From iris.program_logic Require Export weakestpre.
From
iris
.
heap_lang
Require
Import
proofmode
notation
.
From
iris
.
algebra
Require
Import
list
auth
excl
.
From
iris
.
base_logic
Require
Import
invariants
.
From
osiris
.
encodings
Require
Export
encodable
stype
.
From
osiris
.
proto
Require
Export
encodable
stype
.
Section
DualStypeEnc
.
Context
`
{
EncDec
V
}
`
{
PROP
:
bi
}
.
...
...
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