Search code examples
Minimum in non-empty, finite set...


coqminimum

Read More
Contradictory hypothesis using coq inversion tactic...


coqproofcoq-tactic

Read More
How to prove decidability of a partial order inductive predicate?...


coqproofdeterministicformal-verificationpartial-ordering

Read More
Weird proof obligations resulting from a push/pop evaluator in Coq...


coqproofdependent-typeproof-obligation

Read More
Applying a Program Definition fails with "unable to unify Prop with [goal]"...


coqproof

Read More
What is the EvalOp in Coq CompCert...


coqcoq-tacticcoq-extractioncompcert

Read More
Coq: Bypassing the uniform inheritance condition...


coqcoercionsubtype

Read More
A Coq proof of a theorem which turns a formula containing y into a formula containing f(x)...


coq

Read More
Non-positive occurrence due to polymorphic function...


coqalgebraic-data-types

Read More
How to extract Coq's Z into Haskell's Integer...


coqcoq-extraction

Read More
Coq - proving something which has already been defined?...


coqproof

Read More
Understanding "well founded" proofs in Coq...


theorycoq

Read More
Error in defining Ackermann in Coq...


coqackermanntotality

Read More
Defining floats and proofs using flocq...


floating-pointcoq

Read More
From an Inductive predicate to list A -> list A -> bool...


coq

Read More
Decomposing equality of constructors with match expressions in Coq...


coqcoq-tactic

Read More
Understanding Coq through a simple theorem proof...


coqtheorem-proving

Read More
How to prove excluded middle is irrefutable in Coq?...


logiccoqcoq-tactic

Read More
How can I find what file a value is defined in?...


coq

Read More
setoid_rewrite fails in pattern matching scenario...


pattern-matchingcoqsubstitution

Read More
ocamlbuild links libraries in wrong order...


ocamlcoqocamlbuild

Read More
In the coq tactics language, what is the difference between intro and intros...


coqcoq-tactic

Read More
Coq not generating inductive hypothesis...


coqprooftheorem-proving

Read More
Proof automation...


automationcoqproof

Read More
How can I automate counting within proofs in Coq?...


coqcoq-tactic

Read More
How to use auto with repeat in custom tactics?...


coqcoq-tactic

Read More
Compute with a recursive function defined by well-defined induction...


coq

Read More
Proof on booleans, false = true...


coq

Read More
Induction over relations...


coqcoq-tactic

Read More
Break "forall" hypothesis with conjunctions up into components?...


coq

Read More
BackNext