Skip to content

Commit

Permalink
chore(ring_theory/witt_vector): fix a docstring (#9575)
Browse files Browse the repository at this point in the history
  • Loading branch information
jcommelin committed Oct 6, 2021
1 parent 850d5d2 commit 6abd6f2
Show file tree
Hide file tree
Showing 2 changed files with 4 additions and 4 deletions.
2 changes: 1 addition & 1 deletion src/ring_theory/witt_vector/frobenius.lean
Expand Up @@ -79,7 +79,7 @@ private def pnat_multiplicity (n : ℕ+) : ℕ :=
local notation `v` := pnat_multiplicity

/-- An auxiliary polynomial over the integers, that satisfies
`(frobenius_poly_aux p n - X n ^ p) / p = frobenius_poly p n`.
`p * (frobenius_poly_aux p n) + X n ^ p = frobenius_poly p n`.
This makes it easy to show that `frobenius_poly p n` is congruent to `X n ^ p`
modulo `p`. -/
noncomputable def frobenius_poly_aux : ℕ → mv_polynomial ℕ ℤ
Expand Down
6 changes: 3 additions & 3 deletions src/ring_theory/witt_vector/structure_polynomial.lean
Expand Up @@ -180,11 +180,11 @@ begin
exact pow_ne_zero _ (nat.cast_ne_zero.2 hp.1.ne_zero),
end

/-- `witt_structure_int Φ` is a family of polynomials `ℕ → mv_polynomial (idx × ℕ) `
/-- `witt_structure_int Φ` is a family of polynomials `ℕ → mv_polynomial (idx × ℕ) `
that are uniquely characterised by the property that
```
bind₁ (witt_structure_int p Φ) (witt_polynomial p n) =
bind₁ (λ i, (rename (prod.mk i) (witt_polynomial p n))) Φ
bind₁ (witt_structure_int p Φ) (witt_polynomial p n) =
bind₁ (λ i, (rename (prod.mk i) (witt_polynomial p n))) Φ
```
In other words: evaluating the `n`-th Witt polynomial on the family `witt_structure_int Φ`
is the same as evaluating `Φ` on the (appropriately renamed) `n`-th Witt polynomials.
Expand Down

0 comments on commit 6abd6f2

Please sign in to comment.