Skip to content

Commit

Permalink
fix(*): adjust for changed lemmas
Browse files Browse the repository at this point in the history
  • Loading branch information
eric-wieser committed Oct 28, 2020
1 parent 986ed3c commit 7274502
Showing 1 changed file with 4 additions and 4 deletions.
8 changes: 4 additions & 4 deletions src/algebra/monoid_algebra.lean
Original file line number Diff line number Diff line change
Expand Up @@ -434,11 +434,11 @@ The `alg_hom` which maps from a grading of an algebra `A` back to that algebra.
-/
def sum_id {A : Type*} [comm_semiring k] [semiring A] [algebra k A] [monoid G] :
monoid_algebra A G →ₐ[k] A :=
lift_nc ⟨λ g, 1, by simp, λ a b, by simp⟩ (alg_hom.id k A) (by simp)
lift_nc_alg_hom (alg_hom.id k A) ⟨λ g, 1, by simp, λ a b, by simp⟩ (by simp)

lemma sum_id_apply {A : Type*} [comm_semiring k] [semiring A] [algebra k A] [monoid G] (g : monoid_algebra A G) :
sum_id k g = g.sum (λ _ gi, gi) :=
by simp [sum_id, lift_aux]
by simp [sum_id, lift_nc_alg_hom]

section
local attribute [reducible] monoid_algebra
Expand Down Expand Up @@ -870,11 +870,11 @@ The `alg_hom` which maps from a grading of an algebra `A` back to that algebra.
-/
def sum_id {A : Type*} [comm_semiring k] [semiring A] [algebra k A] [add_monoid G] :
add_monoid_algebra A G →ₐ[k] A :=
lift_aux ⟨λ g, 1, by simp, λ a b, by simp⟩ (alg_hom.id k A) (by simp)
lift_nc_alg_hom (alg_hom.id k A) ⟨λ g, 1, by simp, λ a b, by simp⟩ (by simp)

lemma sum_id_apply {A : Type*} [comm_semiring k] [semiring A] [algebra k A] [add_monoid G] (g : add_monoid_algebra A G) :
sum_id k g = g.sum (λ _ gi, gi) :=
by simp [sum_id, lift_aux]
by simp [sum_id, lift_nc_alg_hom]

section
local attribute [reducible] add_monoid_algebra
Expand Down

0 comments on commit 7274502

Please sign in to comment.