Search code examples
How to overload the "+" notation in Coq?...


coq

Read More
Fail to `destruct` due to ill-typedness and even cannot give an exact term in Coq...


coq

Read More
How do I install ocamlfind first properly before other opam packages without root permissions?...


ocamlcoqopamdune

Read More
How to duplicate a hypothesis in Coq?...


coq

Read More
Does `∃! x, ∃! y, P (x, y)` imply `∃! xy, P (fst xy) (snd xy)`?...


coq

Read More
How to call proof asistant Coq from external software...


coq

Read More
Why does Ltac not match the clause?...


coqltac

Read More
How does one expand a `fix` function just one step?...


recursioncoq

Read More
How to prove A \/ False -> A in Coq?...


logiccoqtheorem-proving

Read More
Lean4: Proving that `(xs = ys) = (reverse xs = reverse ys)`...


logiccoqprooftheorem-provinglean

Read More
"Cannot instantiate metavariable P of type ..." when destructing in Coq proof mode...


coq

Read More
Forcing evaluation of terms before extraction, or other ways to test extracted functions?...


coqcoq-extraction

Read More
Is it possible to make Coq accept a class of Fixpoint functions if we provide proofs of argument siz...


coq

Read More
What does InjL and InjR operator means in coq-Iris?...


coqformal-verificationformal-semantics

Read More
using addf_div for rat_numDomainType...


coqssreflect

Read More
Exhaustiveness matching in proof objects for induction in Coq...


coq

Read More
Is it possible to destruct and rewrite simultaneously?...


coq

Read More
induction integer record in coq...


coqcoq-tactic

Read More
Do you need to pass in template types to functions that accept template objects in Coq?...


coq

Read More
Rewrite with variable from inner scope?...


coq

Read More
Fix vs. Fix_sub...


coq

Read More
Two Coq Problems SOS: one is about IndProp, another has something to do with recursion, I guess...


recursioncoq

Read More
Proving theorems containing bitwise operators...


binarycoqcoq-tactic

Read More
How to avoid "Cannot guess decreasing argument of fix." in Coq...


recursioncoqcoqide

Read More
De Bruijn indices in Isabelle and Coq...


coqisabelle

Read More
Coq: Unification fails with record...


recordcoqdependent-typeunification

Read More
How to install the coq 8.14 (or 8.15) package with opam pin when it says it can't find it?...


ocamlcoqopam

Read More
type variable in datatype definition...


coqisabelleformal-languagesformal-verification

Read More
How do I exit coqtop REPL?...


coq

Read More
Proving Union of Ensemble is not Empty_set...


coq

Read More
BackNext