Search code examples
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
Proving Binary Tree Properties...


binary-treecomputer-sciencecoqproof-general

Read More
coq: Tactic to replace true hypothesis in 'and' statement...


coqcoq-tactic

Read More
Tactic for existential hypothesis...


coqcoq-tactic

Read More
Curly brace proof syntax: begin x. = { auto } y. []...


coq

Read More
Why does this Coq Definition fail? Coq Namespace error for Inductive Type...


coq

Read More
Problem with Dependent pattern matching in COQ...


coq

Read More
Remove useless hypothesis from context...


coqcoq-tactic

Read More
How do you selectively simplify arguments to each time a function is called, without evaluating the ...


coqcoq-tactic

Read More
Are arrows in Coq aliases of universal quantifications?...


coq

Read More
Coq: goal is just a type (when using theorems with unnecessary arguments)...


argumentscoqcoq-tactic

Read More
Coq: prove while is equivalent to repeat...


coqsemanticscoq-tacticformal-semantics

Read More
How to use HoTT path induction in Coq?...


coqtype-theory

Read More
"False" in goal: is that a an indication I am doing something wrong?...


coq

Read More
Best practices for parametrized Coq libraries...


coq

Read More
How to prove that another definition of permutation is the same as the Default Permutation Library f...


permutationcoqproofinduction

Read More
Coq: How are the equality tacticts symmetry and transitivity defined?...


coqcoq-tacticltac

Read More
Coq - Rewriting a FMap Within a Relation...


programming-languagescoqproof

Read More
Coq: Cannot infer an internal placeholder of type "nat" in environment: ev : nat -> Pro...


coq

Read More
Coq - Obtaining equality from match statement...


typescastingcoq

Read More
Problems adding new notation in Coq...


coq

Read More
Proof of "less equal" transitive law in Coq...


coqcoq-tactic

Read More
BackNext