Search code examples
Pattern matching multiple constructors in a single clause in Coq...


pattern-matchingcoq

Read More
Proving even + even = even with mutual induction using tactics...


coq

Read More
Coq: Defining a function by pattern matching on the arity of its argument...


functionmatchdefinitioncoq

Read More
Problems with dependent types in Coq proof assistant...


coqdependent-type

Read More
Proof involving unfolding two recursive functions in COQ...


coqproofcoq-tactic

Read More
Coq how to pretty-print a term constructed using tactics?...


coq

Read More
Applying apply tactic to premises instead of the goal...


coq

Read More
Can´t destruct exists in hypothesis...


coq

Read More
Coq proof of forall a b c: nat, b >= c -> a + b - c = a + (b - c)...


coq

Read More
How to match a "match" expression?...


coqltac

Read More
apply tactic cannot find an instance for a variable...


coq

Read More
Rewriting hypothesis with a more concrete expression...


coq

Read More
Proving simple inequality in Ssreflect...


coqssreflect

Read More
Unicode "not equal" notation in Coq (≠)...


unicodecoq

Read More
Proving using contradiction technique...


coq

Read More
Coq MSet of bounded naturals...


modulesetcoq

Read More
Postulating namespaces in Coq...


coqagda

Read More
Introducing new hypothesis in the premises...


coq

Read More
Pattern matching not specialising types...


coqtheorem-provingdependent-type

Read More
How to do induction differently?...


coq

Read More
How to rewrite a goal using function definition?...


coqcoq-tactic

Read More
A special case of Lob's theorem using Coq...


coqlobcoq-tactic

Read More
Coq: Proving an application...


functiondefinitioncoqproof

Read More
Folding back after unfolding...


coq

Read More
Definition function without using a helper function...


coq

Read More
Proof that references the conclusion of a previous proof in Coq...


coq

Read More
Coq beginner - Prove a basic lemma...


coq

Read More
Coq: Cannot find library Jessie_memory_model in loadpath...


linuxcoqframa-c

Read More
Smart modification of Coq environment...


coqltac

Read More
Re-writing without using symmetry tactic...


coqcoq-tactic

Read More
BackNext