SHA256
1
0
forked from pool/coq
Commit Graph

42 Commits

Author SHA256 Message Date
Dominique Leuenberger
018f3b6c32 Accepting request 964734 from science
- Update to version 8.15.1.
  * Fixes an inconsistency when using module subtyping with
    inductive types.
  * Speeds up CoqIDE on large files.
  * Fixes a bug where `coqc -vok` was not creating a .vok file.
  * Fixes a regression in `cbn`.
  * Improves usability of schemes with `elim foo using scheme with
    (P0 := ...)` (the `P0` name was not accessible in 8.15.0).

OBS-URL: https://build.opensuse.org/request/show/964734
OBS-URL: https://build.opensuse.org/package/show/openSUSE:Factory/coq?expand=0&rev=16
2022-03-25 20:54:34 +00:00
Aaron Puchert
660b7caabf - Update to version 8.15.1.
* Fixes an inconsistency when using module subtyping with
    inductive types.
  * Speeds up CoqIDE on large files.
  * Fixes a bug where `coqc -vok` was not creating a .vok file.
  * Fixes a regression in `cbn`.
  * Improves usability of schemes with `elim foo using scheme with
    (P0 := ...)` (the `P0` name was not accessible in 8.15.0).

OBS-URL: https://build.opensuse.org/package/show/science/coq?expand=0&rev=38
2022-03-24 22:47:19 +00:00
Dominique Leuenberger
c2d62a169f Accepting request 946708 from science
- Update to version 8.15.0.
  * The `apply with` tactic no longer renames arguments unless
    the compatibility flag `Apply With Renaming` is set.
  * Improvements to the `auto` tactic family, fixing `Hint Unfold`
    behavior, and generalizing the use of discrimination nets.
  * The `typeclasses eauto` tactic has a new `best_effort` option
    allowing it to return partial solutions to a proof search
    problem, depending on the mode declarations associated to each
    constraint. This mode is used by typeclass resolution during
    type inference to provide more precise error messages.
  * Many commands and options were deprecated or removed after
    deprecation and more consistently support locality attributes.
  * The `Import` command is extended with `import_categories` to
    select the components of a module to import or not, including
    features such as hints, coercions, and notations.
  * A visual Ltac debugger is now available in CoqIDE.
  * For more details, see refman/changes.html in coq-doc.

OBS-URL: https://build.opensuse.org/request/show/946708
OBS-URL: https://build.opensuse.org/package/show/openSUSE:Factory/coq?expand=0&rev=15
2022-01-16 22:18:05 +00:00
Aaron Puchert
da8ddfc177 - Update to version 8.15.0.
* The `apply with` tactic no longer renames arguments unless
    the compatibility flag `Apply With Renaming` is set.
  * Improvements to the `auto` tactic family, fixing `Hint Unfold`
    behavior, and generalizing the use of discrimination nets.
  * The `typeclasses eauto` tactic has a new `best_effort` option
    allowing it to return partial solutions to a proof search
    problem, depending on the mode declarations associated to each
    constraint. This mode is used by typeclass resolution during
    type inference to provide more precise error messages.
  * Many commands and options were deprecated or removed after
    deprecation and more consistently support locality attributes.
  * The `Import` command is extended with `import_categories` to
    select the components of a module to import or not, including
    features such as hints, coercions, and notations.
  * A visual Ltac debugger is now available in CoqIDE.
  * For more details, see refman/changes.html in coq-doc.

OBS-URL: https://build.opensuse.org/package/show/science/coq?expand=0&rev=37
2022-01-15 19:42:50 +00:00
Dominique Leuenberger
9ba52e1735 Accepting request 940115 from science
- Update to version 8.14.1.
  * Fixed the implementation of persistent arrays used by the VM
    and native compute so that it uses a uniform representation.
    Previously, storing primitive floats inside primitive arrays
    could cause memory corruption.
  * Fixed missing registration of universe constraints in Module
    Type elaboration.
  * Made `abstract` more robust with respect to Ltac `constr`
    bindings containing existential variables.
  * Correct support of trailing `let` by tactic `specialize`.
  * Fixed an anomaly with `Extraction Conservative Types` when
    extracting pattern-matching on singleton types.
  * Regular error instead of an anomaly when calling `Separate
    Extraction` in a module.

