src/HOL/Library/Ring_and_Field.thy
changeset 13483 0e6adce08fb0
parent 13476 600f1c93124f
child 14260 3862336cd4bd
equal deleted inserted replaced
13482:2bb7200a99cf 13483:0e6adce08fb0
    88   also have "... = a * 1" by (simp add: mult_commute)
    88   also have "... = a * 1" by (simp add: mult_commute)
    89   finally show ?thesis .
    89   finally show ?thesis .
    90 qed
    90 qed
    91 
    91 
    92 lemma mult_left_commute: "a * (b * c) = b * (a * (c::'a::ring))"
    92 lemma mult_left_commute: "a * (b * c) = b * (a * (c::'a::ring))"
    93 by(rule mk_left_commute[OF mult_assoc mult_commute])
    93   by (rule mk_left_commute [of "op *", OF mult_assoc mult_commute])
    94 
    94 
    95 theorems ring_mult_ac = mult_assoc mult_commute mult_left_commute
    95 theorems ring_mult_ac = mult_assoc mult_commute mult_left_commute
    96 
    96 
    97 lemma right_inverse [simp]: "a \<noteq> 0 ==>  a * inverse (a::'a::field) = 1"
    97 lemma right_inverse [simp]: "a \<noteq> 0 ==>  a * inverse (a::'a::field) = 1"
    98 proof -
    98 proof -