begin
theorem
canceled;
theorem Th2:
Lm1:
for a, b being real number holds 0 <= (a ^2) + (b ^2)
definition
let z be
complex number ;
canceled;func Re z -> set means :
Def2:
it = z if z in REAL otherwise ex
f being
Function of 2,
REAL st
(
z = f &
it = f . 0 );
existence
( ( z in REAL implies ex b1 being set st b1 = z ) & ( not z in REAL implies ex b1 being set ex f being Function of 2,REAL st
( z = f & b1 = f . 0 ) ) )
uniqueness
for b1, b2 being set holds
( ( z in REAL & b1 = z & b2 = z implies b1 = b2 ) & ( not z in REAL & ex f being Function of 2,REAL st
( z = f & b1 = f . 0 ) & ex f being Function of 2,REAL st
( z = f & b2 = f . 0 ) implies b1 = b2 ) )
;
consistency
for b1 being set holds verum
;
func Im z -> set means :
Def3:
it = 0 if z in REAL otherwise ex
f being
Function of 2,
REAL st
(
z = f &
it = f . 1 );
existence
( ( z in REAL implies ex b1 being set st b1 = 0 ) & ( not z in REAL implies ex b1 being set ex f being Function of 2,REAL st
( z = f & b1 = f . 1 ) ) )
uniqueness
for b1, b2 being set holds
( ( z in REAL & b1 = 0 & b2 = 0 implies b1 = b2 ) & ( not z in REAL & ex f being Function of 2,REAL st
( z = f & b1 = f . 1 ) & ex f being Function of 2,REAL st
( z = f & b2 = f . 1 ) implies b1 = b2 ) )
;
consistency
for b1 being set holds verum
;
end;
:: deftheorem COMPLEX1:def 1 :
canceled;
:: deftheorem Def2 defines Re COMPLEX1:def 2 :
for z being complex number
for b2 being set holds
( ( z in REAL implies ( b2 = Re z iff b2 = z ) ) & ( not z in REAL implies ( b2 = Re z iff ex f being Function of 2,REAL st
( z = f & b2 = f . 0 ) ) ) );
:: deftheorem Def3 defines Im COMPLEX1:def 3 :
for z being complex number
for b2 being set holds
( ( z in REAL implies ( b2 = Im z iff b2 = 0 ) ) & ( not z in REAL implies ( b2 = Im z iff ex f being Function of 2,REAL st
( z = f & b2 = f . 1 ) ) ) );
theorem
canceled;
theorem
canceled;
theorem Th5:
Lm2:
for a, b being Element of REAL holds
( Re [*a,b*] = a & Im [*a,b*] = b )
Lm3:
for z being complex number holds [*(Re z),(Im z)*] = z
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem Th9:
:: deftheorem COMPLEX1:def 4 :
canceled;
:: deftheorem defines = COMPLEX1:def 5 :
for z1, z2 being complex number holds
( z1 = z2 iff ( Re z1 = Re z2 & Im z1 = Im z2 ) );
:: deftheorem COMPLEX1:def 6 :
canceled;
:: deftheorem defines 1r COMPLEX1:def 7 :
1r = 1;
Lm4:
0 = [*0,0*]
by ARYTM_0:def 7;
Lm5:
1r = [*1,0*]
by ARYTM_0:def 7;
theorem
canceled;
theorem
canceled;
theorem Th12:
theorem Th13:
theorem
canceled;
theorem Th15:
theorem
canceled;
Lm6:
<i> = [*0,1*]
by ARYTM_0:def 7, XCMPLX_0:def 1;
theorem Th17:
Lm7:
for x being real number
for x1, x2 being Element of REAL st x = [*x1,x2*] holds
( x2 = 0 & x = x1 )
Lm8:
for x9, y9 being Element of REAL
for x, y being real number st x9 = x & y9 = y holds
+ (x9,y9) = x + y
Lm9:
for x being Element of REAL holds opp x = - x
Lm10:
for x9, y9 being Element of REAL
for x, y being real number st x9 = x & y9 = y holds
* (x9,y9) = x * y
Lm11:
for x, y, z being complex number st z = x + y holds
Re z = (Re x) + (Re y)
Lm12:
for x, y, z being complex number st z = x + y holds
Im z = (Im x) + (Im y)
Lm13:
for x, y, z being complex number st z = x * y holds
Re z = ((Re x) * (Re y)) - ((Im x) * (Im y))
Lm14:
for x, y, z being complex number st z = x * y holds
Im z = ((Re x) * (Im y)) + ((Im x) * (Re y))
Lm15:
for z1, z2 being complex number holds z1 + z2 = [*((Re z1) + (Re z2)),((Im z1) + (Im z2))*]
Lm16:
for z1, z2 being complex number holds z1 * z2 = [*(((Re z1) * (Re z2)) - ((Im z1) * (Im z2))),(((Re z1) * (Im z2)) + ((Re z2) * (Im z1)))*]
Lm17:
for z1, z2 being complex number holds
( Re (z1 * z2) = ((Re z1) * (Re z2)) - ((Im z1) * (Im z2)) & Im (z1 * z2) = ((Re z1) * (Im z2)) + ((Re z2) * (Im z1)) )
Lm18:
for z1, z2 being complex number holds
( Re (z1 + z2) = (Re z1) + (Re z2) & Im (z1 + z2) = (Im z1) + (Im z2) )
Lm19:
for x being Real holds Re (x * <i>) = 0
Lm20:
for x being Real holds Im (x * <i>) = x
Lm21:
for x, y being Real holds [*x,y*] = x + (y * <i>)
:: deftheorem COMPLEX1:def 8 :
canceled;
:: deftheorem defines + COMPLEX1:def 9 :
for z1, z2 being Element of COMPLEX holds z1 + z2 = ((Re z1) + (Re z2)) + (((Im z1) + (Im z2)) * <i>);
theorem
canceled;
theorem Th19:
:: deftheorem defines * COMPLEX1:def 10 :
for z1, z2 being Element of COMPLEX holds z1 * z2 = (((Re z1) * (Re z2)) - ((Im z1) * (Im z2))) + ((((Re z1) * (Im z2)) + ((Re z2) * (Im z1))) * <i>);
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem Th24:
theorem
theorem
theorem
canceled;
theorem Th28:
theorem Th29:
theorem Th30:
theorem Th31:
theorem
:: deftheorem Def11 defines - COMPLEX1:def 11 :
for z being Element of COMPLEX holds - z = (- (Re z)) + ((- (Im z)) * <i>);
theorem
canceled;
theorem Th34:
theorem
canceled;
theorem
canceled;
theorem
:: deftheorem Def12 defines - COMPLEX1:def 12 :
for z1, z2 being Element of COMPLEX holds z1 - z2 = ((Re z1) - (Re z2)) + (((Im z1) - (Im z2)) * <i>);
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem Th48:
:: deftheorem Def13 defines " COMPLEX1:def 13 :
for z being Element of COMPLEX holds z " = ((Re z) / (((Re z) ^2) + ((Im z) ^2))) + (((- (Im z)) / (((Re z) ^2) + ((Im z) ^2))) * <i>);
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem Th64:
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem Th79:
theorem Th80:
:: deftheorem Def14 defines / COMPLEX1:def 14 :
for z1, z2 being complex number holds z1 / z2 = ((((Re z1) * (Re z2)) + ((Im z1) * (Im z2))) / (((Re z2) ^2) + ((Im z2) ^2))) + (((((Re z2) * (Im z1)) - ((Re z1) * (Im z2))) / (((Re z2) ^2) + ((Im z2) ^2))) * <i>);
theorem
canceled;
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;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
theorem
:: deftheorem defines *' COMPLEX1:def 15 :
for z being complex number holds z *' = (Re z) - ((Im z) * <i>);
theorem
canceled;
theorem Th112:
theorem
theorem
theorem
theorem
theorem
canceled;
theorem Th118:
theorem Th119:
theorem
theorem Th121:
theorem Th122:
theorem
theorem
theorem
theorem
theorem
theorem
:: deftheorem defines |. COMPLEX1:def 16 :
for z being complex number holds |.z.| = sqrt (((Re z) ^2) + ((Im z) ^2));
theorem Th129:
theorem
theorem
theorem
theorem
theorem Th134:
theorem
Lm22:
for z being complex number holds |.(- z).| = |.z.|
Lm23:
for a being real number st a <= 0 holds
|.a.| = - a
Lm24:
for a being real number holds sqrt (a ^2) = |.a.|
theorem
theorem
theorem
theorem Th139:
Lm25:
for a being real number holds
( - |.a.| <= a & a <= |.a.| )
theorem
theorem
theorem Th142:
theorem Th143:
theorem
theorem Th145:
theorem Th146:
theorem Th147:
theorem
theorem
Lm26:
for b, a being real number holds
( ( - b <= a & a <= b ) iff |.a.| <= b )
theorem
theorem Th151:
theorem Th152:
theorem Th153:
theorem
theorem
theorem
theorem Th157:
theorem
theorem
theorem
theorem Th161:
theorem
theorem
theorem
theorem
theorem