Skip to content

Commit

Permalink
Add some markers of origin.
Browse files Browse the repository at this point in the history
  • Loading branch information
Zimmi48 committed May 14, 2020
1 parent 95c4fc7 commit 26cd7d0
Show file tree
Hide file tree
Showing 7 changed files with 20 additions and 0 deletions.
2 changes: 2 additions & 0 deletions doc/sphinx/language/core/inductive.rst
Expand Up @@ -508,6 +508,8 @@ constructions.
| cons t f' => (tree_size t + forest_size f')
end.

.. extracted from CIC chapter
.. _inductive-definitions:

Theory of inductive definitions
Expand Down
4 changes: 4 additions & 0 deletions doc/sphinx/language/core/modules.rst
Expand Up @@ -50,6 +50,8 @@ A module type abbreviation is written :math:`\ModType{Y}{S}`,
where :math:`Y` is an identifier and :math:`S` is any structure
expression .

.. extracted from Gallina extensions chapter
Using modules
-------------

Expand Down Expand Up @@ -852,6 +854,8 @@ and :math:`Γ_C` is :math:`[c_1 :C_1 ;…;c_n :C_n ]`.
--------------------------
E[] ⊢ p.c_i \triangleright_δ p'.c_i

.. extracted from Gallina extensions chapter
Libraries and qualified names
---------------------------------

Expand Down
2 changes: 2 additions & 0 deletions doc/sphinx/language/extensions/canonical.rst
Expand Up @@ -14,6 +14,8 @@ of another, complementary, use of canonical structures: advanced proof search.
This latter papers also presents many techniques one can employ to tune the
inference of canonical structures.

.. extracted from implicit arguments section
.. _canonical-structure-declaration:

Declaraction of canonical structures
Expand Down
6 changes: 6 additions & 0 deletions doc/sphinx/language/extensions/evars.rst
@@ -1,3 +1,5 @@
.. extracted from Gallina extensions chapter
.. _existential-variables:

Existential variables
Expand Down Expand Up @@ -62,6 +64,8 @@ the syntax :n:`?[@ident]`. This is useful when the existential
variable needs to be explicitly handled later in the script (e.g.
with a named-goal selector, see :ref:`goal-selectors`).

.. extracted from Gallina chapter
.. index:: _

Inferable subterms
Expand All @@ -71,6 +75,8 @@ Expressions often contain redundant pieces of information. Subterms that can be
automatically inferred by Coq can be replaced by the symbol ``_`` and Coq will
guess the missing piece of information.

.. extracted from Gallina extensions chapter
.. _explicit-display-existentials:

Explicit displaying of existential instances for pretty-printing
Expand Down
2 changes: 2 additions & 0 deletions doc/sphinx/language/extensions/match.rst
Expand Up @@ -9,6 +9,8 @@ This section describes the full form of pattern matching in |Coq| terms.

.. |rhs| replace:: right hand sides

.. extracted from Gallina extensions chapter

Variants and extensions of :g:`match`
-------------------------------------

Expand Down
2 changes: 2 additions & 0 deletions doc/sphinx/proof-engine/vernacular-commands.rst
Expand Up @@ -747,6 +747,8 @@ Controlling display
after each tactic. The information is used by the Prooftree tool in Proof
General. (https://askra.de/software/prooftree)

.. extracted from Gallina extensions chapter
.. _printing_constructions_full:

Printing constructions in full
Expand Down
2 changes: 2 additions & 0 deletions doc/sphinx/user-extensions/syntax-extensions.rst
Expand Up @@ -1383,6 +1383,8 @@ Abbreviations
exception, if the right-hand side is just of the form :n:`@@qualid`,
this conventionally stops the inheritance of implicit arguments.

.. extracted from Gallina chapter
Numerals and strings
--------------------

Expand Down

0 comments on commit 26cd7d0

Please sign in to comment.