OBS-URL: https://build.opensuse.org/request/show/940115
OBS-URL: https://build.opensuse.org/package/show/openSUSE:Factory/coq?expand=0&rev=14
2021-12-13 19:44:29 +00:00
Aaron Puchert
4e1d685c4c - Update to version 8.14.1.
* Fixed the implementation of persistent arrays used by the VM
    and native compute so that it uses a uniform representation.
    Previously, storing primitive floats inside primitive arrays
    could cause memory corruption.
  * Fixed missing registration of universe constraints in Module
    Type elaboration.
  * Made `abstract` more robust with respect to Ltac `constr`
    bindings containing existential variables.
  * Correct support of trailing `let` by tactic `specialize`.
  * Fixed an anomaly with `Extraction Conservative Types` when
    extracting pattern-matching on singleton types.
  * Regular error instead of an anomaly when calling `Separate
    Extraction` in a module.

OBS-URL: https://build.opensuse.org/package/show/science/coq?expand=0&rev=36
2021-12-12 21:22:34 +00:00
Dominique Leuenberger
14545c8f27 Accepting request 926632 from science
- Update to version 8.14.0.
  * The internal representation of match has changed to a more
    space-efficient and cleaner structure, allowing the fix of a
    completeness issue with cumulative inductive types in the type-
    checker. The internal representation is now closer to the user-
    level view of match, where the argument context of branches and
    the inductive binders in and as do not carry type annotations.
  * A new coqnative binary performs separate native compilation of
    libraries, starting from a .vo file. It is supported by
    coq_makefile.
  * Improvements to typeclasses and canonical structure resolution,
    allowing more terms to be considered as classes or keys.
  * More control over notations declarations and support for
    primitive types in string and number notations.
  * Removal of deprecated tactics, notably omega, which has been
    replaced by a greatly improved lia, along with many bug fixes.
  * New Ltac2 APIs for interaction with Ltac1, manipulation of
    inductive types and printing.
  * Many changes and additions to the standard library in the
    numbers, vectors and lists libraries. A new signed primitive
    integers library Sint63 is available in addition to the
    unsigned Uint63 library.
  * For more details, see refman/changes.html in coq-doc.

OBS-URL: https://build.opensuse.org/request/show/926632
OBS-URL: https://build.opensuse.org/package/show/openSUSE:Factory/coq?expand=0&rev=13
2021-10-21 21:55:25 +00:00
Aaron Puchert
96b9f456bb - Fix typo in condition.
OBS-URL: https://build.opensuse.org/package/show/science/coq?expand=0&rev=35
2021-10-21 00:03:26 +00:00
Aaron Puchert
f595c547f2 OBS-URL: https://build.opensuse.org/package/show/science/coq?expand=0&rev=34 2021-10-20 23:30:38 +00:00
Dominique Leuenberger
fc4ca13aa9 Accepting request 916845 from science
- Add documentation package based on github.com/coq/doc until we
  can build the documentation directly in OBS.

OBS-URL: https://build.opensuse.org/request/show/916845
OBS-URL: https://build.opensuse.org/package/show/openSUSE:Factory/coq?expand=0&rev=12
2021-09-04 20:35:26 +00:00
Aaron Puchert
eed432c976 - Add documentation package based on github.com/coq/doc until we
can build the documentation directly in OBS.

OBS-URL: https://build.opensuse.org/package/show/science/coq?expand=0&rev=32
2021-09-04 12:54:51 +00:00
Dominique Leuenberger
c2dbf14392 Accepting request 889764 from science
- Update to version 8.13.2.
  * Fix crash when using vm_compute on an irreducible PArray.set.
  * Fix crash when loading .vo files containing a vm_compute
    normalized primitive array.
  * Fix Ltac2.Array.init computational complexity.

OBS-URL: https://build.opensuse.org/request/show/889764
OBS-URL: https://build.opensuse.org/package/show/openSUSE:Factory/coq?expand=0&rev=11
2021-05-02 16:36:08 +00:00
Aaron Puchert
d0636cc204 Accepting request 889763 from home:aaronpuchert
- Update to version 8.13.2.
  * Fix crash when using vm_compute on an irreducible PArray.set.
  * Fix crash when loading .vo files containing a vm_compute
    normalized primitive array.
  * Fix Ltac2.Array.init computational complexity.

OBS-URL: https://build.opensuse.org/request/show/889763
OBS-URL: https://build.opensuse.org/package/show/science/coq?expand=0&rev=30
2021-05-01 21:33:33 +00:00
Dominique Leuenberger
8afc5fda0d Accepting request 875244 from science
- Update to version 8.13.1.
  * Fix arities of VM opcodes for some floating-point operations
    that could cause memory corruption.

