SHA256
1
0
forked from pool/coq
Commit Graph

71 Commits

Author SHA256 Message Date
Ana Guerrero
ea92abb9c6 Accepting request 1199381 from science
- Update to version 8.20.0. The most impactful changes are:
  * A mechanism to add user-defined rewrite rules to Coq's reduction
    mechanisms; see chapter "User-defined rewrite rules".
  * Support for primitive strings in terms.
  * Reduction of the bytecode segment size, which in turn means
    that `.vo` files might now be considerably smaller.
- Notable breaking changes:
  * Syntactic global references passed through the `using` clauses
    of `auto`-like tactics are now handled as plain references
    rather than interpreted terms. In particular, their typeclass
    arguments will not be inferred. In general, the previous
    behaviour can be emulated by replacing `auto using foo` with
    `pose proof foo; auto`.
  * Argument order for the Ltac2 combinators `List.fold_left2` and
    `List.fold_right2` changed to be the same as in OCaml.
  * Importing a module containing a mutable Ltac2 definition does
    not undo its mutations. Replace `Ltac2 mutable foo :=
    some_expr.` with `Ltac2 mutable foo := some_expr. Ltac2 Set foo
    := some_expr.` to recover the previous behaviour.
  * Some renaming in the standard library. Deprecations are
    provided for a smooth transition.
- For more details, see the change log in coq-doc.

OBS-URL: https://build.opensuse.org/request/show/1199381
OBS-URL: https://build.opensuse.org/package/show/openSUSE:Factory/coq?expand=0&rev=29
2024-09-09 12:44:11 +00:00
Aaron Puchert
9c22c89df3 - Update to version 8.20.0. The most impactful changes are:
* A mechanism to add user-defined rewrite rules to Coq's reduction
    mechanisms; see chapter "User-defined rewrite rules".
  * Support for primitive strings in terms.
  * Reduction of the bytecode segment size, which in turn means
    that `.vo` files might now be considerably smaller.
- Notable breaking changes:
  * Syntactic global references passed through the `using` clauses
    of `auto`-like tactics are now handled as plain references
    rather than interpreted terms. In particular, their typeclass
    arguments will not be inferred. In general, the previous
    behaviour can be emulated by replacing `auto using foo` with
    `pose proof foo; auto`.
  * Argument order for the Ltac2 combinators `List.fold_left2` and
    `List.fold_right2` changed to be the same as in OCaml.
  * Importing a module containing a mutable Ltac2 definition does
    not undo its mutations. Replace `Ltac2 mutable foo :=
    some_expr.` with `Ltac2 mutable foo := some_expr. Ltac2 Set foo
    := some_expr.` to recover the previous behaviour.
  * Some renaming in the standard library. Deprecations are
    provided for a smooth transition.
- For more details, see the change log in coq-doc.

OBS-URL: https://build.opensuse.org/package/show/science/coq?expand=0&rev=67
2024-09-07 15:01:23 +00:00
Dominique Leuenberger
516fd9bf5c Accepting request 1184115 from science
- Update to version 8.19.2.
  * Fixed a regression from Coq 8.18 in the presence of a defined
    field in a primitive `Record`.
  * Fixed an issue where the printer was sometimes failing to use a
    prefix or infix custom notation whose right-hand side refers to
    a different custom entry.
  * Fixed `abstract` failure in the presence of admitted goals in
    the surrounding proof.
  * Fixed issues when using Ltac2 in VsCoq due to incorrect state
    handling of Ltac2 notations.
  * Fixed `Include` on a module containing a record declared with
    `Primitive Projections`.
  * Fixed an issue in `Fixpoint` with no arguments.
  * Position error/warning tooltips correctly when multibyte UTF-8
    characters are present.

