Search code examples
Equal indexed inductive types implies equal indices...


coq

Read More
How proof assistants are implemented?...


coqisabelleproof

Read More
What does "==>" mean in coq?...


coq

Read More
Instantiating a commutative ring of Zn with mathcomp...


coqssreflect

Read More
How to access functions inside a record inside a module...


coq

Read More
Proving that size with filter is not equal to (size + 1)...


coqssreflect

Read More
How to import the file in other project/directory by configuring the Makefile or _Coqproject in curr...


coq

Read More
How to concatenate vectors defined as functions from finite types...


coq

Read More
Quantification under sumbool...


coq

Read More
Simplifying expression with lists equality...


coqssreflect

Read More
Locate a Notation that takes an infix argument...


coq

Read More
Coq : How to correctly remember dependent values without messing up the induction hypothesis?...


coqproofdependent-type

Read More
In Coq, are there tactics for working with Rabs, Rineq?...


coqtheorem-provingcoq-tacticreal-number

Read More
How to prove (forall x, P x /\ Q x) -> (forall x, P x)...


proofcoq

Read More
High-speed calculation of Coq's theorems...


profilingcoq

Read More
Rel: le_antisymmetric comprehension...


coqlogical-foundations

Read More
Extra type constructor if parameter matches a pattern...


coq

Read More
What is the difference between Notation and Definition from the point of view of the auto tactic?...


coqcoq-tactic

Read More
Why is vm_compute faster in definitions than in proofs in Coq?...


coq

Read More
How should a user-defined enumerated type be made `finType`?...


coqssreflect

Read More
Chaining definitions in coq...


coq

Read More
Coq/SSReflect: How to do case analysis when reflecting && and /\...


coqcoq-tacticssreflect

Read More
Defining equality relation for infinite trees...


coqcoinduction

Read More
Replace hypothesis with implication without adding its premise as subgoal...


coq

Read More
Transform `not A` into `A -> False` in Coq...


coqtheorem-proving

Read More
Logical Coq Proof related to map function...


functional-programminglogiccoqproof

Read More
Coq: Issue with Require Export...


coqcoqide

Read More
How to reason with complex pattern-matchings?...


coq

Read More
Rev.v le_antisymmetric...


coqlogical-foundations

Read More
Software Foundations: apply ... with ... tactic...


coqlogical-foundations

Read More
BackNext