Skip to content

Commit eaea130

Browse files
authored
Merge pull request #471 from Seasawher/auto-update-branch
2 parents e9f7550 + 5d61911 commit eaea130

File tree

6 files changed

+350
-109
lines changed

6 files changed

+350
-109
lines changed

docs/attributes.md

Lines changed: 38 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1,6 +1,6 @@
11
# Attributes
22

3-
Mathlib version: `a8071348b19ed841a1f46dbd5a25d109bc804711`
3+
Mathlib version: `b30c0393ac6454d5d43ee1d1a6760c1939a2302b`
44

55
## Std.Internal.tree_tac
66
simp theorems used by internal DTreeMap lemmas
@@ -254,6 +254,21 @@ This allows the documentation of core Lean features to be visible without import
254254
are defined in. This is only useful during bootstrapping and should not be used outside of
255255
the Lean source code.
256256

257+
## builtin_doc_code_block
258+
docstring code block expander
259+
260+
## builtin_doc_code_suggestions
261+
docstring code element suggestion provider
262+
263+
## builtin_doc_command
264+
builtin docstring command expander
265+
266+
## builtin_doc_directive
267+
docstring directive expander
268+
269+
## builtin_doc_role
270+
docstring role expander
271+
257272
## builtin_formatter
258273
(builtin) Register a formatter for a parser.
259274
Registers a formatter for a parser.
@@ -569,6 +584,21 @@ special casing. If the term is an `Expr.mdata` with a single key `k`, `mdata.k`
569584
## doElem_parser
570585
parser
571586

587+
## doc_code_block
588+
docstring code block expander
589+
590+
## doc_code_suggestions
591+
docstring code element suggestion provider
592+
593+
## doc_command
594+
docstring command expander
595+
596+
## doc_directive
597+
docstring directive expander
598+
599+
## doc_role
600+
docstring role expander
601+
572602
## elab_as_elim
573603
instructs elaborator that the arguments of the function application should be elaborated as were an eliminator
574604
Instructs the elaborator that applications of this function should be elaborated like an eliminator.
@@ -760,6 +790,13 @@ Lemmas involving `<` or `≤` can also be marked `@[bound]` for use in the relat
760790
## gcongr_forward
761791
adds a gcongr_forward extension
762792
793+
## gen_constructor_elims
794+
generate the `.toCtorIdx` and `.ctor.elim` definitions for the given inductive
795+
Generate the `.toCtorIdx` and `.ctor.elim` definitions for the given inductive.
796+
797+
This attribute is only meant to be used in `Init.Prelude` to build these constructions for
798+
types where we did not generate them imediatelly (due to `set_option genCtorIdx false`).
799+
763800
## ghost_simps
764801
Simplification rules for ghost equations.
765802

docs/commands.md

Lines changed: 11 additions & 15 deletions
Original file line numberDiff line numberDiff line change
@@ -1,6 +1,6 @@
11
# Commands
22

3-
Mathlib version: `a8071348b19ed841a1f46dbd5a25d109bc804711`
3+
Mathlib version: `b30c0393ac6454d5d43ee1d1a6760c1939a2302b`
44

55
## \#adaptation_note
66
Defined in: `adaptationNoteCmd`
@@ -463,7 +463,8 @@ In general, `#guard_msgs` accepts a comma-separated list of configuration clause
463463
```lean
464464
#guard_msgs (configElt,*) in cmd
465465
```
466-
By default, the configuration list is `(check all, whitespace := normalized, ordering := exact)`.
466+
By default, the configuration list is
467+
`(check all, whitespace := normalized, ordering := exact, positions := false)`.
467468

468469
Message filters select messages by severity:
469470
- `info`, `warning`, `error`: (non-trace) messages with the given severity level.
@@ -489,6 +490,11 @@ Message ordering:
489490
- `ordering := sorted` sorts the messages in lexicographic order.
490491
This helps with testing commands that are non-deterministic in their ordering.
491492

493+
Position reporting:
494+
- `positions := true` reports the ranges of all messages relative to the line on which
495+
`#guard_msgs` appears.
496+
- `positions := false` does not report position info.
497+
492498
For example, `#guard_msgs (error, drop all) in cmd` means to check warnings and drop
493499
everything else.
494500

@@ -623,17 +629,6 @@ Another important difference is that the `minImports` *linter* starts counting i
623629
where the option is set to `true` *downwards*, whereas the `#min_imports` *command* looks at the
624630
imports needed from the command *upwards*.
625631

626-
## \#import_diff
627-
Defined in: `«command#import_diff_»`
628-
629-
`#import_diff foo bar ...` computes the new transitive imports that are added to a given file when
630-
modules `foo, bar, ...` are added to the set of imports of the file. More precisely, it computes the
631-
import diff between when `foo, bar, ...` are added to the imports and when `foo, bar, ...` are removed
632-
from the imports.
633-
634-
Note: the command also works when some of the modules passed as arguments are already present in the file's
635-
imports.
636-
637632
## \#info_trees
638633
Defined in: `Lean.infoTreesCmd`
639634

@@ -1657,8 +1652,9 @@ docs of `<declName>` by adding `<prefix_string>` before and `<suffix_string>` af
16571652
## gen_injective_theorems%
16581653
Defined in: `Lean.Parser.Command.genInjectiveTheorems`
16591654

1660-
This is an auxiliary command for generation constructor injectivity theorems for
1655+
This is an auxiliary command to generate constructor injectivity theorems for
16611656
inductive types defined at `Prelude.lean`.
1657+
Temporarily also controls the generation of the `ctorIdx` definition.
16621658
It is meant for bootstrapping purposes only.
16631659

16641660
## grind_pattern
@@ -2318,7 +2314,7 @@ which helps in maintaining the desired abstraction level without affecting globa
23182314
## section
23192315
Defined in: `Lean.Parser.Command.section`
23202316

2321-
A `section`/`end` pair delimits the scope of `variable`, `include, `open`, `set_option`, and `local`
2317+
A `section`/`end` pair delimits the scope of `variable`, `include`, `open`, `set_option`, and `local`
23222318
commands. Sections can be nested. `section <id>` provides a label to the section that has to appear
23232319
with the matching `end`. In either case, the `end` can be omitted, in which case the section is
23242320
closed at the end of the file.

0 commit comments

Comments
 (0)