Search code examples
How does `auto` interract with biconditional (iff)...


coq

Read More
How does decidable equality works with List.remove?...


coq

Read More
not_iff_compat not found in the current environment...


coq

Read More
Counting number of different elements in a list in Coq...


coq

Read More
Using 'unfold' of a Fixpoint inside the recursive step of the induction...


coqcoq-tactic

Read More
Creating a dictionary/map in Coq...


dictionarycoqformal-verification

Read More
Coq: Resolve an expression to multiple instances...


classtype-inferencecoq

Read More
Implicit arguments in a computed type in Coq...


typescoq

Read More
`context` expression in Coq...


coqltac

Read More
Using destruct on pattern match expression with 'convoy pattern'...


coq

Read More
Coq HoTT - How to correctly put a definition inside a theorem?...


coqtype-theory

Read More
Use Identifier before Defining for BNF-Style Definitions...


coq

Read More
coq What tactics should I use forall A : Prop, A -> ~~A...


coq

Read More
Tactic automation: simple decision procedure...


coqcoq-tactic

Read More
Equivalent of `remember (f x) as y eqn:H; clear H; clear x`?...


coqcoq-tacticltac

Read More
When does the termination checker reduce a record accessor...


coqtermination

Read More
Induction principle for nested inductive types...


coqinduction

Read More
Coq item 1.2.10 Type cast...


coq

Read More
How to pattern match multiple values in Idris/Agda/Coq?...


coqagdadependent-typeidris

Read More
What's the difference between Program Fixpoint and Function in Coq?...


coqtotality

Read More
How can I convince Coq that my function is in fact recursive?...


recursioncoqtermination

Read More
Coq simpl for Program Fixpoint...


coqtheorem-provingtotality

Read More
Using coqide, the command `Require Import BigN` worked using coq 8.6 but not in coq 8.7...


coqopam

Read More
Proving Termination of Function in Coq...


recursioncoqtermination

Read More
What does V stand for in the Coq file extension?...


filecoq

Read More
"Ring" tactic in CoqIde not accepted...


coqcoq-tactic

Read More
Eta conversion tactics?...


coqcoq-tactic

Read More
Subtype with Coq...


coqsubtype

Read More
Define product type after importing QArith...


coq

Read More
Coq vector permutations...


listvectorpermutationcoqinduction

Read More
BackNext