Skip to content

Commit

Permalink
fix(ring_theory/ideal/basic): remove universe restriction (#10843)
Browse files Browse the repository at this point in the history
  • Loading branch information
eric-wieser committed Dec 16, 2021
1 parent 905d887 commit 601f2ab
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions src/ring_theory/ideal/basic.lean
Expand Up @@ -241,7 +241,7 @@ show S ≤ S ⊔ T, from le_sup_left
lemma mem_sup_right {S T : ideal R} : ∀ {x : R}, x ∈ T → x ∈ S ⊔ T :=
show T ≤ S ⊔ T, from le_sup_right

lemma mem_supr_of_mem {ι : Type*} {S : ι → ideal R} (i : ι) :
lemma mem_supr_of_mem {ι : Sort*} {S : ι → ideal R} (i : ι) :
∀ {x : R}, x ∈ S i → x ∈ supr S :=
show S i ≤ supr S, from le_supr _ _

Expand All @@ -255,7 +255,7 @@ theorem mem_Inf {s : set (ideal R)} {x : R} :

@[simp] lemma mem_inf {I J : ideal R} {x : R} : x ∈ I ⊓ J ↔ x ∈ I ∧ x ∈ J := iff.rfl

@[simp] lemma mem_infi {ι : Type*} {I : ι → ideal R} {x : R} : x ∈ infi I ↔ ∀ i, x ∈ I i :=
@[simp] lemma mem_infi {ι : Sort*} {I : ι → ideal R} {x : R} : x ∈ infi I ↔ ∀ i, x ∈ I i :=
submodule.mem_infi _

@[simp] lemma mem_bot {x : R} : x ∈ (⊥ : ideal R) ↔ x = 0 :=
Expand Down

0 comments on commit 601f2ab

Please sign in to comment.