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...
Using Printing Width to get the max printing width. Close #18438
Fix #5342 This makes `destruct` and `Scheme` use the same error message as `match`.
This PR adds new vernacular instructions `Sort q1 ... qn.` / `Sorts q1 ... qn.` to declare global fresh sort qualities `q1`, ..., `qn`. Its intended usage is to add...
Depends on a few patches still.
#### Description of the problem A few tactics which do not strictly refine the goal lose the name of the goal. E.g.: ```coq Goal exists x, x = 0. unshelve...
#### Description of the problem ```coq Record T := { f : Type -> Type }. Arguments f _ A. Goal T. split; intro. (* returns "X : Type |-...
Currently it's not possible to write efficient Coq in Ltac2 without making use of terms with unbound references, which are incompatible with tactics like `cbv` and `match!` without `Constr.in_context`, which...
#### Description of the problem Hi, I've just noticed a problem with `Reset` (which is a great feature for testing while writing code!). Basically, as you see below, I can...
#### Description of the problem In the following example (from CUDW2023) rewriting with a local hypothesis does not work using Ltac2 rewrite: ``` Require Import Reals. Require Import QArith. Require...
#### Description of the problem ```coq From Coq Require Import ssreflect. Goal True -> True. move=> H. apply: (H) {H}. (* Error: Anomaly "in retyping: Variable H unbound." *) ```...