Skip to content

Commit

Permalink
feat(algebra/char_p): fields with a hom between them have same char (#…
Browse files Browse the repository at this point in the history
  • Loading branch information
jcommelin committed Oct 13, 2020
1 parent dd8bf2c commit 9f9344d
Showing 1 changed file with 8 additions and 0 deletions.
8 changes: 8 additions & 0 deletions src/algebra/char_p.lean
Expand Up @@ -163,6 +163,14 @@ begin
rw fact at *, linarith,
end

lemma ring_hom.char_p_iff_char_p {K L : Type*} [field K] [field L] (f : K →+* L) (p : ℕ) :
char_p K p ↔ char_p L p :=
begin
split;
{ introI _c, constructor, intro n,
rw [← @char_p.cast_eq_zero_iff _ _ p _c n, ← f.injective.eq_iff, f.map_nat_cast, f.map_zero] }
end

section frobenius

variables (R : Type u) [comm_ring R] {S : Type v} [comm_ring S] (f : R →* S) (g : R →+* S)
Expand Down

0 comments on commit 9f9344d

Please sign in to comment.