Skip to content

Commit b7a945f

Browse files
authored
Merge pull request #545 from Seasawher/auto-update-branch
2 parents 3dc3475 + 2e85417 commit b7a945f

File tree

5 files changed

+14
-8
lines changed

5 files changed

+14
-8
lines changed

docs/attributes.md

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

3-
Mathlib version: `6a263ebffc52b615a6cda0fc9a15d3879d674d10`
3+
Mathlib version: `90f5d6d994d62d023ec24dc2fac75d053e04c801`
44

55
## Std.Internal.tree_tac
66
simp theorems used by internal DTreeMap lemmas
@@ -1544,6 +1544,9 @@ have to be assigned in the same file as the declaration.
15441544
Similar to `registerParametricAttribute` except that attributes do not
15451545
have to be assigned in the same file as the declaration.
15461546

1547+
## to_fun
1548+
generate a copy of a lemma where point-free functions are expanded to their `fun` form
1549+
15471550
## trans
15481551
transitive relation
15491552

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: `6a263ebffc52b615a6cda0fc9a15d3879d674d10`
3+
Mathlib version: `90f5d6d994d62d023ec24dc2fac75d053e04c801`
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: `6a263ebffc52b615a6cda0fc9a15d3879d674d10`
3+
Mathlib version: `90f5d6d994d62d023ec24dc2fac75d053e04c801`
44

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

docs/tactics.md

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

3-
Mathlib version: `6a263ebffc52b615a6cda0fc9a15d3879d674d10`
3+
Mathlib version: `90f5d6d994d62d023ec24dc2fac75d053e04c801`
44

55
## \#adaptation_note
66
Defined in: `«tactic#adaptation_note_»`
@@ -1061,8 +1061,11 @@ Defined in: `byContra!`
10611061
If the target of the main goal is a proposition `p`,
10621062
`by_contra!` reduces the goal to proving `False` using the additional hypothesis `this : ¬ p`.
10631063
`by_contra! h` can be used to name the hypothesis `h : ¬ p`.
1064-
The hypothesis `¬ p` will be negation normalized using `push_neg`.
1064+
The hypothesis `¬ p` will be normalized using `push_neg`.
10651065
For instance, `¬ a < b` will be changed to `b ≤ a`.
1066+
`by_contra!` can be used with `rcases` patterns.
1067+
For instance, `by_contra! rfl` on `⊢ s.Nonempty` will substitute the equality `s = ∅`,
1068+
and `by_contra! ⟨hp, hq⟩` on `⊢ ¬ p ∨ ¬ q` will introduce `hp : p` and `hq : q`.
10661069
`by_contra! h : q` will normalize negations in `¬ p`, normalize negations in `q`,
10671070
and then check that the two normalized forms are equal.
10681071
The resulting hypothesis is the pre-normalized form, `q`.
@@ -2719,15 +2722,15 @@ Patterns can be used like in the `intro` tactic. Example, given a goal
27192722
Defined in: `Mathlib.Tactic.GCongr.tacticGcongr___With___`
27202723

27212724
The `gcongr` tactic applies "generalized congruence" rules, reducing a relational goal
2722-
between a LHS and RHS. For example,
2725+
between an LHS and RHS. For example,
27232726
```
27242727
example {a b x c d : ℝ} (h1 : a + 1 ≤ b + 1) (h2 : c + 2 ≤ d + 2) :
27252728
x ^ 2 * a + c ≤ x ^ 2 * b + d := by
27262729
gcongr
27272730
· linarith
27282731
· linarith
27292732
```
2730-
This example has the goal of proving the relation `` between a LHS and RHS both of the pattern
2733+
This example has the goal of proving the relation `` between an LHS and RHS both of the pattern
27312734
```
27322735
x ^ 2 * ?_ + ?_
27332736
```

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

0 commit comments

Comments
 (0)