Skip to content

Commit

Permalink
Merge pull request #2257 from lgaeher/iris-4.0.0
Browse files Browse the repository at this point in the history
Release Iris 4.0.0 and std++ 1.8.0
  • Loading branch information
palmskog authored Aug 18, 2022
2 parents f60c78e + 04ad322 commit fe08c35
Show file tree
Hide file tree
Showing 3 changed files with 120 additions and 0 deletions.
31 changes: 31 additions & 0 deletions released/packages/coq-iris-heap-lang/coq-iris-heap-lang.4.0.0/opam
Original file line number Diff line number Diff line change
@@ -0,0 +1,31 @@
opam-version: "2.0"
maintainer: "Ralf Jung <[email protected]>"
authors: "The Iris Team"
license: "BSD-3-Clause"
homepage: "https://iris-project.org/"
bug-reports: "https://gitlab.mpi-sws.org/iris/iris/issues"
dev-repo: "git+https://gitlab.mpi-sws.org/iris/iris.git"

synopsis: "The canonical example language for Iris"
description: """
This package defines HeapLang, a concurrent lambda calculus with references, and
uses Iris to build a program logic for HeapLang programs.
"""
tags: [
"date:2022-08-17"
"logpath:iris.heap_lang"
]

depends: [
"coq-iris" {= version}
]

build: ["./make-package" "iris_heap_lang" "-j%{jobs}%"]
install: ["./make-package" "iris_heap_lang" "install"]

url {
src:
"https://gitlab.mpi-sws.org/iris/iris/-/archive/iris-4.0.0.tar.gz"
checksum:
"sha512=919ab6a7657d7bc6df3be576a752df884e44b638318574fcf0682cc04be3a272270986fb23a0010b09b4fd80c6a0dafe04b7364764381e6831e81e1f942ebffc"
}
42 changes: 42 additions & 0 deletions released/packages/coq-iris/coq-iris.4.0.0/opam
Original file line number Diff line number Diff line change
@@ -0,0 +1,42 @@
opam-version: "2.0"
maintainer: "Ralf Jung <[email protected]>"
authors: "The Iris Team"
license: "BSD-3-Clause"
homepage: "https://iris-project.org/"
bug-reports: "https://gitlab.mpi-sws.org/iris/iris/issues"
dev-repo: "git+https://gitlab.mpi-sws.org/iris/iris.git"

synopsis: "A Higher-Order Concurrent Separation Logic Framework with support for interactive proofs"
description: """
Iris is a framework for reasoning about the safety of concurrent programs using
concurrent separation logic. It can be used to develop a program logic, for
defining logical relations, and for reasoning about type systems, among other
applications. This package includes the base logic, Iris Proof Mode (IPM) /
MoSeL, and a general language-independent program logic; see coq-iris-heap-lang
for an instantiation of the program logic to a particular programming language.
"""
tags: [
"date:2022-08-17"
"logpath:iris.prelude"
"logpath:iris.algebra"
"logpath:iris.si_logic"
"logpath:iris.bi"
"logpath:iris.proofmode"
"logpath:iris.base_logic"
"logpath:iris.program_logic"
]

depends: [
"coq" { (>= "8.13" & < "8.17~") | (= "dev") }
"coq-stdpp" { (= "1.8.0") | (= "dev") }
]

build: ["./make-package" "iris" "-j%{jobs}%"]
install: ["./make-package" "iris" "install"]

url {
src:
"https://gitlab.mpi-sws.org/iris/iris/-/archive/iris-4.0.0.tar.gz"
checksum:
"sha512=919ab6a7657d7bc6df3be576a752df884e44b638318574fcf0682cc04be3a272270986fb23a0010b09b4fd80c6a0dafe04b7364764381e6831e81e1f942ebffc"
}
47 changes: 47 additions & 0 deletions released/packages/coq-stdpp/coq-stdpp.1.8.0/opam
Original file line number Diff line number Diff line change
@@ -0,0 +1,47 @@
opam-version: "2.0"
maintainer: "Ralf Jung <[email protected]>"
authors: "The std++ team"
license: "BSD-3-Clause"
homepage: "https://gitlab.mpi-sws.org/iris/stdpp"
bug-reports: "https://gitlab.mpi-sws.org/iris/stdpp/issues"
dev-repo: "git+https://gitlab.mpi-sws.org/iris/stdpp.git"

synopsis: "An extended \"Standard Library\" for Coq"
description: """
The key features of this library are as follows:

- It provides a great number of definitions and lemmas for common data
structures such as lists, finite maps, finite sets, and finite multisets.
- It uses type classes for common notations (like `∅`, `∪`, and Haskell-style
monad notations) so that these can be overloaded for different data structures.
- It uses type classes to keep track of common properties of types, like it
having decidable equality or being countable or finite.
- Most data structures are represented in canonical ways so that Leibniz
equality can be used as much as possible (for example, for maps we have
`m1 = m2` iff `∀ i, m1 !! i = m2 !! i`). On top of that, the library provides
setoid instances for most types and operations.
- It provides various tactics for common tasks, like an ssreflect inspired
`done` tactic for finishing trivial goals, a simple breadth-first solver
`naive_solver`, an equality simplifier `simplify_eq`, a solver `solve_proper`
for proving compatibility of functions with respect to relations, and a solver
`set_solver` for goals involving set operations.
- It is entirely dependency- and axiom-free.
"""
tags: [
"date:2022-08-17"
"logpath:stdpp"
]

depends: [
"coq" { (>= "8.12" & < "8.17~") | (= "dev") }
]

build: ["./make-package" "stdpp" "-j%{jobs}%"]
install: ["./make-package" "stdpp" "install"]

url {
src:
"https://gitlab.mpi-sws.org/iris/stdpp/-/archive/coq-stdpp-1.8.0.tar.gz"
checksum:
"sha512=c894cc0574ab00efa41c807628f97abdeff917bee71b40e2f98251bcdc91ebfb7a2964683e61e7cefbe6e578b2e123098ddd7694252406f8c4835176c1d0df37"
}

0 comments on commit fe08c35

Please sign in to comment.