Search code examples
What is Isabelle/HOL command for Compute in Coq?...


coqisabelle

Read More
Infinite recursive types in Coq (for Bananas and Lenses)...


coqrecursion-schemes

Read More
How to define an affine set in coq...


coq

Read More
Coq: Proving relation between < and ≤...


coqproofcoq-tactic

Read More
Coq: Proving simple theorem using Fixpoints and Induction...


coqproofcoq-tactic

Read More
Software Foundations: proving leb_complete and leb_correct...


coqlogical-foundations

Read More
Logic: auxilliry lemma for tr_rev_correct...


coqlogical-foundations

Read More
Tactics: stuck in eqb_trans...


coqlogical-foundations

Read More
Using a 3 symbols notation [constr:operconstr] expected after [constr:operconstr]...


coqnotation

Read More
proof Lemma which based on Fixpoint definitions...


coqcoq-tacticproof-general

Read More
Solving linear equation systems in Coq...


coqlinear-equation

Read More
Proof Process busy on combine_split...


coqproof-general

Read More
How to prove `(fun _ : nat => False) = Empty_set nat` in Coq?...


coq

Read More
Induction on a datatype with non-uniform type parameters produces ill-typed terms...


coqtheorem-proving

Read More
Simpler proof of `0<a -> 1<a+1`...


coqssreflect

Read More
How to reason across equality proofs?...


coq

Read More
How to use 'apply ... with' and 'apply ... in' together?...


coq

Read More
How can I create a polymorphic "map xs f" function?...


coqparametric-polymorphism

Read More
Trouble in implementing dependently typed lookup in Coq using Equations...


coqdependent-type

Read More
Coq: Create a super-type of boolean and nat...


typescoqmixed

Read More
Defining recursive function over product type...


coqterminationtotality

Read More
DeMorgan's law for quantifiers in Coq...


coqquantifiersfirst-order-logicdemorgans-law

Read More
Proving that a reversible list is a palindrome in Coq...


coqpalindrometheorem-provinglogical-foundations

Read More
Lemma about list and rev(list)...


coq

Read More
How to set implicit parameters for constructor...


coqlogical-foundations

Read More
How to avoid necessity to put module prefix...


coq

Read More
Understanding specialize tactic...


coqcoq-tacticlogical-foundations

Read More
Coq: About "%" and "mod" as a notation symbol...


coqnotation

Read More
I want to prove some properties about list, but am stuck at induction...


coq

Read More
use module signature definition in module implementation...


coq

Read More
BackNext