OBS-URL: https://build.opensuse.org/request/show/875244
OBS-URL: https://build.opensuse.org/package/show/openSUSE:Factory/coq?expand=0&rev=10
2021-02-26 20:59:54 +00:00
Aaron Puchert
7777299bac - Update to version 8.13.1.
* Fix arities of VM opcodes for some floating-point operations
    that could cause memory corruption.

OBS-URL: https://build.opensuse.org/package/show/science/coq?expand=0&rev=28
2021-02-25 23:36:41 +00:00
Dominique Leuenberger
f8c1a8965d Accepting request 870152 from science
OBS-URL: https://build.opensuse.org/request/show/870152
OBS-URL: https://build.opensuse.org/package/show/openSUSE:Factory/coq?expand=0&rev=9
2021-02-08 10:47:41 +00:00
Aaron Puchert
2b13e5c237 Accepting request 870151 from home:aaronpuchert
- Update to version 8.13.0.
  * Introduction of primitive persistent arrays in the core
    language, implemented using imperative persistent arrays.
  * Introduction of definitional proof irrelevance for the equality
    type defined in the SProp sort.
  * Cumulative record and inductive type declarations can now
    specify the variance of their universes.
  * Various bugfixes and uniformization of behavior with respect to
    the use of implicit arguments and the handling of existential
    variables in declarations, unification and tactics.
  * New warning for unused variables in catch-all match branches
    that match multiple distinct patterns.
  * New warning for Hint commands outside sections without a
    locality attribute, whose goal is to eventually remove the
    fragile default behavior of importing hints only when using
    Require. The recommended fix is to declare hints as export,
    instead of the current default global, meaning that they are
    imported through Require Import only, not Require.
  * General support for boolean attributes.
  * Many improvements to the handling of notations, including
    number notations, recursive notations and notations with
    bindings. A new algorithm chooses the most precise notation
    available to print an expression, which might introduce changes
    in printing behavior.
  * Tactic improvements in lia and its zify preprocessing step,
    now supporting reasoning on boolean operators such as Z.leb and
    supporting primitive integers Int63.
  * Typing flags can now be specified per-constant / inductive.
  * Improvements to the reference manual including updated syntax
    descriptions that match Coq's grammar in several chapters, and
    splitting parts of the tactics chapter to independent sections.
- Add build flag to turn off building of the IDE.

OBS-URL: https://build.opensuse.org/request/show/870151
OBS-URL: https://build.opensuse.org/package/show/science/coq?expand=0&rev=26
2021-02-07 23:06:30 +00:00
Dominique Leuenberger
cd33483f40 Accepting request 855595 from science
- Update to version 8.12.2.

OBS-URL: https://build.opensuse.org/request/show/855595
OBS-URL: https://build.opensuse.org/package/show/openSUSE:Factory/coq?expand=0&rev=8
2020-12-14 17:09:33 +00:00
Aaron Puchert
e78df31e71 - Update to version 8.12.2. Fixes two impacting 8.12 regressions:
* Fixed a regression causing notations mentioning a coercion to
    be ignored.
  * Fixed a regression causing incomplete inference of implicit
    arguments in exists.

OBS-URL: https://build.opensuse.org/package/show/science/coq?expand=0&rev=24
2020-12-13 17:13:48 +00:00
Dominique Leuenberger
e01d1ee19a Accepting request 849178 from science
- Update to version 8.12.1. This contains mostly bug fixes:
  * Polymorphic side-effects inside monomorphic definitions were
    incorrectly handled as not inlined. This allowed deriving an
    inconsistency.
  * Regression in error reporting after SSReflect's case tactic.
    A generic error message "Could not fill dependent hole in
    apply" was reported for any error following case or elim.
  * Several bugs with Search.
  * The details environment introduced in coqdoc in Coq 8.12 can
    now be used as advertised in the reference manual.
  * View menu "Display parentheses" introduced in CoqIDE in
    Coq 8.12 now works correctly.
- Use memoryperjob constraint instead of %limit_build macro.

OBS-URL: https://build.opensuse.org/request/show/849178
OBS-URL: https://build.opensuse.org/package/show/openSUSE:Factory/coq?expand=0&rev=7
2020-12-04 20:27:53 +00:00
Aaron Puchert
c3225375ef - Update to version 8.12.1. This contains mostly bug fixes:
* Polymorphic side-effects inside monomorphic definitions were
    incorrectly handled as not inlined. This allowed deriving an
    inconsistency.
  * Regression in error reporting after SSReflect's case tactic.
    A generic error message "Could not fill dependent hole in
    apply" was reported for any error following case or elim.
  * Several bugs with Search.
  * The details environment introduced in coqdoc in Coq 8.12 can
    now be used as advertised in the reference manual.
  * View menu "Display parentheses" introduced in CoqIDE in
    Coq 8.12 now works correctly.

