Skip to content

Commit

Permalink
doc(ComputeDegree): typos (#21095)
Browse files Browse the repository at this point in the history
  • Loading branch information
adomani committed Jan 26, 2025
1 parent 1a2855b commit 7564134
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions Mathlib/Tactic/ComputeDegree.lean
Original file line number Diff line number Diff line change
Expand Up @@ -440,14 +440,14 @@ def miscomputedDegree? (deg : Expr) : List Expr → List MessageData
* `degree f ≤ d`,
* `coeff f d = r`, if `d` is the degree of `f`.
The tactic may leave goals of the form `d' = d` `d' ≤ d`, or `r ≠ 0`, where `d'` in `ℕ` or
The tactic may leave goals of the form `d' = d`, `d' ≤ d`, or `r ≠ 0`, where `d'` in `ℕ` or
`WithBot ℕ` is the tactic's guess of the degree, and `r` is the coefficient's guess of the
leading coefficient of `f`.
`compute_degree` applies `norm_num` to the left-hand side of all side goals, trying to close them.
The variant `compute_degree!` first applies `compute_degree`.
Then it uses `norm_num` on all the whole remaining goals and tries `assumption`.
Then it uses `norm_num` on all the remaining goals and tries `assumption`.
-/
syntax (name := computeDegree) "compute_degree" "!"? : tactic

Expand Down

0 comments on commit 7564134

Please sign in to comment.