aboutsummaryrefslogtreecommitdiffhomepage
path: root/doc/sphinx/language/gallina-specification-language.rst
Commit message (Collapse)AuthorAge
* Tactic deprecation machineryGravatar Maxime Dénès2018-07-12
| | | | | | | | | | | | | | | | | | | | | | | | | | | We make it possible to deprecate tactics defined by `Ltac`, `Tactic Notation` or ML. For the first two variants, we anticipate the syntax of attributes: `#[deprecated(since = "XX", note = "YY")]` In ML, the syntax is: ``` let reflexivity_depr = let open CWarnings in { since = "8.5"; note = "Use admit instead." } TACTIC EXTEND reflexivity DEPRECATED reflexivity_depr [ "reflexivity" ] -> [ Tactics.intros_reflexivity ] END ``` A warning is shown at the point where the tactic is used (either a direct call or when defining another tactic): Tactic `foo` is deprecated since XX. YY YY is typically meant to be "Use bar instead.".
* Describe attributes in the documentation.Gravatar Vincent Laporte2018-07-03
|
* Merge PR #7703: Add an option to force parameters to be uniformGravatar Matthieu Sozeau2018-07-02
|\
| * Document option Uniform Inductive ParametersGravatar Jasper Hugunin2018-07-01
| |
* | doc: typesetting and hyperlinks in Syntax ExtensionsGravatar Lysxia2018-06-30
|/
* Improve the last section of the Gallina chapter.Gravatar Théo Zimmermann2018-05-28
|
* Chapter 1 of the refman compiles without reporting any undocumented object.Gravatar Théo Zimmermann2018-05-28
|
* Improve sections on (Co)Fixpoint of the Gallina chapter.Gravatar Théo Zimmermann2018-05-28
|
* Improve subsection on co-inductive types of the Gallina chapter.Gravatar Théo Zimmermann2018-05-27
|
* Improve subsection on mutual inductive types of the Gallina chapter.Gravatar Théo Zimmermann2018-05-27
|
* Move 'new in Coq 8.1' subsection to an appropriate place.Gravatar Théo Zimmermann2018-05-27
|
* Document Variant properly.Gravatar Théo Zimmermann2018-05-27
| | | | | | Cf. Enrico's remark at https://github.com/coq/coq/pull/7536#issuecomment-389826121 This commit also marginally improves the Record doc (a lot more remains to do).
* Improve inductive types subsection of the Gallina chapter.Gravatar Théo Zimmermann2018-05-27
|
* Improve subsection Definitions of the Gallina chapter.Gravatar Théo Zimmermann2018-05-26
|
* Improve subsection Assumptions of the Gallina chapter.Gravatar Théo Zimmermann2018-05-26
|
* Improve the section Terms of the Gallina chapter.Gravatar Théo Zimmermann2018-05-26
| | | | Including adding missing irrefutable-patterns to the grammar of binders.
* [doc] Allow more than one signature and name per Sphinx objectGravatar Clément Pit-Claudel2018-05-25
| | | | As discussed in GH-7556.
* Document the new nested-proof error message.Gravatar Théo Zimmermann2018-05-21
|
* Document nested proofs and associated option.Gravatar Théo Zimmermann2018-05-17
|
* [doc] Address feedback on doc writer guideGravatar Clément Pit-Claudel2018-05-15
| | | | Co-Authored-By: @Zimmi48
* Remove duplicate entries for Proof, Qed, Defined, Admitted.Gravatar Théo Zimmermann2018-05-14
| | | | And marginal improvements in the last section of the Gallina chapter.
* [sphinx] Fix new warnings related to tacn, cmd, opt...Gravatar Théo Zimmermann2018-05-09
|
* Clean-up around cmd documentation.Gravatar Théo Zimmermann2018-05-05
| | | | In particular, remove trailing dots.
* Fix error messages and make them consistent.Gravatar Théo Zimmermann2018-05-05
| | | | All the error messages start with a capitalized letter and end with a dot.
* [sphinx] Fix some references.Gravatar Théo Zimmermann2018-05-05
|
* [Sphinx] Clean-up indicesGravatar Maxime Dénès2018-04-16
|
* [Sphinx] Fix all remaining warnings.Gravatar Maxime Dénès2018-04-14
|
* [sphinx] Fix many warnings.Gravatar Théo Zimmermann2018-04-14
| | | | | Including cross-reference TODOs. I took down the number of warnings from 300 to 50.
* [Sphinx] Add Chapter 1Gravatar Maxime Dénès2018-04-13
|
* [Sphinx] Move chapter 1 to new infrastructureGravatar Maxime Dénès2018-04-13