theorem Th4:
for
A being
Ring for
X being non
empty set for
f being
Function of
A,
X for
a,
b,
c being
Element of
X st
f is
bijective holds
addemb (
f,
a,
(addemb (f,b,c)))
= addemb (
f,
(addemb (f,a,b)),
c)
definition
let A be
Ring;
let X be non
empty set ;
let f be
Function of
A,
X;
existence
ex b1 being BinOp of X st
for a, b being Element of X holds b1 . (a,b) = addemb (f,a,b)
uniqueness
for b1, b2 being BinOp of X st ( for a, b being Element of X holds b1 . (a,b) = addemb (f,a,b) ) & ( for a, b being Element of X holds b2 . (a,b) = addemb (f,a,b) ) holds
b1 = b2
end;
definition
let A be
Ring;
let X be non
empty set ;
let f be
Function of
A,
X;
existence
ex b1 being BinOp of X st
for a, b being Element of X holds b1 . (a,b) = multemb (f,a,b)
uniqueness
for b1, b2 being BinOp of X st ( for a, b being Element of X holds b1 . (a,b) = multemb (f,a,b) ) & ( for a, b being Element of X holds b2 . (a,b) = multemb (f,a,b) ) holds
b1 = b2
end;
Lm1:
for R, S being AbGroup
for f being Homomorphism of R,S holds 0. S in rng f
Lm2:
for R, S being AbGroup
for f being Homomorphism of R,S holds rng f is Preserv of the addF of S
theorem Th11:
for
A being
AbGroup for
X being non
empty set for
f being
Function of
A,
X for
a,
b,
c being
Element of
X st
f is
bijective holds
addemb (
f,
a,
(addemb (f,b,c)))
= addemb (
f,
(addemb (f,a,b)),
c)
definition
let A be
AbGroup;
let X be non
empty set ;
let f be
Function of
A,
X;
existence
ex b1 being BinOp of X st
for a, b being Element of X holds b1 . (a,b) = addemb (f,a,b)
uniqueness
for b1, b2 being BinOp of X st ( for a, b being Element of X holds b1 . (a,b) = addemb (f,a,b) ) & ( for a, b being Element of X holds b2 . (a,b) = addemb (f,a,b) ) holds
b1 = b2
end;