Skip to content

Commit

Permalink
Merge PR #18074: Explain "Constant" in Locate output
Browse files Browse the repository at this point in the history
Reviewed-by: ppedrot
Co-authored-by: ppedrot <ppedrot@users.noreply.github.com>
  • Loading branch information
coqbot-app[bot] and ppedrot committed May 22, 2024
2 parents f1649da + 38d5aec commit 1bae91e
Showing 1 changed file with 4 additions and 0 deletions.
4 changes: 4 additions & 0 deletions doc/sphinx/proof-engine/vernacular-commands.rst
Original file line number Diff line number Diff line change
Expand Up @@ -417,6 +417,10 @@ Requests to the environment
are reported only when the containing module has been imported
(e.g. with :cmd:`Require Import` or :cmd:`Import`).

Objects defined with commands such as :cmd:`Definition`, :cmd:`Parameter`,
:cmd:`Record`, :cmd:`Theorem` and their numerous variants are shown
as `Constant` in the output.

:n:`@qualid`
refers to object names that end with :n:`@qualid`.

Expand Down

0 comments on commit 1bae91e

Please sign in to comment.