Search code examples
Coq prove a false list assumption...


coq

Read More
Trivial lemma on real numbers on Coq...


coq

Read More
Definition of equality among vectors...


coq

Read More
diffefentiation of (1/2)*(x-y)^2 on x is x - y...


coq

Read More
How can I construct terms in first-order logic using Coq?...


coqfirst-order-logic

Read More
Coq: Syntax error 'Type' or 'Types' expected after 'Implicit'...


coq

Read More
Make two arbitrary variables the same in Coq...


coq

Read More
Coq destruct with an excluding precondition...


coq

Read More
`match goal` doesn't match let destructuring expression...


coqcoq-tactic

Read More
Coq - How can you apply an implication with a match clause?...


coqcoq-tactic

Read More
How does 'elim' in Coq work on existential quantifier?...


coqfirst-order-logic

Read More
Stuck with a proof...


coq

Read More
Dependent functions in Coq...


coq

Read More
Different arguments, but behavior of function is same...


coq

Read More
How does the grading script of the LF series work for manually graded exercises?...


coqlogical-foundations

Read More
Is there a good strategy for proving the given theorem?...


sortingcoq

Read More
Can't bind variable to wrapped open formula...


coq

Read More
Equality on complex functions with complex type...


coq

Read More
Equality on complex functions...


coq

Read More
How to prove equivalence between those two types - algorithm' and algorithm''?...


coq

Read More
Z_3: left inversion lemma...


coq

Read More
Coq unable to unify -- how to change hypothesis?...


coqcoq-tactic

Read More
How to apply a constructor in an hypothesis?...


coqproofcoq-tactic

Read More
Messing around with category theory...


coqcategory-theory

Read More
Z_3: left id proof...


coq

Read More
Inductive proposition for sublists in Coq...


coqcoq-tacticinductive-logic-programming

Read More
Proof irrelevance for boolean equality...


coqproof

Read More
How can I prevent Coq notations in closed scopes interfering with notations in open ones?...


coq

Read More
normalize (normalize n) = normalize (n)...


coq

Read More
Prove equality of lists with list_beq...


coq

Read More
BackNext