src/HOL/Algebra/Ring.thy
changeset 23957 54fab60ddc97
parent 23350 50c5b0912a0c
child 26202 51f8a696cd8d
equal deleted inserted replaced
23956:48494ccfabaf 23957:54fab60ddc97
   469   finally have "x \<otimes> (\<ominus> y) \<oplus> x \<otimes> y = \<zero>" .
   469   finally have "x \<otimes> (\<ominus> y) \<oplus> x \<otimes> y = \<zero>" .
   470   with R have "x \<otimes> (\<ominus> y) \<oplus> x \<otimes> y \<oplus> \<ominus> (x \<otimes> y) = \<zero> \<oplus> \<ominus> (x \<otimes> y)" by simp
   470   with R have "x \<otimes> (\<ominus> y) \<oplus> x \<otimes> y \<oplus> \<ominus> (x \<otimes> y) = \<zero> \<oplus> \<ominus> (x \<otimes> y)" by simp
   471   with R show ?thesis by (simp add: a_assoc r_neg )
   471   with R show ?thesis by (simp add: a_assoc r_neg )
   472 qed
   472 qed
   473 
   473 
   474 lemma (in ring) minus_eq:
   474 lemma (in abelian_group) minus_eq:
   475   "[| x \<in> carrier R; y \<in> carrier R |] ==> x \<ominus> y = x \<oplus> \<ominus> y"
   475   "[| x \<in> carrier G; y \<in> carrier G |] ==> x \<ominus> y = x \<oplus> \<ominus> y"
   476   by (simp only: a_minus_def)
   476   by (simp only: a_minus_def)
   477 
   477 
   478 text {* Setup algebra method:
   478 text {* Setup algebra method:
   479   compute distributive normal form in locale contexts *}
   479   compute distributive normal form in locale contexts *}
   480 
   480