Skip to content

Commit

Permalink
Update Basic.lean
Browse files Browse the repository at this point in the history
  • Loading branch information
eric-wieser authored Jan 24, 2024
1 parent 2c2a1ce commit 640e2db
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Mathlib/Algebra/Group/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -471,7 +471,7 @@ theorem one_div_one_div : 1 / (1 / a) = a := by simp
#align one_div_one_div one_div_one_div
#align zero_sub_zero_sub zero_sub_zero_sub

@[to_additive (attr := simp)]
@[to_additive]
theorem div_eq_div_iff_comm : a / b = c / d ↔ b / a = d / c :=
inv_inj.symm.trans <| by simp only [inv_div]

Expand Down

0 comments on commit 640e2db

Please sign in to comment.