help1:
for R being domRing
for n being Element of NAT holds (<%(0. R),(1. R)%> `^ n) . n = 1. R
help2:
for R being domRing
for n, i being Element of NAT st i <> n holds
(<%(0. R),(1. R)%> `^ n) . i = 0. R
help3a:
for R being domRing
for n being Element of NAT st n <> 0 holds
for a being Element of R holds eval ((<%(0. R),(1. R)%> `^ n),a) = a |^ n
ThR1:
for R being Ring holds R is Subring of R
by LIOUVIL2:18;
Th28:
for L being non empty ZeroStr
for a being Element of L holds
( (a | L) . 0 = a & ( for n being Nat st n <> 0 holds
(a | L) . n = 0. L ) )
Lm10:
for R being Ring
for S being RingExtension of R
for T being Subset of S
for x being Element of (RAdj (R,T)) holds x is Element of S
Lm11:
for R being Ring
for S being RingExtension of R
for T being Subset of S
for a, b being Element of S
for x, y being Element of (RAdj (R,T)) st a = x & b = y holds
a + b = x + y
Lm12:
for R being Ring
for S being RingExtension of R
for T being Subset of S
for a, b being Element of S
for x, y being Element of (RAdj (R,T)) st a = x & b = y holds
a * b = x * y
Lm10f:
for R being Field
for S being FieldExtension of R
for T being Subset of S
for x being Element of (FAdj (R,T)) holds x is Element of S
Lm11f:
for R being Field
for S being FieldExtension of R
for T being Subset of S
for a, b being Element of S
for x, y being Element of (FAdj (R,T)) st a = x & b = y holds
a + b = x + y
Lm12f:
for R being Field
for S being FieldExtension of R
for T being Subset of S
for a, b being Element of S
for x, y being Element of (FAdj (R,T)) st a = x & b = y holds
a * b = x * y
lcsub1:
for F being Field
for E being FieldExtension of F
for a being Element of E
for n being Element of NAT holds a |^ n in the carrier of (FAdj (F,{a}))
lemphi1:
for F being Field
for E being FieldExtension of F
for a being Element of E holds rng (hom_Ext_eval (a,F)) = { (Ext_eval (p,a)) where p is Polynomial of F : verum }
lemphi2:
for F being Field
for E being FieldExtension of F
for a being Element of E holds rng (hom_Ext_eval (a,F)) c= the carrier of (RAdj (F,{a}))
lemphi3:
for F being Field
for E being Polynom-Ring b1 -homomorphic FieldExtension of F
for a being Element of E holds F is Subring of Image (hom_Ext_eval (a,F))
lemlin:
for F being Field
for E being b1 -finite FieldExtension of F
for A being finite Subset of (VecSp (E,F)) st card A > dim (VecSp (E,F)) holds
A is linearly-dependent
Lm12a:
for F being Ring
for E being RingExtension of F
for a, b being Element of E
for s being Element of F
for v being Element of (VecSp (E,F)) st a = s & b = v holds
a * b = s * v
Lm12b:
for F being Ring
for E being RingExtension of F
for a, b being Element of E
for x, y being Element of F st a = x & b = y holds
a * b = x * y
lemminirred:
for F being Field
for E being FieldExtension of F
for a being b1 -algebraic Element of E holds MinPoly (a,F) is irreducible
lembas1b:
for F being Field
for E being FieldExtension of F
for a being b1 -algebraic Element of E
for p being Polynomial of F st deg p < deg (MinPoly (a,F)) holds
Ext_eval ((Leading-Monomial p),a) in Lin (Base a)
lembas1a:
for F being Field
for E being Polynom-Ring b1 -homomorphic FieldExtension of F
for a being b1 -algebraic Element of E
for p being Polynomial of F st deg p < deg (MinPoly (a,F)) holds
Ext_eval (p,a) in Lin (Base a)