OBS-URL: https://build.opensuse.org/request/show/1184115
OBS-URL: https://build.opensuse.org/package/show/openSUSE:Factory/coq?expand=0&rev=28
2024-07-01 09:21:23 +00:00
Aaron Puchert
4fddaa2fa7 - Update to version 8.19.2.
* Fixed a regression from Coq 8.18 in the presence of a defined
    field in a primitive `Record`.
  * Fixed an issue where the printer was sometimes failing to use a
    prefix or infix custom notation whose right-hand side refers to
    a different custom entry.
  * Fixed `abstract` failure in the presence of admitted goals in
    the surrounding proof.
  * Fixed issues when using Ltac2 in VsCoq due to incorrect state
    handling of Ltac2 notations.
  * Fixed `Include` on a module containing a record declared with
    `Primitive Projections`.
  * Fixed an issue in `Fixpoint` with no arguments.
  * Position error/warning tooltips correctly when multibyte UTF-8
    characters are present.

OBS-URL: https://build.opensuse.org/package/show/science/coq?expand=0&rev=65
2024-06-30 17:29:40 +00:00
Ana Guerrero
2c5836b4d9 Accepting request 1156169 from science
- Update to version 8.19.1.
  * Fixed incorrect abstraction of sort variables for opaque
    constants leading to an inconsistency.
  * Fixed memory corruption with `vm_compute` (rare but more
    likely with OCaml 5.1).
  * "Found no matching notation to enable or disable" is now a
    warning instead of an error.
  * Fixed undeclared universe with multiple uses of `abstract`.
  * Fixed incorrect printing of constructor values with multiple
    arguments, and over-parenthesizing of constructor printing.
  * Fixed incorrect declared type for Ltac2.FMap.fold.

OBS-URL: https://build.opensuse.org/request/show/1156169
OBS-URL: https://build.opensuse.org/package/show/openSUSE:Factory/coq?expand=0&rev=27
2024-03-08 17:09:09 +00:00
Aaron Puchert
8870b507b6 - Update to version 8.19.1.
* Fixed incorrect abstraction of sort variables for opaque
    constants leading to an inconsistency.
  * Fixed memory corruption with `vm_compute` (rare but more
    likely with OCaml 5.1).
  * "Found no matching notation to enable or disable" is now a
    warning instead of an error.
  * Fixed undeclared universe with multiple uses of `abstract`.
  * Fixed incorrect printing of constructor values with multiple
    arguments, and over-parenthesizing of constructor printing.
  * Fixed incorrect declared type for Ltac2.FMap.fold.

OBS-URL: https://build.opensuse.org/package/show/science/coq?expand=0&rev=63
2024-03-07 23:33:38 +00:00
Ana Guerrero
4a9b6a9784 Accepting request 1142140 from science
- Update to version 8.19.0. The most impactful changes:
  * Sort polymorphism makes it possible to share common constructs
    over `Type`, `Prop` and `SProp`.
  * The notation `term%_scope` to set a scope only temporarily (in
    addition to `term%scope` for opening a scope applying to all
    subterms).
  * `lazy`, `simpl`, `cbn` and `cbv` and the associated `Eval` and
    `eval` reductions learned to do head reduction when given flag
    `head`.
  * New Ltac2 APIs, improved Ltac2 `exact` and dynamic building of
    Ltac2 term patterns.
  * New performance evaluation facilities: `Instructions` to count
    CPU instructions used by a command and Profiling system to
    produce trace files.
  * New command `Attributes` to assign attributes such as
    `deprecated` to a library file.
- Notable breaking changes:
  * `replace` with `by tac` does not automatically attempt to solve
    the generated equality subgoal using the hypotheses. Use `by
    first [assumption | symmetry;assumption | tac]` if you need the
    previous behaviour.
  * Removed old deprecated files from the standard library. 
- Use %fdupes in the documentation package.

