Zulip Chat Archive

Stream: Is there code for X?

Topic: characteristic two


Eric Wieser (Nov 22 2021 at 16:28):

Do we have this anywhere?

lemma char_two_neg {R} [ring R] [char_p R 2] (x : R) : -x = x :=
by rw [neg_eq_iff_add_eq_zero, two_smul  x, nsmul_eq_smul_cast R 2 x, char_p.cast_eq_zero,
  zero_smul]

lemma char_two_sub {R} [ring R] [char_p R 2] (x y : R) : x - y = x + y :=
by rw [sub_eq_add_neg, char_two_neg]

Last updated: Dec 20 2023 at 11:08 UTC