Search code examples
Syntax of the case tactic in coq...

coqcoq-tactic

Read More
Understanding nat_ind2 in Logical Foundations...

coqlogical-foundationsproof-assistant

Read More
Split multiple conjuncts in the goal...

coqcoq-tactic

Read More
What `dependent induction` tactic does in Coq and how to use it...

coqcoq-tacticinduction

Read More
Coq can't define an inductive proposition...

coq

Read More
The `specialize` tatic in Coq does not work well with typeclasses?...

coqtypeclass

Read More
What's the exact rule of applying a theorem in Coq?...

coq

Read More
Coq inductive not right form...

coqinduction

Read More
Why I can't use exact P if P is a Prop?...

coq

Read More
Why we can't use "simpl" on `j = j -> x = y`?...

coq

Read More
Why can't I perform rewrite tactic here?...

coq

Read More
Prove theorem about the last element of a list...

coq

Read More
How do I apply (S n' <=? m) = true to S n' <= m?...

coqlogical-foundations

Read More
Coq : Using a parametrized Type from within a Module...

coq

Read More
How to prove this in Coq...

coqcoqide

Read More
Software Foundations (lf): proving leb_plus_exists and plus_leb_exists...

coqlogical-foundations

Read More
Coq QArith division by zero is zero, why?...

coqdivide-by-zerorational-numbers

Read More
Coq/Ltac: is it possible to design a tactic that says the goal is proved when a decision procedure p...

coqltac

Read More
Proving some theorems on the function index in Coq...

coq

Read More
Why does coq not recognize that `None = Some v` is false?...

coqproof-assistant

Read More
Does import not only import but also change existing definitions?...

coq

Read More
In Coq, what would be the steps to prove the correctness of a function that solves puzzles like Sudo...

coq

Read More
Dependent equality with 2 different type functions...

coqdependent-type

Read More
Equivalence of inductive and recursive...

coq

Read More
How would I prove that b = c if (andb b c = orb b c) in coq?...

coqproofproof-of-correctness

Read More
How to prove (X × Y = ∅) <-> (X = ∅) ∨ (Y = ∅)...

coqset-theory

Read More
Iris/Coq replacing literal...

coq

Read More
How do I install a library in coq? (MacOS)...

coqvscoq

Read More
Is there a three-valued case analysis on patterns (a < b) (a = b) (a > b)?...

coqnested-ifcoq-tactic

Read More
How can I give an alias to a type in coq...

aliastypedefcoq

Read More
BackNext