Documentation

Mathlib.Algebra.Category.ModuleCat.Simple

Simple objects in the category of R-modules #

We prove simple modules are exactly simple objects in the category of R-modules.

A simple module is a simple object in the category of modules.

Equations
  • =

A simple object in the category of modules is a simple module.

Equations
  • =
theorem simple_of_finrank_eq_one {R : Type u_1} [Ring R] {k : Type u_3} [Field k] [Algebra k R] {V : ModuleCat R} (h : FiniteDimensional.finrank k V = 1) :

Any k-algebra module which is 1-dimensional over k is simple.