aboutsummaryrefslogtreecommitdiff
path: root/doc/sphinx/language
diff options
context:
space:
mode:
authorEmilio Jesus Gallego Arias2020-11-26 21:32:37 +0100
committerEmilio Jesus Gallego Arias2020-11-26 22:08:01 +0100
commit1f0f1ae93f757be8101d598f8aaf5b564bde9dcd (patch)
tree5afe9610e6412cf6e15bd3e158f04e32bd2d17e2 /doc/sphinx/language
parent50af46a596af607493ce46da782389e8a82e8354 (diff)
[attributes] [typing] Rename `typing` to `bypass_check`
As discussed in the Coq meeting.
Diffstat (limited to 'doc/sphinx/language')
-rw-r--r--doc/sphinx/language/core/coinductive.rst4
-rw-r--r--doc/sphinx/language/core/definitions.rst6
-rw-r--r--doc/sphinx/language/core/inductive.rst12
3 files changed, 11 insertions, 11 deletions
diff --git a/doc/sphinx/language/core/coinductive.rst b/doc/sphinx/language/core/coinductive.rst
index e9737f8712..cf46580bdb 100644
--- a/doc/sphinx/language/core/coinductive.rst
+++ b/doc/sphinx/language/core/coinductive.rst
@@ -27,8 +27,8 @@ More information on co-inductive definitions can be found in
This command supports the :attr:`universes(polymorphic)`,
:attr:`universes(template)`, :attr:`universes(cumulative)`,
- :attr:`private(matching)`, :attr:`typing(universes)`,
- :attr:`typing(positive)`, and :attr:`using` attributes.
+ :attr:`private(matching)`, :attr:`bypass_check(universes)`,
+ :attr:`bypass_check(positivity)`, and :attr:`using` attributes.
.. example::
diff --git a/doc/sphinx/language/core/definitions.rst b/doc/sphinx/language/core/definitions.rst
index 95bb1b0e0c..76aa543b8b 100644
--- a/doc/sphinx/language/core/definitions.rst
+++ b/doc/sphinx/language/core/definitions.rst
@@ -91,7 +91,7 @@ Section :ref:`typing-rules`.
These commands also support the :attr:`universes(polymorphic)`,
:attr:`program` (see :ref:`program_definition`), :attr:`canonical`,
- :attr:`typing(universes)`, :attr:`typing(guarded)`, and
+ :attr:`bypass_check(universes)`, :attr:`bypass_check(guard)`, and
:attr:`using` attributes.
If :n:`@term` is omitted, :n:`@type` is required and Coq enters proof editing mode.
@@ -163,8 +163,8 @@ Chapter :ref:`Tactics`. The basic assertion command is:
correct at some time of the interactive development of a proof, use the
command :cmd:`Guarded`.
- This command accepts the :attr:`typing(universes)`,
- :attr:`typing(guarded)`, and :attr:`using` attributes.
+ This command accepts the :attr:`bypass_check(universes)`,
+ :attr:`bypass_check(guard)`, and :attr:`using` attributes.
.. exn:: The term @term has type @type which should be Set, Prop or Type.
:undocumented:
diff --git a/doc/sphinx/language/core/inductive.rst b/doc/sphinx/language/core/inductive.rst
index 86de059f28..4bee7cc1b1 100644
--- a/doc/sphinx/language/core/inductive.rst
+++ b/doc/sphinx/language/core/inductive.rst
@@ -32,7 +32,7 @@ Inductive types
This command supports the :attr:`universes(polymorphic)`,
:attr:`universes(template)`, :attr:`universes(cumulative)`,
- :attr:`typing(positive)`, :attr:`typing(universes)`, and
+ :attr:`bypass_check(positivity)`, :attr:`bypass_check(universes)`, and
:attr:`private(matching)` attributes.
Mutually inductive types can be defined by including multiple :n:`@inductive_definition`\s.
@@ -54,7 +54,7 @@ Inductive types
condition* (see Section :ref:`positivity`). This condition
ensures the soundness of the inductive definition.
Positivity checking can be disabled using the :flag:`Positivity
- Checking` flag or the :attr:`typing(positive)` attribute (see
+ Checking` flag or the :attr:`bypass_check(positivity)` attribute (see
:ref:`controlling-typing-flags`).
.. exn:: The conclusion of @type is not valid; it must be built from @ident.
@@ -394,7 +394,7 @@ constructions.
to :n:`fun {* @binder } => @term`.
This command accepts the :attr:`program`,
- :attr:`typing(universes)`, and :attr:`typing(guarded)` attributes.
+ :attr:`bypass_check(universes)`, and :attr:`bypass_check(guard)` attributes.
To be accepted, a :cmd:`Fixpoint` definition has to satisfy syntactical
constraints on a special argument called the decreasing argument. They
@@ -852,7 +852,7 @@ between universes for inductive types in the Type hierarchy.
.. coqtop:: none
- #[typing(positive=no)] Inductive I : Prop := not_I_I (not_I : I -> False) : I.
+ #[bypass_check(positivity)] Inductive I : Prop := not_I_I (not_I : I -> False) : I.
.. coqtop:: all
@@ -886,7 +886,7 @@ between universes for inductive types in the Type hierarchy.
.. coqtop:: none
- #[typing(positive=no)] Inductive Lam := lam (_ : Lam -> Lam).
+ #[bypass_check(positivity)] Inductive Lam := lam (_ : Lam -> Lam).
.. coqtop:: all
@@ -915,7 +915,7 @@ between universes for inductive types in the Type hierarchy.
.. coqtop:: none
- #[typing(positive=no)] Inductive A: Type := introA: ((A -> Prop) -> Prop) -> A.
+ #[bypass_check(positivity)] Inductive A: Type := introA: ((A -> Prop) -> Prop) -> A.
.. coqtop:: all