theorem Th121:
for
a,
b being
Nat st
a < b &
b <> 0 holds
(2 * a) div b < 2
LmAssoc:
for G being Group
for g1, g2, g3, g4, g5 being Element of G holds (g1 * ((g2 * g3) * g4)) * g5 = (((g1 * g2) * g3) * g4) * g5
theorem thUnitalMagmaIsGroupCond:
Th61:
for G being Group
for H1, H2 being Subgroup of G holds H1 * H2 c= the carrier of (H1 "\/" H2)
Lm1:
for G1, G2 being Group
for x being Element of product (Carrier <*G1,G2*>) holds
( x . 1 in G1 & x . 2 in G2 & dom x = {1,2} )
Lm2:
for A, G being Group
for a being Element of A
for g being Element of G holds <*a,g*> in product (Carrier <*A,G*>)
Lm3:
for G1, G2 being Group
for phi being Homomorphism of G1,G2
for a being Element of G1 holds phi . a in G2
;
definition
let G,
A be
Group;
let phi be
Homomorphism of
A,
(AutGroup G);
existence
ex b1 being non empty strict multMagma st
( the carrier of b1 = product (Carrier <*G,A*>) & ( for f, g being Element of product (Carrier <*G,A*>) ex h being Function ex a1 being Element of A ex g2 being Element of G st
( h = the multF of b1 . (f,g) & a1 = f . 2 & g2 = g . 1 & h . 1 = the multF of G . ((f . 1),((phi . a1) . g2)) & h . 2 = the multF of A . ((f . 2),(g . 2)) ) ) )
uniqueness
for b1, b2 being non empty strict multMagma st the carrier of b1 = product (Carrier <*G,A*>) & ( for f, g being Element of product (Carrier <*G,A*>) ex h being Function ex a1 being Element of A ex g2 being Element of G st
( h = the multF of b1 . (f,g) & a1 = f . 2 & g2 = g . 1 & h . 1 = the multF of G . ((f . 1),((phi . a1) . g2)) & h . 2 = the multF of A . ((f . 2),(g . 2)) ) ) & the carrier of b2 = product (Carrier <*G,A*>) & ( for f, g being Element of product (Carrier <*G,A*>) ex h being Function ex a1 being Element of A ex g2 being Element of G st
( h = the multF of b2 . (f,g) & a1 = f . 2 & g2 = g . 1 & h . 1 = the multF of G . ((f . 1),((phi . a1) . g2)) & h . 2 = the multF of A . ((f . 2),(g . 2)) ) ) holds
b1 = b2
end;
::
deftheorem Def1 defines
semidirect_product GROUP_24:def 1 :
for G, A being Group
for phi being Homomorphism of A,(AutGroup G)
for b4 being non empty strict multMagma holds
( b4 = semidirect_product (G,A,phi) iff ( the carrier of b4 = product (Carrier <*G,A*>) & ( for f, g being Element of product (Carrier <*G,A*>) ex h being Function ex a1 being Element of A ex g2 being Element of G st
( h = the multF of b4 . (f,g) & a1 = f . 2 & g2 = g . 1 & h . 1 = the multF of G . ((f . 1),((phi . a1) . g2)) & h . 2 = the multF of A . ((f . 2),(g . 2)) ) ) ) );
theorem Th14:
for
G,
A being
Group for
phi being
Homomorphism of
A,
(AutGroup G) for
x,
y being
Element of
(semidirect_product (G,A,phi)) for
a1,
a2 being
Element of
A for
g1,
g2,
g3 being
Element of
G st
x = <*g1,a1*> &
y = <*g2,a2*> &
g3 = (phi . a1) . g2 holds
x * y = <*(g1 * g3),(a1 * a2)*>
Lm4:
for G, A being Group
for phi being Homomorphism of A,(AutGroup G)
for x, e being Element of (semidirect_product (G,A,phi)) st e = <*(1_ G),(1_ A)*> holds
( x * e = x & e * x = x )
theorem Th20:
for
G,
A being
Group for
phi being
Homomorphism of
A,
(AutGroup G) for
x,
y being
Element of
(semidirect_product (G,A,phi)) for
a being
Element of
A for
g being
Element of
G st
x = <*g,a*> &
y = <*((phi . (a ")) . (g ")),(a ")*> holds
(
x * y = 1_ (semidirect_product (G,A,phi)) &
y * x = 1_ (semidirect_product (G,A,phi)) )
theorem Th23:
for
G,
A being
Group for
phi being
Homomorphism of
A,
(AutGroup G) for
g1,
g2 being
Element of
G for
x,
y,
z being
Element of
(semidirect_product (G,A,phi)) st
x = <*g1,(1_ A)*> &
y = <*g2,(1_ A)*> &
z = <*(g1 * g2),(1_ A)*> holds
x * y = z
theorem Th26:
for
G,
A being
Group for
phi being
Homomorphism of
A,
(AutGroup G) for
a1,
a2 being
Element of
A for
x,
y,
z being
Element of
(semidirect_product (G,A,phi)) st
x = <*(1_ G),a1*> &
y = <*(1_ G),a2*> &
z = <*(1_ G),(a1 * a2)*> holds
x * y = z
definition
let G,
A be
Group;
let phi be
Homomorphism of
A,
(AutGroup G);
existence
ex b1 being Function of G,(semidirect_product (G,A,phi)) st
for g being Element of G holds b1 . g = <*g,(1_ A)*>
uniqueness
for b1, b2 being Function of G,(semidirect_product (G,A,phi)) st ( for g being Element of G holds b1 . g = <*g,(1_ A)*> ) & ( for g being Element of G holds b2 . g = <*g,(1_ A)*> ) holds
b1 = b2
end;
definition
let G,
A be
Group;
let phi be
Homomorphism of
A,
(AutGroup G);
existence
ex b1 being Function of A,(semidirect_product (G,A,phi)) st
for a being Element of A holds b1 . a = <*(1_ G),a*>
uniqueness
for b1, b2 being Function of A,(semidirect_product (G,A,phi)) st ( for a being Element of A holds b1 . a = <*(1_ G),a*> ) & ( for a being Element of A holds b2 . a = <*(1_ G),a*> ) holds
b1 = b2
end;
theorem UniversalPropertyQuotientGroups:
theorem
for
H,
G being
Group for
N being
strict Group for
f being
Homomorphism of
N,
G for
g being
Homomorphism of
H,
G for
phi being
Homomorphism of
H,
(AutGroup N) st ( for
n being
Element of
N for
h being
Element of
H holds
f . ((phi . h) . n) = ((g . h) * (f . n)) * (g . (h ")) ) holds
ex
k being
Homomorphism of
(semidirect_product (N,H,phi)),
G st
(
f = k * (incl1 (N,H,phi)) &
g = k * (incl2 (N,H,phi)) )
Lm6:
for n being non zero even Nat holds 1 in Segm n
ThTrivialCriterion:
for G being Group holds
( G is trivial iff card G = 1 )
by GROUP_6:11;
theorem ThTrivialCyclicGroupCriterion1:
theorem ThTrivialCyclicGroupCriterion:
theorem ThMultTableINTGroup2:
theorem ThInverseOpGSquaresToIdentity:
theorem ThCommutationEq2:
definition
let n be non
zero ExtNat;
existence
ex b1 being strict Group st
( ( n = +infty implies b1 = semidirect_product (INT.Group,(INT.Group 2),(inversions INT.Group)) ) & ( n <> +infty implies ex n1 being non zero Nat st
( n = n1 & b1 = semidirect_product ((INT.Group n1),(INT.Group 2),(inversions (INT.Group n1))) ) ) )
uniqueness
for b1, b2 being strict Group st ( n = +infty implies b1 = semidirect_product (INT.Group,(INT.Group 2),(inversions INT.Group)) ) & ( n <> +infty implies ex n1 being non zero Nat st
( n = n1 & b1 = semidirect_product ((INT.Group n1),(INT.Group 2),(inversions (INT.Group n1))) ) ) & ( n = +infty implies b2 = semidirect_product (INT.Group,(INT.Group 2),(inversions INT.Group)) ) & ( n <> +infty implies ex n1 being non zero Nat st
( n = n1 & b2 = semidirect_product ((INT.Group n1),(INT.Group 2),(inversions (INT.Group n1))) ) ) holds
b1 = b2
;
end;