Search code examples
The Coq :> symbol...


syntaxsymbolscoq

Read More
Defining the syntax with constraints...


coq

Read More
Parametric HOAS in Coq - is it possible to repeat type name inside the body of type declaration?...


coq

Read More
Difference between sumbool and intuitionnistic disjunction...


coq

Read More
Coq: Non-list Data structures living in Set?...


functional-programmingcoqdependent-typetheorem-proving

Read More
Tactic to prove a boolean implication...


coqcoq-tactic

Read More
Unicity of non-equality proofs...


coq

Read More
Representing Functions as Types...


functionhaskellcoqtype-theory

Read More
Unfolding a definition without reduction...


coqcoq-tactic

Read More
Coq list sorting practices & sortBy?...


sortingcoq

Read More
Sorted List in Coq...


sortingcoq

Read More
Using forall within recursive Function definition...


coqformal-methodscoq-plugin

Read More
where is Coq aac_tactics installed?...


coqopamcoq-plugin

Read More
rewrite works for integer but not for rationals for Coq aac_tactics...


coqcoq-tacticcoq-plugin

Read More
singleton list (`A) in Coq?...


listcoq

Read More
What are background goals, shelved goals, and abandoned goals in Coq?...


coqcoq-extraction

Read More
Binary search Tree in Coq. Trouble to use ( e0 : (val ?= n) = true ) to prove val = n...


coq

Read More
Folding only applications...


coqcoq-tactic

Read More
Specifying polarity in a module type...


coq

Read More
Are Coercions allowed within polymorphic datatypes in coq?...


coq

Read More
Define recursive notation with two recursive variables in Coq...


coq

Read More
Stuck on a simple proof about regular expressions...


coq

Read More
How to leverage auto's searching and hint databases in custom tactics?...


coqcoq-tactic

Read More
Dependent Pair Types...


typescoq

Read More
How to use Cycle / Swap tactics?...


coqcoq-tactic

Read More
A simple case of universe inconsistency...


coq

Read More
Destruct if condition in program fixpoint coq...


coq

Read More
Why, in Coq, a record projection expects a Type as argument?...


coq

Read More
Proper instance for "nested" matching...


coqcoq-tactic

Read More
Use proof of if expression = true in then part coq...


coq

Read More
BackNext