![]() |
Metamath
Proof Explorer Theorem List (p. 467 of 479) | < Previous Next > |
Bad symbols? Try the
GIF version. |
||
Mirrors > Metamath Home Page > MPE Home Page > Theorem List Contents > Recent Proofs This page: Page List |
Color key: | ![]() (1-30166) |
![]() (30167-31689) |
![]() (31690-47842) |
Type | Label | Description |
---|---|---|
Statement | ||
Definition | df-assintop 46601* | Function mapping a set to the class of all associative (closed internal binary) operations for this set, see definition 5 in [BourbakiAlg1] p. 4, where it is called "an associative law of composition". (Contributed by AV, 20-Jan-2020.) |
β’ assIntOp = (π β V β¦ {π β ( clIntOp βπ) β£ π assLaw π}) | ||
Theorem | intopval 46602 | The internal (binary) operations for a set. (Contributed by AV, 20-Jan-2020.) |
β’ ((π β π β§ π β π) β (π intOp π) = (π βm (π Γ π))) | ||
Theorem | intop 46603 | An internal (binary) operation for a set. (Contributed by AV, 20-Jan-2020.) |
β’ ( β¬ β (π intOp π) β β¬ :(π Γ π)βΆπ) | ||
Theorem | clintopval 46604 | The closed (internal binary) operations for a set. (Contributed by AV, 20-Jan-2020.) |
β’ (π β π β ( clIntOp βπ) = (π βm (π Γ π))) | ||
Theorem | assintopval 46605* | The associative (closed internal binary) operations for a set. (Contributed by AV, 20-Jan-2020.) |
β’ (π β π β ( assIntOp βπ) = {π β ( clIntOp βπ) β£ π assLaw π}) | ||
Theorem | assintopmap 46606* | The associative (closed internal binary) operations for a set, expressed with set exponentiation. (Contributed by AV, 20-Jan-2020.) |
β’ (π β π β ( assIntOp βπ) = {π β (π βm (π Γ π)) β£ π assLaw π}) | ||
Theorem | isclintop 46607 | The predicate "is a closed (internal binary) operations for a set". (Contributed by FL, 2-Nov-2009.) (Revised by AV, 20-Jan-2020.) |
β’ (π β π β ( β¬ β ( clIntOp βπ) β β¬ :(π Γ π)βΆπ)) | ||
Theorem | clintop 46608 | A closed (internal binary) operation for a set. (Contributed by AV, 20-Jan-2020.) |
β’ ( β¬ β ( clIntOp βπ) β β¬ :(π Γ π)βΆπ) | ||
Theorem | assintop 46609 | An associative (closed internal binary) operation for a set. (Contributed by AV, 20-Jan-2020.) |
β’ ( β¬ β ( assIntOp βπ) β ( β¬ :(π Γ π)βΆπ β§ β¬ assLaw π)) | ||
Theorem | isassintop 46610* | The predicate "is an associative (closed internal binary) operations for a set". (Contributed by FL, 2-Nov-2009.) (Revised by AV, 20-Jan-2020.) |
β’ (π β π β ( β¬ β ( assIntOp βπ) β ( β¬ :(π Γ π)βΆπ β§ βπ₯ β π βπ¦ β π βπ§ β π ((π₯ β¬ π¦) β¬ π§) = (π₯ β¬ (π¦ β¬ π§))))) | ||
Theorem | clintopcllaw 46611 | The closure law holds for a closed (internal binary) operation for a set. (Contributed by AV, 20-Jan-2020.) |
β’ ( β¬ β ( clIntOp βπ) β β¬ clLaw π) | ||
Theorem | assintopcllaw 46612 | The closure low holds for an associative (closed internal binary) operation for a set. (Contributed by FL, 2-Nov-2009.) (Revised by AV, 20-Jan-2020.) |
β’ ( β¬ β ( assIntOp βπ) β β¬ clLaw π) | ||
Theorem | assintopasslaw 46613 | The associative low holds for a associative (closed internal binary) operation for a set. (Contributed by FL, 2-Nov-2009.) (Revised by AV, 20-Jan-2020.) |
β’ ( β¬ β ( assIntOp βπ) β β¬ assLaw π) | ||
Theorem | assintopass 46614* | An associative (closed internal binary) operation for a set is associative. (Contributed by FL, 2-Nov-2009.) (Revised by AV, 20-Jan-2020.) |
β’ ( β¬ β ( assIntOp βπ) β βπ₯ β π βπ¦ β π βπ§ β π ((π₯ β¬ π¦) β¬ π§) = (π₯ β¬ (π¦ β¬ π§))) | ||
Syntax | cmgm2 46615 | Extend class notation with class of all magmas. |
class MgmALT | ||
Syntax | ccmgm2 46616 | Extend class notation with class of all commutative magmas. |
class CMgmALT | ||
Syntax | csgrp2 46617 | Extend class notation with class of all semigroups. |
class SGrpALT | ||
Syntax | ccsgrp2 46618 | Extend class notation with class of all commutative semigroups. |
class CSGrpALT | ||
Definition | df-mgm2 46619 | A magma is a set equipped with a closed operation. Definition 1 of [BourbakiAlg1] p. 1, or definition of a groupoid in section I.1 of [Bruck] p. 1. Note: The term "groupoid" is now widely used to refer to other objects: (small) categories all of whose morphisms are invertible, or groups with a partial function replacing the binary operation. Therefore, we will only use the term "magma" for the present notion in set.mm. (Contributed by AV, 6-Jan-2020.) |
β’ MgmALT = {π β£ (+gβπ) clLaw (Baseβπ)} | ||
Definition | df-cmgm2 46620 | A commutative magma is a magma with a commutative operation. Definition 8 of [BourbakiAlg1] p. 7. (Contributed by AV, 20-Jan-2020.) |
β’ CMgmALT = {π β MgmALT β£ (+gβπ) comLaw (Baseβπ)} | ||
Definition | df-sgrp2 46621 | A semigroup is a magma with an associative operation. Definition in section II.1 of [Bruck] p. 23, or of an "associative magma" in definition 5 of [BourbakiAlg1] p. 4, or of a semigroup in section 1.3 of [Hall] p. 7. (Contributed by AV, 6-Jan-2020.) |
β’ SGrpALT = {π β MgmALT β£ (+gβπ) assLaw (Baseβπ)} | ||
Definition | df-csgrp2 46622 | A commutative semigroup is a semigroup with a commutative operation. (Contributed by AV, 20-Jan-2020.) |
β’ CSGrpALT = {π β SGrpALT β£ (+gβπ) comLaw (Baseβπ)} | ||
Theorem | ismgmALT 46623 | The predicate "is a magma". (Contributed by AV, 16-Jan-2020.) (New usage is discouraged.) (Proof modification is discouraged.) |
β’ π΅ = (Baseβπ) & β’ β¬ = (+gβπ) β β’ (π β π β (π β MgmALT β β¬ clLaw π΅)) | ||
Theorem | iscmgmALT 46624 | The predicate "is a commutative magma". (Contributed by AV, 20-Jan-2020.) (New usage is discouraged.) (Proof modification is discouraged.) |
β’ π΅ = (Baseβπ) & β’ β¬ = (+gβπ) β β’ (π β CMgmALT β (π β MgmALT β§ β¬ comLaw π΅)) | ||
Theorem | issgrpALT 46625 | The predicate "is a semigroup". (Contributed by AV, 16-Jan-2020.) (New usage is discouraged.) (Proof modification is discouraged.) |
β’ π΅ = (Baseβπ) & β’ β¬ = (+gβπ) β β’ (π β SGrpALT β (π β MgmALT β§ β¬ assLaw π΅)) | ||
Theorem | iscsgrpALT 46626 | The predicate "is a commutative semigroup". (Contributed by AV, 20-Jan-2020.) (New usage is discouraged.) (Proof modification is discouraged.) |
β’ π΅ = (Baseβπ) & β’ β¬ = (+gβπ) β β’ (π β CSGrpALT β (π β SGrpALT β§ β¬ comLaw π΅)) | ||
Theorem | mgm2mgm 46627 | Equivalence of the two definitions of a magma. (Contributed by AV, 16-Jan-2020.) |
β’ (π β MgmALT β π β Mgm) | ||
Theorem | sgrp2sgrp 46628 | Equivalence of the two definitions of a semigroup. (Contributed by AV, 16-Jan-2020.) |
β’ (π β SGrpALT β π β Smgrp) | ||
Theorem | idfusubc0 46629* | The identity functor for a subcategory is an "inclusion functor" from the subcategory into its supercategory. (Contributed by AV, 29-Mar-2020.) |
β’ π = (πΆ βΎcat π½) & β’ πΌ = (idfuncβπ) & β’ π΅ = (Baseβπ) β β’ (π½ β (SubcatβπΆ) β πΌ = β¨( I βΎ π΅), (π₯ β π΅, π¦ β π΅ β¦ ( I βΎ (π₯(Hom βπ)π¦)))β©) | ||
Theorem | idfusubc 46630* | The identity functor for a subcategory is an "inclusion functor" from the subcategory into its supercategory. (Contributed by AV, 29-Mar-2020.) |
β’ π = (πΆ βΎcat π½) & β’ πΌ = (idfuncβπ) & β’ π΅ = (Baseβπ) β β’ (π½ β (SubcatβπΆ) β πΌ = β¨( I βΎ π΅), (π₯ β π΅, π¦ β π΅ β¦ ( I βΎ (π₯π½π¦)))β©) | ||
Theorem | inclfusubc 46631* | The "inclusion functor" from a subcategory of a category into the category itself. (Contributed by AV, 30-Mar-2020.) |
β’ (π β π½ β (SubcatβπΆ)) & β’ π = (πΆ βΎcat π½) & β’ π΅ = (Baseβπ) & β’ (π β πΉ = ( I βΎ π΅)) & β’ (π β πΊ = (π₯ β π΅, π¦ β π΅ β¦ ( I βΎ (π₯π½π¦)))) β β’ (π β πΉ(π Func πΆ)πΊ) | ||
Theorem | lmod0rng 46632 | If the scalar ring of a module is the zero ring, the module is the zero module, i.e. the base set of the module is the singleton consisting of the identity element only. (Contributed by AV, 17-Apr-2019.) |
β’ ((π β LMod β§ Β¬ (Scalarβπ) β NzRing) β (Baseβπ) = {(0gβπ)}) | ||
Theorem | nzrneg1ne0 46633 | The additive inverse of the 1 in a nonzero ring is not zero ( -1 =/= 0 ). (Contributed by AV, 29-Apr-2019.) |
β’ (π β NzRing β ((invgβπ )β(1rβπ )) β (0gβπ )) | ||
Theorem | 0ringdif 46634 | A zero ring is a ring which is not a nonzero ring. (Contributed by AV, 17-Apr-2020.) |
β’ π΅ = (Baseβπ ) & β’ 0 = (0gβπ ) β β’ (π β (Ring β NzRing) β (π β Ring β§ π΅ = { 0 })) | ||
Theorem | 0ringbas 46635 | The base set of a zero ring, a ring which is not a nonzero ring, is the singleton of the zero element. (Contributed by AV, 17-Apr-2020.) |
β’ π΅ = (Baseβπ ) & β’ 0 = (0gβπ ) β β’ (π β (Ring β NzRing) β π΅ = { 0 }) | ||
Theorem | 0ring1eq0 46636 | In a zero ring, a ring which is not a nonzero ring, the ring unity equals the zero element. (Contributed by AV, 17-Apr-2020.) |
β’ π΅ = (Baseβπ ) & β’ 0 = (0gβπ ) & β’ 1 = (1rβπ ) β β’ (π β (Ring β NzRing) β 1 = 0 ) | ||
Theorem | nrhmzr 46637 | There is no ring homomorphism from the zero ring into a nonzero ring. (Contributed by AV, 18-Apr-2020.) |
β’ ((π β (Ring β NzRing) β§ π β NzRing) β (π RingHom π ) = β ) | ||
According to Wikipedia, "... in abstract algebra, a rng (or pseudo-ring or non-unital ring) is an algebraic structure satisfying the same properties as a [unital] ring, without assuming the existence of a multiplicative identity. The term "rng" (pronounced rung) is meant to suggest that it is a "ring" without "i", i.e. without the requirement for an "identity element"." (see https://en.wikipedia.org/wiki/Rng_(algebra), 6-Jan-2020). | ||
Syntax | crng 46638 | Extend class notation with class of all non-unital rings. |
class Rng | ||
Definition | df-rng 46639* | Define class of all non-unital rings. A non-unital ring (or rng, or pseudoring) is a set equipped with two everywhere-defined internal operations, whose first one is an additive abelian group operation and the second one is a multiplicative semigroup operation, and where the addition is left- and right-distributive for the multiplication. Definition of a pseudo-ring in section I.8.1 of [BourbakiAlg1] p. 93 or the definition of a ring in part Preliminaries of [Roman] p. 18. As almost always in mathematics, "non-unital" means "not necessarily unital". Therefore, by talking about a ring (in general) or a non-unital ring the "unital" case is always included. In contrast to a unital ring, the commutativity of addition must be postulated and cannot be proven from the other conditions. (Contributed by AV, 6-Jan-2020.) |
β’ Rng = {π β Abel β£ ((mulGrpβπ) β Smgrp β§ [(Baseβπ) / π][(+gβπ) / π][(.rβπ) / π‘]βπ₯ β π βπ¦ β π βπ§ β π ((π₯π‘(π¦ππ§)) = ((π₯π‘π¦)π(π₯π‘π§)) β§ ((π₯ππ¦)π‘π§) = ((π₯π‘π§)π(π¦π‘π§))))} | ||
Theorem | isrng 46640* | The predicate "is a non-unital ring." (Contributed by AV, 6-Jan-2020.) |
β’ π΅ = (Baseβπ ) & β’ πΊ = (mulGrpβπ ) & β’ + = (+gβπ ) & β’ Β· = (.rβπ ) β β’ (π β Rng β (π β Abel β§ πΊ β Smgrp β§ βπ₯ β π΅ βπ¦ β π΅ βπ§ β π΅ ((π₯ Β· (π¦ + π§)) = ((π₯ Β· π¦) + (π₯ Β· π§)) β§ ((π₯ + π¦) Β· π§) = ((π₯ Β· π§) + (π¦ Β· π§))))) | ||
Theorem | rngabl 46641 | A non-unital ring is an (additive) abelian group. (Contributed by AV, 17-Feb-2020.) |
β’ (π β Rng β π β Abel) | ||
Theorem | rngmgp 46642 | A non-unital ring is a semigroup under multiplication. (Contributed by AV, 17-Feb-2020.) |
β’ πΊ = (mulGrpβπ ) β β’ (π β Rng β πΊ β Smgrp) | ||
Theorem | rngmgpf 46643 | Restricted functionality of the multiplicative group on non-unital rings (mgpf 20070 analog). (Contributed by AV, 22-Feb-2025.) |
β’ (mulGrp βΎ Rng):RngβΆSmgrp | ||
Theorem | rnggrp 46644 | A non-unital ring is a (additive) group. (Contributed by AV, 16-Feb-2025.) |
β’ (π β Rng β π β Grp) | ||
Theorem | ringrng 46645 | A unital ring is a non-unital ring. (Contributed by AV, 6-Jan-2020.) |
β’ (π β Ring β π β Rng) | ||
Theorem | ringssrng 46646 | The unital rings are non-unital rings. (Contributed by AV, 20-Mar-2020.) |
β’ Ring β Rng | ||
Theorem | isringrng 46647* | The predicate "is a unital ring" as extension of the predicate "is a non-unital ring". (Contributed by AV, 17-Feb-2020.) |
β’ π΅ = (Baseβπ ) & β’ Β· = (.rβπ ) β β’ (π β Ring β (π β Rng β§ βπ₯ β π΅ βπ¦ β π΅ ((π₯ Β· π¦) = π¦ β§ (π¦ Β· π₯) = π¦))) | ||
Theorem | rngass 46648 | Associative law for the multiplication operation of a non-unital ring. (Contributed by NM, 27-Aug-2011.) (Revised by AV, 13-Feb-2025.) |
β’ π΅ = (Baseβπ ) & β’ Β· = (.rβπ ) β β’ ((π β Rng β§ (π β π΅ β§ π β π΅ β§ π β π΅)) β ((π Β· π) Β· π) = (π Β· (π Β· π))) | ||
Theorem | rngdi 46649 | Distributive law for the multiplication operation of a non-unital ring (left-distributivity). (Contributed by AV, 14-Feb-2025.) |
β’ π΅ = (Baseβπ ) & β’ + = (+gβπ ) & β’ Β· = (.rβπ ) β β’ ((π β Rng β§ (π β π΅ β§ π β π΅ β§ π β π΅)) β (π Β· (π + π)) = ((π Β· π) + (π Β· π))) | ||
Theorem | rngdir 46650 | Distributive law for the multiplication operation of a non-unital ring (right-distributivity). (Contributed by AV, 17-Apr-2020.) |
β’ π΅ = (Baseβπ ) & β’ + = (+gβπ ) & β’ Β· = (.rβπ ) β β’ ((π β Rng β§ (π β π΅ β§ π β π΅ β§ π β π΅)) β ((π + π) Β· π) = ((π Β· π) + (π Β· π))) | ||
Theorem | rngacl 46651 | Closure of the addition operation of a non-unital ring. (Contributed by AV, 16-Feb-2025.) |
β’ π΅ = (Baseβπ ) & β’ + = (+gβπ ) β β’ ((π β Rng β§ π β π΅ β§ π β π΅) β (π + π) β π΅) | ||
Theorem | rng0cl 46652 | The zero element of a non-unital ring belongs to its base set. (Contributed by AV, 16-Feb-2025.) |
β’ π΅ = (Baseβπ ) & β’ 0 = (0gβπ ) β β’ (π β Rng β 0 β π΅) | ||
Theorem | rngcl 46653 | Closure of the multiplication operation of a non-unital ring. (Contributed by AV, 17-Apr-2020.) |
β’ π΅ = (Baseβπ ) & β’ Β· = (.rβπ ) β β’ ((π β Rng β§ π β π΅ β§ π β π΅) β (π Β· π) β π΅) | ||
Theorem | rnglz 46654 | The zero of a non-unital ring is a left-absorbing element. (Contributed by AV, 17-Apr-2020.) |
β’ π΅ = (Baseβπ ) & β’ Β· = (.rβπ ) & β’ 0 = (0gβπ ) β β’ ((π β Rng β§ π β π΅) β ( 0 Β· π) = 0 ) | ||
Theorem | rngrz 46655 | The zero of a non-unital ring is a right-absorbing element. (Contributed by AV, 16-Feb-2025.) |
β’ π΅ = (Baseβπ ) & β’ Β· = (.rβπ ) & β’ 0 = (0gβπ ) β β’ ((π β Rng β§ π β π΅) β (π Β· 0 ) = 0 ) | ||
Theorem | rngmneg1 46656 | Negation of a product in a non-unital ring (mulneg1 11649 analog). In contrast to ringmneg1 20115, the proof does not (and cannot) make use of the existence of a ring unity. (Contributed by AV, 17-Feb-2025.) |
β’ π΅ = (Baseβπ ) & β’ Β· = (.rβπ ) & β’ π = (invgβπ ) & β’ (π β π β Rng) & β’ (π β π β π΅) & β’ (π β π β π΅) β β’ (π β ((πβπ) Β· π) = (πβ(π Β· π))) | ||
Theorem | rngmneg2 46657 | Negation of a product in a non-unital ring (mulneg2 11650 analog). In contrast to ringmneg1 20115, the proof does not (and cannot) make use of the existence of a ring unity. (Contributed by AV, 17-Feb-2025.) |
β’ π΅ = (Baseβπ ) & β’ Β· = (.rβπ ) & β’ π = (invgβπ ) & β’ (π β π β Rng) & β’ (π β π β π΅) & β’ (π β π β π΅) β β’ (π β (π Β· (πβπ)) = (πβ(π Β· π))) | ||
Theorem | rngm2neg 46658 | Double negation of a product in a non-unital ring (mul2neg 11652 analog). (Contributed by AV, 17-Feb-2025.) |
β’ π΅ = (Baseβπ ) & β’ Β· = (.rβπ ) & β’ π = (invgβπ ) & β’ (π β π β Rng) & β’ (π β π β π΅) & β’ (π β π β π΅) β β’ (π β ((πβπ) Β· (πβπ)) = (π Β· π)) | ||
Theorem | rngansg 46659 | Every additive subgroup of a non-unital ring is normal. (Contributed by AV, 25-Feb-2025.) |
β’ (π β Rng β (NrmSGrpβπ ) = (SubGrpβπ )) | ||
Theorem | rngsubdi 46660 | Ring multiplication distributes over subtraction. (subdi 11646 analog.) (Contributed by Jeff Madsen, 19-Jun-2010.) (Revised by Mario Carneiro, 2-Jul-2014.) ringsubdi 20118 generalized for non-unital rings. (Revised by AV, 23-Feb-2025.) |
β’ π΅ = (Baseβπ ) & β’ Β· = (.rβπ ) & β’ β = (-gβπ ) & β’ (π β π β Rng) & β’ (π β π β π΅) & β’ (π β π β π΅) & β’ (π β π β π΅) β β’ (π β (π Β· (π β π)) = ((π Β· π) β (π Β· π))) | ||
Theorem | rngsubdir 46661 | Ring multiplication distributes over subtraction. (subdir 11647 analog.) (Contributed by Jeff Madsen, 19-Jun-2010.) (Revised by Mario Carneiro, 2-Jul-2014.) ringsubdir 20119 generalized for non-unital rings. (Revised by AV, 23-Feb-2025.) |
β’ π΅ = (Baseβπ ) & β’ Β· = (.rβπ ) & β’ β = (-gβπ ) & β’ (π β π β Rng) & β’ (π β π β π΅) & β’ (π β π β π΅) & β’ (π β π β π΅) β β’ (π β ((π β π) Β· π) = ((π Β· π) β (π Β· π))) | ||
Theorem | isrngd 46662* | Properties that determine a non-unital ring. (Contributed by AV, 14-Feb-2025.) |
β’ (π β π΅ = (Baseβπ )) & β’ (π β + = (+gβπ )) & β’ (π β Β· = (.rβπ )) & β’ (π β π β Abel) & β’ ((π β§ π₯ β π΅ β§ π¦ β π΅) β (π₯ Β· π¦) β π΅) & β’ ((π β§ (π₯ β π΅ β§ π¦ β π΅ β§ π§ β π΅)) β ((π₯ Β· π¦) Β· π§) = (π₯ Β· (π¦ Β· π§))) & β’ ((π β§ (π₯ β π΅ β§ π¦ β π΅ β§ π§ β π΅)) β (π₯ Β· (π¦ + π§)) = ((π₯ Β· π¦) + (π₯ Β· π§))) & β’ ((π β§ (π₯ β π΅ β§ π¦ β π΅ β§ π§ β π΅)) β ((π₯ + π¦) Β· π§) = ((π₯ Β· π§) + (π¦ Β· π§))) β β’ (π β π β Rng) | ||
Theorem | rngpropd 46663* | If two structures have the same base set, and the values of their group (addition) and ring (multiplication) operations are equal for all pairs of elements of the base set, one is a non-unital ring iff the other one is. (Contributed by AV, 15-Feb-2025.) |
β’ (π β π΅ = (BaseβπΎ)) & β’ (π β π΅ = (BaseβπΏ)) & β’ ((π β§ (π₯ β π΅ β§ π¦ β π΅)) β (π₯(+gβπΎ)π¦) = (π₯(+gβπΏ)π¦)) & β’ ((π β§ (π₯ β π΅ β§ π¦ β π΅)) β (π₯(.rβπΎ)π¦) = (π₯(.rβπΏ)π¦)) β β’ (π β (πΎ β Rng β πΏ β Rng)) | ||
Theorem | opprrng 46664 | An opposite non-unital ring is a non-unital ring. (Contributed by AV, 15-Feb-2025.) |
β’ π = (opprβπ ) β β’ (π β Rng β π β Rng) | ||
Theorem | opprrngb 46665 | A class is a non-unital ring if and only if its opposite is a non-unital ring. Bidirectional form of opprrng 46664. (Contributed by AV, 15-Feb-2025.) |
β’ π = (opprβπ ) β β’ (π β Rng β π β Rng) | ||
Theorem | prdsmulrngcl 46666 | Closure of the multiplication in a structure product of non-unital rings. (Contributed by AV, 21-Feb-2025.) |
β’ π = (πXsπ ) & β’ π΅ = (Baseβπ) & β’ Β· = (.rβπ) & β’ (π β π β π) & β’ (π β πΌ β π) & β’ (π β π :πΌβΆRng) & β’ (π β πΉ β π΅) & β’ (π β πΊ β π΅) β β’ (π β (πΉ Β· πΊ) β π΅) | ||
Theorem | prdsrngd 46667 | A product of non-unital rings is a non-unital ring. (Contributed by AV, 22-Feb-2025.) |
β’ π = (πXsπ ) & β’ (π β πΌ β π) & β’ (π β π β π) & β’ (π β π :πΌβΆRng) β β’ (π β π β Rng) | ||
Theorem | imasrng 46668* | The image structure of a non-unital ring is a non-unital ring (imasring 20142 analog). (Contributed by AV, 22-Feb-2025.) |
β’ (π β π = (πΉ βs π )) & β’ (π β π = (Baseβπ )) & β’ + = (+gβπ ) & β’ Β· = (.rβπ ) & β’ (π β πΉ:πβontoβπ΅) & β’ ((π β§ (π β π β§ π β π) β§ (π β π β§ π β π)) β (((πΉβπ) = (πΉβπ) β§ (πΉβπ) = (πΉβπ)) β (πΉβ(π + π)) = (πΉβ(π + π)))) & β’ ((π β§ (π β π β§ π β π) β§ (π β π β§ π β π)) β (((πΉβπ) = (πΉβπ) β§ (πΉβπ) = (πΉβπ)) β (πΉβ(π Β· π)) = (πΉβ(π Β· π)))) & β’ (π β π β Rng) β β’ (π β π β Rng) | ||
Theorem | imasrngf1 46669 | The image of a non-unital ring under an injection is a non-unital ring (imasmndf1 18663 analog). (Contributed by AV, 22-Feb-2025.) |
β’ π = (πΉ βs π ) & β’ π = (Baseβπ ) β β’ ((πΉ:πβ1-1βπ΅ β§ π β Rng) β π β Rng) | ||
Theorem | xpsrngd 46670 | A product of two non-unital rings is a non-unital ring (xpsmnd 18664 analog). (Contributed by AV, 22-Feb-2025.) |
β’ π = (π Γs π ) & β’ (π β π β Rng) & β’ (π β π β Rng) β β’ (π β π β Rng) | ||
Theorem | qusrng 46671* | The quotient structure of a non-unital ring is a non-unital ring (qusring2 20146 analog). (Contributed by AV, 23-Feb-2025.) |
β’ (π β π = (π /s βΌ )) & β’ (π β π = (Baseβπ )) & β’ + = (+gβπ ) & β’ Β· = (.rβπ ) & β’ (π β βΌ Er π) & β’ (π β ((π βΌ π β§ π βΌ π) β (π + π) βΌ (π + π))) & β’ (π β ((π βΌ π β§ π βΌ π) β (π Β· π) βΌ (π Β· π))) & β’ (π β π β Rng) β β’ (π β π β Rng) | ||
Theorem | zringrng 46672 | The ring of integers is a non-unital ring. (Contributed by AV, 17-Mar-2025.) |
β’ β€ring β Rng | ||
Syntax | crngh 46673 | non-unital ring homomorphisms. |
class RngHomo | ||
Syntax | crngs 46674 | non-unital ring isomorphisms. |
class RngIsom | ||
Definition | df-rnghomo 46675* | Define the set of non-unital ring homomorphisms from π to π . (Contributed by AV, 20-Feb-2020.) |
β’ RngHomo = (π β Rng, π β Rng β¦ β¦(Baseβπ) / π£β¦β¦(Baseβπ ) / π€β¦{π β (π€ βm π£) β£ βπ₯ β π£ βπ¦ β π£ ((πβ(π₯(+gβπ)π¦)) = ((πβπ₯)(+gβπ )(πβπ¦)) β§ (πβ(π₯(.rβπ)π¦)) = ((πβπ₯)(.rβπ )(πβπ¦)))}) | ||
Definition | df-rngisom 46676* | Define the set of non-unital ring isomorphisms from π to π . (Contributed by AV, 20-Feb-2020.) |
β’ RngIsom = (π β V, π β V β¦ {π β (π RngHomo π ) β£ β‘π β (π RngHomo π)}) | ||
Theorem | rnghmrcl 46677 | Reverse closure of a non-unital ring homomorphism. (Contributed by AV, 22-Feb-2020.) |
β’ (πΉ β (π RngHomo π) β (π β Rng β§ π β Rng)) | ||
Theorem | rnghmfn 46678 | The mapping of two non-unital rings to the non-unital ring homomorphisms between them is a function. (Contributed by AV, 1-Mar-2020.) |
β’ RngHomo Fn (Rng Γ Rng) | ||
Theorem | rnghmval 46679* | The set of the non-unital ring homomorphisms between two non-unital rings. (Contributed by AV, 22-Feb-2020.) |
β’ π΅ = (Baseβπ ) & β’ Β· = (.rβπ ) & β’ β = (.rβπ) & β’ πΆ = (Baseβπ) & β’ + = (+gβπ ) & β’ β = (+gβπ) β β’ ((π β Rng β§ π β Rng) β (π RngHomo π) = {π β (πΆ βm π΅) β£ βπ₯ β π΅ βπ¦ β π΅ ((πβ(π₯ + π¦)) = ((πβπ₯) β (πβπ¦)) β§ (πβ(π₯ Β· π¦)) = ((πβπ₯) β (πβπ¦)))}) | ||
Theorem | isrnghm 46680* | A function is a non-unital ring homomorphism iff it is a group homomorphism and preserves multiplication. (Contributed by AV, 22-Feb-2020.) |
β’ π΅ = (Baseβπ ) & β’ Β· = (.rβπ ) & β’ β = (.rβπ) β β’ (πΉ β (π RngHomo π) β ((π β Rng β§ π β Rng) β§ (πΉ β (π GrpHom π) β§ βπ₯ β π΅ βπ¦ β π΅ (πΉβ(π₯ Β· π¦)) = ((πΉβπ₯) β (πΉβπ¦))))) | ||
Theorem | isrnghmmul 46681 | A function is a non-unital ring homomorphism iff it preserves both addition and multiplication. (Contributed by AV, 27-Feb-2020.) |
β’ π = (mulGrpβπ ) & β’ π = (mulGrpβπ) β β’ (πΉ β (π RngHomo π) β ((π β Rng β§ π β Rng) β§ (πΉ β (π GrpHom π) β§ πΉ β (π MgmHom π)))) | ||
Theorem | rnghmmgmhm 46682 | A non-unital ring homomorphism is a homomorphism of multiplicative magmas. (Contributed by AV, 27-Feb-2020.) |
β’ π = (mulGrpβπ ) & β’ π = (mulGrpβπ) β β’ (πΉ β (π RngHomo π) β πΉ β (π MgmHom π)) | ||
Theorem | rnghmval2 46683 | The non-unital ring homomorphisms between two non-unital rings. (Contributed by AV, 1-Mar-2020.) |
β’ ((π β Rng β§ π β Rng) β (π RngHomo π) = ((π GrpHom π) β© ((mulGrpβπ ) MgmHom (mulGrpβπ)))) | ||
Theorem | isrngisom 46684 | An isomorphism of non-unital rings is a homomorphism whose converse is also a homomorphism. (Contributed by AV, 22-Feb-2020.) |
β’ ((π β π β§ π β π) β (πΉ β (π RngIsom π) β (πΉ β (π RngHomo π) β§ β‘πΉ β (π RngHomo π )))) | ||
Theorem | rngimrcl 46685 | Reverse closure for an isomorphism of non-unital rings. (Contributed by AV, 22-Feb-2020.) |
β’ (πΉ β (π RngIsom π) β (π β V β§ π β V)) | ||
Theorem | rnghmghm 46686 | A non-unital ring homomorphism is an additive group homomorphism. (Contributed by AV, 23-Feb-2020.) |
β’ (πΉ β (π RngHomo π) β πΉ β (π GrpHom π)) | ||
Theorem | rnghmf 46687 | A ring homomorphism is a function. (Contributed by AV, 23-Feb-2020.) |
β’ π΅ = (Baseβπ ) & β’ πΆ = (Baseβπ) β β’ (πΉ β (π RngHomo π) β πΉ:π΅βΆπΆ) | ||
Theorem | rnghmmul 46688 | A homomorphism of non-unital rings preserves multiplication. (Contributed by AV, 23-Feb-2020.) |
β’ π = (Baseβπ ) & β’ Β· = (.rβπ ) & β’ Γ = (.rβπ) β β’ ((πΉ β (π RngHomo π) β§ π΄ β π β§ π΅ β π) β (πΉβ(π΄ Β· π΅)) = ((πΉβπ΄) Γ (πΉβπ΅))) | ||
Theorem | isrnghm2d 46689* | Demonstration of non-unital ring homomorphism. (Contributed by AV, 23-Feb-2020.) |
β’ π΅ = (Baseβπ ) & β’ Β· = (.rβπ ) & β’ Γ = (.rβπ) & β’ (π β π β Rng) & β’ (π β π β Rng) & β’ ((π β§ (π₯ β π΅ β§ π¦ β π΅)) β (πΉβ(π₯ Β· π¦)) = ((πΉβπ₯) Γ (πΉβπ¦))) & β’ (π β πΉ β (π GrpHom π)) β β’ (π β πΉ β (π RngHomo π)) | ||
Theorem | isrnghmd 46690* | Demonstration of non-unital ring homomorphism. (Contributed by AV, 23-Feb-2020.) |
β’ π΅ = (Baseβπ ) & β’ Β· = (.rβπ ) & β’ Γ = (.rβπ) & β’ (π β π β Rng) & β’ (π β π β Rng) & β’ ((π β§ (π₯ β π΅ β§ π¦ β π΅)) β (πΉβ(π₯ Β· π¦)) = ((πΉβπ₯) Γ (πΉβπ¦))) & β’ πΆ = (Baseβπ) & β’ + = (+gβπ ) & ⒠⨣ = (+gβπ) & β’ (π β πΉ:π΅βΆπΆ) & β’ ((π β§ (π₯ β π΅ β§ π¦ β π΅)) β (πΉβ(π₯ + π¦)) = ((πΉβπ₯) ⨣ (πΉβπ¦))) β β’ (π β πΉ β (π RngHomo π)) | ||
Theorem | rnghmf1o 46691 | A non-unital ring homomorphism is bijective iff its converse is also a non-unital ring homomorphism. (Contributed by AV, 27-Feb-2020.) |
β’ π΅ = (Baseβπ ) & β’ πΆ = (Baseβπ) β β’ (πΉ β (π RngHomo π) β (πΉ:π΅β1-1-ontoβπΆ β β‘πΉ β (π RngHomo π ))) | ||
Theorem | isrngim 46692 | An isomorphism of non-unital rings is a bijective homomorphism. (Contributed by AV, 23-Feb-2020.) |
β’ π΅ = (Baseβπ ) & β’ πΆ = (Baseβπ) β β’ ((π β π β§ π β π) β (πΉ β (π RngIsom π) β (πΉ β (π RngHomo π) β§ πΉ:π΅β1-1-ontoβπΆ))) | ||
Theorem | rngimf1o 46693 | An isomorphism of non-unital rings is a bijection. (Contributed by AV, 23-Feb-2020.) |
β’ π΅ = (Baseβπ ) & β’ πΆ = (Baseβπ) β β’ (πΉ β (π RngIsom π) β πΉ:π΅β1-1-ontoβπΆ) | ||
Theorem | rngimrnghm 46694 | An isomorphism of non-unital rings is a homomorphism. (Contributed by AV, 23-Feb-2020.) |
β’ π΅ = (Baseβπ ) & β’ πΆ = (Baseβπ) β β’ (πΉ β (π RngIsom π) β πΉ β (π RngHomo π)) | ||
Theorem | rngimcnv 46695 | The converse of an isomorphism of non-unital rings is an isomorphism of non-unital rings. (Contributed by AV, 27-Feb-2025.) |
β’ (πΉ β (π RngIsom π) β β‘πΉ β (π RngIsom π)) | ||
Theorem | rnghmco 46696 | The composition of non-unital ring homomorphisms is a homomorphism. (Contributed by AV, 27-Feb-2020.) |
β’ ((πΉ β (π RngHomo π) β§ πΊ β (π RngHomo π)) β (πΉ β πΊ) β (π RngHomo π)) | ||
Theorem | idrnghm 46697 | The identity homomorphism on a non-unital ring. (Contributed by AV, 27-Feb-2020.) |
β’ π΅ = (Baseβπ ) β β’ (π β Rng β ( I βΎ π΅) β (π RngHomo π )) | ||
Theorem | c0mgm 46698* | The constant mapping to zero is a magma homomorphism into a monoid. Remark: Instead of the assumption that T is a monoid, it would be sufficient that T is a magma with a right or left identity. (Contributed by AV, 17-Apr-2020.) |
β’ π΅ = (Baseβπ) & β’ 0 = (0gβπ) & β’ π» = (π₯ β π΅ β¦ 0 ) β β’ ((π β Mgm β§ π β Mnd) β π» β (π MgmHom π)) | ||
Theorem | c0mhm 46699* | The constant mapping to zero is a monoid homomorphism. (Contributed by AV, 16-Apr-2020.) |
β’ π΅ = (Baseβπ) & β’ 0 = (0gβπ) & β’ π» = (π₯ β π΅ β¦ 0 ) β β’ ((π β Mnd β§ π β Mnd) β π» β (π MndHom π)) | ||
Theorem | c0ghm 46700* | The constant mapping to zero is a group homomorphism. (Contributed by AV, 16-Apr-2020.) |
β’ π΅ = (Baseβπ) & β’ 0 = (0gβπ) & β’ π» = (π₯ β π΅ β¦ 0 ) β β’ ((π β Grp β§ π β Grp) β π» β (π GrpHom π)) |
< Previous Next > |
Copyright terms: Public domain | < Previous Next > |