Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit a500c24

Browse files
authored
Update units.lean (#1938)
1 parent 50bbb8d commit a500c24

File tree

1 file changed

+2
-0
lines changed

1 file changed

+2
-0
lines changed

src/algebra/group/units.lean

Lines changed: 2 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -107,6 +107,8 @@ units.ext $ nat.eq_one_of_dvd_one ⟨u.inv, u.val_inv.symm⟩
107107
def units.mk_of_mul_eq_one [comm_monoid α] (a b : α) (hab : a * b = 1) : units α :=
108108
⟨a, b, hab, (mul_comm b a).trans hab⟩
109109

110+
@[simp] lemma units.coe_mk_of_mul_eq_one [comm_monoid α] {a b : α} (h : a * b = 1) :
111+
(units.mk_of_mul_eq_one a b h : α) = a := rfl
110112

111113
section monoid
112114
variables [monoid α] {a b c : α}

0 commit comments

Comments
 (0)