Search code examples
How to prove the goals in more elegant way using ssreflect?...

coqcoq-tacticssreflect

Read More
How to continue case analysis of a nested match in coq?...

coqcoq-tactic

Read More
Coq: Is there a way to define "map" for Ensemble...

coq

Read More
Why is `specialize` not an invalid tactic within a proof?...

coqcoq-tactic

Read More
Proof objects in the identity type...

coq

Read More
Custom tactics provided by libraries...

coqcoq-tactic

Read More
Can't find Lemma for set equality in stdpp library...

coq

Read More
How to create a new hypothesis from apply?...

coq

Read More
How to prove forall x y, x<=y -> div2 x <= div2 y in coq?...

coq

Read More
Coq matrix manipulation...

matrixcoq

Read More
Software Foundations Basics - Theorem lower_grade_lowers need to prove implication Eq = Lt -> Eq ...

coqcoq-tacticlogical-foundations

Read More
How to represent 2D array in Verifiable C...

coqverifiable-c

Read More
How to proof by natural number case analysis in Coq?...

coq

Read More
How to install Coq...

coqcoqide

Read More
Software Foundations Basics Exercise - How do I access letter from grade?...

coqlogical-foundations

Read More
List without gaps in Coq...

coqdependent-typetype-theory

Read More
Forall and exists in a Coq proof...

coq

Read More
How to extract the exact information of `GenArg`?...

ocamlabstract-syntax-treecoq

Read More
How to generate the AST of a Coq source code?...

ocamlabstract-syntax-treecoq

Read More
PLF: [S <: S->S] Subtyping Example Hint...

coq

Read More
Coq: A \/ A -> A...

coq

Read More
Programming in the Calculus of Inductive Constructions with Coq...

coqdependent-typetheorem-proving

Read More
What's the role of unification in Coq's core type system?...

coqdependent-typetype-systemstheorem-provingunification

Read More
Rewrite proposition using equivalence in Coq...

coq

Read More
Coq simpl / unfold only once. (Replace part of goal with the result of one iteration of a function.)...

coqproofcoq-tacticinduction

Read More
Is Prop a subtype of Set?...

coqdependent-type

Read More
What is the meaning of "|-" in coq, and how do I find the definitions for the other seemin...

coq

Read More
Why the `Let-in` construct cannot be defined as a derived form in a dependently-typed language?...

coqdependent-typetype-systems

Read More
Domain of a map in Coq...

coqcoq-tactic

Read More
Ergonomic way to define elements of dependent records in proof mode?...

coq

Read More
BackNext