Search code examples
How to prove in Coq ~~(P \/ ~P)...


logiccoq

Read More
Why Coq doesn't allow inversion, destruct, etc. when the goal is a Type?...


coqproofinversion

Read More
Coq: trying to use dependent induction...


coqdependent-type

Read More
Import <Module> vs. Include <Module> in Coq Module system...


coq

Read More
Addition of natural numbers in Coq...


coq

Read More
Check cnat. and got Type return...


coqlogical-foundations

Read More
How to prove an absurd rule in Coq...


coq

Read More
Coq - Coercion of list nat...


listtypescoqcoercion

Read More
Is it possible to remove/override an existing coercion?...


coqcoercion

Read More
Why Coq does not infer the type parameter...


coq

Read More
Relations with dependent types in Coq...


coqdependent-type

Read More
How do you define an ordered pair in Coq?...


coq

Read More
How can I write a tactic which works both in a goal and a hypothesis?...


coqcoq-tactic

Read More
How to prove shorter nat comparisons like 10000 > 1 for sigma types in Coq?...


coq

Read More
Coq's proof #Coq...


coqcoq-tactic

Read More
How to save the current goal / subgoal as an `assert` lemma...


coqcoq-tactic

Read More
How can I proove forall a b, a <=? b = true -> a <=? S b = true in Coq...


coq

Read More
Trace inclusion between program and state machine...


coq

Read More
Proving S (n + m) = n + (S m), how to rewrite n+1 = S(n)?...


coqgallina

Read More
Cannot rewrite goal with assertion?...


coq

Read More
Understanding the intros keyword work in Coq...


coqgallina

Read More
How can I prove excluded middle with the given hypothesis (forall P Q : Prop, (P -> Q) -> (~P ...


coqlogical-foundations

Read More
Double induction in Coq...


doublerecurrencecoqinduction

Read More
Why is UIP unprovable in Coq? Why does the match construct generalize types?...


coq

Read More
What does the term "?T@{x:=t}", or a type with a question mark and at sign surrounding it ...


coq

Read More
How to Import Coq library HoTT in CoqIde...


coqcoq-tacticformal-verificationformal-methodscoqide

Read More
Proving a theorem containing not exists...


coq

Read More
Is there a shorter proof to this Coq theorem?...


coq

Read More
Coq: Associativity of relational composition...


functional-programmingcoqalgebraformal-verificationformal-methods

Read More
Are those two proofs equivalent?...


coq

Read More
BackNext