Skip to content

Commit c9d34cd

Browse files
authored
Merge pull request #562 from Seasawher/auto-update-branch
2 parents f346fb3 + a8a3d33 commit c9d34cd

File tree

5 files changed

+20
-8
lines changed

5 files changed

+20
-8
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: `07f1b273c8871bec3f61440bb61babe43ae4d932`
3+
Mathlib version: `11d700a58e53f1903b9d99aacb82e03bdf4cca64`
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: `07f1b273c8871bec3f61440bb61babe43ae4d932`
3+
Mathlib version: `11d700a58e53f1903b9d99aacb82e03bdf4cca64`
44

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

docs/options.md

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

3-
Mathlib version: `07f1b273c8871bec3f61440bb61babe43ae4d932`
3+
Mathlib version: `11d700a58e53f1903b9d99aacb82e03bdf4cca64`
44

55
## Elab.async
66
type: `Bool`

docs/tactics.md

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

3-
Mathlib version: `07f1b273c8871bec3f61440bb61babe43ae4d932`
3+
Mathlib version: `11d700a58e53f1903b9d99aacb82e03bdf4cca64`
44

55
## \#adaptation_note
66
Defined in: `«tactic#adaptation_note_»`
@@ -3242,7 +3242,8 @@ Defined in: `Mathlib.Tactic.grwSeq`
32423242

32433243
`grw [e]` works just like `rw [e]`, but `e` can be a relation other than `=` or ``.
32443244

3245-
For example,
3245+
For example:
3246+
32463247
```lean
32473248
variable {a b c d n : ℤ}
32483249
@@ -3256,6 +3257,17 @@ example (h₁ : a ∣ b) (h₂ : b ∣ a ^ 2 * c) : a ∣ b ^ 2 * c := by
32563257
grw [h₁] at *
32573258
exact h₂
32583259
```
3260+
3261+
To replace the RHS with the LHS of the given relation, use the `` notation (just like in `rw`):
3262+
3263+
```
3264+
example (h₁ : a < b) (h₂ : b ≤ c) : a + d ≤ c + d := by
3265+
grw [← h₂, ← h₁]
3266+
```
3267+
3268+
The strict inequality `a < b` is turned into the non-strict inequality `a ≤ b` to rewrite with it.
3269+
A future version of `grw` may get special support for making better use of strict inequalities.
3270+
32593271
To rewrite only in the `n`-th position, use `nth_grw n`.
32603272
This is useful when `grw` tries to rewrite in a position that is not valid for the given relation.
32613273

lake-manifest.json

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -5,7 +5,7 @@
55
"type": "git",
66
"subDir": null,
77
"scope": "",
8-
"rev": "07f1b273c8871bec3f61440bb61babe43ae4d932",
8+
"rev": "11d700a58e53f1903b9d99aacb82e03bdf4cca64",
99
"name": "mathlib",
1010
"manifestFile": "lake-manifest.json",
1111
"inputRev": "master",
@@ -15,7 +15,7 @@
1515
"type": "git",
1616
"subDir": null,
1717
"scope": "leanprover-community",
18-
"rev": "e2a2ee109182182dd0e347e8149d312d72bfbfb2",
18+
"rev": "b3dd6c3ebc0a71685e86bea9223be39ea4c299fb",
1919
"name": "plausible",
2020
"manifestFile": "lake-manifest.json",
2121
"inputRev": "main",
@@ -75,7 +75,7 @@
7575
"type": "git",
7676
"subDir": null,
7777
"scope": "leanprover-community",
78-
"rev": "78129e1913fe4988ac238156ec5f223ec02d286c",
78+
"rev": "6cae843edf5b3abc871c557614eaffdcb4492d89",
7979
"name": "batteries",
8080
"manifestFile": "lake-manifest.json",
8181
"inputRev": "main",

0 commit comments

Comments
 (0)