coq
coq copied to clipboard
Coq is a formal proof management system. It provides a formal language to write mathematical definitions, executable algorithms and theorems together with an environment for semi-interactive developme...
https://github.com/coq/coq/blob/d712096e84579b346bf87341165228c55403dded/user-contrib/Ltac2/Constr.v#L92-L95 It should be possible to add a let-binding to the context and not just a lambda binding cc @coq/ltac2-maintainers
#### Description of the problem I am not sure where is the right place to report this, but I feel like there are some pains caused by the dune migration...
This is an experimental branch, not to be merged directly.
In particular we remove the `coqlib` field which was just used to suppress a warning. This brings `coqdep/loadpath` closer to `vernac/loadpath.ml`, but still a way to go. Many differences are...
Add computational content to `List.v`: mainly `Type` is used instead of `Prop` as much as possible. **Kind:** feature. - [ ] Entry added in the changelog
Setting this flag in `auto` (and `eauto`) makes the resolution be slightly closer to `simple (e)apply`. Also, this behavior is closer to `typeclasses eauto`. Fixes #16323 Fixes #16062 Currently, `debug...
Not sure this will have much impact but let's see
#### Description of the problem Consider the code ```coq Fixpoint mkgoal (n : nat) : Prop := match n with | O => True /\ True -> True | S...
#### Version ~~~~~ The Coq Proof Assistant, version 8.8.1 (July 2018) compiled on Jul 5 2018 7:25:50 with OCaml 4.06.0 ~~~~~ #### Operating system Arch Linux, up to date as...
Note: the issue was created automatically with bugzilla2github tool Original bug ID: BZ#2727 From: @fpottier Reported version: 8.5 CC: @herbelin, @pirbo