Lm1:
2 -' 1 = 2 - 1
by XREAL_0:def 2;
Lm2:
3 -' 1 = 3 - 1
by XREAL_0:def 2;
theorem Th2:
for
a,
b being
Real holds
( not
|.a.| = b or
a = b or
a = - b )
theorem Th29:
for
L being non
empty right_zeroed addLoopStr for
z0,
z1,
z2,
z3,
z4,
z5 being
Element of
L holds
<%z0,z1,z2%> + <%z3,z4,z5%> = <%(z0 + z3),(z1 + z4),(z2 + z5)%>
theorem
for
L being non
empty right_complementable add-associative right_zeroed addLoopStr for
z0,
z1,
z2,
z3,
z4,
z5 being
Element of
L holds
<%z0,z1,z2%> - <%z3,z4,z5%> = <%(z0 - z3),(z1 - z4),(z2 - z5)%>
lemmul:
for L being non empty right_complementable add-associative right_zeroed distributive doubleLoopStr
for p, q being Polynomial of L st p <> 0_. L & q <> 0_. L holds
(p *' q) . ((((len p) + (len q)) - 1) -' 1) = (p . ((len p) -' 1)) * (q . ((len q) -' 1))
Lm4:
for r being Real st 0 <= r & r <= 2 * PI & r / PI is rational & cos r is rational holds
cos r in {0,1,(- 1),(1 / 2),(- (1 / 2))}
Lm5:
for r being Real st 0 <= r & r <= 2 * PI & r / PI is rational & sin r is rational holds
sin r in {0,1,(- 1),(1 / 2),(- (1 / 2))}