Skip to content

Commit

Permalink
Update Mathlib/Data/Sign.lean
Browse files Browse the repository at this point in the history
Co-authored-by: Eric Wieser <[email protected]>
  • Loading branch information
madvorak and eric-wieser authored Jan 3, 2025
1 parent cc712ea commit 044e56e
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Mathlib/Data/Sign.lean
Original file line number Diff line number Diff line change
Expand Up @@ -434,7 +434,7 @@ theorem sign_pow (x : α) (n : ℕ) : sign (x ^ n) = sign x ^ n := map_pow signH
lemma zero_mem_setRange_signTypeCast : (0 : α) ∈ Set.range SignType.cast :=
0, rfl⟩

lemma in_set_range_singType_cast_mul_in_set_range_singType_cast {a b : α}
lemma mul_mem_setRange_signTypeCast {a b : α}
(ha : a ∈ Set.range SignType.cast) (hb : b ∈ Set.range SignType.cast) :
a * b ∈ Set.range SignType.cast := by
obtain ⟨a', rfl⟩ := ha
Expand Down

0 comments on commit 044e56e

Please sign in to comment.