Skip to content

Commit

Permalink
feat(field_theory/mv_polynomial): char_p instance (#3491)
Browse files Browse the repository at this point in the history
Co-authored-by: Johan Commelin <johan@commelin.net>



Co-authored-by: Rob Lewis <rob.y.lewis@gmail.com>
  • Loading branch information
robertylewis and robertylewis committed Jul 21, 2020
1 parent 1a31e69 commit d57130b
Showing 1 changed file with 9 additions and 0 deletions.
9 changes: 9 additions & 0 deletions src/field_theory/mv_polynomial.lean
Expand Up @@ -260,3 +260,12 @@ begin
end

end mv_polynomial

namespace mv_polynomial

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

instance [char_p R p] : char_p (mv_polynomial σ R) p :=
{ cast_eq_zero_iff := λ n, by rw [← C_eq_coe_nat, ← C_0, C_inj, char_p.cast_eq_zero_iff R p] }

end mv_polynomial

0 comments on commit d57130b

Please sign in to comment.