Unbundled subgroups (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 unbundled multiplicative and additive subgroups. Instead of using this file,
please use Subgroup G
and AddSubgroup A
, defined in GroupTheory.Subgroup.Basic
.
Main definitions #
IsAddSubgroup (S : Set A)
: the predicate that S
is the underlying subset of an additive
subgroup of A
. The bundled variant AddSubgroup A
should be used in preference to this.
IsSubgroup (S : Set G)
: the predicate that S
is the underlying subset of a subgroup
of G
. The bundled variant Subgroup G
should be used in preference to this.
Tags #
subgroup, subgroups, IsSubgroup
- zero_mem : 0 ∈ s✝
The proposition that
s
is closed under negation.
s
is an additive subgroup: a set containing 0 and closed under addition and negation.
Instances For
- one_mem : 1 ∈ s✝
The proposition that
s
is closed under inverse.
s
is a subgroup: a set containing 1 and closed under multiplication and inverse.
Instances For
- zero_mem : 0 ∈ s✝
The proposition that
s
is closed under (additive) conjugation.
IsNormalAddSubgroup (s : Set A)
expresses the fact that s
is a normal additive subgroup
of the additive group A
. Important: the preferred way to say this in Lean is via bundled
subgroups S : AddSubgroup A
and hs : S.normal
, and not via this structure.
Instances For
- one_mem : 1 ∈ s✝
The proposition that
s
is closed under conjugation.
IsNormalSubgroup (s : Set G)
expresses the fact that s
is a normal subgroup
of the group G
. Important: the preferred way to say this in Lean is via bundled
subgroups S : Subgroup G
and not via this structure.
Instances For
the trivial additive subgroup
Instances For
The underlying set of the center of an additive group.
Instances For
The underlying set of the center of a group.
Instances For
- basic: ∀ {A : Type u_3} [inst : AddGroup A] {s : Set A} {a : A}, a ∈ s → AddGroup.InClosure s a
- zero: ∀ {A : Type u_3} [inst : AddGroup A] {s : Set A}, AddGroup.InClosure s 0
- neg: ∀ {A : Type u_3} [inst : AddGroup A] {s : Set A} {a : A}, AddGroup.InClosure s a → AddGroup.InClosure s (-a)
- add: ∀ {A : Type u_3} [inst : AddGroup A] {s : Set A} {a b : A}, AddGroup.InClosure s a → AddGroup.InClosure s b → AddGroup.InClosure s (a + b)
If A
is an additive group and s : Set A
, then InClosure s : Set A
is the underlying
subset of the subgroup generated by s
.
Instances For
- basic: ∀ {G : Type u_1} [inst : Group G] {s : Set G} {a : G}, a ∈ s → Group.InClosure s a
- one: ∀ {G : Type u_1} [inst : Group G] {s : Set G}, Group.InClosure s 1
- inv: ∀ {G : Type u_1} [inst : Group G] {s : Set G} {a : G}, Group.InClosure s a → Group.InClosure s a⁻¹
- mul: ∀ {G : Type u_1} [inst : Group G] {s : Set G} {a b : G}, Group.InClosure s a → Group.InClosure s b → Group.InClosure s (a * b)
If G
is a group and s : Set G
, then InClosure s : Set G
is the underlying
subset of the subgroup generated by s
.
Instances For
AddGroup.closure s
is the additive subgroup generated by s
, i.e., the
smallest additive subgroup containing s
.
Instances For
Group.closure s
is the subgroup generated by s
, i.e. the smallest subgroup containing s
.
Instances For
Instances For
The normal closure of a set is a subgroup.
The normal closure of s is a normal subgroup.
The normal closure of s is the smallest normal subgroup containing s.
Create a bundled additive subgroup from a set s
and [IsAddSubgroup s]
.
Instances For
Create a bundled subgroup from a set s
and [IsSubgroup s]
.