Skip to content

Commit 762534b

Browse files
authored
Merge pull request #501 from Seasawher/auto-update-branch
2 parents b6a8493 + d9e5483 commit 762534b

File tree

5 files changed

+13
-5
lines changed

5 files changed

+13
-5
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: `ed5b08ca63c16a9533ab652a7c140afca119b817`
3+
Mathlib version: `acb60b64877e03f0184702506a006f157e37e044`
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: `ed5b08ca63c16a9533ab652a7c140afca119b817`
3+
Mathlib version: `acb60b64877e03f0184702506a006f157e37e044`
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: `ed5b08ca63c16a9533ab652a7c140afca119b817`
3+
Mathlib version: `acb60b64877e03f0184702506a006f157e37e044`
44

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

docs/tactics.md

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

3-
Mathlib version: `ed5b08ca63c16a9533ab652a7c140afca119b817`
3+
Mathlib version: `acb60b64877e03f0184702506a006f157e37e044`
44

55
## \#adaptation_note
66
Defined in: `«tactic#adaptation_note_»`
@@ -5791,13 +5791,21 @@ according to the syntax of the expression `x`, if the atoms composing the expres
57915791
numeric lower bounds which can be proved positive/nonnegative/nonzero by `norm_num`. This tactic
57925792
either closes the goal or fails.
57935793

5794+
`positivity [t₁, …, tₙ]` first executes `have := t₁; …; have := tₙ` in the current goal,
5795+
then runs `positivity`. This is useful when `positivity` needs derived premises such as `0 < y`
5796+
for division/reciprocal, or `0 ≤ x` for real powers.
5797+
57945798
Examples:
57955799
```lean
57965800
example {a : ℤ} (ha : 3 < a) : 0 ≤ a ^ 3 + a := by positivity
57975801
57985802
example {a : ℤ} (ha : 1 < a) : 0 < |(3:ℤ) + a| := by positivity
57995803
58005804
example {b : ℤ} : 0 ≤ max (-3) (b ^ 2) := by positivity
5805+
5806+
example {a b c d : ℝ} (hab : 0 < a * b) (hb : 0 ≤ b) (hcd : c < d) :
5807+
0 < a ^ c + 1 / (d - c) := by
5808+
positivity [sub_pos_of_lt hcd, pos_of_mul_pos_left hab hb]
58015809
```
58025810

58035811
## pull

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": "ed5b08ca63c16a9533ab652a7c140afca119b817",
8+
"rev": "acb60b64877e03f0184702506a006f157e37e044",
99
"name": "mathlib",
1010
"manifestFile": "lake-manifest.json",
1111
"inputRev": "master",

0 commit comments

Comments
 (0)