begin
Lm1:
now
set G =
multMagma(#
REAL,
addreal #);
thus
for
h,
g,
f being
Element of
multMagma(#
REAL,
addreal #) holds
(h * g) * f = h * (g * f)
ex e being Element of multMagma(# REAL,addreal #) st
for h being Element of multMagma(# REAL,addreal #) holds
( h * e = h & e * h = h & ex g being Element of multMagma(# REAL,addreal #) st
( h * g = e & g * h = e ) )
reconsider e =
0 as
Element of
multMagma(#
REAL,
addreal #) ;
take e =
e;
for h being Element of multMagma(# REAL,addreal #) holds
( h * e = h & e * h = h & ex g being Element of multMagma(# REAL,addreal #) st
( h * g = e & g * h = e ) )let h be
Element of
multMagma(#
REAL,
addreal #);
( h * e = h & e * h = h & ex g being Element of multMagma(# REAL,addreal #) st
( h * g = e & g * h = e ) )reconsider A =
h as
Real ;
thus h * e =
A + 0
by BINOP_2:def 9
.=
h
;
( e * h = h & ex g being Element of multMagma(# REAL,addreal #) st
( h * g = e & g * h = e ) )thus e * h =
0 + A
by BINOP_2:def 9
.=
h
;
ex g being Element of multMagma(# REAL,addreal #) st
( h * g = e & g * h = e )reconsider g =
- A as
Element of
multMagma(#
REAL,
addreal #) ;
take g =
g;
( h * g = e & g * h = e )thus h * g =
A + (- A)
by BINOP_2:def 9
.=
e
;
g * h = ethus g * h =
(- A) + A
by BINOP_2:def 9
.=
e
;
verum
end;
:: deftheorem GROUP_1:def 1 :
canceled;
:: deftheorem Def2 defines unital GROUP_1:def 2 :
for IT being multMagma holds
( IT is unital iff ex e being Element of IT st
for h being Element of IT holds
( h * e = h & e * h = h ) );
:: deftheorem Def3 defines Group-like GROUP_1:def 3 :
for IT being multMagma holds
( IT is Group-like iff ex e being Element of IT st
for h being Element of IT holds
( h * e = h & e * h = h & ex g being Element of IT st
( h * g = e & g * h = e ) ) );
:: deftheorem Def4 defines associative GROUP_1:def 4 :
for IT being multMagma holds
( IT is associative iff for x, y, z being Element of IT holds (x * y) * z = x * (y * z) );
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
theorem
theorem Th7:
:: deftheorem Def5 defines 1_ GROUP_1:def 5 :
for G being multMagma st G is unital holds
for b2 being Element of G holds
( b2 = 1_ G iff for h being Element of G holds
( h * b2 = h & b2 * h = h ) );
theorem
canceled;
theorem
canceled;
theorem
:: deftheorem Def6 defines " GROUP_1:def 6 :
for G being Group
for h, b3 being Element of G holds
( b3 = h " iff ( h * b3 = 1_ G & b3 * h = 1_ G ) );
theorem
canceled;
theorem
theorem
canceled;
theorem Th14:
for
G being
Group for
h,
g,
f being
Element of
G st (
h * g = h * f or
g * h = f * h ) holds
g = f
theorem
theorem Th16:
theorem
theorem
theorem
theorem Th20:
theorem Th21:
for
G being
Group for
h,
f,
g being
Element of
G holds
(
h * f = g iff
f = (h ") * g )
theorem Th22:
for
G being
Group for
f,
h,
g being
Element of
G holds
(
f * h = g iff
f = g * (h ") )
theorem
theorem
theorem Th25:
theorem Th26:
theorem Th27:
theorem Th28:
:: deftheorem Def7 defines inverse_op GROUP_1:def 7 :
for G being Group
for b2 being UnOp of G holds
( b2 = inverse_op G iff for h being Element of G holds b2 . h = h " );
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem Th32:
theorem Th33:
theorem
canceled;
theorem Th35:
theorem
canceled;
theorem
definition
let G be non
empty multMagma ;
func power G -> Function of
[: the carrier of G,NAT:], the
carrier of
G means :
Def8:
for
h being
Element of
G holds
(
it . (
h,
0)
= 1_ G & ( for
n being
Element of
NAT holds
it . (
h,
(n + 1))
= (it . (h,n)) * h ) );
existence
ex b1 being Function of [: the carrier of G,NAT:], the carrier of G st
for h being Element of G holds
( b1 . (h,0) = 1_ G & ( for n being Element of NAT holds b1 . (h,(n + 1)) = (b1 . (h,n)) * h ) )
uniqueness
for b1, b2 being Function of [: the carrier of G,NAT:], the carrier of G st ( for h being Element of G holds
( b1 . (h,0) = 1_ G & ( for n being Element of NAT holds b1 . (h,(n + 1)) = (b1 . (h,n)) * h ) ) ) & ( for h being Element of G holds
( b2 . (h,0) = 1_ G & ( for n being Element of NAT holds b2 . (h,(n + 1)) = (b2 . (h,n)) * h ) ) ) holds
b1 = b2
end;
:: deftheorem Def8 defines power GROUP_1:def 8 :
for G being non empty multMagma
for b2 being Function of [: the carrier of G,NAT:], the carrier of G holds
( b2 = power G iff for h being Element of G holds
( b2 . (h,0) = 1_ G & ( for n being Element of NAT holds b2 . (h,(n + 1)) = (b2 . (h,n)) * h ) ) );
:: deftheorem Def9 defines |^ GROUP_1:def 9 :
for G being Group
for i being Integer
for h being Element of G holds
( ( 0 <= i implies h |^ i = (power G) . (h,(abs i)) ) & ( not 0 <= i implies h |^ i = ((power G) . (h,(abs i))) " ) );
:: deftheorem defines |^ GROUP_1:def 10 :
for G being Group
for n being Nat
for h being Element of G holds h |^ n = (power G) . (h,n);
Lm2:
for n being Nat
for G being Group
for h being Element of G holds h |^ (n + 1) = (h |^ n) * h
Lm3:
for G being Group
for h being Element of G holds h |^ 0 = 1_ G
by Def8;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
Lm4:
for n being Nat
for G being Group holds (1_ G) |^ n = 1_ G
theorem
theorem Th44:
theorem Th45:
theorem
theorem
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
Lm5:
for n, m being Nat
for G being Group
for h being Element of G holds h |^ (n + m) = (h |^ n) * (h |^ m)
Lm6:
for n being Nat
for G being Group
for h being Element of G holds
( h |^ (n + 1) = (h |^ n) * h & h |^ (n + 1) = h * (h |^ n) )
Lm7:
for n, m being Nat
for G being Group
for h being Element of G holds h |^ (n * m) = (h |^ n) |^ m
Lm8:
for n being Nat
for G being Group
for h being Element of G holds (h ") |^ n = (h |^ n) "
Lm9:
for n being Nat
for G being Group
for g, h being Element of G st g * h = h * g holds
g * (h |^ n) = (h |^ n) * g
Lm10:
for n, m being Nat
for G being Group
for g, h being Element of G st g * h = h * g holds
(g |^ n) * (h |^ m) = (h |^ m) * (g |^ n)
Lm11:
for n being Nat
for G being Group
for g, h being Element of G st g * h = h * g holds
(g * h) |^ n = (g |^ n) * (h |^ n)
theorem Th60:
theorem
theorem Th62:
Lm12:
for i being Integer
for G being Group
for h being Element of G holds h |^ (- i) = (h |^ i) "
Lm13:
for j being Integer holds
( j >= 1 or j = 0 or j < 0 )
Lm14:
for j being Integer
for G being Group
for h being Element of G holds h |^ (j - 1) = (h |^ j) * (h |^ (- 1))
Lm15:
for j being Integer holds
( j >= 0 or j = - 1 or j < - 1 )
Lm16:
for j being Integer
for G being Group
for h being Element of G holds h |^ (j + 1) = (h |^ j) * (h |^ 1)
theorem Th63:
theorem
canceled;
theorem
canceled;
theorem
Lm17:
for i being Integer
for G being Group
for h being Element of G holds (h ") |^ i = (h |^ i) "
theorem
theorem
canceled;
theorem
canceled;
theorem
theorem
canceled;
theorem
theorem Th73:
theorem Th74:
theorem
canceled;
theorem
canceled;
theorem
:: deftheorem Def11 defines being_of_order_0 GROUP_1:def 11 :
for G being Group
for h being Element of G holds
( h is being_of_order_0 iff for n being Nat st h |^ n = 1_ G holds
n = 0 );
theorem
canceled;
theorem
canceled;
:: deftheorem Def12 defines ord GROUP_1:def 12 :
for G being Group
for h being Element of G
for b3 being Element of NAT holds
( ( h is being_of_order_0 implies ( b3 = ord h iff b3 = 0 ) ) & ( not h is being_of_order_0 implies ( b3 = ord h iff ( h |^ b3 = 1_ G & b3 <> 0 & ( for m being Nat st h |^ m = 1_ G & m <> 0 holds
b3 <= m ) ) ) ) );
theorem
canceled;
theorem
canceled;
theorem Th82:
theorem
canceled;
theorem
theorem
theorem
:: deftheorem GROUP_1:def 13 :
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
:: deftheorem GROUP_1:def 14 :
canceled;
:: deftheorem GROUP_1:def 15 :
canceled;
:: deftheorem Def16 defines commutative GROUP_1:def 16 :
for IT being multMagma holds
( IT is commutative iff for x, y being Element of IT holds x * y = y * x );
theorem
canceled;
theorem
theorem
canceled;
theorem
theorem
canceled;
theorem
theorem
begin
theorem Th98:
theorem
theorem
:: deftheorem defines unity-preserving GROUP_1:def 17 :
for G, H being multMagma
for IT being Function of G,H holds
( IT is unity-preserving iff IT . (1_ G) = 1_ H );