Search code examples
Coq proving nonsensical inductive property implication?...


coqcoq-tacticlogical-foundations

Read More
Finding rewrite rules...


coq

Read More
Define polymorphic inductive type tree in coq...


coq

Read More
Coq leb <=? does not give me an hypothesis after case or induction...


coq

Read More
Postulate and prove theorem about equality for different types (Prove commutativity for the sum of t...


coq

Read More
Case splitting on if-then-else condition...


coq

Read More
Coq: evaluating/simplifying `Prop` tautologies...


coqtheorem-proving

Read More
Recursive definition of nat_to_bin is ill-formed...


binarycoq

Read More
Anyone know how mult works in coq?...


coq

Read More
Define a polymorphic type in coq...


coq

Read More
Does ssreflect assume excluded middle?...


coqssreflect

Read More
Define list length in recursion in Coq Not sure if my function is wrong and got stuck...


coqcoq-tactic

Read More
Theorem + induction vs Fixpoint + destruct in Coq...


coqcoq-tactic

Read More
How to constrain a type field to a power of two in a type system?...


typescripthaskellconstraintscoqtype-systems

Read More
Translating proof from Nat to Rat...


coqssreflect

Read More
How to prove for all functions P, Q from typical type to `Prop`, "forall a, b, P(a) or Q(b) hol...


coq

Read More
Compiling multiple Coq files does not work...


coq

Read More
Defining integers inductively in Coq (inductive definitions subject to relations)...


integercoqinduction

Read More
Coq: Rewriting between two equivalent setoids...


coq

Read More
"Non strictly positive occurrence of ..."...


coq

Read More
Removing trivial match clause in Coq...


pattern-matchingcoq

Read More
Coq can't see that two types are the same...


typesfunctional-programmingcoq

Read More
how to proof (f1+f1 = f2+f2 -> f1 = f2) in coq...


coq

Read More
Is it possible to prove `forall n: nat, le n 0 -> n = 0.` in Coq without using inversion?...


coqcoq-tactic

Read More
Proofs of structural properties of arguments in match in coq...


functional-programmingcoqdependent-typerefinement-type

Read More
Introducing a new assumption/hypothesis by adding it as subgoal...


coq

Read More
Difference between propositionals True/False and booleans true/false in Coq...


coq

Read More
Why can I use the constructor tactic to prove reflexivity?...


coqcoq-tactic

Read More
Using the same variable multiple times in a definition to represent equality...


coq

Read More
Printing ssrnat's ".+1" definition...


printingcoqssreflect

Read More
BackNext