Skip to content

Commit

Permalink
feat(algebra/char_p): add two helper lemmas about the cast of the cha…
Browse files Browse the repository at this point in the history
…racteristics being zero (#14464)

- `(ring_char R : R) = 0` and
- If there exists a positive `n` lifting to zero, then the characteristics is positive.



Co-authored-by: Jon Eugster <eugster.jon@gmail.com>
  • Loading branch information
Jon Eugster and joneugster committed Jun 6, 2022
1 parent 769a934 commit 789af09
Showing 1 changed file with 4 additions and 0 deletions.
4 changes: 4 additions & 0 deletions src/algebra/char_p/basic.lean
Expand Up @@ -122,6 +122,10 @@ theorem dvd {x : ℕ} (hx : (x : R) = 0) : ring_char R ∣ x :=
@[simp]
lemma eq_zero [char_zero R] : ring_char R = 0 := eq R 0

@[simp]
lemma nat.cast_ring_char : (ring_char R : R) = 0 :=
by rw ring_char.spec

end ring_char

theorem add_pow_char_of_commute [semiring R] {p : ℕ} [fact p.prime]
Expand Down

0 comments on commit 789af09

Please sign in to comment.