Search code examples
Axiom reuse with Typeclasses in Coq...


coq

Read More
Coq: can I use a type argument as the type of successive argument?...


coqtypingparametric-polymorphismadhoc-polymorphism

Read More
Looking for some match trick or convoy pattern...


coq

Read More
Non strictly positive occurrence problem in Coq inductive definition...


coq

Read More
coq Basics: bin_to_nat function...


coqlogical-foundations

Read More
Interpret term as type in Coq...


coq

Read More
Prove equality on list constructed with a map...


coqcoq-tactic

Read More
How do I simplify a hypothesis of the form True -> P in Coq?...


coqcoq-tactic

Read More
What does plus '+' operator mean between two propositions in Coq...


coq

Read More
Coq Set Inheritance...


inheritancecoq

Read More
Eliding a proof when generating HTML using coqdoc...


coq

Read More
Back to Coq proof checker after 5-8 years away: how to prove that (forall n, m : N, (n - (S m)) = pr...


coq

Read More
Avoid printing notation in Coq with Proof General...


coqproof-general

Read More
what is the type of a here...


typescoq

Read More
Automatically specialize forall when the parameters are in scope...


coqcoq-tactic

Read More
proving strong induction in coq from scratch...


coqinduction

Read More
Does Gallina have holes like in Agda?...


coq

Read More
How do you prove in Coq that (e: p = p) = eq_refl?...


coq

Read More
Is there a strong relation with bools and Prop in Coq?...


coq

Read More
types as parameters in coq...


polymorphismcoqdependent-typeparametric-polymorphism

Read More
Coq constructor can't take two arguments of different types?...


coq

Read More
Generic equality lifting in coq...


coq

Read More
How to prove non-equality of terms produced by two different constructors of the same inductive in c...


coq

Read More
(A -> B) /\ (B -> C) -> (A -> C) in Coq?...


coqcoq-tactic

Read More
How do I describe a multiplication of vectorized matrices?...


coqssreflect

Read More
Coq use refine with bi-implication...


coqcoq-tactic

Read More
coqc: -Q.PLF: no such file or directory...


coqcoqide

Read More
COQ Proof Assistant - Apply the hyppothesis...


coqcoq-tactic

Read More
Nested recursion and `Program Fixpoint` or `Function`...


recursioncoqisabelletermination

Read More
Unable to prove that only 0 is less than 1 with mathcomp's finTypes...


coqproof

Read More
BackNext