OBS-URL: https://build.opensuse.org/package/show/science/coq?expand=0&rev=22
2020-11-17 22:12:19 +00:00
Aaron Puchert
2cfc0855cf Accepting request 828043 from home:marxin:memory-constraint
Use memoryperjob constraint instead of %limit_build macro.

OBS-URL: https://build.opensuse.org/request/show/828043
OBS-URL: https://build.opensuse.org/package/show/science/coq?expand=0&rev=21
2020-08-20 12:25:06 +00:00
Dominique Leuenberger
da3c57af9f Accepting request 824553 from science
- Update to version 8.12.0.
  * New binder notation for non-maximal implicit arguments using []
    allowing to set and see the implicit status of arguments
    immediately.
  * New notation Inductive "I A | x : s := ..." to distinguish the
    uniform from the non-uniform parameters in inductive
    definitions.
  * More robust and expressive treatment of implicit inductive
    parameters in inductive declarations.
  * Improvements in the treatment of implicit arguments and
    partially applied constants in notations, parsing of
    hexadecimal number notation and better handling of scopes and
    coercions for printing.
  * A correct and efficient coercion coherence checking algorithm,
    avoiding spurious or duplicate warnings.
  * An improved Search command which accepts complex queries. This
    takes precedence over the now deprecated ssreflect search.
  * Many additions and improvements of the standard library.
  * Improvements to the reference manual include a more logical
    organization of chapters along with updated syntax descriptions
    that match Coq's grammar in most but not all chapters.

OBS-URL: https://build.opensuse.org/request/show/824553
OBS-URL: https://build.opensuse.org/package/show/openSUSE:Factory/coq?expand=0&rev=6
2020-08-06 08:42:44 +00:00
Aaron Puchert
226481272d - Update to version 8.12.0.
* New binder notation for non-maximal implicit arguments using []
    allowing to set and see the implicit status of arguments
    immediately.
  * New notation Inductive "I A | x : s := ..." to distinguish the
    uniform from the non-uniform parameters in inductive
    definitions.
  * More robust and expressive treatment of implicit inductive
    parameters in inductive declarations.
  * Improvements in the treatment of implicit arguments and
    partially applied constants in notations, parsing of
    hexadecimal number notation and better handling of scopes and
    coercions for printing.
  * A correct and efficient coercion coherence checking algorithm,
    avoiding spurious or duplicate warnings.
  * An improved Search command which accepts complex queries. This
    takes precedence over the now deprecated ssreflect search.
  * Many additions and improvements of the standard library.
  * Improvements to the reference manual include a more logical
    organization of chapters along with updated syntax descriptions
    that match Coq's grammar in most but not all chapters.

OBS-URL: https://build.opensuse.org/package/show/science/coq?expand=0&rev=19
2020-08-05 21:55:19 +00:00
Dominique Leuenberger
b413004247 Accepting request 812064 from science
- Update to version 8.11.2.
  * Fixed a kernel issue where using Require inside a section
    caused an anomaly when closing the section.
  * Fixed normalization in conclusion of custom induction scheme.
  * Fixed a loss of location of some tactic errors.
  * Ignore -native-compiler option when built without native
    compute support.
  * Fixed a segfault issue with CoqIDE completion.
  * Highlighting style is now consistently applied to all three
    buffers of CoqIDE.

OBS-URL: https://build.opensuse.org/request/show/812064
OBS-URL: https://build.opensuse.org/package/show/openSUSE:Factory/coq?expand=0&rev=5
2020-06-07 19:37:49 +00:00
Aaron Puchert
de34c223a6 - Update to version 8.11.2.
* Fixed a kernel issue where using Require inside a section
    caused an anomaly when closing the section.
  * Fixed normalization in conclusion of custom induction scheme.
  * Fixed a loss of location of some tactic errors.
  * Ignore -native-compiler option when built without native
    compute support.
  * Fixed a segfault issue with CoqIDE completion.
  * Highlighting style is now consistently applied to all three
    buffers of CoqIDE.

