Search code examples
Coq: rewriting under a pointwise_relation...


coqrewriting

Read More
How does one compute/create a concrete/actual string in coq to pass to functions or store in a varia...


coq

Read More
Why S n' =? S n' simplifies to n' =? n' in Coq?...


coq

Read More
Stuck on the proof of a simple Lemma: which induction should I use?...


coq

Read More
Agda: Failed to solve the following constraints: P x <= _X_53 (blocked on _X_53)...


coqagdatype-theoryhomotopy-type-theoryagda-mode

Read More
Coq: Implementation of splitstring and proof that nothing gets deleted...


coqproofinduction

Read More
Proving enumerate(...) to range(len(...)) equality...


coqcoq-tactic

Read More
Understanding how pattern matching works in Coq...


pattern-matchingcoq

Read More
Cannot focus on a remaining unfocused goal in Coq...


coqlogical-foundations

Read More
Best way to make a relation associative in Coq...


coq

Read More
Evaluate constant inequation in Coq...


coq

Read More
RelationClasses versus CRelationClasses...


coq

Read More
Coq - prove that there exists a maximal element in a non empty sequence...


coqssreflect

Read More
Case analysis on max - ssreflect...


coqssreflect

Read More
redundant eval $(opam env) needed in Dockerfile...


bashdockerdockerfilecoqopam

Read More
How to improve this proof?...


coq

Read More
Define a function based on a relation in Coq...


coq

Read More
How does one import the lia tactic given that the omega tactic was reprecated in Coq?...


coq

Read More
Assume the negation of the goal in Coq...


coq

Read More
Can I prove a lemma without an additional inductive type...


coq

Read More
Unfolding terms created with `assert` in Coq...


coqcoq-tactichomotopy-type-theory

Read More
Can't find a way to 'reverse' a constructor...


coq

Read More
User defined language in pandoc code-block...


markdowncoqpandoc

Read More
How to delay a lambda evaluation so I can substitute lambdas...


coq

Read More
Proofs of simple arithmetic expressions...


coqproof

Read More
Add an assertion and its negation to Coq...


coq

Read More
Coq make failing on Omega...


coq

Read More
Fail to prove a permutation property...


coq

Read More
Equivalence but not congruence...


coq

Read More
Prove recursive function exists using only `nat_ind`...


recursioncoqinduction

Read More
BackNext