Skip to content

Commit

Permalink
feat: add a simp attribute to isUnit_iff_ne_zero (#11756)
Browse files Browse the repository at this point in the history
  • Loading branch information
edgarcosta committed Mar 29, 2024
1 parent 1c32311 commit 575260d
Show file tree
Hide file tree
Showing 2 changed files with 2 additions and 1 deletion.
2 changes: 1 addition & 1 deletion Mathlib/Algebra/Algebra/Quasispectrum.lean
Expand Up @@ -279,7 +279,7 @@ lemma quasispectrum_eq_spectrum_union_zero (R : Type*) {A : Type*} [Semifield R]
[Algebra R A] (a : A) : quasispectrum R a = spectrum R a ∪ {0} := by
convert quasispectrum_eq_spectrum_union R a
ext x
simpa using isUnit_iff_ne_zero |>.symm |> not_iff_not.mpr
simp

namespace Unitization

Expand Down
1 change: 1 addition & 0 deletions Mathlib/Algebra/GroupWithZero/Units/Basic.lean
Expand Up @@ -249,6 +249,7 @@ theorem IsUnit.mk0 (x : G₀) (hx : x ≠ 0) : IsUnit x :=
(Units.mk0 x hx).isUnit
#align is_unit.mk0 IsUnit.mk0

@[simp]
theorem isUnit_iff_ne_zero : IsUnit a ↔ a ≠ 0 :=
Units.exists_iff_ne_zero
#align is_unit_iff_ne_zero isUnit_iff_ne_zero
Expand Down

0 comments on commit 575260d

Please sign in to comment.