Stuck at a simple inequality of natural number proof in Coq...
Read MoreCoq - VSCode highlight Compute command in blue...
Read MoreTurn `P(?x)` into `exists x,P(x)` to give different instantiations for different subgoals in Coq...
Read MoreWhy doesn't Coq notation defined by other notation working well?...
Read More"Cannot guess decreasing argument of fix" error when defining a Fixpoint for extracting th...
Read MoreWrong Typeclass Instance used in Coq Proof...
Read MoreCoq's Search command and modules...
Read MoreHow to make OCaml (or Coq) code from the llvmir code using vellvm framework...
Read MoreCoq repeating "destruct" for disjunctive hypothesis causing unwanted destruction in the en...
Read MoreIs there a lightweight way to define a mutable dictionary that can return all of its keys in Coq?...
Read MoreConstructing proof terms inside a recursive function...
Read MoreCoq notation defined inside a module expecting type without module prefix...
Read MoreCan a dependently typed language be Turing complete?...
Read MoreBeta-reduction after delta-reduction in unfold tactic...
Read MoreEquality for elements of sig type in Coq...
Read MoreDefining mutually recursive types in Coq?...
Read MoreHow to mix sections with hints in Coq?...
Read MoreNon-trivial Fixpoint on nested recursive types...
Read MoreIs there an intuitionistic proof of `(A -> B \/ C) -> (A -> B) \/ (A -> C)`?...
Read MoreInteractionTrees library - simple program on ASM...
Read MoreHow to instruct `auto` to simplify the goal during proof search?...
Read MoreIs is possible to rename a coq term?...
Read MoreWhat are the practical limitations of a non-turing complete language like Coq?...
Read MoreCoq : mutually recursive definitions with [mrec] in InteractionTrees Library...
Read MoreIs there a function that returns a list of values with specific type in OCaml?...
Read MoreFormualting a logic in farmer astronaught...
Read MoreWhat's the correct setup for Kami (Coq framework for Bluespec) to be able to run on WSL Ubuntu?...
Read MoreCoq: keeping information in a match statement...
Read MoreShowing polynomial equality in coq/ssreflect...
Read More