begin
definition
canceled;canceled;func hcflat -> BinOp of
NAT means :
Def3:
for
m,
n being
Nat holds
it . (
m,
n)
= m gcd n;
existence
ex b1 being BinOp of NAT st
for m, n being Nat holds b1 . (m,n) = m gcd n
uniqueness
for b1, b2 being BinOp of NAT st ( for m, n being Nat holds b1 . (m,n) = m gcd n ) & ( for m, n being Nat holds b2 . (m,n) = m gcd n ) holds
b1 = b2
func lcmlat -> BinOp of
NAT means :
Def4:
for
m,
n being
Nat holds
it . (
m,
n)
= m lcm n;
existence
ex b1 being BinOp of NAT st
for m, n being Nat holds b1 . (m,n) = m lcm n
uniqueness
for b1, b2 being BinOp of NAT st ( for m, n being Nat holds b1 . (m,n) = m lcm n ) & ( for m, n being Nat holds b2 . (m,n) = m lcm n ) holds
b1 = b2
end;
:: deftheorem NAT_LAT:def 1 :
canceled;
:: deftheorem NAT_LAT:def 2 :
canceled;
:: deftheorem Def3 defines hcflat NAT_LAT:def 3 :
for b1 being BinOp of NAT holds
( b1 = hcflat iff for m, n being Nat holds b1 . (m,n) = m gcd n );
:: deftheorem Def4 defines lcmlat NAT_LAT:def 4 :
for b1 being BinOp of NAT holds
( b1 = lcmlat iff for m, n being Nat holds b1 . (m,n) = m lcm n );
:: deftheorem defines Nat_Lattice NAT_LAT:def 5 :
Nat_Lattice = LattStr(# NAT,lcmlat,hcflat #);
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
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
theorem
canceled;
theorem
canceled;
theorem
:: deftheorem defines 0_NN NAT_LAT:def 6 :
0_NN = 1;
:: deftheorem defines 1_NN NAT_LAT:def 7 :
1_NN = 0 ;
theorem
canceled;
theorem
canceled;
theorem
Lm1:
for a being Element of Nat_Lattice holds
( 0_NN "/\" a = 0_NN & a "/\" 0_NN = 0_NN )
by NEWTON:64;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem Th61:
theorem Th62:
theorem Th63:
theorem
for
p,
q,
r being
Element of
Nat_Lattice holds
(
lcmlat . (
p,
(lcmlat . (q,r)))
= lcmlat . (
(lcmlat . (q,p)),
r) &
lcmlat . (
p,
(lcmlat . (q,r)))
= lcmlat . (
(lcmlat . (p,r)),
q) &
lcmlat . (
p,
(lcmlat . (q,r)))
= lcmlat . (
(lcmlat . (r,q)),
p) &
lcmlat . (
p,
(lcmlat . (q,r)))
= lcmlat . (
(lcmlat . (r,p)),
q) )
theorem Th65:
theorem
for
p,
q,
r being
Element of
Nat_Lattice holds
(
hcflat . (
p,
(hcflat . (q,r)))
= hcflat . (
(hcflat . (q,p)),
r) &
hcflat . (
p,
(hcflat . (q,r)))
= hcflat . (
(hcflat . (p,r)),
q) &
hcflat . (
p,
(hcflat . (q,r)))
= hcflat . (
(hcflat . (r,q)),
p) &
hcflat . (
p,
(hcflat . (q,r)))
= hcflat . (
(hcflat . (r,p)),
q) )
theorem
theorem
:: deftheorem NAT_LAT:def 8 :
canceled;
:: deftheorem Def9 defines NATPLUS NAT_LAT:def 9 :
for b1 being Subset of NAT holds
( b1 = NATPLUS iff for n being Nat holds
( n in b1 iff 0 < n ) );
:: deftheorem Def10 defines @ NAT_LAT:def 10 :
for k being Nat st k > 0 holds
@ k = k;
definition
canceled;func hcflatplus -> BinOp of
NATPLUS means :
Def12:
for
m,
n being
NatPlus holds
it . (
m,
n)
= m gcd n;
existence
ex b1 being BinOp of NATPLUS st
for m, n being NatPlus holds b1 . (m,n) = m gcd n
uniqueness
for b1, b2 being BinOp of NATPLUS st ( for m, n being NatPlus holds b1 . (m,n) = m gcd n ) & ( for m, n being NatPlus holds b2 . (m,n) = m gcd n ) holds
b1 = b2
func lcmlatplus -> BinOp of
NATPLUS means :
Def13:
for
m,
n being
NatPlus holds
it . (
m,
n)
= m lcm n;
existence
ex b1 being BinOp of NATPLUS st
for m, n being NatPlus holds b1 . (m,n) = m lcm n
uniqueness
for b1, b2 being BinOp of NATPLUS st ( for m, n being NatPlus holds b1 . (m,n) = m lcm n ) & ( for m, n being NatPlus holds b2 . (m,n) = m lcm n ) holds
b1 = b2
end;
:: deftheorem NAT_LAT:def 11 :
canceled;
:: deftheorem Def12 defines hcflatplus NAT_LAT:def 12 :
for b1 being BinOp of NATPLUS holds
( b1 = hcflatplus iff for m, n being NatPlus holds b1 . (m,n) = m gcd n );
:: deftheorem Def13 defines lcmlatplus NAT_LAT:def 13 :
for b1 being BinOp of NATPLUS holds
( b1 = lcmlatplus iff for m, n being NatPlus holds b1 . (m,n) = m lcm n );
:: deftheorem defines NatPlus_Lattice NAT_LAT:def 14 :
NatPlus_Lattice = LattStr(# NATPLUS,lcmlatplus,hcflatplus #);
:: deftheorem defines @ NAT_LAT:def 15 :
for m being Element of NatPlus_Lattice holds @ m = m;
theorem
theorem
Lm2:
( ( for a, b being Element of NatPlus_Lattice holds a "\/" b = b "\/" a ) & ( for a, b, c being Element of NatPlus_Lattice holds a "\/" (b "\/" c) = (a "\/" b) "\/" c ) )
by NEWTON:56;
Lm3:
( ( for a, b being Element of NatPlus_Lattice holds (a "/\" b) "\/" b = b ) & ( for a, b being Element of NatPlus_Lattice holds a "/\" b = b "/\" a ) )
by NEWTON:66;
Lm4:
( ( for a, b, c being Element of NatPlus_Lattice holds a "/\" (b "/\" c) = (a "/\" b) "/\" c ) & ( for a, b being Element of NatPlus_Lattice holds a "/\" (a "\/" b) = a ) )
by NEWTON:61, NEWTON:67;
:: deftheorem Def16 defines SubLattice NAT_LAT:def 16 :
for L, b2 being Lattice holds
( b2 is SubLattice of L iff ( the carrier of b2 c= the carrier of L & the L_join of b2 = the L_join of L || the carrier of b2 & the L_meet of b2 = the L_meet of L || the carrier of b2 ) );
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
theorem