Search code examples
Stuck at a simple inequality of natural number proof in Coq...

coqcoq-tactic

Read More
Coq - VSCode highlight Compute command in blue...

visual-studio-codecoq

Read More
Turn `P(?x)` into `exists x,P(x)` to give different instantiations for different subgoals in Coq...

logiccoqformal-verification

Read More
Why doesn't Coq notation defined by other notation working well?...

mathcoqnotation

Read More
"Cannot guess decreasing argument of fix" error when defining a Fixpoint for extracting th...

coq

Read More
Wrong Typeclass Instance used in Coq Proof...

functional-programmingcoqtypeclassdependent-typetheorem-proving

Read More
Coq's Search command and modules...

modulecoq

Read More
How to make OCaml (or Coq) code from the llvmir code using vellvm framework...

coq

Read More
Coq repeating "destruct" for disjunctive hypothesis causing unwanted destruction in the en...

coq

Read More
Is there a lightweight way to define a mutable dictionary that can return all of its keys in Coq?...

coq

Read More
Constructing proof terms inside a recursive function...

coq

Read More
Coq notation defined inside a module expecting type without module prefix...

coq

Read More
How does one implement Coq?...

coq

Read More
Can a dependently typed language be Turing complete?...

haskellocamlcoqagdadependent-type

Read More
Beta-reduction after delta-reduction in unfold tactic...

coq

Read More
Equality for elements of sig type in Coq...

coqsubtype

Read More
Defining mutually recursive types in Coq?...

coq

Read More
How to mix sections with hints in Coq?...

coq

Read More
Non-trivial Fixpoint on nested recursive types...

coqtheorem-proving

Read More
Is there an intuitionistic proof of `(A -> B \/ C) -> (A -> B) \/ (A -> C)`?...

coq

Read More
InteractionTrees library - simple program on ASM...

coq

Read More
How to instruct `auto` to simplify the goal during proof search?...

coqproof

Read More
Is is possible to rename a coq term?...

coqproofcoq-tactic

Read More
What are the practical limitations of a non-turing complete language like Coq?...

programming-languagesfunctional-programmingturing-completecoq

Read More
Coq : mutually recursive definitions with [mrec] in InteractionTrees Library...

coqmutual-recursion

Read More
Is there a function that returns a list of values with specific type in OCaml?...

ocamlcoq

Read More
Formualting a logic in farmer astronaught...

logicboolean-logiccoq

Read More
What's the correct setup for Kami (Coq framework for Bluespec) to be able to run on WSL Ubuntu?...

ubuntumakefilewindows-subsystem-for-linuxcoqbluespec

Read More
Coq: keeping information in a match statement...

recursioncoq

Read More
Showing polynomial equality in coq/ssreflect...

coqssreflect

Read More
BackNext