Understanding nat_ind2 in Logical Foundations...
Read MoreSplit multiple conjuncts in the goal...
Read MoreWhat `dependent induction` tactic does in Coq and how to use it...
Read MoreCoq can't define an inductive proposition...
Read MoreThe `specialize` tatic in Coq does not work well with typeclasses?...
Read MoreWhat's the exact rule of applying a theorem in Coq?...
Read MoreWhy I can't use exact P if P is a Prop?...
Read MoreWhy we can't use "simpl" on `j = j -> x = y`?...
Read MoreWhy can't I perform rewrite tactic here?...
Read MoreProve theorem about the last element of a list...
Read MoreHow do I apply (S n' <=? m) = true to S n' <= m?...
Read MoreCoq : Using a parametrized Type from within a Module...
Read MoreSoftware Foundations (lf): proving leb_plus_exists and plus_leb_exists...
Read MoreCoq QArith division by zero is zero, why?...
Read MoreCoq/Ltac: is it possible to design a tactic that says the goal is proved when a decision procedure p...
Read MoreProving some theorems on the function index in Coq...
Read MoreWhy does coq not recognize that `None = Some v` is false?...
Read MoreDoes import not only import but also change existing definitions?...
Read MoreIn Coq, what would be the steps to prove the correctness of a function that solves puzzles like Sudo...
Read MoreDependent equality with 2 different type functions...
Read MoreEquivalence of inductive and recursive...
Read MoreHow would I prove that b = c if (andb b c = orb b c) in coq?...
Read MoreHow to prove (X × Y = ∅) <-> (X = ∅) ∨ (Y = ∅)...
Read MoreHow do I install a library in coq? (MacOS)...
Read MoreIs there a three-valued case analysis on patterns (a < b) (a = b) (a > b)?...
Read MoreHow can I give an alias to a type in coq...
Read More