Search code examples
Proving that s-expressions printing is injective...


coq

Read More
How to apply an axiom to simplify a match in Coq?...


coq

Read More
Arithmetic expressions and big-step semantic...


mathexpressioncoqsemantics

Read More
Idempotency of normalizing a binary number in coq...


coq

Read More
Can any one help me how to prove this therom in coq...


coq

Read More
Unable to provide long (1024+ character) inputs to the OCaml toplevel and coqtop (and Proof General)...


emacsocamlttycoqproof-general

Read More
Not pretty-printing a field of a record...


coq

Read More
How to express that one element of an inductive relation can't be derived from another in Coq?...


coqinduction

Read More
Weird goal `Some 0 = true` generated in proof...


coq

Read More
How to prove Theorem plus_lt : forall n1 n2 m, n1 + n2 < m -> n1 < m /\ n2 < m...


coqcoq-tactic

Read More
Can't figure out why re-write does not work...


coqcoq-tactic

Read More
How to prove `plus_le_compat_l : forall n m p, n <= m -> p + n <= p + m.`...


coqcoq-tactic

Read More
What does the tactic destruct do in the proof below?...


coqcoq-tactic

Read More
Suppress Warning At Import...


coq

Read More
Why is my definition not allowed because of strict positivity?...


coqagdatype-theory

Read More
Equal implies Less-Than-Or-Equal in Coq...


coq

Read More
How to tell Coq that it's okay to remove the `n`s?...


coqcoq-tactic

Read More
How to split equality of two lists?...


coqcoq-tactic

Read More
SF Volume 1: Logic: How to prove tr_rev <-> rev?...


coqcoq-tacticproof-of-correctnessproof-general

Read More
How to generalize a variable on both sides of an equation in Coq?...


coq

Read More
Software Foundations Volume 1: Tactics: injection_ex3...


coqcoq-tacticproof-general

Read More
Trying to define a "rect2"-like function on heterogeneous vectors...


coqdependent-type

Read More
erewrite that asks for hypothesis first?...


coqcoq-tactic

Read More
Is it possible to turn unification errors into goals in Coq?...


coqcoq-tactic

Read More
ssreflect inversion, I need two equations instead of one...


coqssreflect

Read More
Binary tree inversion in Coq...


binary-treecoqtheorem-proving

Read More
Add notation to a scope globally in Coq...


coq

Read More
Proving MStar' in Logical Foundations (IndProp.v)...


coqlogical-foundations

Read More
Problems with missing information in Obligations when defining using Program in Coq...


coq

Read More
Adding "in" part to tactic to specify where to apply it...


coqltac

Read More
BackNext