Skip to content

Commit 003fce4

Browse files
authored
Merge pull request #538 from Seasawher/auto-update-branch
2 parents 69d47fa + ffafc7d commit 003fce4

File tree

5 files changed

+13
-61
lines changed

5 files changed

+13
-61
lines changed

docs/attributes.md

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

3-
Mathlib version: `c1ee2821db22c395b37586d80ae2b7f9a24ee2cb`
3+
Mathlib version: `786ca91ad0b41b6ee048e3dcdd23cc71807fddbb`
44

55
## Std.Internal.tree_tac
66
simp theorems used by internal DTreeMap lemmas

docs/commands.md

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1,6 +1,6 @@
11
# Commands
22

3-
Mathlib version: `c1ee2821db22c395b37586d80ae2b7f9a24ee2cb`
3+
Mathlib version: `786ca91ad0b41b6ee048e3dcdd23cc71807fddbb`
44

55
## \#adaptation_note
66
Defined in: `adaptationNoteCmd`

docs/options.md

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

3-
Mathlib version: `c1ee2821db22c395b37586d80ae2b7f9a24ee2cb`
3+
Mathlib version: `786ca91ad0b41b6ee048e3dcdd23cc71807fddbb`
44

55
## Elab.async
66
type: `Bool`
@@ -1269,6 +1269,13 @@ default: `true`
12691269

12701270
Linter used by translate attributes that checks if the given declaration name is equal to the automatically generated name
12711271

1272+
## linter.translateReorder
1273+
type: `Bool`
1274+
1275+
default: `true`
1276+
1277+
Linter used by translate attributes that checks if the given reorder is equal to the automatically generated one
1278+
12721279
## linter.unnecessarySeqFocus
12731280
type: `Bool`
12741281

@@ -4002,13 +4009,6 @@ default: `false`
40024009

40034010
enable/disable tracing for the given module and submodules
40044011

4005-
## trace.Tactic.propose
4006-
type: `Bool`
4007-
4008-
default: `false`
4009-
4010-
enable/disable tracing for the given module and submodules
4011-
40124012
## trace.Tactic.rewrites
40134013
type: `Bool`
40144014

docs/tactics.md

Lines changed: 1 addition & 49 deletions
Original file line numberDiff line numberDiff line change
@@ -1,6 +1,6 @@
11
# Tactics
22

3-
Mathlib version: `c1ee2821db22c395b37586d80ae2b7f9a24ee2cb`
3+
Mathlib version: `786ca91ad0b41b6ee048e3dcdd23cc71807fddbb`
44

55
## \#adaptation_note
66
Defined in: `«tactic#adaptation_note_»`
@@ -3306,59 +3306,11 @@ The tactic supports all the same syntax variants and options as the `have` term.
33063306
which may be important for performance reasons.
33073307
Consider using the equivalent `let +nondep` to indicate the intent.
33083308

3309-
## have!?
3310-
Defined in: `Mathlib.Tactic.Propose.«tacticHave!?:_Using__»`
3311-
3312-
* `have? using a, b, c` tries to find a lemma
3313-
which makes use of each of the local hypotheses `a, b, c`,
3314-
and reports any results via trace messages.
3315-
* `have? : h using a, b, c` only returns lemmas whose type matches `h` (which may contain `_`).
3316-
* `have?! using a, b, c` will also call `have` to add results to the local goal state.
3317-
3318-
Note that `have?` (unlike `apply?`) does not inspect the goal at all,
3319-
only the types of the lemmas in the `using` clause.
3320-
3321-
`have?` should not be left in proofs; it is a search tool, like `apply?`.
3322-
3323-
Suggestions are printed as `have := f a b c`.
3324-
33253309
## have'
33263310
Defined in: `Lean.Parser.Tactic.tacticHave'`
33273311

33283312
Similar to `have`, but using `refine'`
33293313

3330-
## have?
3331-
Defined in: `Mathlib.Tactic.Propose.propose'`
3332-
3333-
* `have? using a, b, c` tries to find a lemma
3334-
which makes use of each of the local hypotheses `a, b, c`,
3335-
and reports any results via trace messages.
3336-
* `have? : h using a, b, c` only returns lemmas whose type matches `h` (which may contain `_`).
3337-
* `have?! using a, b, c` will also call `have` to add results to the local goal state.
3338-
3339-
Note that `have?` (unlike `apply?`) does not inspect the goal at all,
3340-
only the types of the lemmas in the `using` clause.
3341-
3342-
`have?` should not be left in proofs; it is a search tool, like `apply?`.
3343-
3344-
Suggestions are printed as `have := f a b c`.
3345-
3346-
## have?!
3347-
Defined in: `Mathlib.Tactic.Propose.«tacticHave?!:_Using__»`
3348-
3349-
* `have? using a, b, c` tries to find a lemma
3350-
which makes use of each of the local hypotheses `a, b, c`,
3351-
and reports any results via trace messages.
3352-
* `have? : h using a, b, c` only returns lemmas whose type matches `h` (which may contain `_`).
3353-
* `have?! using a, b, c` will also call `have` to add results to the local goal state.
3354-
3355-
Note that `have?` (unlike `apply?`) does not inspect the goal at all,
3356-
only the types of the lemmas in the `using` clause.
3357-
3358-
`have?` should not be left in proofs; it is a search tool, like `apply?`.
3359-
3360-
Suggestions are printed as `have := f a b c`.
3361-
33623314
## haveI
33633315
Defined in: `Lean.Parser.Tactic.tacticHaveI__`
33643316

lake-manifest.json

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -5,7 +5,7 @@
55
"type": "git",
66
"subDir": null,
77
"scope": "",
8-
"rev": "c1ee2821db22c395b37586d80ae2b7f9a24ee2cb",
8+
"rev": "786ca91ad0b41b6ee048e3dcdd23cc71807fddbb",
99
"name": "mathlib",
1010
"manifestFile": "lake-manifest.json",
1111
"inputRev": "master",
@@ -75,7 +75,7 @@
7575
"type": "git",
7676
"subDir": null,
7777
"scope": "leanprover-community",
78-
"rev": "30cfb2255996f3e6217a77fd940fde1f3e12ccc2",
78+
"rev": "26884086fb66f99b56ed363c5e54bfcc70238599",
7979
"name": "batteries",
8080
"manifestFile": "lake-manifest.json",
8181
"inputRev": "main",

0 commit comments

Comments
 (0)