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
Iris
RefinedC
Commits
6cfc6d3e
Commit
6cfc6d3e
authored
Oct 29, 2020
by
Rodolphe Lepigre
Browse files
Require Coq 8.12
parent
4e25788d
Pipeline
#36778
passed with stage
in 33 minutes and 37 seconds
Changes
3
Pipelines
5
Hide whitespace changes
Inline
Side-by-side
refinedc.opam
View file @
6cfc6d3e
...
...
@@ -16,7 +16,7 @@ bug-reports: "https://gitlab.mpi-sws.org/iris/refinedc/issues"
dev-repo: "git+https://gitlab.mpi-sws.org/iris/refinedc.git"
depends: [
"coq" { (>= "8.1
1
.0" & < "8.1
2
~") }
"coq" { (>= "8.1
2
.0" & < "8.1
3
~") }
"coq-iris" { (= "dev.2020-10-01.3.8f6c063a") | (= "dev") }
"dune" {>= "2.7.0"}
"cerberus" {= "~dev"}
...
...
theories/lang/base.v
View file @
6cfc6d3e
...
...
@@ -379,7 +379,7 @@ Definition keep_factor2 (n : nat) (def : nat) : nat :=
Lemma
Pos_pow_add_r
a
b
c
:
(
a
^
(
b
+
c
)
=
a
^
b
*
a
^
c
)%
positive
.
Proof
.
zify
.
rewrite
!
Pos2Z
.
inj_pow
Pos2Z
.
inj_add
Z
.
pow_add_r
;
lia
.
Qed
.
Proof
.
zify
.
rewrite
Z
.
pow_add_r
;
lia
.
Qed
.
Lemma
Pos_factor2_mult_xI
a
b
:
Pos_factor2
(
a
~
1
*
b
)
=
Pos_factor2
b
.
...
...
theories/lithium/simpl_instances.v
View file @
6cfc6d3e
...
...
@@ -93,7 +93,6 @@ Proof.
unfold
CanSolve
in
*.
rewrite
/
Z
.
divide
.
split
.
-
move
=>
HT
[
x
Hx
].
apply
:
(
HT
(
Z
.
to_nat
x
)).
rewrite
-
Z2Nat
.
inj_mul
;
try
lia
.
apply
(
Z
.
mul_nonneg_cancel_r
_
a
)
;
lia
.
-
move
=>
HT
n
?.
apply
HT
.
eexists
n
.
lia
.
Qed
.
...
...
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