Skip to content

Commit

Permalink
feat: DirectSum.toAddMonoid is injective (#9385)
Browse files Browse the repository at this point in the history
From LeanAPAP
  • Loading branch information
YaelDillies committed Jan 10, 2024
1 parent d819f3c commit b271734
Showing 1 changed file with 8 additions and 1 deletion.
9 changes: 8 additions & 1 deletion Mathlib/Algebra/DirectSum/Basic.lean
Expand Up @@ -23,7 +23,8 @@ This notation is in the `DirectSum` locale, accessible after `open DirectSum`.
* https://en.wikipedia.org/wiki/Direct_sum
-/

open BigOperators
open Function
open scoped BigOperators

universe u v w u₁

Expand Down Expand Up @@ -213,6 +214,12 @@ theorem toAddMonoid.unique (f : ⨁ i, β i) : ψ f = toAddMonoid (fun i => ψ.c
simp [toAddMonoid, of]
#align direct_sum.to_add_monoid.unique DirectSum.toAddMonoid.unique

lemma toAddMonoid_injective : Injective (toAddMonoid : (∀ i, β i →+ γ) → (⨁ i, β i) →+ γ) :=
DFinsupp.liftAddHom.injective

@[simp] lemma toAddMonoid_inj {f g : ∀ i, β i →+ γ} : toAddMonoid f = toAddMonoid g ↔ f = g :=
toAddMonoid_injective.eq_iff

end ToAddMonoid

section FromAddMonoid
Expand Down

0 comments on commit b271734

Please sign in to comment.