coq
                                
                                 coq copied to clipboard
                                
                                    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...
Hi, the idea of an introduction pattern following the `'pat`-style quantification is in the air for some time. This PR is proposing a (very) raw first proof of concept. Basic...
#### Description of the problem ```coq Goal True. Proof. ``` gives ``` Error: Anomaly "Stm.join: tip not cached" Please report at http://coq.inria.fr/bugs/. ``` cc @coq/stm-maintainers #### Coq Version https://gitlab.com/coq/coq/-/jobs/2740357137/artifacts/download i.e....
#### Description of the problem The folded and unfolded state of `Hint Opaque` projections are not unified by `autoapply`. ```coq From Coq Require Import ssreflect. #[local] Set Primitive Projections. Class...
Note: the issue was created automatically with bugzilla2github tool Original bug ID: BZ#3104 From: @ezyang Reported version: trunk CC: @JasonGross, @ppedrot
#### Version Coq 8.8+alpha (commit a2b02cb91) #### Operating system macOS #### Description of the problem `auto using pf` is more powerful than adding pf as a hint because it doesn't...
#### Description of the problem Possibly related: https://github.com/coq/coq/issues/6544 (but here the behavior is the other way around). The documentation of `Hint Immediate` states that > adds the tactic [simple apply](https://coq.inria.fr/distrib/current/refman/proof-engine/tactics.html#coq:tacv.simple-apply)...
#### Description of the problem When `auto` is called on a goal containing an evar, the outcome is difficult to predict and the debug log on `exact` is misleading. ```coq...
#### Description of the problem Universe Polymorphism, JMeq, and a simple dependent type cause (previously working) proofs to fail at QED time. The exact error message is `Anomaly "File "kernel/term_typing.ml",...
**Kind**: enhancement This is an experimental change of heuristic about when a notation defined using the `Notation "..." := ...` syntax is liable to modify a generic printing rule. The...
**Kind:** cleanup This is part 2 of proposal at #15562. It includes: - removal redundancy between termops and econstr - move of `it_mkLambda`/`it_mkProd` combinators from `termops.ml` to `eConstr.ml` when on...