Skip to content

Commit

Permalink
feat(linear_algebra/basic): define algebra structure on endomorphisms…
Browse files Browse the repository at this point in the history
… of module (leanprover-community#1618)

* feat(linear_algebra/basic): define algebra structure on endomorphisms of module

* Update algebra.lean
  • Loading branch information
Oliver Nash authored and anrddh committed May 15, 2020
1 parent 59ae66f commit aef258a
Showing 1 changed file with 7 additions and 0 deletions.
7 changes: 7 additions & 0 deletions src/ring_theory/algebra.lean
Original file line number Diff line number Diff line change
Expand Up @@ -146,6 +146,13 @@ variables {R A}

end algebra

instance module.endomorphism_algebra (R : Type u) (M : Type v)
[comm_ring R] [add_comm_group M] [module R M] : algebra R (M →ₗ[R] M) :=
{ to_fun := (λ r, r • linear_map.id),
hom := by apply is_ring_hom.mk; intros; ext; simp [mul_smul, add_smul],
commutes' := by intros; ext; simp,
smul_def' := by intros; ext; simp }

set_option old_structure_cmd true
/-- Defining the homomorphism in the category R-Alg. -/
structure alg_hom (R : Type u) (A : Type v) (B : Type w)
Expand Down

0 comments on commit aef258a

Please sign in to comment.