How to prove the goals in more elegant way using ssreflect?...
Read MoreHow to continue case analysis of a nested match in coq?...
Read MoreCoq: Is there a way to define "map" for Ensemble...
Read MoreWhy is `specialize` not an invalid tactic within a proof?...
Read MoreProof objects in the identity type...
Read MoreCustom tactics provided by libraries...
Read MoreCan't find Lemma for set equality in stdpp library...
Read MoreHow to create a new hypothesis from apply?...
Read MoreHow to prove forall x y, x<=y -> div2 x <= div2 y in coq?...
Read MoreSoftware Foundations Basics - Theorem lower_grade_lowers need to prove implication Eq = Lt -> Eq ...
Read MoreHow to represent 2D array in Verifiable C...
Read MoreHow to proof by natural number case analysis in Coq?...
Read MoreSoftware Foundations Basics Exercise - How do I access letter from grade?...
Read MoreHow to extract the exact information of `GenArg`?...
Read MoreHow to generate the AST of a Coq source code?...
Read MorePLF: [S <: S->S] Subtyping Example Hint...
Read MoreProgramming in the Calculus of Inductive Constructions with Coq...
Read MoreWhat's the role of unification in Coq's core type system?...
Read MoreRewrite proposition using equivalence in Coq...
Read MoreCoq simpl / unfold only once. (Replace part of goal with the result of one iteration of a function.)...
Read MoreWhat is the meaning of "|-" in coq, and how do I find the definitions for the other seemin...
Read MoreWhy the `Let-in` construct cannot be defined as a derived form in a dependently-typed language?...
Read MoreErgonomic way to define elements of dependent records in proof mode?...
Read More