Skip to content
GitLab
Menu
Projects
Groups
Snippets
Help
Help
Support
Community forum
Keyboard shortcuts
?
Submit feedback
Contribute to GitLab
Sign in / Register
Toggle navigation
Menu
Open sidebar
Janno
iris-coq
Commits
78f10027
Commit
78f10027
authored
Dec 12, 2016
by
Ralf Jung
Browse files
rename op_rules -> lifting
parent
6b8069fa
Changes
5
Hide whitespace changes
Inline
Side-by-side
_CoqProject
View file @
78f10027
...
...
@@ -95,8 +95,8 @@ theories/program_logic/gen_heap.v
theories/program_logic/ownp.v
theories/heap_lang/lang.v
theories/heap_lang/tactics.v
theories/heap_lang/lifting.v
theories/heap_lang/wp_tactics.v
theories/heap_lang/op_rules.v
theories/heap_lang/notation.v
theories/heap_lang/lib/spawn.v
theories/heap_lang/lib/par.v
...
...
theories/heap_lang/adequacy.v
View file @
78f10027
From
iris
.
program_logic
Require
Export
weakestpre
adequacy
gen_heap
.
From
iris
.
heap_lang
Require
Export
op_rules
.
From
iris
.
heap_lang
Require
Export
lifting
.
From
iris
.
algebra
Require
Import
auth
.
From
iris
.
heap_lang
Require
Import
proofmode
notation
.
From
iris
.
proofmode
Require
Import
tactics
.
...
...
theories/heap_lang/
op_rules
.v
→
theories/heap_lang/
lifting
.v
View file @
78f10027
...
...
@@ -52,7 +52,7 @@ Local Hint Constructors head_step.
Local
Hint
Resolve
alloc_fresh
.
Local
Hint
Resolve
to_of_val
.
Section
rules
.
Section
lifting
.
Context
`
{
heapG
Σ
}.
Implicit
Types
P
Q
:
iProp
Σ
.
Implicit
Types
Φ
:
val
→
iProp
Σ
.
...
...
@@ -276,4 +276,4 @@ Proof.
intros
.
rewrite
-
wp_bin_op
//
;
[].
destruct
(
bool_decide_reflect
(
v1
=
v2
))
;
by
eauto
.
Qed
.
End
rules
.
End
lifting
.
theories/heap_lang/proofmode.v
View file @
78f10027
From
iris
.
program_logic
Require
Export
weakestpre
.
From
iris
.
proofmode
Require
Import
coq_tactics
.
From
iris
.
proofmode
Require
Export
tactics
.
From
iris
.
heap_lang
Require
Export
wp_tactics
op_rules
.
From
iris
.
heap_lang
Require
Export
wp_tactics
lifting
.
Import
uPred
.
Ltac
wp_strip_later
::
=
iNext
.
...
...
theories/heap_lang/wp_tactics.v
View file @
78f10027
From
iris
.
heap_lang
Require
Export
tactics
op_rules
.
From
iris
.
heap_lang
Require
Export
tactics
lifting
.
Import
uPred
.
(** wp-specific helper tactics *)
...
...
Write
Preview
Supports
Markdown
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