OBS-URL: https://build.opensuse.org/package/show/science/coq?expand=0&rev=17
2020-06-06 12:12:35 +00:00
Dominique Leuenberger
7aa2118d49 Accepting request 792575 from science
- Update to version 8.11.1, with upstream support for OCaml 4.10.
  * Allow more inductive types in Unset Positivity Checking mode.
  * Fixed bugs in dealing with precedence of notations in custom
    entries.
  * In primitive floats, print a warning when parsing a decimal
    value that is not exactly a binary64 floating-point number.
    For instance, parsing 0.1 will print a warning whereas parsing
    0.5 won't.
  * Fixed an issue in CoqIDE about compiling file paths containing
    spaces.
  * Fixed an issue where Extraction Implicit on the constructor of
    a record was leading to an anomaly.
- Remove now obsolete ocaml-410-build.patch.

OBS-URL: https://build.opensuse.org/request/show/792575
OBS-URL: https://build.opensuse.org/package/show/openSUSE:Factory/coq?expand=0&rev=4
2020-04-09 21:17:16 +00:00
Aaron Puchert
402a945db4 - Update to version 8.11.1, with upstream support for OCaml 4.10.
* Allow more inductive types in Unset Positivity Checking mode.
  * Fixed bugs in dealing with precedence of notations in custom
    entries.
  * In primitive floats, print a warning when parsing a decimal
    value that is not exactly a binary64 floating-point number.
    For instance, parsing 0.1 will print a warning whereas parsing
    0.5 won't.
  * Fixed an issue in CoqIDE about compiling file paths containing
    spaces.
  * Fixed an issue where Extraction Implicit on the constructor of
    a record was leading to an anomaly.
- Remove now obsolete ocaml-410-build.patch.

OBS-URL: https://build.opensuse.org/package/show/science/coq?expand=0&rev=15
2020-04-08 23:19:34 +00:00
Dominique Leuenberger
81797fca28 Accepting request 789593 from science
- The num library is required for OCaml 4.06 or later.
- Add ocaml-410-build.patch: fix build with OCaml 4.10.

OBS-URL: https://build.opensuse.org/request/show/789593
OBS-URL: https://build.opensuse.org/package/show/openSUSE:Factory/coq?expand=0&rev=3
2020-03-30 21:02:48 +00:00
Aaron Puchert
9476266733 - Add patch tag.
OBS-URL: https://build.opensuse.org/package/show/science/coq?expand=0&rev=13
2020-03-29 22:22:42 +00:00
Aaron Puchert
c327875f86 - Always require ocamlfind(num), seems we can't use %pkg_vcmp here.
OBS-URL: https://build.opensuse.org/package/show/science/coq?expand=0&rev=12
2020-03-29 22:17:57 +00:00
Aaron Puchert
504ea95368 - The num library is required for OCaml 4.06 or later.
- Add ocaml-410-build.patch: fix build with OCaml 4.10.

OBS-URL: https://build.opensuse.org/package/show/science/coq?expand=0&rev=11
2020-03-29 22:08:07 +00:00
Dominique Leuenberger
d261ad0795 Accepting request 774603 from science
- Update to version 8.11.0.
  * Ltac2, a new tactic language for writing more robust larger
    scale tactics, with built-in support for datatypes and the
    multi-goal tactic monad.
  * Primitive floats are integrated in terms and follow the binary64
    format of the IEEE 754 standard, as specified in the
    Coq.Float.Floats library.
  * Many other cleanups and improvements have been performed and
    are further described in the changelog.
  * Special note on compatibility: Fixed bugs of Export and Import
    that can have a significant impact on user developments.
- Drop unneeded empty *.vos files.
- Update to version 8.10.2.
  * Fixed a critical bug of template polymorphism and nonlinear
    universes;
  * Fixed a few anomalies;
  * Fixed an 8.10 regression related to the printing of coercions
    associated to notations;
  * Fixed uneven dimensions of CoqIDE panels when window has been
    resized;
  * Fixed queries in CoqIDE.
- Update to version 8.10.0.
  * some quality-of-life bug fixes;
  * a critical bug fix related to template polymorphism;
  * native 63-bit machine integers;
  * a new sort of definitionally proof-irrelevant propositions: SProp;
  * private universes for opaque polymorphic constants;
  * string notations and numeral notations;
  * a new simplex-based proof engine for the tactics lia, nia, lra
    and nra;
  * new introduction patterns for SSReflect;
  * a tactic to rewrite under binders: under;
  * easy input of non-ASCII symbols in CoqIDE, which now uses GTK3.
