Skip to content

Commit

Permalink
feat(ring_theory/graded_algebra): definitions and basic operations of…
Browse files Browse the repository at this point in the history
… homogeneous ideal (#10784)

This defines homogeneous ideals (`homogeneous_ideal`) of a graded algebra.



Co-authored-by: jjaassoonn <jujian.zhang1998@out.com>
Co-authored-by: Eric Wieser <wieser.eric@gmail.com>
  • Loading branch information
3 people committed Feb 23, 2022
1 parent e167efa commit 0d5bed0
Show file tree
Hide file tree
Showing 3 changed files with 489 additions and 0 deletions.
4 changes: 4 additions & 0 deletions src/algebra/graded_monoid.lean
Expand Up @@ -518,6 +518,10 @@ variables {R S : Type*} [set_like S R]
/-- An element `a : R` is said to be homogeneous if there is some `i : ι` such that `a ∈ A i`. -/
def set_like.is_homogeneous (A : ι → S) (a : R) : Prop := ∃ i, a ∈ A i

@[simp] lemma set_like.is_homogeneous_coe {A : ι → S} {i} (x : A i) :
set_like.is_homogeneous A (x : R) :=
⟨i, x.prop⟩

lemma set_like.is_homogeneous_one [has_zero ι] [has_one R]
(A : ι → S) [set_like.has_graded_one A] : set_like.is_homogeneous A (1 : R) :=
0, set_like.has_graded_one.one_mem⟩
Expand Down

0 comments on commit 0d5bed0

Please sign in to comment.