Skip to content

Commit

Permalink
whitespace
Browse files Browse the repository at this point in the history
  • Loading branch information
eric-wieser committed Jan 24, 2024
1 parent 6c7feff commit 2c2a1ce
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions Mathlib/Algebra/GroupWithZero/Units/Lemmas.lean
Original file line number Diff line number Diff line change
Expand Up @@ -198,8 +198,8 @@ theorem div_eq_div_iff (hb : b ≠ 0) (hd : d ≠ 0) : a / b = c / d ↔ a * d =

/-- The `CommGroupWithZero` version of `div_eq_div_iff_div_eq_div`. -/
theorem div_eq_div_iff_div_eq_div' (hb : b ≠ 0) (hc : c ≠ 0) : a / b = c / d ↔ a / c = b / d := by
conv_lhs => rw [←mul_left_inj' hb, div_mul_cancel _ hb]
conv_rhs => rw [←mul_left_inj' hc, div_mul_cancel _ hc]
conv_lhs => rw [← mul_left_inj' hb, div_mul_cancel _ hb]
conv_rhs => rw [← mul_left_inj' hc, div_mul_cancel _ hc]
rw [mul_comm _ c, div_mul_eq_mul_div, mul_div_assoc]

theorem div_div_cancel' (ha : a ≠ 0) : a / (a / b) = b :=
Expand Down

0 comments on commit 2c2a1ce

Please sign in to comment.