Search code examples
Coq: Defining a type class instance...


classtypescoq

Read More
How to express inheritance in Coq?...


coq

Read More
Nested recursion with partial application...


recursioncoq

Read More
Which vector library to use in coq?...


listvectorcoqproofdependent-type

Read More
How can I break `forall i: nat i < S k -> H` in Coq into `i < k and i=k`?...


coqcoq-tactic

Read More
Instantiating an existential with a specific proof...


coqltac

Read More
The reference "X" was not found in the current environment...


coqcoqide

Read More
Coq: Is it possible to prove that, if two records are different, then one of their fields is differe...


recordcoq

Read More
forall equality in Coq...


coq

Read More
Is there a good way to block beta-reduction from automatically occurring in goals?...


coq

Read More
Coq: Trouble w/ a dependent pattern match...


pattern-matchingcoq

Read More
how to figure out what "=" means in different types in coq...


coq

Read More
coq induction with passing in equality...


coqinduction

Read More
Coq: Fixing a recursive notation...


parsingrecursiondefinitioncoqnotation

Read More
How can I implement a coq tactic that iterates over the hypotheses?...


coqcoq-tacticltac

Read More
Is is possible to implement a Coq tactic that inspects a HintDb? If so, how?...


coqcoq-tacticltac

Read More
Converting Coq to Idris...


coqidris

Read More
Can I use a notation for an Inductive type to define that type in Coq?...


coqnotationdependent-type

Read More
prove that a list returned from a recursively defined function is fixed length in Coq...


coqcoq-tactic

Read More
generalizing expressions under binders...


coqcoq-tacticltac

Read More
What is difference between `destruct` and `case_eq` tactics in Coq?...


coq

Read More
Coq: How to prove if statements involving strings?...


coqcoq-tactic

Read More
Coq: How to prove max a b <= a+b?...


coqcoq-tactic

Read More
Prove existential quantifier using Coq...


coq

Read More
Why inversion tactic doesn't work in the following Coq proof?...


coq

Read More
Porting (simply-typed) lambda calculus term saturation proof from Coq to Agda...


recursioncoqagdatermination

Read More
How does elim work in Coq on /\ and \/?...


coqcoq-tactic

Read More
how to define piecewise function from naturals to naturals in coq...


coq

Read More
Is there a minimal complete set of tactics in Coq?...


coqcoq-tactic

Read More
How can I compare (equality) of two elements of same Set in Coq?...


coq

Read More
BackNext