- Update to version 8.10.1.
  * Fix proof of False when using SProp
  * Fix an anomaly when unsolved evar in Add Ring
  * Fix Ltac regression in binding free names in uconstr
  * Fix handling of unicode input before space
  * Fix custom extraction of inductives to JSON
- Update version requirements.

OBS-URL: https://build.opensuse.org/request/show/774603
OBS-URL: https://build.opensuse.org/package/show/openSUSE:Factory/coq?expand=0&rev=2
2020-02-15 21:26:16 +00:00
Aaron Puchert
fcdc0a168f Accepting request 774600 from home:aaronpuchert
- Update to version 8.11.0.
  * Ltac2, a new tactic language for writing more robust larger
    scale tactics, with built-in support for datatypes and the
    multi-goal tactic monad.
  * Primitive floats are integrated in terms and follow the binary64
    format of the IEEE 754 standard, as specified in the
    Coq.Float.Floats library.
  * Many other cleanups and improvements have been performed and
    are further described in the changelog.
  * Special note on compatibility: Fixed bugs of Export and Import
    that can have a significant impact on user developments.
- Drop unneeded empty *.vos files.
- Update to version 8.10.2.
  * Fixed a critical bug of template polymorphism and nonlinear
    universes;
  * Fixed a few anomalies;
  * Fixed an 8.10 regression related to the printing of coercions
    associated to notations;
  * Fixed uneven dimensions of CoqIDE panels when window has been
    resized;
  * Fixed queries in CoqIDE.
- Update to version 8.10.0.
  * some quality-of-life bug fixes;
  * a critical bug fix related to template polymorphism;
  * native 63-bit machine integers;
  * a new sort of definitionally proof-irrelevant propositions: SProp;
  * private universes for opaque polymorphic constants;
  * string notations and numeral notations;
  * a new simplex-based proof engine for the tactics lia, nia, lra
    and nra;
  * new introduction patterns for SSReflect;
  * a tactic to rewrite under binders: under;
  * easy input of non-ASCII symbols in CoqIDE, which now uses GTK3.
- Update to version 8.10.1.
  * Fix proof of False when using SProp
  * Fix an anomaly when unsolved evar in Add Ring
  * Fix Ltac regression in binding free names in uconstr
  * Fix handling of unicode input before space
  * Fix custom extraction of inductives to JSON
- Update version requirements.

OBS-URL: https://build.opensuse.org/request/show/774600
OBS-URL: https://build.opensuse.org/package/show/science/coq?expand=0&rev=9
2020-02-15 19:32:26 +00:00
Dominique Leuenberger
cac1a7f4c9 Accepting request 747961 from science
- Initial release based on version 8.9.1.

OBS-URL: https://build.opensuse.org/request/show/747961
OBS-URL: https://build.opensuse.org/package/show/openSUSE:Factory/coq?expand=0&rev=1
2019-11-30 09:36:53 +00:00
Aaron Puchert
f2a34ee4a1 - Fix findlib build dependency.
OBS-URL: https://build.opensuse.org/package/show/science/coq?expand=0&rev=7
2019-11-13 01:44:06 +00:00
Aaron Puchert
bc5f5c08e6 - Use memory-constraints package to limit number of threads.
- Add dependencies to fix installation issues.

OBS-URL: https://build.opensuse.org/package/show/science/coq?expand=0&rev=6
2019-11-03 18:30:53 +00:00
Aaron Puchert
c14d724bca - Fix typo.
OBS-URL: https://build.opensuse.org/package/show/science/coq?expand=0&rev=5
2019-09-25 21:33:11 +00:00
Aaron Puchert
ded928ac6b - Adjust number of jobs manually.
OBS-URL: https://build.opensuse.org/package/show/science/coq?expand=0&rev=4
2019-09-25 21:30:35 +00:00
Aaron Puchert
a6698df172 - Remove line break, apparently that doesn't work.
OBS-URL: https://build.opensuse.org/package/show/science/coq?expand=0&rev=3
2019-09-25 20:43:30 +00:00
Aaron Puchert
057e1be183 - Prevent OOM by limiting the number of threads.
OBS-URL: https://build.opensuse.org/package/show/science/coq?expand=0&rev=2
2019-09-25 20:17:00 +00:00
928f86c4f8 Accepting request 733035 from home:aaronpuchert
- Initial release based on version 8.9.1.

OBS-URL: https://build.opensuse.org/request/show/733035
OBS-URL: https://build.opensuse.org/package/show/science/coq?expand=0&rev=1
2019-09-25 09:10:33 +00:00