Search code examples
No implicits in dependent "match" pattern with ssreflect...


coqssreflect

Read More
when is the `:` (colon) in necessary in ssreflect/Coq?...


coqssreflect

Read More
Lexicographical comparison of tuples of nats...


coq

Read More
Coq: defining a function from a sigma type to its second projection (and making it a coercion)...


typescoqproofcoercionsubtype

Read More
Adding complete disjunctive assumption in Coq...


coqtheorem-proving

Read More
Getting a stronger induction principle in Coq...


coqtheorem-proving

Read More
Writing well-founded programs in Coq using Fix or Program Fixpoint...


coq

Read More
Multiple Where-clauses for Reserved Notation in Coq?...


coqnotationdependent-type

Read More
Syntax Error with `<` in Coq Notations...


parsingsyntaxoperatorscoqnotation

Read More
Coq proof that the Selection monad is an applicative and a monad...


functorcoqapplicativetheorem-proving

Read More
Coq Real numbers -lexing and parsing 3.14...


coqreal-number

Read More
Coquelicot library for basic undergraduate calculus...


coqreal-number

Read More
Pattern-match on type in order to implement equality for existentially typed constructor in Coq...


coq

Read More
How to introduce n distinct symbols in Coq...


coq

Read More
Supplying section arguments for examples...


coq

Read More
Coq won't compute a typeclass function if the typeclass has a Prop...


typeclasscoq

Read More
Agda-like programming in Coq/Proof General?...


coqagdadependent-typeproof-generalcoqide

Read More
How do I the calculate the sqrt of a natural or rational number in coq?...


coqsquare-rootsqrt

Read More
State-machines in Coq...


state-machinecoq

Read More
Can Coq be used (easily) as a model checker?...


coqmodel-checking

Read More
Universe inconsistency (because of strict positivity restriction?)...


coq

Read More
Coq: fixed universe hierarchy w/ explicit universes...


typescoq

Read More
How to build a function implicitly in Coq?...


coq

Read More
Why is it impossible to perform induction on a term that is used in conclusion?...


coq

Read More
Coq eapply generates a goal with a question mark while proving existence of a function...


coq

Read More
Proper way to use FMap in Coq 8.6?...


dictionarycoq

Read More
Finite map example...


dictionarycoq

Read More
How can I read Coq's definition of proj1_sig?...


coqtheorem-proving

Read More
Prove equality on Sigma-types...


coq

Read More
How do I prove that two Fibonacci implementations are equal in Coq?...


functional-programmingfibonaccicoq

Read More
BackNext