definition
let L1,
L2,
T1,
T2 be
RelStr ;
let f be
Function of
L1,
T1;
let g be
Function of
L2,
T2;
[:redefine func [:f,g:] -> Function of
[:L1,L2:],
[:T1,T2:];
coherence
[:f,g:] is Function of [:L1,L2:],[:T1,T2:]
end;
theorem Th37:
for
L being
complete continuous LATTICE for
R being
Subset of
[:L,L:] for
k being
kernel Function of
L,
L st
k is
directed-sups-preserving &
R = [:k,k:] " (id the carrier of L) holds
ex
LR being
strict complete continuous LATTICE st
( the
carrier of
LR = Class (EqRel R) & the
InternalRel of
LR = { [(Class ((EqRel R),x)),(Class ((EqRel R),y))] where x, y is Element of L : k . x <= k . y } & ( for
g being
Function of
L,
LR st ( for
x being
Element of
L holds
g . x = Class (
(EqRel R),
x) ) holds
g is
CLHomomorphism of
L,
LR ) )
definition
let L be
complete continuous LATTICE;
let R be non
empty Subset of
[:L,L:];
assume A1:
R is
CLCongruence
;
existence
ex b1 being strict complete continuous LATTICE st
( the carrier of b1 = Class (EqRel R) & ( for x, y being Element of b1 holds
( x <= y iff "/\" (x,L) <= "/\" (y,L) ) ) )
uniqueness
for b1, b2 being strict complete continuous LATTICE st the carrier of b1 = Class (EqRel R) & ( for x, y being Element of b1 holds
( x <= y iff "/\" (x,L) <= "/\" (y,L) ) ) & the carrier of b2 = Class (EqRel R) & ( for x, y being Element of b2 holds
( x <= y iff "/\" (x,L) <= "/\" (y,L) ) ) holds
b1 = b2
end;
:: Lemma 2.10, p. 61, see WAYBEL15:16