Search code examples
How to exhaust the match with in coq using something like default or or clause?...

coq

Read More
Using or_comm in Coq...

coq

Read More
How to dependent match on a list with two elements?...

coq

Read More
multiplication of two binary numbers...

coqimplementation

Read More
How to do an inductive proof...

coqproofinduction

Read More
Found a constructor of inductive type bool while a constructor of list is expected...

coqinductive-logic-programming

Read More
setoid_rewrite: rewrite under bindings with 2 parameters...

coq

Read More
How to compile Coq files with Proof General + Emacs?...

coq

Read More
rewriting hypothesis to false with a contradictory theorem...

coqssreflect

Read More
How to get a better proof style in Coq?...

coq

Read More
Pose proof in Coq...

coq

Read More
Using tuples when constructing inductive types...

coq

Read More
Using the commutativity of the AND operator in Coq...

coq

Read More
How to solve a simple inequality in COQ with the same variable which is adding on both sides of the ...

coqcoq-tactic

Read More
Coq: easiest way to construct members of a decidable sigma type?...

coq

Read More
How to prove insert_BST in Coq...

logiccoqproofcoq-tacticproof-of-correctness

Read More
Coq Program Fixpoint vs equations as far as best way to get reduction lemmas?...

coqedit-distanceproof-of-correctness

Read More
How to solve the very simple Syntax error: 'end' expected after [branches] (in [term_match])...

coq

Read More
How to simplify A + 0 > 0 into A > 0?...

coqsimplification

Read More
Removing the last element of a sized list in Coq...

coq

Read More
How to prove a constant function that neither injective nor surjective in Coq?...

coq

Read More
Warning : “Set this option from the IDE menu instead” in coq...

coqcoq-tacticcoqide

Read More
Concatenation of 2 lists in lambda-calculus...

coqlambda-calculuscoqide

Read More
Number of element in a list in lambd-calculus?...

coqlambda-calculus

Read More
how to create a polymorphe couple such as "( a : type A, b : type B ) " in lambda-calculus...

coqlambda-calculuscoqide

Read More
Creating Coq tactic: how to use a newly generated name?...

coqproofcoq-tactic

Read More
Why does Coq remove/clear my asserted lemmas in my proof after the base case is proved?...

coqcoq-tactic

Read More
How can I rewrite "+ 1" (plus one) to "S" (succ) in Coq?...

coqcoq-tacticsuccessor-arithmetics

Read More
What is the right proof term so that the ssreflect tutorial work with the exact: hAiB example?...

coqcoq-tactic

Read More
How do you lookup the definition or implementation of Coq proof tactics?...

mathcoqproof

Read More
BackNext