OBS-URL: https://build.opensuse.org/request/show/1142140
OBS-URL: https://build.opensuse.org/package/show/openSUSE:Factory/coq?expand=0&rev=26
2024-01-29 21:28:51 +00:00
Aaron Puchert
10555467e2 - Cover stdlib with %fdupes.
OBS-URL: https://build.opensuse.org/package/show/science/coq?expand=0&rev=61
2024-01-28 20:56:18 +00:00
Aaron Puchert
042203acb7 - Update to version 8.19.0. The most impactful changes:
* Sort polymorphism makes it possible to share common constructs
    over `Type`, `Prop` and `SProp`.
  * The notation `term%_scope` to set a scope only temporarily (in
    addition to `term%scope` for opening a scope applying to all
    subterms).
  * Tactics `lazy`, `simpl`, `cbn` and `cbv` and the associated
    `Eval` and `eval` reductions learned to do head reduction when
    given flag head.
  * New Ltac2 APIs, improved Ltac2 `exact` and dynamic building of
    Ltac2 term patterns.
  * New performance evaluation facilities: `Instructions` to count
    CPU instructions used by a command (Linux only) and Profiling
    system to produce trace files.
  * New command `Attributes` to assign attributes such as
    `deprecated` to a library file.
- Notable breaking changes:
  * `replace` with `by tac` does not automatically attempt to solve
    the generated equality subgoal using the hypotheses. Use `by
    first [assumption | symmetry;assumption | tac]` if you need the
    previous behaviour.
  * Removed old deprecated files from the standard library. 
- Use %fdupes in the documentation package.

OBS-URL: https://build.opensuse.org/package/show/science/coq?expand=0&rev=60
2024-01-28 20:41:21 +00:00
Ana Guerrero
53f3b27cea Accepting request 1125372 from science
- Revert last change: this is now set in ocaml-rpm-macros.
- Increase stack size limit in QEMU user space builds. Here ulimit
  has no effect, so we add a wrapper around ocamlopt.opt to PATH
  that adds "-s ..." to the qemu-<arch> command line.

OBS-URL: https://build.opensuse.org/request/show/1125372
OBS-URL: https://build.opensuse.org/package/show/openSUSE:Factory/coq?expand=0&rev=25
2023-11-13 21:21:57 +00:00
Aaron Puchert
37bbcb7cbf - Do the right thing if qemu_user_space_build is defined as 0.
OBS-URL: https://build.opensuse.org/package/show/science/coq?expand=0&rev=58
2023-11-12 23:14:09 +00:00
Aaron Puchert
669ef86008 - Increase stack size limit in QEMU user space builds. Here ulimit
has no effect, so we add a wrapper around ocamlopt.opt to PATH
  that adds "-s ..." to the qemu-<arch> command line.

OBS-URL: https://build.opensuse.org/package/show/science/coq?expand=0&rev=57
2023-11-12 22:55:08 +00:00
Aaron Puchert
d5b741161a - Revert last change: this is now set in ocaml-rpm-macros.
OBS-URL: https://build.opensuse.org/package/show/science/coq?expand=0&rev=56
2023-11-11 00:35:56 +00:00
Ana Guerrero
36d9e6cc14 Accepting request 1121332 from science
- Increase stack size limit to fix build on riscv64.

OBS-URL: https://build.opensuse.org/request/show/1121332
OBS-URL: https://build.opensuse.org/package/show/openSUSE:Factory/coq?expand=0&rev=24
2023-10-31 19:25:29 +00:00
Aaron Puchert
ad9d18ea83 - Increase stack size limit to fix build on riscv64.
OBS-URL: https://build.opensuse.org/package/show/science/coq?expand=0&rev=54
2023-10-30 22:28:37 +00:00
Dominique Leuenberger
b65f8cd660 Accepting request 1111685 from science
- Update to version 8.18.0.
  * The default locality of `Hint` and `Instance` commands was
    switched to `export`.
  * The universe unification algorithm can now delay the commitment
    to a sort (the algorithm used to pick `Type`). Thanks to this
    feature many `Prop` and `SProp` annotations can be now omitted.
  * Ltac2 supports array literals, maps and sets of primitive
    datatypes such as names (of constants, inductive types, etc)
    and fine-grained control over profiling.
  * The warning system offers new categories, enabling finer
    (de)activation of specific warnings. This should be
    particularly useful to handle deprecations.
  * Many new lemmas useful for teaching analysis with Coq are now
    part of the standard library about real numbers.
  * The `#[deprecated]` attribute can now be applied to definitions.

