This an informal draft, established through informal discussions with the community, of what the documentation could look in terms of content. It is not fixed and will evolve with the project through discussions and according to the need of the users.
- Preliminary
- Trying it out (games), Installing, Courses and Books
- Writing proofs in Coq
- Basic tactics
- Solvers and Decision procedures
- SSReflect
- MetaProgramming
- Programming in Coq
- Writing programs in Coq
- Extraction
- Programming by dependent pattern matching with Equations
- Tools for verifying software
- Verified software in Coq
- Coq functionalities
- Stuff that make your life easier
- Packaging mathematical structures
- Computing in Coq
- Others
- Coq's theory
- Sorts in Coq
- (Co)Inductive Types
- Coq and Axioms
- Coq and Paradoxes
- Libraries
- General purpose librairies, real numbers, ...
- Trying it out (games)
- Installing
- Courses and Books
- Reasoning about Logic
- Reasoning about Equality
- Reasoning about Inductive Types
- Proof Search tactics (assumption, easy, trivial, intuition ?)
- Tactics for Forward Reasoning
- Combining Tactics
- Advanced Proof search tactics :
- auto / eauto / typeclasses eauto
- Domain Specific Solvers :
- congruence, bauto, tauto, first-order, lia, itauto, etc...
- Algebraic Solvers :
- Ring etc... Algebra-tactics
- SMT Solvers
- CoqHammer
- I guess there is much to say 😄
- Ltac
- Ltac2
- MTac2
- CoqElpi :
- Tutorial
- How to do sth that Elpi is good at
- MetaCoq
- Writing programs in Coq
- Termination / Well-founded
- Pattern matching in Coq
- Coinductive Types
- Programming by dependent pattern matching with Equations
- Extraction
- Tools for verifying software
- Verified software in Coq
- Searching for lemmas
- Implicit Arguments
- Notations
- Sections
- Modules
- Records
- Type Classes
- Canonical Structures
- Hierarchy builders
- Native compute
- Vm compute
- CoqEal
- Trocq
- Program derivation
- dpdgraphs
- UniCoq
- ParamCoq
- Types and cumulativity
- Prop
- SProp
- Polymorphism of Sorts
- Inductive Types
- Inductives Types, Induction, Pattern Matching, WellFounded Recursion
- Coinduction Types
- Main Axioms and Compatibilities
- Extentionality Principles
- Classical Logic
- Axiom of Choice
- Axiom K / UIP
- Univalence Axiom
- Universe Paradoxes (Type:Type, etc...)
- Guard Conditions Paradoxes (Non Strict Positivity, etc...)
- Positive CoInductive Types
There is work to be done to understand how to introduce the different and many libraries existing in the Coq ecosystem
- StdLib
- MathComp
- UniMath
- Coq Hott
- Corn
- ExtLib
- Stdpp ?
- Coquelicot
- Flocq
- Gappa
- Coq Interval
- Coq prime numbers generator
- Coqprime
- RegLanguage