Th1:
for n being Nat holds n = { m where m is Nat : m < n }
by AXIOMS:4;
theorem Th3:
for
n being
Nat for
x,
y being
object st
n = {x,y} &
x <> y & not (
x = 0 &
y = 1 ) holds
(
x = 1 &
y = 0 )
definition
let R be non
almost_trivial Ring;
let x be non
trivial Element of
R;
let o be
object ;
let a,
b be
Element of
carr (
x,
o);
func addR (
a,
b)
-> Element of
carr (
x,
o)
equals :
Def4:
the
addF of
R . (
x,
x)
if (
a = o &
b = o & the
addF of
R . (
x,
x)
<> x )
the
addF of
R . (
a,
x)
if (
a <> o &
b = o & the
addF of
R . (
a,
x)
<> x )
the
addF of
R . (
x,
b)
if (
a = o &
b <> o & the
addF of
R . (
x,
b)
<> x )
the
addF of
R . (
a,
b)
if (
a <> o &
b <> o & the
addF of
R . (
a,
b)
<> x )
otherwise o;
coherence
( ( a = o & b = o & the addF of R . (x,x) <> x implies the addF of R . (x,x) is Element of carr (x,o) ) & ( a <> o & b = o & the addF of R . (a,x) <> x implies the addF of R . (a,x) is Element of carr (x,o) ) & ( a = o & b <> o & the addF of R . (x,b) <> x implies the addF of R . (x,b) is Element of carr (x,o) ) & ( a <> o & b <> o & the addF of R . (a,b) <> x implies the addF of R . (a,b) is Element of carr (x,o) ) & ( ( not a = o or not b = o or not the addF of R . (x,x) <> x ) & ( not a <> o or not b = o or not the addF of R . (a,x) <> x ) & ( not a = o or not b <> o or not the addF of R . (x,b) <> x ) & ( not a <> o or not b <> o or not the addF of R . (a,b) <> x ) implies o is Element of carr (x,o) ) )
consistency
for b1 being Element of carr (x,o) holds
( ( a = o & b = o & the addF of R . (x,x) <> x & a <> o & b = o & the addF of R . (a,x) <> x implies ( b1 = the addF of R . (x,x) iff b1 = the addF of R . (a,x) ) ) & ( a = o & b = o & the addF of R . (x,x) <> x & a = o & b <> o & the addF of R . (x,b) <> x implies ( b1 = the addF of R . (x,x) iff b1 = the addF of R . (x,b) ) ) & ( a = o & b = o & the addF of R . (x,x) <> x & a <> o & b <> o & the addF of R . (a,b) <> x implies ( b1 = the addF of R . (x,x) iff b1 = the addF of R . (a,b) ) ) & ( a <> o & b = o & the addF of R . (a,x) <> x & a = o & b <> o & the addF of R . (x,b) <> x implies ( b1 = the addF of R . (a,x) iff b1 = the addF of R . (x,b) ) ) & ( a <> o & b = o & the addF of R . (a,x) <> x & a <> o & b <> o & the addF of R . (a,b) <> x implies ( b1 = the addF of R . (a,x) iff b1 = the addF of R . (a,b) ) ) & ( a = o & b <> o & the addF of R . (x,b) <> x & a <> o & b <> o & the addF of R . (a,b) <> x implies ( b1 = the addF of R . (x,b) iff b1 = the addF of R . (a,b) ) ) )
;
end;
::
deftheorem Def4 defines
addR FIELD_3:def 5 :
for R being non almost_trivial Ring
for x being non trivial Element of R
for o being object
for a, b being Element of carr (x,o) holds
( ( a = o & b = o & the addF of R . (x,x) <> x implies addR (a,b) = the addF of R . (x,x) ) & ( a <> o & b = o & the addF of R . (a,x) <> x implies addR (a,b) = the addF of R . (a,x) ) & ( a = o & b <> o & the addF of R . (x,b) <> x implies addR (a,b) = the addF of R . (x,b) ) & ( a <> o & b <> o & the addF of R . (a,b) <> x implies addR (a,b) = the addF of R . (a,b) ) & ( ( not a = o or not b = o or not the addF of R . (x,x) <> x ) & ( not a <> o or not b = o or not the addF of R . (a,x) <> x ) & ( not a = o or not b <> o or not the addF of R . (x,b) <> x ) & ( not a <> o or not b <> o or not the addF of R . (a,b) <> x ) implies addR (a,b) = o ) );
definition
let R be non
almost_trivial Ring;
let x be non
trivial Element of
R;
let o be
object ;
existence
ex b1 being BinOp of (carr (x,o)) st
for a, b being Element of carr (x,o) holds b1 . (a,b) = addR (a,b)
uniqueness
for b1, b2 being BinOp of (carr (x,o)) st ( for a, b being Element of carr (x,o) holds b1 . (a,b) = addR (a,b) ) & ( for a, b being Element of carr (x,o) holds b2 . (a,b) = addR (a,b) ) holds
b1 = b2
end;
definition
let R be non
almost_trivial Ring;
let x be non
trivial Element of
R;
let o be
object ;
let a,
b be
Element of
carr (
x,
o);
func multR (
a,
b)
-> Element of
carr (
x,
o)
equals :
Def6:
the
multF of
R . (
x,
x)
if (
a = o &
b = o & the
multF of
R . (
x,
x)
<> x )
the
multF of
R . (
a,
x)
if (
a <> o &
b = o & the
multF of
R . (
a,
x)
<> x )
the
multF of
R . (
x,
b)
if (
a = o &
b <> o & the
multF of
R . (
x,
b)
<> x )
the
multF of
R . (
a,
b)
if (
a <> o &
b <> o & the
multF of
R . (
a,
b)
<> x )
otherwise o;
coherence
( ( a = o & b = o & the multF of R . (x,x) <> x implies the multF of R . (x,x) is Element of carr (x,o) ) & ( a <> o & b = o & the multF of R . (a,x) <> x implies the multF of R . (a,x) is Element of carr (x,o) ) & ( a = o & b <> o & the multF of R . (x,b) <> x implies the multF of R . (x,b) is Element of carr (x,o) ) & ( a <> o & b <> o & the multF of R . (a,b) <> x implies the multF of R . (a,b) is Element of carr (x,o) ) & ( ( not a = o or not b = o or not the multF of R . (x,x) <> x ) & ( not a <> o or not b = o or not the multF of R . (a,x) <> x ) & ( not a = o or not b <> o or not the multF of R . (x,b) <> x ) & ( not a <> o or not b <> o or not the multF of R . (a,b) <> x ) implies o is Element of carr (x,o) ) )
consistency
for b1 being Element of carr (x,o) holds
( ( a = o & b = o & the multF of R . (x,x) <> x & a <> o & b = o & the multF of R . (a,x) <> x implies ( b1 = the multF of R . (x,x) iff b1 = the multF of R . (a,x) ) ) & ( a = o & b = o & the multF of R . (x,x) <> x & a = o & b <> o & the multF of R . (x,b) <> x implies ( b1 = the multF of R . (x,x) iff b1 = the multF of R . (x,b) ) ) & ( a = o & b = o & the multF of R . (x,x) <> x & a <> o & b <> o & the multF of R . (a,b) <> x implies ( b1 = the multF of R . (x,x) iff b1 = the multF of R . (a,b) ) ) & ( a <> o & b = o & the multF of R . (a,x) <> x & a = o & b <> o & the multF of R . (x,b) <> x implies ( b1 = the multF of R . (a,x) iff b1 = the multF of R . (x,b) ) ) & ( a <> o & b = o & the multF of R . (a,x) <> x & a <> o & b <> o & the multF of R . (a,b) <> x implies ( b1 = the multF of R . (a,x) iff b1 = the multF of R . (a,b) ) ) & ( a = o & b <> o & the multF of R . (x,b) <> x & a <> o & b <> o & the multF of R . (a,b) <> x implies ( b1 = the multF of R . (x,b) iff b1 = the multF of R . (a,b) ) ) )
;
end;
::
deftheorem Def6 defines
multR FIELD_3:def 7 :
for R being non almost_trivial Ring
for x being non trivial Element of R
for o being object
for a, b being Element of carr (x,o) holds
( ( a = o & b = o & the multF of R . (x,x) <> x implies multR (a,b) = the multF of R . (x,x) ) & ( a <> o & b = o & the multF of R . (a,x) <> x implies multR (a,b) = the multF of R . (a,x) ) & ( a = o & b <> o & the multF of R . (x,b) <> x implies multR (a,b) = the multF of R . (x,b) ) & ( a <> o & b <> o & the multF of R . (a,b) <> x implies multR (a,b) = the multF of R . (a,b) ) & ( ( not a = o or not b = o or not the multF of R . (x,x) <> x ) & ( not a <> o or not b = o or not the multF of R . (a,x) <> x ) & ( not a = o or not b <> o or not the multF of R . (x,b) <> x ) & ( not a <> o or not b <> o or not the multF of R . (a,b) <> x ) implies multR (a,b) = o ) );
definition
let R be non
almost_trivial Ring;
let x be non
trivial Element of
R;
let o be
object ;
existence
ex b1 being BinOp of (carr (x,o)) st
for a, b being Element of carr (x,o) holds b1 . (a,b) = multR (a,b)
uniqueness
for b1, b2 being BinOp of (carr (x,o)) st ( for a, b being Element of carr (x,o) holds b1 . (a,b) = multR (a,b) ) & ( for a, b being Element of carr (x,o) holds b2 . (a,b) = multR (a,b) ) holds
b1 = b2
end;
definition
let F be non
almost_trivial Field;
let x be non
trivial Element of
F;
let o be
object ;
existence
ex b1 being strict doubleLoopStr st
( the carrier of b1 = carr (x,o) & the addF of b1 = addR (x,o) & the multF of b1 = multR (x,o) & the OneF of b1 = 1. F & the ZeroF of b1 = 0. F )
uniqueness
for b1, b2 being strict doubleLoopStr st the carrier of b1 = carr (x,o) & the addF of b1 = addR (x,o) & the multF of b1 = multR (x,o) & the OneF of b1 = 1. F & the ZeroF of b1 = 0. F & the carrier of b2 = carr (x,o) & the addF of b2 = addR (x,o) & the multF of b2 = multR (x,o) & the OneF of b2 = 1. F & the ZeroF of b2 = 0. F holds
b1 = b2
;
end;
Lem2:
for R being Ring
for p being Polynomial of R
for r being Rational st r in RAT+ & p = r holds
r = [1,2]
Lem3:
for R being Ring
for p being Polynomial of R holds p <> [1,2]
Lem4:
for R being Ring
for p being Polynomial of R
for r being Real st r in REAL+ holds
p <> r