OBS-URL: https://build.opensuse.org/request/show/1111685
OBS-URL: https://build.opensuse.org/package/show/openSUSE:Factory/coq?expand=0&rev=23
2023-09-20 11:25:12 +00:00
Aaron Puchert
111d6555f8 - Update to version 8.18.0.
* The default locality of `Hint` and `Instance` commands was
    switched to `export`.
  * The universe unification algorithm can now delay the commitment
    to a sort (the algorithm used to pick `Type`). Thanks to this
    feature many `Prop` and `SProp` annotations can be now omitted.
  * Ltac2 supports array literals, maps and sets of primitive
    datatypes such as names (of constants, inductive types, etc)
    and fine-grained control over profiling.
  * The warning system offers new categories, enabling finer
    (de)activation of specific warnings. This should be
    particularly useful to handle deprecations.
  * Many new lemmas useful for teaching analysis with Coq are now
    part of the standard library about real numbers.
  * The `#[deprecated]` attribute can now be applied to definitions.

OBS-URL: https://build.opensuse.org/package/show/science/coq?expand=0&rev=52
2023-09-17 00:40:53 +00:00
Dominique Leuenberger
01c47874b8 Accepting request 1095883 from science
- Update to version 8.17.1.
  * Fixed incorrect paths emitted by coqdep in some cases for META
    files which prevented dune builds for plugins from working
    correctly.
  * Fixed shadowing of record fields in extraction to OCaml.
  * Fixed an impossible-to-turn-off debug message "backtracking and
    redoing byextend on ...".
  * Fixed a major memory regression affecting MathComp 2.
- Classify desktop entry under Science instead of Education.
- Add screenshot URL to AppStream metadata.

OBS-URL: https://build.opensuse.org/request/show/1095883
OBS-URL: https://build.opensuse.org/package/show/openSUSE:Factory/coq?expand=0&rev=22
2023-06-29 15:28:52 +00:00
Aaron Puchert
edfae7dd86 - Update to version 8.17.1.
* Fixed incorrect paths emitted by coqdep in some cases for META
    files which prevented dune builds for plugins from working
    correctly.
  * Fixed shadowing of record fields in extraction to OCaml.
  * Fixed an impossible-to-turn-off debug message "backtracking and
    redoing byextend on ...".
  * Fixed a major memory regression affecting MathComp 2.
- Classify desktop entry under Science instead of Education.
- Add screenshot URL to AppStream metadata.

OBS-URL: https://build.opensuse.org/package/show/science/coq?expand=0&rev=50
2023-06-28 23:04:37 +00:00
Dominique Leuenberger
46ec0e01a2 Accepting request 1075082 from science
- Update to version 8.17.0.
  * Fixed a logical inconsistency due to `vm_compute` in presence
    of side-effects in the enviroment (e.g. using Back or Fail).
  * It is now possible to dynamically enable or disable notations.
  * Support multiple scopes in `Arguments` and `Bind Scope`.
  * The tactics chapter of the manual has many improvements in
    presentation and wording. The documented grammar is semi-
    automatically checked for consistency with the implementation.
  * Fixes to the `auto` and `eauto` tactics, to respect hint
    priorities and the documented use of simple apply. This is a
    potentially breaking change.
  * New Ltac2 APIs, deep pattern-matching with `as` clauses and
    handling of literals, support for record types and preterms.
  * Move from :> to :: syntax for declaring typeclass fields as
    instances, fixing a confusion with declaration of coercions.
  * Standard library improvements.

