Skip to content

Commit b2d55cd

Browse files
committed
[rename] algebra scalars function -> algebra scalar lifting function
1 parent 7db4cd4 commit b2d55cd

File tree

1 file changed

+17
-16
lines changed

1 file changed

+17
-16
lines changed

set.mm

Lines changed: 17 additions & 16 deletions
Original file line numberDiff line numberDiff line change
@@ -283995,7 +283995,7 @@ the same dimension over the same (nonzero) ring. (Contributed by AV,
283995283995
$( Algebraic span function. $)
283996283996
casp $a class AlgSpan $.
283997283997

283998-
$( Class of algebra scalars function. $)
283998+
$( Class of algebra scalar lifting function. $)
283999283999
cascl $a class algSc $.
284000284000

284001284001
${
@@ -284407,8 +284407,8 @@ the same dimension over the same (nonzero) ring. (Contributed by AV,
284407284407
asclfval.k $e |- K = ( Base ` F ) $.
284408284408
asclfval.s $e |- .x. = ( .s ` W ) $.
284409284409
asclfval.o $e |- .1. = ( 1r ` W ) $.
284410-
$( Function value of the algebra scalars function. (Contributed by Mario
284411-
Carneiro, 8-Mar-2015.) $)
284410+
$( Function value of the algebra scalar lifting function. (Contributed by
284411+
Mario Carneiro, 8-Mar-2015.) $)
284412284412
asclfval $p |- A = ( x e. K |-> ( x .x. .1. ) ) $=
284413284413
( vw cascl cfv cmpt cbs csca eqtr4di c0 cv cvv wcel wceq cur cvsca fveq2d
284414284414
co fveq2 eqidd oveq123d mpteq12dv df-ascl mptfvmpt wn mpt0 eqtrid mpteq1d
@@ -284430,7 +284430,7 @@ the same dimension over the same (nonzero) ring. (Contributed by AV,
284430284430
asclfn.a $e |- A = ( algSc ` W ) $.
284431284431
asclfn.f $e |- F = ( Scalar ` W ) $.
284432284432
asclfn.k $e |- K = ( Base ` F ) $.
284433-
$( Unconditional functionality of the algebra scalars function.
284433+
$( Unconditional functionality of the algebra scalar lifting function.
284434284434
(Contributed by Mario Carneiro, 9-Mar-2015.) $)
284435284435
asclfn $p |- A Fn K $=
284436284436
( vx cv cur cfv cvsca co ovex eqid asclfval fnmpti ) HCHIZDJKZDLKZMARSTNH
@@ -284446,7 +284446,7 @@ the same dimension over the same (nonzero) ring. (Contributed by AV,
284446284446
${
284447284447
asclf.k $e |- K = ( Base ` F ) $.
284448284448
asclf.b $e |- B = ( Base ` W ) $.
284449-
$( The algebra scalars function is a function into the base set.
284449+
$( The algebra scalar lifting function is a function into the base set.
284450284450
(Contributed by Mario Carneiro, 4-Jul-2015.) $)
284451284451
asclf $p |- ( ph -> A : K --> B ) $=
284452284452
( vx cv cur cfv cvsca wcel adantr eqid co clmod simpr ringidcl lmodvscl
@@ -284455,8 +284455,8 @@ the same dimension over the same (nonzero) ring. (Contributed by AV,
284455284455
NUMDEFGHKUTUSUJUK $.
284456284456
$}
284457284457

284458-
$( The algebra scalars function is a group homomorphism. (Contributed by
284459-
Mario Carneiro, 4-Jul-2015.) $)
284458+
$( The algebra scalar lifting function is a group homomorphism.
284459+
(Contributed by Mario Carneiro, 4-Jul-2015.) $)
284460284460
asclghm $p |- ( ph -> A e. ( F GrpHom W ) ) $=
284461284461
( vx vy cplusg cfv cbs eqid crg wcel syl co wceq asclval lmodring ringgrp
284462284462
clmod asclf cv cur cvsca adantr simprl simprr ringidcl lmodvsdir syl13anc
@@ -284529,7 +284529,7 @@ the same dimension over the same (nonzero) ring. (Contributed by AV,
284529284529
ascldimul.k $e |- K = ( Base ` F ) $.
284530284530
ascldimul.t $e |- .X. = ( .r ` W ) $.
284531284531
ascldimul.s $e |- .x. = ( .r ` F ) $.
284532-
$( The algebra scalars function distributes over multiplication.
284532+
$( The algebra scalar lifting function distributes over multiplication.
284533284533
(Contributed by Mario Carneiro, 8-Mar-2015.) (Proof shortened by SN,
284534284534
5-Nov-2023.) $)
284535284535
ascldimul $p |- ( ( W e. AssAlg /\ R e. K /\ S e. K ) ->
@@ -284564,8 +284564,8 @@ the same dimension over the same (nonzero) ring. (Contributed by AV,
284564284564
$d x y A $. $d x y F $. $d x y W $.
284565284565
asclrhm.a $e |- A = ( algSc ` W ) $.
284566284566
asclrhm.f $e |- F = ( Scalar ` W ) $.
284567-
$( The algebra scalars function is a ring homomorphism. (Contributed by
284568-
Mario Carneiro, 8-Mar-2015.) $)
284567+
$( The algebra scalar lifting function is a ring homomorphism.
284568+
(Contributed by Mario Carneiro, 8-Mar-2015.) $)
284569284569
asclrhm $p |- ( W e. AssAlg -> A e. ( F RingHom W ) ) $=
284570284570
( vx vy casa wcel cbs cfv cmulr cur assasca assaring assalmod ascl1 cv co
284571284571
eqid wceq ascldimul 3expb asclghm isrhm2d ) CHIZFGBJKZBCBLKZCLKZBMKZACMKZ
@@ -292258,7 +292258,7 @@ series in the subring which are also polynomials (in the parent ring).
292258292258
( crg wcel cid cfv ply1sca2 ply1ring ply1lmod cbs cnx baseid strfvi
292259292259
asclf ) DJKABDLMECGCDFNCDFOCDFPDQRQMESHTIUA $.
292260292260

292261-
$( The value of the algebra scalars function for (univariate)
292261+
$( The value of the algebra scalar lifting function for (univariate)
292262292262
polynomials applied to a scalar results in a constant polynomial.
292263292263
(Contributed by AV, 27-Nov-2019.) $)
292264292264
ply1sclcl $p |- ( ( R e. Ring /\ S e. K ) -> ( A ` S ) e. B ) $=
@@ -301895,8 +301895,9 @@ are univariate (or multivariate) polynomials. See Wikipedia "Polynomial
301895301895
pmat0opsc.z $e |- .0. = ( 0g ` R ) $.
301896301896
$( The zero polynomial matrix over a ring represented as operation with
301897301897
"lifted scalars" (i.e. elements of the ring underlying the polynomial
301898-
ring embedded into the polynomial ring by the scalar injection/algebraic
301899-
scalars function ` algSc ` ). (Contributed by AV, 16-Nov-2019.) $)
301898+
ring embedded into the polynomial ring by the scalar injection/algebra
301899+
scalar lifting function ` algSc ` ). (Contributed by AV,
301900+
16-Nov-2019.) $)
301900301901
pmat0opsc $p |- ( ( N e. Fin /\ R e. Ring )
301901301902
-> ( 0g ` C ) = ( i e. N , j e. N |-> ( A ` .0. ) ) ) $=
301902301903
( cfn wcel crg wa c0g cfv cmpo eqid pmat0op wceq ply1scl0 eqcomd mpoeq3dv
@@ -835256,8 +835257,8 @@ have GLB (expanded version). (Contributed by Zhi Wang,
835256835257
${
835257835258
$d A x $. $d C x $. $d M x $. $d W x $. $d ph x $.
835258835259
asclcntr.m $e |- M = ( mulGrp ` W ) $.
835259-
$( The algebra scalars function maps into the center of the algebra.
835260-
Equivalently, a lifted scalar is a center of the algebra.
835260+
$( The algebra scalar lifting function maps into the center of the
835261+
algebra. Equivalently, a lifted scalar is a center of the algebra.
835261835262
(Contributed by Zhi Wang, 11-Sep-2025.) $)
835262835263
asclcntr $p |- ( ph -> ( A ` C ) e. ( Cntr ` M ) ) $=
835263835264
( vx cbs cfv eqid wcel co adantr ccntr asclelbas cv wa casa cmulr simpr
@@ -835280,7 +835281,7 @@ have GLB (expanded version). (Contributed by Zhi Wang,
835280835281
a "vector" element of ` W ` , of the "scalar" ` C ` , which is now an
835281835282
upper triangular matrix, with the "vector" ` X e. ( Base `` W ) ` .
835282835283

835283-
Equivalently, the algebra scalars function is not necessarily
835284+
Equivalently, the algebra scalar lifting function is not necessarily
835284835285
injective unless the algebra is faithful. Therefore, all "scalar
835285835286
injection" was renamed.
835286835287

0 commit comments

Comments
 (0)