Is there a way for Coq to recall it already proved a property for the same element in the same proof...
Read MoreCoerce rat to realType im math-comp/analysis...
Read MoreLtac tactic that accepts an arbitrary number of quantifiers...
Read MoreProving extensional equality of two functions...
Read MoreRecursion and Pattern matching in Coq...
Read MoreMorphism signature for dependently-typed vectors in coq...
Read MoreHow to parse a string into a list of lists in Coq?...
Read MoreIs there a library for sets that works with bool in Coq?...
Read MoreHow to write the iota descriptor in Coq?...
Read MoreHow to deal with lemma only used once in Coq?...
Read More'coqc' does not find findlib.conf...
Read MoreHow to scope Search to the current module only...
Read MoreHow to proof recursively defined functions' prop in Coq...
Read MoreCoq returns cannot guess decreasing argument of fix. How to fix my function?...
Read MoreDecreasing argument (and what is a Program Fixpoint)...
Read MoreWhy do these theorems of propositional logic allow for the same proof in Coq?...
Read MoreHow to distribute an AND operator in Coq?...
Read MoreProving n + S n = S (n + n) without n + S m = S (n + m)...
Read MoreDisjunction and the error `No product after head reduction'...
Read MoreHow to create a custom Ltac to recursively destruct conjunctions?...
Read MoreHow can I write a filter function for sequences represented as functions in Coq?...
Read MoreUnclear error message regarding format and notation...
Read MoreComplete Atomic Boolean algebras in Coq...
Read MoreUnderstanding a message on CoqIde...
Read MoreUsing the transitivity of equivalence to rewrite a goal...
Read MoreHow to break up an implication into two subgoals in Coq?...
Read MoreIs there a way to redirect Coqide messages and errors to the same output?...
Read More