begin
theorem Th1:
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem Th7:
theorem Th8:
theorem Th9:
theorem Th10:
theorem Th11:
theorem Th12:
theorem Th13:
Lm1:
for n being Element of NAT
for x1, x2 being Element of REAL n st x1 <> x2 holds
|.(x1 - x2).| <> 0
theorem Th14:
theorem Th15:
theorem Th16:
theorem Th17:
theorem Th18:
theorem Th19:
theorem
theorem Th21:
theorem Th22:
theorem Th23:
theorem
theorem Th25:
theorem Th26:
theorem Th27:
theorem Th28:
theorem Th29:
for
a1,
a2,
a3,
b1,
b2,
b3 being
Real for
n being
Element of
NAT for
x1,
x2,
x3 being
Element of
REAL n holds
(((a1 * x1) + (a2 * x2)) + (a3 * x3)) + (((b1 * x1) + (b2 * x2)) + (b3 * x3)) = (((a1 + b1) * x1) + ((a2 + b2) * x2)) + ((a3 + b3) * x3)
theorem Th30:
theorem Th31:
for
a1,
a2,
a3,
b1,
b2,
b3 being
Real for
n being
Element of
NAT for
x1,
x2,
x3 being
Element of
REAL n holds
(((a1 * x1) + (a2 * x2)) + (a3 * x3)) - (((b1 * x1) + (b2 * x2)) + (b3 * x3)) = (((a1 - b1) * x1) + ((a2 - b2) * x2)) + ((a3 - b3) * x3)
theorem Th32:
for
a1,
a2,
a3 being
Real for
n being
Element of
NAT for
x1,
x2,
x3 being
Element of
REAL n st
(a1 + a2) + a3 = 1 holds
((a1 * x1) + (a2 * x2)) + (a3 * x3) = (x1 + (a2 * (x2 - x1))) + (a3 * (x3 - x1))
theorem Th33:
for
a2,
a3 being
Real for
n being
Element of
NAT for
x,
x1,
x2,
x3 being
Element of
REAL n st
x = (x1 + (a2 * (x2 - x1))) + (a3 * (x3 - x1)) holds
ex
a1 being
Real st
(
x = ((a1 * x1) + (a2 * x2)) + (a3 * x3) &
(a1 + a2) + a3 = 1 )
theorem
theorem Th35:
theorem Th36:
:: deftheorem Def1 defines // EUCLIDLP:def 1 :
for n being Element of NAT
for x1, x2 being Element of REAL n holds
( x1 // x2 iff ( x1 <> 0* n & x2 <> 0* n & ex r being Real st x1 = r * x2 ) );
theorem Th37:
theorem Th38:
:: deftheorem Def2 defines are_lindependent2 EUCLIDLP:def 2 :
for n being Element of NAT
for x1, x2 being Element of REAL n holds
( x1,x2 are_lindependent2 iff for a1, a2 being Real st (a1 * x1) + (a2 * x2) = 0* n holds
( a1 = 0 & a2 = 0 ) );
Lm2:
for n being Element of NAT
for x1, x2 being Element of REAL n st x1,x2 are_lindependent2 holds
x1 <> 0* n
theorem
theorem Th40:
theorem Th41:
for
a1,
a2,
b1,
b2 being
Real for
n being
Element of
NAT for
y2,
x1,
x2,
y1,
y1 being
Element of
REAL n st
y1,
y2 are_lindependent2 &
y1 = (a1 * x1) + (a2 * x2) &
y2 = (b1 * x1) + (b2 * x2) holds
ex
c1,
c2,
d1,
d2 being
Real st
(
x1 = (c1 * y1) + (c2 * y2) &
x2 = (d1 * y1) + (d2 * y2) )
theorem Th42:
theorem
theorem
theorem Th45:
for
n being
Element of
NAT for
x1,
x0,
x3,
x2,
y0,
y1,
y2,
y3 being
Element of
REAL n st
x1 - x0,
x3 - x2 are_lindependent2 &
y0 in Line (
x0,
x1) &
y1 in Line (
x0,
x1) &
y0 <> y1 &
y2 in Line (
x2,
x3) &
y3 in Line (
x2,
x3) &
y2 <> y3 holds
y1 - y0,
y3 - y2 are_lindependent2
Lm3:
for n being Element of NAT
for x1, x2 being Element of REAL n st x1 // x2 holds
x1,x2 are_ldependent2
theorem
Lm4:
for n being Element of NAT
for x1, x2 being Element of REAL n st x1,x2 are_ldependent2 & x1 <> 0* n & x2 <> 0* n holds
x1 // x2
theorem
theorem Th48:
:: deftheorem Def3 defines _|_ EUCLIDLP:def 3 :
for n being Element of NAT
for x1, x2 being Element of REAL n holds
( x1 _|_ x2 iff ( x1 <> 0* n & x2 <> 0* n & x1,x2 are_orthogonal ) );
theorem Th49:
theorem Th50:
theorem
:: deftheorem defines line_of_REAL EUCLIDLP:def 4 :
for n being Element of NAT holds line_of_REAL n = { (Line (x1,x2)) where x1, x2 is Element of REAL n : verum } ;
theorem Th52:
theorem Th53:
theorem Th54:
theorem
theorem Th56:
theorem Th57:
theorem Th58:
theorem Th59:
theorem Th60:
:: deftheorem defines dist_v EUCLIDLP:def 5 :
for n being Element of NAT
for x being Element of REAL n
for L being Element of line_of_REAL n holds dist_v (x,L) = { |.(x - x0).| where x0 is Element of REAL n : x0 in L } ;
:: deftheorem defines dist EUCLIDLP:def 6 :
for n being Element of NAT
for x being Element of REAL n
for L being Element of line_of_REAL n holds dist (x,L) = lower_bound (dist_v (x,L));
theorem
theorem Th62:
theorem
theorem
definition
let n be
Element of
NAT ;
let L1,
L2 be
Element of
line_of_REAL n;
pred L1 // L2 means :
Def7:
ex
x1,
x2,
y1,
y2 being
Element of
REAL n st
(
L1 = Line (
x1,
x2) &
L2 = Line (
y1,
y2) &
x2 - x1 // y2 - y1 );
symmetry
for L1, L2 being Element of line_of_REAL n st ex x1, x2, y1, y2 being Element of REAL n st
( L1 = Line (x1,x2) & L2 = Line (y1,y2) & x2 - x1 // y2 - y1 ) holds
ex x1, x2, y1, y2 being Element of REAL n st
( L2 = Line (x1,x2) & L1 = Line (y1,y2) & x2 - x1 // y2 - y1 )
;
end;
:: deftheorem Def7 defines // EUCLIDLP:def 7 :
for n being Element of NAT
for L1, L2 being Element of line_of_REAL n holds
( L1 // L2 iff ex x1, x2, y1, y2 being Element of REAL n st
( L1 = Line (x1,x2) & L2 = Line (y1,y2) & x2 - x1 // y2 - y1 ) );
theorem
definition
let n be
Element of
NAT ;
let L1,
L2 be
Element of
line_of_REAL n;
pred L1 _|_ L2 means :
Def8:
ex
x1,
x2,
y1,
y2 being
Element of
REAL n st
(
L1 = Line (
x1,
x2) &
L2 = Line (
y1,
y2) &
x2 - x1 _|_ y2 - y1 );
symmetry
for L1, L2 being Element of line_of_REAL n st ex x1, x2, y1, y2 being Element of REAL n st
( L1 = Line (x1,x2) & L2 = Line (y1,y2) & x2 - x1 _|_ y2 - y1 ) holds
ex x1, x2, y1, y2 being Element of REAL n st
( L2 = Line (x1,x2) & L1 = Line (y1,y2) & x2 - x1 _|_ y2 - y1 )
;
end;
:: deftheorem Def8 defines _|_ EUCLIDLP:def 8 :
for n being Element of NAT
for L1, L2 being Element of line_of_REAL n holds
( L1 _|_ L2 iff ex x1, x2, y1, y2 being Element of REAL n st
( L1 = Line (x1,x2) & L2 = Line (y1,y2) & x2 - x1 _|_ y2 - y1 ) );
theorem Th66:
theorem Th67:
theorem Th68:
theorem Th69:
theorem Th70:
theorem Th71:
theorem Th72:
theorem
theorem
theorem Th75:
theorem Th76:
theorem Th77:
theorem
theorem Th79:
theorem Th80:
theorem Th81:
theorem Th82:
theorem
for
n being
Element of
NAT for
x2,
x1,
x3,
y2,
y3 being
Element of
REAL n for
L1,
L2 being
Element of
line_of_REAL n st
x2 - x1,
x3 - x1 are_lindependent2 &
y2 in Line (
x1,
x2) &
y3 in Line (
x1,
x3) &
L1 = Line (
x2,
x3) &
L2 = Line (
y2,
y3) holds
(
L1 // L2 iff ex
a being
Real st
(
a <> 0 &
y2 - x1 = a * (x2 - x1) &
y3 - x1 = a * (x3 - x1) ) )
theorem Th84:
theorem Th85:
theorem Th86:
:: deftheorem defines plane EUCLIDLP:def 9 :
for n being Element of NAT
for x1, x2, x3 being Element of REAL n holds plane (x1,x2,x3) = { x where x is Element of REAL n : ex a1, a2, a3 being Real st
( (a1 + a2) + a3 = 1 & x = ((a1 * x1) + (a2 * x2)) + (a3 * x3) ) } ;
:: deftheorem Def10 defines being_plane EUCLIDLP:def 10 :
for n being Element of NAT
for A being Subset of (REAL n) holds
( A is being_plane iff ex x1, x2, x3 being Element of REAL n st
( x2 - x1,x3 - x1 are_lindependent2 & A = plane (x1,x2,x3) ) );
theorem Th87:
theorem Th88:
for
n being
Element of
NAT for
x1,
y1,
y2,
y3,
x2,
x3 being
Element of
REAL n st
x1 in plane (
y1,
y2,
y3) &
x2 in plane (
y1,
y2,
y3) &
x3 in plane (
y1,
y2,
y3) holds
plane (
x1,
x2,
x3)
c= plane (
y1,
y2,
y3)
theorem
theorem Th90:
for
n being
Element of
NAT for
y1,
x1,
x2,
x3,
y2 being
Element of
REAL n st
y1 in plane (
x1,
x2,
x3) &
y2 in plane (
x1,
x2,
x3) holds
Line (
y1,
y2)
c= plane (
x1,
x2,
x3)
theorem
theorem
theorem Th93:
theorem
:: deftheorem defines plane_of_REAL EUCLIDLP:def 11 :
for n being Element of NAT holds plane_of_REAL n = { P where P is Subset of (REAL n) : ex x1, x2, x3 being Element of REAL n st P = plane (x1,x2,x3) } ;
theorem Th95:
theorem Th96:
theorem Th97:
theorem
theorem
for
n being
Element of
NAT for
x1,
x2,
x3 being
Element of
REAL n holds
(
Line (
x1,
x2)
c= plane (
x1,
x2,
x3) &
Line (
x2,
x3)
c= plane (
x1,
x2,
x3) &
Line (
x3,
x1)
c= plane (
x1,
x2,
x3) )
theorem Th100:
:: deftheorem Def12 defines are_coplane EUCLIDLP:def 12 :
for n being Element of NAT
for L1, L2 being Element of line_of_REAL n holds
( L1,L2 are_coplane iff ex x1, x2, x3 being Element of REAL n st
( L1 c= plane (x1,x2,x3) & L2 c= plane (x1,x2,x3) ) );
theorem Th101:
theorem Th102:
theorem Th103:
theorem Th104:
theorem Th105:
theorem Th106:
theorem Th107:
theorem
theorem
theorem
theorem Th111:
theorem Th112:
theorem Th113:
theorem Th114:
theorem Th115:
theorem Th116:
theorem Th117:
theorem Th118:
theorem