OBS-URL: https://build.opensuse.org/request/show/1075082
OBS-URL: https://build.opensuse.org/package/show/openSUSE:Factory/coq?expand=0&rev=21
2023-03-29 21:27:14 +00:00
Aaron Puchert
312f3c055e - Update to version 8.17.0.
* Fixed a logical inconsistency due to `vm_compute` in presence
    of side-effects in the enviroment (e.g. using Back or Fail).
  * It is now possible to dynamically enable or disable notations.
  * Support multiple scopes in `Arguments` and `Bind Scope`.
  * The tactics chapter of the manual has many improvements in
    presentation and wording. The documented grammar is semi-
    automatically checked for consistency with the implementation.
  * Fixes to the `auto` and `eauto` tactics, to respect hint
    priorities and the documented use of simple apply. This is a
    potentially breaking change.
  * New Ltac2 APIs, deep pattern-matching with `as` clauses and
    handling of literals, support for record types and preterms.
  * Move from :> to :: syntax for declaring typeclass fields as
    instances, fixing a confusion with declaration of coercions.
  * Standard library improvements.

OBS-URL: https://build.opensuse.org/package/show/science/coq?expand=0&rev=48
2023-03-29 01:36:33 +00:00
Dominique Leuenberger
0236a47897 Accepting request 1061434 from science
- Build with ocaml-rpm-macros to get proper Requires and Provides
  for coq-devel. This should prevent incompatibilities with other
  Ocaml libraries when building native objects against coq-devel.

OBS-URL: https://build.opensuse.org/request/show/1061434
OBS-URL: https://build.opensuse.org/package/show/openSUSE:Factory/coq?expand=0&rev=20
2023-01-27 09:16:34 +00:00
Aaron Puchert
02f83d6668 - Build with ocaml-rpm-macros to get proper Requires and Provides
for coq-devel. This should prevent incompatibilities with other
  Ocaml libraries when building native objects against coq-devel.

OBS-URL: https://build.opensuse.org/package/show/science/coq?expand=0&rev=46
2023-01-26 23:03:52 +00:00
Dominique Leuenberger
2cf283a0cb Accepting request 1038367 from science
- Update to version 8.16.1.
  * Fixed the conversion of `Prod` values in the native compiler.
  * Added `SProp` check for opaque names in conversion.
  * Pass the correct environment to compute η-expansion of
    cofixpoints in VM and native compilation.
  * Fixed an inconsistency with conversion of primitive arrays, and
    associated incomplete strong normalization of primitive arrays
    with `lazy`.
  * `Print Assumptions` treats opaque definitions with missing
    proofs (as found in .vos files, produced using -vos) as axioms
    instead of ignoring them.

OBS-URL: https://build.opensuse.org/request/show/1038367
OBS-URL: https://build.opensuse.org/package/show/openSUSE:Factory/coq?expand=0&rev=19
2022-11-27 11:53:03 +00:00
Aaron Puchert
44fe8f3492 - Update to version 8.16.1.
* Fixed the conversion of `Prod` values in the native compiler.
  * Added `SProp` check for opaque names in conversion.
  * Pass the correct environment to compute η-expansion of
    cofixpoints in VM and native compilation.
  * Fixed an inconsistency with conversion of primitive arrays, and
    associated incomplete strong normalization of primitive arrays
    with `lazy`.
  * `Print Assumptions` treats opaque definitions with missing
    proofs (as found in .vos files, produced using -vos) as axioms
    instead of ignoring them.

OBS-URL: https://build.opensuse.org/package/show/science/coq?expand=0&rev=44
2022-11-26 22:51:51 +00:00
Dominique Leuenberger
fe1a6bfdf5 Accepting request 1002206 from science
- Update to version 8.16.0.
  * The guard checker (see `Guarded`) now ensures strong
    normalization under any reduction strategy.
  * Irrelevant terms (in the `SProp` sort) are now squashed to a
    dummy value during conversion, fixing a subject reduction 
    issue and making proof conversion faster.
  * Introduction of reversible coercions, which allow coercions 
    relying on meta-level resolution such as type-classes or 
    canonical structures. Also allow coercions that do not fullfill
    the uniform inheritance condition.
  * Generalized rewriting support for rewriting with `Type`-valued 
    relations and in `Type` contexts, using the
    `Classes.CMorphisms` library.
  * Added the boolean equality scheme command for decidable 
    inductive types.
  * Added a `Print Notation` command.
  * Incompatibilities in name generation for Program obligations,
    `eauto` treatment of tactic failure levels, use of `ident` in
    notations, parsing of module expressions.
  * Standard library reorganization and deprecations.
  * Improve the treatment of standard library numbers by
    `Extraction`.
