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
Marianna Rapoport
iris-coq
Commits
fd86b7bb
Commit
fd86b7bb
authored
Aug 19, 2016
by
Ralf Jung
Browse files
do "Print Assumptions" outside of sections
parent
4206ef52
Changes
2
Hide whitespace changes
Inline
Side-by-side
.gitlab-ci.yml
View file @
fd86b7bb
...
...
@@ -6,7 +6,7 @@ buildjob:
script
:
-
coqc -v
-
'
time
make
-j8
TIMED=y
2>&1
|
tee
build-log.txt'
-
'
grep
Axiom
build-log.txt
&&
exit
1'
-
'
f
grep
Axiom
build-log.txt
&&
exit
1'
-
'
cat
build-log.txt
|
egrep
"[a-zA-Z0-9_/-]+
\(user:
[0-9]"
|
tee
build-time.txt'
-
make verify
only
:
...
...
tests/barrier_client.v
View file @
fd86b7bb
...
...
@@ -59,7 +59,7 @@ End client.
Section
ClosedProofs
.
Definition
Σ
:
gFunctors
:
=
#[
heap
Σ
;
barrier
Σ
;
spawn
Σ
].
Let
Σ
:
gFunctors
:
=
#[
heap
Σ
;
barrier
Σ
;
spawn
Σ
].
Lemma
client_adequate
σ
:
adequate
client
σ
(
λ
_
,
True
).
Proof
.
...
...
@@ -67,6 +67,6 @@ Proof.
apply
(
client_safe
(
nroot
.@
"barrier"
))
;
auto
with
ndisj
.
Qed
.
Print
Assumptions
client_adequate
.
End
ClosedProofs
.
Print
Assumptions
client_adequate
.
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