lean2/tests/lean/run/rewrite5.lean

9 lines
175 B
Text
Raw Normal View History

import algebra.group
variable {A : Type}
variable [s : group A]
include s
theorem mul.right_inv₁ (a : A) : a * a⁻¹ = 1 :=
by rewrite [-{a}inv_inv at {1}, mul.left_inv]