ch1:
for X being non empty set
for C being ascending Chain of X
for x being object
for i, j being Nat st i <= j & x in C . i holds
x in C . j
hom3:
for E, F being Field
for f being additive multiplicative Function of E,F holds
( ( f . (1. E) = 0. F & f = E --> (0. F) ) or ( f . (1. E) = 1. F & f is monomorphism ) )
ker1:
for R, S being non empty doubleLoopStr
for f being Function of R,S
for x being Element of R st x in ker f holds
f . x = 0. S
T0:
for R being Ring
for S being b1 -homomorphic Ring
for f being Homomorphism of R,S holds 0. S in rng f
T1:
for R being Ring
for S being b1 -homomorphic Ring
for f being Homomorphism of R,S holds 1. S in rng f
T3:
for R being Ring
for S being b1 -homomorphic Ring
for f being Homomorphism of R,S holds rng f is Preserv of the addF of S
T4:
for R being Ring
for S being b1 -homomorphic Ring
for f being Homomorphism of R,S holds rng f is Preserv of the multF of S
T5:
for R being Ring
for S being b1 -homomorphic Ring
for f being Homomorphism of R,S
for a, b being Element of (Image f)
for x, y being Element of S st a = x & b = y holds
( a + b = x + y & a * b = x * y )
T6:
for R being Ring
for S being b1 -homomorphic Ring
for f being Homomorphism of R,S
for a being Element of (Image f) ex x being Element of R st f . x = a
definition
let R be
Ring;
let S be
R -homomorphic Ring;
let f be
Homomorphism of
R,
S;
existence
ex b1 being Function of (R / (ker f)),(Image f) st
for a being Element of R holds b1 . (Class ((EqRel (R,(ker f))),a)) = f . a
uniqueness
for b1, b2 being Function of (R / (ker f)),(Image f) st ( for a being Element of R holds b1 . (Class ((EqRel (R,(ker f))),a)) = f . a ) & ( for a being Element of R holds b2 . (Class ((EqRel (R,(ker f))),a)) = f . a ) holds
b1 = b2
end;
lemintr:
for x, y being Integer
for a, b being Element of INT.Ring st x <> 0 & x = a & y = b holds
( x divides y iff a divides b )
fact1:
for R being non empty right_unital doubleLoopStr
for a being Element of R holds
( a is irreducible iff <*a*> is_a_factorization_of a )
lemfactunique1:
for R being domRing
for a, b, x being Element of R
for F being non empty FinSequence of R st x is prime & x divides a & a is_associated_to b & F is_a_factorization_of b holds
ex i being Element of dom F st F . i is_associated_to x
lemfactunique:
for R being PIDomain
for x, y being Element of R
for F, G being non empty FinSequence of R st F is_a_factorization_of x & G is_a_factorization_of y & x is_associated_to y holds
ex p being Function of (dom F),(dom G) st
( p is bijective & ( for i being Element of dom F holds G . (p . i) is_associated_to F . i ) )
thEucl2:
for L being Field ex f being Function of (Polynom-Ring L),NAT st
for p, q being Element of (Polynom-Ring L) st q <> 0. (Polynom-Ring L) holds
ex u, r being Element of (Polynom-Ring L) st
( p = (u * q) + r & ( r = 0. (Polynom-Ring L) or f . r < f . q ) )