package coq
Install
Dune Dependency
Authors
Maintainers
Sources
sha256=36577b55f4a4b1c64682c387de7abea932d0fd42fc0cd5406927dca344f53587
doc/coq-core.vernac/Attributes/index.html
Module Attributes
Source
The type of parsing attribute data
and vernac_flag_value =
| VernacFlagEmpty
| VernacFlagLeaf of vernac_flag_type
| VernacFlagList of vernac_flags
The type of attributes. When parsing attributes if an 'a attribute
is present then an 'a
value will be produced. In the most general case, an attribute transforms the raw flags along with its value.
Errors on unsupported attributes.
Errors if the list of flags is nonempty.
Definitions for some standard attributes.
With the warning for Hint (and not for Instance etc)
Enable/Disable universe checking
For internal use when messing with the global option.
Parse attributes allowing only locality.
Parse attributes allowing only polymorphism. Uses the global flag for the default value.
Ignores unsupported attributes.
Returns unsupported attributes.
* Defining attributes.
A parser for some key in an attribute. It is given a nonempty 'a option
when the attribute is multiply set for some command.
eg in #[polymorphic] Monomorphic Definition foo := ...
, when parsing Monomorphic
it will be given Some true
.
Make an attribute from a list of key parsers together with their associated key.
Define boolean attribute name
, of the form name={yes,no}
. The attribute may only be set once for a command.
qualified_attribute qual att
treats #[qual(atts)]
like att
treats atts
.
Combinators to help define your own parsers. See the implementation of bool_attribute
for practical use.
assert_empty key v
errors if v
is not empty. key
is used in the error message as the name of the attribute.
assert_once ~name v
errors if v
is not empty. name
is used in the error message as the name of the attribute. Used to ensure that a given attribute is not reapeated.
single_key_parser ~name ~key v
makes a parser for attribute name
giving the constant value v
for key key
taking no arguments. name
may only be given once.
Make an attribute using the internal representation, thus with access to the full power of attributes. Unstable.
Compatibility values for parsing Polymorphic
.
For internal use.