aboutsummaryrefslogtreecommitdiff
path: root/doc/sphinx/proof-engine
diff options
context:
space:
mode:
authorPaolo G. Giarrusso2020-07-11 18:10:18 +0200
committerGitHub2020-07-11 18:10:18 +0200
commitf91f2ac64fbc7035c77592195c67050640abc3cb (patch)
tree722f93abd2f359bc51ea616cfa514558644430dc /doc/sphinx/proof-engine
parentf4593ab277c12eda7e000011eeb2276716ac9a09 (diff)
tactics.rst: `Require A` is enough for `A`'s hints
As the text says later: > Hints should only be made available when the module they are defined in is imported, not just required.
Diffstat (limited to 'doc/sphinx/proof-engine')
-rw-r--r--doc/sphinx/proof-engine/tactics.rst2
1 files changed, 1 insertions, 1 deletions
diff --git a/doc/sphinx/proof-engine/tactics.rst b/doc/sphinx/proof-engine/tactics.rst
index 4af3ebc47b..25c4de7389 100644
--- a/doc/sphinx/proof-engine/tactics.rst
+++ b/doc/sphinx/proof-engine/tactics.rst
@@ -4162,7 +4162,7 @@ Hint locality
Hints provided by the ``Hint`` commands are erased when closing a section.
Conversely, all hints of a module ``A`` that are not defined inside a
section (and not defined with option ``Local``) become available when the
-module ``A`` is imported (using e.g. ``Require Import A.``).
+module ``A`` is required (using e.g. ``Require A.``).
As of today, hints only have a binary behavior regarding locality, as
described above: either they disappear at the end of a section scope,