Search code examples
Error: Cannot coerce to an evaluable reference in coq...


coqcompcert

Read More
Casting types in coq...


coqcoq-tacticcompcert

Read More
In Coq, is there a way to get rid of "useless" preconditions in a hypothesis?...


coq

Read More
Why can't I use `app` together with `fold_right` in Coq?...


coq

Read More
Proving equality on coinductive lazy lists in Coq...


coqlazy-sequencescoinduction

Read More
Fixpoint on Types...


typescoq

Read More
How to prove forall x, (R x \/ ~ R x) [in the Coq proof assistant]?...


coqproof

Read More
Coq --- Arguments directive...


argumentscoqimplicit-typing

Read More
a + b = 0 -> a = 0 and b = 0 in Coq...


coq

Read More
Declaring a well colored digraph in coq...


coq

Read More
How to access the elements of a record in coq...


coq

Read More
Change a function at one point...


coq

Read More
How to prove x + y - z = x + (y - z) in Coq...


coqproof

Read More
how to finish this proof in Coq...


coq

Read More
Solving (BEq a a0 = BTrue \/ BEq a a0 = BFalse) in Coq...


coqproof

Read More
Coq: Error: The reference [Lemma/Theorem] was not found in the current environment...


coq

Read More
Prove "rev (rev l) = l" in Coq...


coqinduction

Read More
Reference in Coq Lists library not found...


coq

Read More
Coq variable exists in list...


coqformal-verification

Read More
Proving for all elements of a list in coq...


coq

Read More
comparing two unequal values in coq...


coqcompcert

Read More
How to change display style in Coq IDE to match Coqtop?...


coqcoqide

Read More
Coq notation format for double square braces...


formatcoqnotation

Read More
Different induction principles for Prop and Type...


coq

Read More
Simple identity in Coq...


coqtheorem-proving

Read More
Definition by property in coq...


coq

Read More
disjunction of empty and non-empty list in coq...


coq

Read More
Coq adding a new variable instead of using the correct one...


coq

Read More
Unfold a notation within a scope...


coq

Read More
Solving equality / inequality in goal, coq code...


coqformal-verificationcompcert

Read More
BackNext