Search code examples
Vector: take out some elements from a vector with two methods...


coq

Read More
A list transformed from a vector equals to a list transformed from a vector casted its type...


coq

Read More
How to prove that the subsequence of an empty list is empty?...


coqcoq-tactic

Read More
Equality on type which is not inductive type...


coq

Read More
Quick Chick eqBoolArrowA_correct theorem...


coqlogical-foundations

Read More
Vector: theorem about splitting and appending vectors...


coq

Read More
Teach Coq that associative law of natural numbers holds...


coq

Read More
How can I build a list of bytes from its specification in Coq...


coqproofcoq-tacticformal-verification

Read More
What does Proof. simpl. reflexivity. Qed. mean in Coq?...


coq

Read More
Take a conjunction of two hypotheses and create a new hypothesis in Coq...


coqcoq-tactic

Read More
Vector : t A n = t A (n+0)?...


coq

Read More
Append and Split is same as doing nothing...


coq

Read More
Can I use destruct here given the constraint I have for index range of a list?...


coqproofcoq-tacticformal-verification

Read More
If two constructor expressions of an inductive type are equal in Coq, can I do rewriting based on th...


coqproofcoq-tacticformal-verification

Read More
Coq error: Unable to unify "true" with "is_true (0 < a - b - 3)"...


coqproofcoq-tacticformal-verification

Read More
is there any tactic in Coq that can transform a bool expression to a Prop one?...


coqproofcoq-tacticformal-verification

Read More
Coq: How do I prove that forall n m : nat, (n > m) -> (S n > S m)?...


numberscoqproof

Read More
How to index a tuple with ssreflect ordinals...


coqssreflect

Read More
Coq: Ltac for transitivity of implication (a.k.a. hypothetical syllogism)...


matchcoqltacimplication

Read More
Defining Addition Over Integers in Coq...


coq

Read More
Transform the lemma leaving previous state on Coq...


coqdependent-type

Read More
Can I print the partial definition of not finished proof in coq?...


coq

Read More
A proof about a mutually inductive proposition...


coqinduction

Read More
Can we ban arguments that don't meet conditions?...


coqdependent-type

Read More
Vector error : The type of this term is a product...


coqdependent-typeconvoy-pattern

Read More
Partial differentiation using Coqelicot on Coq...


coqdifferentiation

Read More
Reusing lia tactic to prove decidability...


coq

Read More
exact value of the derivative on Coq...


coq

Read More
Differential calculus on Coq...


coq

Read More
Pattern match with two list whose type is dependent type on Coq...


coqdependent-type

Read More
BackNext