- Coq requires ocamlfind at runtime now.

OBS-URL: https://build.opensuse.org/request/show/1002206
OBS-URL: https://build.opensuse.org/package/show/openSUSE:Factory/coq?expand=0&rev=18
2022-09-09 16:28:00 +00:00
Aaron Puchert
6dee5e36dc - Update to version 8.16.0.
* The guard checker (see `Guarded`) now ensures strong
    normalization under any reduction strategy.
  * Irrelevant terms (in the `SProp` sort) are now squashed to a
    dummy value during conversion, fixing a subject reduction 
    issue and making proof conversion faster.
  * Introduction of reversible coercions, which allow coercions 
    relying on meta-level resolution such as type-classes or 
    canonical structures. Also allow coercions that do not fullfill
    the uniform inheritance condition.
  * Generalized rewriting support for rewriting with `Type`-valued 
    relations and in `Type` contexts, using the
    `Classes.CMorphisms` library.
  * Added the boolean equality scheme command for decidable 
    inductive types.
  * Added a `Print Notation` command.
  * Incompatibilities in name generation for Program obligations,
    `eauto` treatment of tactic failure levels, use of `ident` in
    notations, parsing of module expressions.
  * Standard library reorganization and deprecations.
  * Improve the treatment of standard library numbers by
    `Extraction`.
- Coq requires ocamlfind at runtime now.

OBS-URL: https://build.opensuse.org/package/show/science/coq?expand=0&rev=42
2022-09-08 21:21:24 +00:00
Dominique Leuenberger
da554d4f31 Accepting request 980409 from science
- Update to version 8.15.2.
  * Tactics `intuition` and `dintuition` use
    `Tauto.intuition_solver` (defined as `auto with *`) instead of
    hardcoding `auto with *`. This makes it possible to change the
    default solver with `Ltac Tauto.intuition_solver ::= ...`.
  * Fixed an uncaught exception `UnableToUnify` with
    bidirectionality hints.
  * Fixed multiple CoqIDE bugs.
  * Fixed an incorrect implementation of `SFClassify`, allowing for
    a proof of `False` since 8.11.0, due to Axioms present in
    `Float.Axioms`.
- Rename coq.desktop to fr.inria.coq.coqide.desktop as the
  documentation suggests, add an accompanying metainfo file.
- Declare documentation as noarch.

OBS-URL: https://build.opensuse.org/request/show/980409
OBS-URL: https://build.opensuse.org/package/show/openSUSE:Factory/coq?expand=0&rev=17
2022-06-02 19:54:19 +00:00
Aaron Puchert
9b2016e937 - Update to version 8.15.2.
* Tactics `intuition` and `dintuition` use
    `Tauto.intuition_solver` (defined as `auto with *`) instead of
    hardcoding `auto with *`. This makes it possible to change the
    default solver with `Ltac Tauto.intuition_solver ::= ...`.
  * Fixed an uncaught exception `UnableToUnify` with
    bidirectionality hints.
  * Fixed multiple CoqIDE bugs.
  * Fixed an incorrect implementation of `SFClassify`, allowing for
    a proof of `False` since 8.11.0, due to Axioms present in
    `Float.Axioms`.
- Rename coq.desktop to fr.inria.coq.coqide.desktop as the
  documentation suggests, add an accompanying metainfo file.
- Declare documentation as noarch.

OBS-URL: https://build.opensuse.org/package/show/science/coq?expand=0&rev=40
2022-06-01 21:48:29 +00:00
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