Skip to content

Commit e910bde

Browse files
authored
Merge pull request #3337 from proux01/validsdp104
Add validsdp 1.0.4
2 parents 7fff806 + 9a62242 commit e910bde

File tree

2 files changed

+116
-0
lines changed
  • released/packages
    • coq-libvalidsdp/coq-libvalidsdp.1.0.4
    • coq-validsdp/coq-validsdp.1.0.4

2 files changed

+116
-0
lines changed
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,53 @@
1+
opam-version: "2.0"
2+
maintainer: [
3+
"Pierre Roux <[email protected]>"
4+
"Érik Martin-Dorel <[email protected]>"
5+
]
6+
7+
homepage: "https://sourcesup.renater.fr/validsdp/"
8+
dev-repo: "git+https://github.com/validsdp/validsdp.git"
9+
bug-reports: "https://github.com/validsdp/validsdp/issues"
10+
license: "LGPL-2.1-or-later"
11+
12+
build: [
13+
[make "-C" "libvalidsdp" "-j%{jobs}%"]
14+
]
15+
install: [make "-C" "libvalidsdp" "install"]
16+
depends: [
17+
"coq" {>= "8.18" & < "8.21~"}
18+
"coq-bignums"
19+
"coq-flocq" {>= "3.3.0"}
20+
"coq-coquelicot" {>= "3.0"}
21+
"coq-interval" {>= "4.0.0" & < "5~"}
22+
"coq-mathcomp-field" {>= "2.1" & < "2.4~"}
23+
("coq-mathcomp-analysis" {>= "1.0.0" & < "1.7~"}
24+
| "coq-mathcomp-reals-stdlib" {>= "1.8.0"})
25+
]
26+
synopsis: "LibValidSDP"
27+
description: """
28+
LibValidSDP is a library for the Coq formal proof assistant. It provides
29+
results mostly about rounding errors in the Cholesky decomposition algorithm
30+
used in the ValidSDP library which itself implements Coq tactics to prove
31+
multivariate inequalities using SDP solvers.
32+
33+
Once installed, the following modules can be imported :
34+
From libValidSDP Require Import Rstruct.v misc.v real_matrix.v bounded.v float_spec.v fsum.v fcmsum.v binary64.v cholesky.v float_infnan_spec.v binary64_infnan.v cholesky_infnan.v flx64.v zulp.v coqinterval_infnan.v.
35+
"""
36+
37+
tags: [
38+
"keyword:libValidSDP"
39+
"keyword:ValidSDP"
40+
"keyword:floating-point arithmetic"
41+
"keyword:Cholesky decomposition"
42+
"category:libValidSDP"
43+
"category:Miscellaneous/Coq Extensions"
44+
"logpath:libValidSDP"
45+
]
46+
authors: [
47+
"Pierre Roux <[email protected]>"
48+
"Érik Martin-Dorel <[email protected]>"
49+
]
50+
url {
51+
src: "https://github.com/validsdp/validsdp/releases/download/v1.0.4/validsdp-1.0.4.tar.gz"
52+
checksum: "sha512=47f9c3b0f67cc41bec5dc97d7df4dcfec05443b2b799320b34efe0cc843f24ae11c1b6340c8c6103789338fccb5dc657729ff96e56d6d8c840d7f0dce4bf0cbd"
53+
}
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,63 @@
1+
opam-version: "2.0"
2+
maintainer: [
3+
"Érik Martin-Dorel <[email protected]>"
4+
"Pierre Roux <[email protected]>"
5+
]
6+
7+
homepage: "https://sourcesup.renater.fr/validsdp/"
8+
dev-repo: "git+https://github.com/validsdp/validsdp.git"
9+
bug-reports: "https://github.com/validsdp/validsdp/issues"
10+
license: "LGPL-2.1-or-later"
11+
12+
build: [
13+
["sh" "-c" "./configure"]
14+
[make "-j%{jobs}%"]
15+
]
16+
run-test: [make "-j%{jobs}%" "test"]
17+
install: [make "install"]
18+
19+
depends: [
20+
"ocaml"
21+
"coq" {>= "8.18" & < "8.21~"}
22+
"coq-bignums"
23+
"coq-flocq" {>= "3.3.0"}
24+
"coq-interval" {>= "4.0.0" & < "5~"}
25+
"coq-mathcomp-field" {>= "2.1" & < "2.4~"}
26+
("coq-mathcomp-analysis" {>= "1.0.0" & < "1.7~"}
27+
| "coq-mathcomp-reals-stdlib" {>= "1.8.0"})
28+
"coq-libvalidsdp" {= version}
29+
"coq-mathcomp-multinomials" {>= "2.0"}
30+
"coq-coqeal" {>= "2.0.2"}
31+
"osdp" {>= "1.1.1"}
32+
"ocamlfind" {build}
33+
"conf-autoconf" {build & dev}
34+
]
35+
synopsis: "ValidSDP"
36+
description: """
37+
ValidSDP is a library for the Coq formal proof assistant. It provides
38+
reflexive tactics to prove multivariate inequalities involving
39+
real-valued variables and rational constants, using SDP solvers as
40+
untrusted back-ends and verified checkers based on libValidSDP.
41+
42+
Once installed, you can import the following modules:
43+
From Coq Require Import Reals.
44+
From ValidSDP Require Import validsdp.
45+
"""
46+
47+
tags: [
48+
"keyword:libValidSDP"
49+
"keyword:ValidSDP"
50+
"keyword:floating-point arithmetic"
51+
"keyword:Cholesky decomposition"
52+
"category:Miscellaneous/Coq Extensions"
53+
"category:ValidSDP"
54+
"logpath:ValidSDP"
55+
]
56+
authors: [
57+
"Érik Martin-Dorel <[email protected]>"
58+
"Pierre Roux <[email protected]>"
59+
]
60+
url {
61+
src: "https://github.com/validsdp/validsdp/releases/download/v1.0.4/validsdp-1.0.4.tar.gz"
62+
checksum: "sha512=47f9c3b0f67cc41bec5dc97d7df4dcfec05443b2b799320b34efe0cc843f24ae11c1b6340c8c6103789338fccb5dc657729ff96e56d6d8c840d7f0dce4bf0cbd"
63+
}

0 commit comments

Comments
 (0)