Unbundled subrings (deprecated) #
This file is deprecated, and is no longer imported by anything in mathlib other than other deprecated files, and test files. You should not need to import it.
This file defines predicates for unbundled subrings. Instead of using this file, please use
subring
, defined in ring_theory.subring.basic
, for subrings of rings.
Main definitions #
is_subring (S : set R) : Prop
: the predicate that S
is the underlying set of a subring
of the ring R
. The bundled variant subring R
should be used in preference to this.
Tags #
is_subring
- to_is_add_subgroup : is_add_subgroup S
- to_is_submonoid : is_submonoid S
S
is a subring: a set containing 1 and closed under multiplication, addition and additive
inverse.
theorem
ring_hom.is_subring_preimage
{R : Type u}
{S : Type v}
[ring R]
[ring S]
(f : R →+* S)
{s : set S}
(hs : is_subring s) :
is_subring (⇑f ⁻¹' s)
theorem
ring_hom.is_subring_image
{R : Type u}
{S : Type v}
[ring R]
[ring S]
(f : R →+* S)
{s : set R}
(hs : is_subring s) :
is_subring (⇑f '' s)
theorem
ring_hom.is_subring_set_range
{R : Type u}
{S : Type v}
[ring R]
[ring S]
(f : R →+* S) :
is_subring (set.range ⇑f)
theorem
is_subring.inter
{R : Type u}
[ring R]
{S₁ S₂ : set R}
(hS₁ : is_subring S₁)
(hS₂ : is_subring S₂) :
is_subring (S₁ ∩ S₂)
theorem
is_subring.Inter
{R : Type u}
[ring R]
{ι : Sort u_1}
{S : ι → set R}
(h : ∀ (y : ι), is_subring (S y)) :
is_subring (set.Inter S)
theorem
is_subring_Union_of_directed
{R : Type u}
[ring R]
{ι : Type u_1}
[hι : nonempty ι]
{s : ι → set R}
(h : ∀ (i : ι), is_subring (s i))
(directed : ∀ (i j : ι), ∃ (k : ι), s i ⊆ s k ∧ s j ⊆ s k) :
is_subring (⋃ (i : ι), s i)
The smallest subring containing a given subset of a ring, considered as a set. This function
is deprecated; use subring.closure
.
Equations
@[protected]
theorem
ring.in_closure.rec_on
{R : Type u}
[ring R]
{s : set R}
{C : R → Prop}
{x : R}
(hx : x ∈ ring.closure s)
(h1 : C 1)
(hneg1 : C (-1))
(hs : ∀ (z : R), z ∈ s → ∀ (n : R), C n → C (z * n))
(ha : ∀ {x y : R}, C x → C y → C (x + y)) :
C x
theorem
ring.closure_subset
{R : Type u}
[ring R]
{s t : set R}
(ht : is_subring t) :
s ⊆ t → ring.closure s ⊆ t
theorem
ring.closure_subset_iff
{R : Type u}
[ring R]
{s t : set R}
(ht : is_subring t) :
ring.closure s ⊆ t ↔ s ⊆ t
theorem
ring.image_closure
{R : Type u}
[ring R]
{S : Type u_1}
[ring S]
(f : R →+* S)
(s : set R) :
⇑f '' ring.closure s = ring.closure (⇑f '' s)