Skip to content

Commit c966125

Browse files
authored
Merge pull request #549 from Seasawher/auto-update-branch
2 parents df432ac + 544ef12 commit c966125

File tree

5 files changed

+32
-12
lines changed

5 files changed

+32
-12
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: `a7f816c359320b9c0383f3c052d5a0574db65b97`
3+
Mathlib version: `89ec9c848cb1c5922fa50b91eb5156a46bd71e85`
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: `a7f816c359320b9c0383f3c052d5a0574db65b97`
3+
Mathlib version: `89ec9c848cb1c5922fa50b91eb5156a46bd71e85`
44

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

docs/options.md

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

3-
Mathlib version: `a7f816c359320b9c0383f3c052d5a0574db65b97`
3+
Mathlib version: `89ec9c848cb1c5922fa50b91eb5156a46bd71e85`
44

55
## Elab.async
66
type: `Bool`
@@ -1219,13 +1219,34 @@ default: `1`
12191219

12201220

12211221

1222+
## linter.tacticAnalysis.tryAtEachStep.selfReplacements
1223+
type: `Bool`
1224+
1225+
default: `true`
1226+
1227+
1228+
1229+
## linter.tacticAnalysis.tryAtEachStep.showTiming
1230+
type: `Bool`
1231+
1232+
default: `true`
1233+
1234+
1235+
12221236
## linter.tacticAnalysis.tryAtEachStepAesop
12231237
type: `Bool`
12241238

12251239
default: `false`
12261240

12271241

12281242

1243+
## linter.tacticAnalysis.tryAtEachStepFromEnv
1244+
type: `Bool`
1245+
1246+
default: `false`
1247+
1248+
1249+
12291250
## linter.tacticAnalysis.tryAtEachStepGrind
12301251
type: `Bool`
12311252

@@ -2066,7 +2087,7 @@ type: `Bool`
20662087

20672088
default: `false`
20682089

2069-
Make `push_neg` use `not_and_or` rather than the default `not_and`.
2090+
Set `distrib` to true in `push_neg` and related tactics.
20702091

20712092
## quotPrecheck
20722093
type: `Bool`

docs/tactics.md

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

3-
Mathlib version: `a7f816c359320b9c0383f3c052d5a0574db65b97`
3+
Mathlib version: `89ec9c848cb1c5922fa50b91eb5156a46bd71e85`
44

55
## \#adaptation_note
66
Defined in: `«tactic#adaptation_note_»`
@@ -1047,10 +1047,10 @@ Defined in: `«tacticBy_cases_:_»`
10471047
`by_cases (h :)? p` splits the main goal into two cases, assuming `h : p` in the first branch, and `h : ¬ p` in the second branch.
10481048

10491049
## by_cases!
1050-
Defined in: `byCases!`
1050+
Defined in: `Mathlib.Tactic.ByCases.byCases!`
10511051

10521052
`by_cases! h : p` runs the `by_cases h : p` tactic, followed by
1053-
`try push_neg at h` in the second subgoal. For example,
1053+
`push_neg at h` in the second subgoal. For example,
10541054
- `by_cases! h : a < b` creates one goal with hypothesis `h : a < b` and
10551055
another with `h : b ≤ a`.
10561056
- `by_cases! h : a ≠ b` creates one goal with hypothesis `h : a ≠ b` and
@@ -1066,7 +1066,7 @@ introducing a hypothesis `h : ¬p` and proving `False`.
10661066
* If `h` is omitted, the introduced variable will be called `this`.
10671067

10681068
## by_contra!
1069-
Defined in: `byContra!`
1069+
Defined in: `Mathlib.Tactic.ByContra.byContra!`
10701070

10711071
If the target of the main goal is a proposition `p`,
10721072
`by_contra!` reduces the goal to proving `False` using the additional hypothesis `this : ¬ p`.
@@ -6022,7 +6022,7 @@ which can also cope with identities of the form
60226022
where `a = a'`, `b = b'`, and `c = c'` can be proved using `pure_coherence`
60236023

60246024
## push
6025-
Defined in: `Mathlib.Tactic.Push.push`
6025+
Defined in: `Mathlib.Tactic.Push.pushStx`
60266026

60276027
`push` pushes the given constant away from the head of the expression. For example
60286028
- `push _ ∈ _` rewrites `x ∈ {y} ∪ zᶜ` into `x = y ∨ ¬ x ∈ z`.
@@ -6085,8 +6085,7 @@ For instance, a hypothesis `h : ¬ ∀ x, ∃ y, x ≤ y` will be transformed by
60856085
`push_neg` is a special case of the more general `push` tactic, namely `push Not`.
60866086
The `push` tactic can be extended using the `@[push]` attribute. `push` has special-casing
60876087
built in for `push Not`, so that it can preserve binder names, and so that `¬ (p ∧ q)` can be
6088-
transformed to either `p → ¬ q` (the default) or `¬ p ∨ ¬ q`. To get `¬ p ∨ ¬ q`, use
6089-
`set_option push_neg.use_distrib true`.
6088+
transformed to either `p → ¬ q` (default) or `¬ p ∨ ¬ q` (`push_neg +distrib`).
60906089

60916090
Tactics that introduce a negation usually have a version that automatically calls `push_neg` on
60926091
that negation. These include `by_cases!`, `contrapose!` and `by_contra!`.

lake-manifest.json

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -5,7 +5,7 @@
55
"type": "git",
66
"subDir": null,
77
"scope": "",
8-
"rev": "a7f816c359320b9c0383f3c052d5a0574db65b97",
8+
"rev": "89ec9c848cb1c5922fa50b91eb5156a46bd71e85",
99
"name": "mathlib",
1010
"manifestFile": "lake-manifest.json",
1111
"inputRev": "master",

0 commit comments

Comments
 (0)