Documentation

Mathlib.Deprecated.Submonoid

Unbundled submonoids (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 submonoids. Instead of using this file, please use Submonoid G and AddSubmonoid A, defined in GroupTheory.Submonoid.Basic.

Main definitions #

IsAddSubmonoid (S : Set M) : the predicate that S is the underlying subset of an additive submonoid of M. The bundled variant AddSubmonoid M should be used in preference to this.

IsSubmonoid (S : Set M) : the predicate that S is the underlying subset of a submonoid of M. The bundled variant Submonoid M should be used in preference to this.

Tags #

Submonoid, Submonoids, IsSubmonoid

structure IsAddSubmonoid {A : Type u_2} [AddMonoid A] (s : Set A) :

s is an additive submonoid: a set containing 0 and closed under addition. Note that this structure is deprecated, and the bundled variant AddSubmonoid A should be preferred.

  • zero_mem : 0 s

    The proposition that s contains 0.

  • add_mem : ∀ {a b : A}, a sb sa + b s

    The proposition that s is closed under addition.

Instances For
    structure IsSubmonoid {M : Type u_1} [Monoid M] (s : Set M) :

    s is a submonoid: a set containing 1 and closed under multiplication. Note that this structure is deprecated, and the bundled variant Submonoid M should be preferred.

    • one_mem : 1 s

      The proposition that s contains 1.

    • mul_mem : ∀ {a b : M}, a sb sa * b s

      The proposition that s is closed under multiplication.

    Instances For
      theorem IsAddSubmonoid.inter {M : Type u_1} [AddMonoid M] {s₁ : Set M} {s₂ : Set M} (is₁ : IsAddSubmonoid s₁) (is₂ : IsAddSubmonoid s₂) :
      IsAddSubmonoid (s₁ s₂)

      The intersection of two AddSubmonoids of an AddMonoid M is an AddSubmonoid of M.

      theorem IsSubmonoid.inter {M : Type u_1} [Monoid M] {s₁ : Set M} {s₂ : Set M} (is₁ : IsSubmonoid s₁) (is₂ : IsSubmonoid s₂) :
      IsSubmonoid (s₁ s₂)

      The intersection of two submonoids of a monoid M is a submonoid of M.

      theorem IsAddSubmonoid.iInter {M : Type u_1} [AddMonoid M] {ι : Sort u_3} {s : ιSet M} (h : ∀ (y : ι), IsAddSubmonoid (s y)) :

      The intersection of an indexed set of AddSubmonoids of an AddMonoid M is an AddSubmonoid of M.

      theorem IsSubmonoid.iInter {M : Type u_1} [Monoid M] {ι : Sort u_3} {s : ιSet M} (h : ∀ (y : ι), IsSubmonoid (s y)) :

      The intersection of an indexed set of submonoids of a monoid M is a submonoid of M.

      abbrev isAddSubmonoid_iUnion_of_directed.match_3 {M : Type u_2} {ι : Type u_1} {s : ιSet M} :
      ∀ {b : M} (motive : (∃ (i : ι), b s i)Prop) (x : ∃ (i : ι), b s i), (∀ (j : ι) (hj : b s j), motive )motive x
      Equations
      • =
      Instances For
        abbrev isAddSubmonoid_iUnion_of_directed.match_2 {M : Type u_2} {ι : Type u_1} {s : ιSet M} (i : ι) (j : ι) (motive : (∃ (k : ι), s i s k s j s k)Prop) :
        ∀ (x : ∃ (k : ι), s i s k s j s k), (∀ (k : ι) (hk : s i s k s j s k), motive )motive x
        Equations
        • =
        Instances For
          abbrev isAddSubmonoid_iUnion_of_directed.match_1 {ι : Type u_1} (motive : Nonempty ιProp) :
          ∀ ( : Nonempty ι), (∀ (i : ι), motive )motive
          Equations
          • =
          Instances For
            theorem isAddSubmonoid_iUnion_of_directed {M : Type u_1} [AddMonoid M] {ι : Type u_3} [hι : Nonempty ι] {s : ιSet M} (hs : ∀ (i : ι), IsAddSubmonoid (s i)) (Directed : ∀ (i j : ι), ∃ (k : ι), s i s k s j s k) :
            IsAddSubmonoid (⋃ (i : ι), s i)

            The union of an indexed, directed, nonempty set of AddSubmonoids of an AddMonoid M is an AddSubmonoid of M.

            theorem isSubmonoid_iUnion_of_directed {M : Type u_1} [Monoid M] {ι : Type u_3} [hι : Nonempty ι] {s : ιSet M} (hs : ∀ (i : ι), IsSubmonoid (s i)) (Directed : ∀ (i j : ι), ∃ (k : ι), s i s k s j s k) :
            IsSubmonoid (⋃ (i : ι), s i)

            The union of an indexed, directed, nonempty set of submonoids of a monoid M is a submonoid of M.

            def multiples {M : Type u_1} [AddMonoid M] (x : M) :
            Set M

            The set of natural number multiples 0, x, 2x, ... of an element x of an AddMonoid.

            Equations
            Instances For
              def powers {M : Type u_1} [Monoid M] (x : M) :
              Set M

              The set of natural number powers 1, x, x², ... of an element x of a monoid.

              Equations
              Instances For
                theorem multiples.zero_mem {M : Type u_1} [AddMonoid M] {x : M} :

                0 is in the set of natural number multiples of an element of an AddMonoid.

                theorem powers.one_mem {M : Type u_1} [Monoid M] {x : M} :

                1 is in the set of natural number powers of an element of a monoid.

                theorem multiples.self_mem {M : Type u_1} [AddMonoid M] {x : M} :

                An element of an AddMonoid is in the set of that element's natural number multiples.

                theorem powers.self_mem {M : Type u_1} [Monoid M] {x : M} :

                An element of a monoid is in the set of that element's natural number powers.

                theorem multiples.add_mem {M : Type u_1} [AddMonoid M] {x : M} {y : M} {z : M} :
                y multiples xz multiples xy + z multiples x

                The set of natural number multiples of an element of an AddMonoid is closed under addition.

                abbrev multiples.add_mem.match_1 {M : Type u_1} [AddMonoid M] {x : M} {z : M} (motive : z multiples xProp) :
                ∀ (x_1 : z multiples x), (∀ (n₂ : ) (h₂ : n₂ x = z), motive )motive x_1
                Equations
                • =
                Instances For
                  theorem powers.mul_mem {M : Type u_1} [Monoid M] {x : M} {y : M} {z : M} :
                  y powers xz powers xy * z powers x

                  The set of natural number powers of an element of a monoid is closed under multiplication.

                  The set of natural number multiples of an element of an AddMonoid M is an AddSubmonoid of M.

                  theorem powers.isSubmonoid {M : Type u_1} [Monoid M] (x : M) :

                  The set of natural number powers of an element of a monoid M is a submonoid of M.

                  theorem Univ.isAddSubmonoid {M : Type u_1} [AddMonoid M] :

                  An AddMonoid is an AddSubmonoid of itself.

                  theorem Univ.isSubmonoid {M : Type u_1} [Monoid M] :
                  IsSubmonoid Set.univ

                  A monoid is a submonoid of itself.

                  theorem IsAddSubmonoid.preimage {M : Type u_1} [AddMonoid M] {N : Type u_3} [AddMonoid N] {f : MN} (hf : IsAddMonoidHom f) {s : Set N} (hs : IsAddSubmonoid s) :

                  The preimage of an AddSubmonoid under an AddMonoid hom is an AddSubmonoid of the domain.

                  theorem IsSubmonoid.preimage {M : Type u_1} [Monoid M] {N : Type u_3} [Monoid N] {f : MN} (hf : IsMonoidHom f) {s : Set N} (hs : IsSubmonoid s) :

                  The preimage of a submonoid under a monoid hom is a submonoid of the domain.

                  theorem IsAddSubmonoid.image {M : Type u_1} [AddMonoid M] {γ : Type u_3} [AddMonoid γ] {f : Mγ} (hf : IsAddMonoidHom f) {s : Set M} (hs : IsAddSubmonoid s) :

                  The image of an AddSubmonoid under an AddMonoid hom is an AddSubmonoid of the codomain.

                  abbrev IsAddSubmonoid.image.match_1 {M : Type u_2} {γ : Type u_1} {f : Mγ} {s : Set M} (b : γ) (motive : b f '' sProp) :
                  ∀ (x : b f '' s), (∀ (y : M) (hy : y s f y = b), motive )motive x
                  Equations
                  • =
                  Instances For
                    theorem IsSubmonoid.image {M : Type u_1} [Monoid M] {γ : Type u_3} [Monoid γ] {f : Mγ} (hf : IsMonoidHom f) {s : Set M} (hs : IsSubmonoid s) :

                    The image of a submonoid under a monoid hom is a submonoid of the codomain.

                    theorem Range.isAddSubmonoid {M : Type u_1} [AddMonoid M] {γ : Type u_3} [AddMonoid γ] {f : Mγ} (hf : IsAddMonoidHom f) :

                    The image of an AddMonoid hom is an AddSubmonoid of the codomain.

                    theorem Range.isSubmonoid {M : Type u_1} [Monoid M] {γ : Type u_3} [Monoid γ] {f : Mγ} (hf : IsMonoidHom f) :

                    The image of a monoid hom is a submonoid of the codomain.

                    abbrev IsAddSubmonoid.nsmul_mem.match_1 (motive : Prop) :
                    ∀ (x : ), (Unitmotive 0)(∀ (n : ), motive (Nat.succ n))motive x
                    Equations
                    • =
                    Instances For
                      theorem IsAddSubmonoid.nsmul_mem {M : Type u_1} [AddMonoid M] {s : Set M} {a : M} (hs : IsAddSubmonoid s) (h : a s) {n : } :
                      n a s

                      An AddSubmonoid is closed under multiplication by naturals.

                      theorem IsSubmonoid.pow_mem {M : Type u_1} [Monoid M] {s : Set M} {a : M} (hs : IsSubmonoid s) (h : a s) {n : } :
                      a ^ n s

                      Submonoids are closed under natural powers.

                      theorem IsAddSubmonoid.multiples_subset {M : Type u_1} [AddMonoid M] {s : Set M} {a : M} (hs : IsAddSubmonoid s) (h : a s) :

                      The set of natural number multiples of an element of an AddSubmonoid is a subset of the AddSubmonoid.

                      theorem IsSubmonoid.powers_subset {M : Type u_1} [Monoid M] {s : Set M} {a : M} (hs : IsSubmonoid s) (h : a s) :

                      The set of natural number powers of an element of a Submonoid is a subset of the Submonoid.

                      @[deprecated IsSubmonoid.powers_subset]
                      theorem IsSubmonoid.power_subset {M : Type u_1} [Monoid M] {s : Set M} {a : M} (hs : IsSubmonoid s) (h : a s) :

                      Alias of IsSubmonoid.powers_subset.


                      The set of natural number powers of an element of a Submonoid is a subset of the Submonoid.

                      theorem IsAddSubmonoid.list_sum_mem {M : Type u_1} [AddMonoid M] {s : Set M} (hs : IsAddSubmonoid s) {l : List M} :
                      (xl, x s)List.sum l s

                      The sum of a list of elements of an AddSubmonoid is an element of the AddSubmonoid.

                      abbrev IsAddSubmonoid.list_sum_mem.match_1 {M : Type u_1} {s : Set M} (motive : (x : List M) → (x_1x, x_1 s)Prop) :
                      ∀ (x : List M) (x_1 : x_1x, x_1 s), (∀ (x : x[], x s), motive [] x)(∀ (a : M) (l : List M) (h : xa :: l, x s), motive (a :: l) h)motive x x_1
                      Equations
                      • =
                      Instances For
                        theorem IsSubmonoid.list_prod_mem {M : Type u_1} [Monoid M] {s : Set M} (hs : IsSubmonoid s) {l : List M} :
                        (xl, x s)List.prod l s

                        The product of a list of elements of a submonoid is an element of the submonoid.

                        theorem IsAddSubmonoid.multiset_sum_mem {M : Type u_3} [AddCommMonoid M] {s : Set M} (hs : IsAddSubmonoid s) (m : Multiset M) :
                        (am, a s)Multiset.sum m s

                        The sum of a multiset of elements of an AddSubmonoid of an AddCommMonoid is an element of the AddSubmonoid.

                        theorem IsSubmonoid.multiset_prod_mem {M : Type u_3} [CommMonoid M] {s : Set M} (hs : IsSubmonoid s) (m : Multiset M) :
                        (am, a s)Multiset.prod m s

                        The product of a multiset of elements of a submonoid of a CommMonoid is an element of the submonoid.

                        abbrev IsAddSubmonoid.finset_sum_mem.match_1 {M : Type u_2} {A : Type u_1} {s : Set M} (f : AM) (motive : (x : Finset A) → (bx, f b s)Prop) :
                        ∀ (x : Finset A) (x_1 : bx, f b s), (∀ (m : Multiset A) (hm : Multiset.Nodup m) (x : b{ val := m, nodup := hm }, f b s), motive { val := m, nodup := hm } x)motive x x_1
                        Equations
                        • =
                        Instances For
                          theorem IsAddSubmonoid.finset_sum_mem {M : Type u_3} {A : Type u_4} [AddCommMonoid M] {s : Set M} (hs : IsAddSubmonoid s) (f : AM) (t : Finset A) :
                          (bt, f b s)(Finset.sum t fun (b : A) => f b) s

                          The sum of elements of an AddSubmonoid of an AddCommMonoid indexed by a Finset is an element of the AddSubmonoid.

                          theorem IsSubmonoid.finset_prod_mem {M : Type u_3} {A : Type u_4} [CommMonoid M] {s : Set M} (hs : IsSubmonoid s) (f : AM) (t : Finset A) :
                          (bt, f b s)(Finset.prod t fun (b : A) => f b) s

                          The product of elements of a submonoid of a CommMonoid indexed by a Finset is an element of the submonoid.

                          inductive AddMonoid.InClosure {A : Type u_2} [AddMonoid A] (s : Set A) :
                          AProp

                          The inductively defined membership predicate for the submonoid generated by a subset of a monoid.

                          Instances For
                            inductive Monoid.InClosure {M : Type u_1} [Monoid M] (s : Set M) :
                            MProp

                            The inductively defined membership predicate for the Submonoid generated by a subset of an monoid.

                            Instances For
                              def AddMonoid.Closure {M : Type u_1} [AddMonoid M] (s : Set M) :
                              Set M

                              The inductively defined AddSubmonoid generated by a subset of an AddMonoid.

                              Equations
                              Instances For
                                def Monoid.Closure {M : Type u_1} [Monoid M] (s : Set M) :
                                Set M

                                The inductively defined submonoid generated by a subset of a monoid.

                                Equations
                                Instances For
                                  theorem AddMonoid.subset_closure {M : Type u_1} [AddMonoid M] {s : Set M} :

                                  A subset of an AddMonoid is contained in the AddSubmonoid it generates.

                                  theorem Monoid.subset_closure {M : Type u_1} [Monoid M] {s : Set M} :

                                  A subset of a monoid is contained in the submonoid it generates.

                                  theorem AddMonoid.closure_subset {M : Type u_1} [AddMonoid M] {s : Set M} {t : Set M} (ht : IsAddSubmonoid t) (h : s t) :

                                  The AddSubmonoid generated by a set is contained in any AddSubmonoid that contains the set.

                                  theorem Monoid.closure_subset {M : Type u_1} [Monoid M] {s : Set M} {t : Set M} (ht : IsSubmonoid t) (h : s t) :

                                  The submonoid generated by a set is contained in any submonoid that contains the set.

                                  theorem AddMonoid.closure_mono {M : Type u_1} [AddMonoid M] {s : Set M} {t : Set M} (h : s t) :

                                  Given subsets t and s of an AddMonoid M, if s ⊆ t, the AddSubmonoid of M generated by s is contained in the AddSubmonoid generated by t.

                                  theorem Monoid.closure_mono {M : Type u_1} [Monoid M] {s : Set M} {t : Set M} (h : s t) :

                                  Given subsets t and s of a monoid M, if s ⊆ t, the submonoid of M generated by s is contained in the submonoid generated by t.

                                  The AddSubmonoid generated by an element of an AddMonoid equals the set of natural number multiples of the element.

                                  theorem Monoid.closure_singleton {M : Type u_1} [Monoid M] {x : M} :

                                  The submonoid generated by an element of a monoid equals the set of natural number powers of the element.

                                  theorem AddMonoid.image_closure {M : Type u_1} [AddMonoid M] {A : Type u_3} [AddMonoid A] {f : MA} (hf : IsAddMonoidHom f) (s : Set M) :

                                  The image under an AddMonoid hom of the AddSubmonoid generated by a set equals the AddSubmonoid generated by the image of the set under the AddMonoid hom.

                                  theorem Monoid.image_closure {M : Type u_1} [Monoid M] {A : Type u_3} [Monoid A] {f : MA} (hf : IsMonoidHom f) (s : Set M) :

                                  The image under a monoid hom of the submonoid generated by a set equals the submonoid generated by the image of the set under the monoid hom.

                                  theorem AddMonoid.exists_list_of_mem_closure {M : Type u_1} [AddMonoid M] {s : Set M} {a : M} (h : a AddMonoid.Closure s) :
                                  ∃ (l : List M), (xl, x s) List.sum l = a

                                  Given an element a of the AddSubmonoid of an AddMonoid M generated by a set s, there exists a list of elements of s whose sum is a.

                                  theorem Monoid.exists_list_of_mem_closure {M : Type u_1} [Monoid M] {s : Set M} {a : M} (h : a Monoid.Closure s) :
                                  ∃ (l : List M), (xl, x s) List.prod l = a

                                  Given an element a of the submonoid of a monoid M generated by a set s, there exists a list of elements of s whose product is a.

                                  abbrev AddMonoid.mem_closure_union_iff.match_1 {M : Type u_1} [AddCommMonoid M] {s : Set M} {t : Set M} (tl : List M) (motive : (∃ y ∈ AddMonoid.Closure s, ∃ z ∈ AddMonoid.Closure t, y + z = List.sum tl)Prop) :
                                  ∀ (x : ∃ y ∈ AddMonoid.Closure s, ∃ z ∈ AddMonoid.Closure t, y + z = List.sum tl), (∀ (y : M) (hy : y AddMonoid.Closure s) (z : M) (hz : z AddMonoid.Closure t) (hyzx : y + z = List.sum tl), motive )motive x
                                  Equations
                                  • =
                                  Instances For
                                    abbrev AddMonoid.mem_closure_union_iff.match_3 {M : Type u_1} [AddCommMonoid M] {s : Set M} {t : Set M} {x : M} (motive : (∃ y ∈ AddMonoid.Closure s, ∃ z ∈ AddMonoid.Closure t, y + z = x)Prop) :
                                    ∀ (x_1 : ∃ y ∈ AddMonoid.Closure s, ∃ z ∈ AddMonoid.Closure t, y + z = x), (∀ (y : M) (hy : y AddMonoid.Closure s) (z : M) (hz : z AddMonoid.Closure t) (hyzx : y + z = x), motive )motive x_1
                                    Equations
                                    • =
                                    Instances For
                                      abbrev AddMonoid.mem_closure_union_iff.match_2 {M : Type u_1} [AddCommMonoid M] {s : Set M} {t : Set M} {x : M} (motive : (∃ (l : List M), (xl, x s t) List.sum l = x)Prop) :
                                      ∀ (x_1 : ∃ (l : List M), (xl, x s t) List.sum l = x), (∀ (L : List M) (HL1 : xL, x s t) (HL2 : List.sum L = x), motive )motive x_1
                                      Equations
                                      • =
                                      Instances For
                                        theorem AddMonoid.mem_closure_union_iff {M : Type u_3} [AddCommMonoid M] {s : Set M} {t : Set M} {x : M} :
                                        x AddMonoid.Closure (s t) ∃ y ∈ AddMonoid.Closure s, ∃ z ∈ AddMonoid.Closure t, y + z = x

                                        Given sets s, t of a commutative AddMonoid M, x ∈ M is in the AddSubmonoid of M generated by s ∪ t iff there exists an element of the AddSubmonoid generated by s and an element of the AddSubmonoid generated by t whose sum is x.

                                        theorem Monoid.mem_closure_union_iff {M : Type u_3} [CommMonoid M] {s : Set M} {t : Set M} {x : M} :
                                        x Monoid.Closure (s t) ∃ y ∈ Monoid.Closure s, ∃ z ∈ Monoid.Closure t, y * z = x

                                        Given sets s, t of a commutative monoid M, x ∈ M is in the submonoid of M generated by s ∪ t iff there exists an element of the submonoid generated by s and an element of the submonoid generated by t whose product is x.

                                        def AddSubmonoid.of {M : Type u_1} [AddMonoid M] {s : Set M} (h : IsAddSubmonoid s) :

                                        Create a bundled additive submonoid from a set s and [IsAddSubmonoid s].

                                        Equations
                                        • AddSubmonoid.of h = { toAddSubsemigroup := { carrier := s, add_mem' := }, zero_mem' := }
                                        Instances For
                                          def Submonoid.of {M : Type u_1} [Monoid M] {s : Set M} (h : IsSubmonoid s) :

                                          Create a bundled submonoid from a set s and [IsSubmonoid s].

                                          Equations
                                          • Submonoid.of h = { toSubsemigroup := { carrier := s, mul_mem' := }, one_mem' := }
                                          Instances For
                                            theorem Submonoid.isSubmonoid {M : Type u_1} [Monoid M] (S : Submonoid M) :