Skip to content

Commit

Permalink
doc(ring_theory/witt_vector/witt_polynomial): move module docstring up (
Browse files Browse the repository at this point in the history
  • Loading branch information
jcommelin committed Feb 19, 2021
1 parent 0df1998 commit aaab837
Showing 1 changed file with 11 additions and 11 deletions.
22 changes: 11 additions & 11 deletions src/ring_theory/witt_vector/witt_polynomial.lean
Expand Up @@ -10,17 +10,6 @@ import data.mv_polynomial.comm_ring
import data.mv_polynomial.expand
import data.zmod.basic

open mv_polynomial
open finset (hiding map)
open finsupp (single)

open_locale big_operators

local attribute [-simp] coe_eval₂_hom

variables (p : ℕ)
variables (R : Type*) [comm_ring R]

/-!
# Witt polynomials
Expand Down Expand Up @@ -61,6 +50,17 @@ In this file we use the following notation
-/

open mv_polynomial
open finset (hiding map)
open finsupp (single)

open_locale big_operators

local attribute [-simp] coe_eval₂_hom

variables (p : ℕ)
variables (R : Type*) [comm_ring R]

/-- `witt_polynomial p R n` is the `n`-th Witt polynomial
with respect to a prime `p` with coefficients in a commutative ring `R`.
It is defined as:
Expand Down

0 comments on commit aaab837

Please sign in to comment.