begin
definition
let G be non
empty BCIStr_0 ;
func BCI-power G -> Function of
[: the carrier of G,NAT:], the
carrier of
G means :
Def1:
for
x being
Element of
G holds
(
it . (
x,
0)
= 0. G & ( for
n being
Element of
NAT holds
it . (
x,
(n + 1))
= x \ ((it . (x,n)) `) ) );
existence
ex b1 being Function of [: the carrier of G,NAT:], the carrier of G st
for x being Element of G holds
( b1 . (x,0) = 0. G & ( for n being Element of NAT holds b1 . (x,(n + 1)) = x \ ((b1 . (x,n)) `) ) )
uniqueness
for b1, b2 being Function of [: the carrier of G,NAT:], the carrier of G st ( for x being Element of G holds
( b1 . (x,0) = 0. G & ( for n being Element of NAT holds b1 . (x,(n + 1)) = x \ ((b1 . (x,n)) `) ) ) ) & ( for x being Element of G holds
( b2 . (x,0) = 0. G & ( for n being Element of NAT holds b2 . (x,(n + 1)) = x \ ((b2 . (x,n)) `) ) ) ) holds
b1 = b2
end;
:: deftheorem Def1 defines BCI-power BCIALG_6:def 1 :
for G being non empty BCIStr_0
for b2 being Function of [: the carrier of G,NAT:], the carrier of G holds
( b2 = BCI-power G iff for x being Element of G holds
( b2 . (x,0) = 0. G & ( for n being Element of NAT holds b2 . (x,(n + 1)) = x \ ((b2 . (x,n)) `) ) ) );
:: deftheorem Def2 defines |^ BCIALG_6:def 2 :
for X being BCI-algebra
for i being Integer
for x being Element of X holds
( ( 0 <= i implies x |^ i = (BCI-power X) . (x,(abs i)) ) & ( not 0 <= i implies x |^ i = (BCI-power X) . ((x `),(abs i)) ) );
:: deftheorem defines |^ BCIALG_6:def 3 :
for X being BCI-algebra
for n being Nat
for x being Element of X holds x |^ n = (BCI-power X) . (x,n);
theorem Th1:
theorem Th2:
theorem Th3:
theorem Th4:
theorem Th5:
theorem
theorem Th7:
theorem
theorem
theorem Th10:
theorem
theorem
theorem Th13:
theorem Th14:
Lm1:
for X being BCI-algebra
for a being Element of AtomSet X
for n, m being Nat holds a |^ (n + m) = (a |^ m) \ ((a |^ n) `)
Lm2:
for X being BCI-algebra
for a being Element of AtomSet X
for m, n being Nat holds (a |^ m) |^ n = a |^ (m * n)
theorem Th15:
theorem
theorem Th17:
theorem Th18:
theorem
theorem Th20:
theorem Th21:
Lm3:
for X being BCI-algebra
for a being Element of AtomSet X
for i, j being Integer st i > 0 & j > 0 holds
(a |^ i) \ (a |^ j) = a |^ (i - j)
theorem Th22:
theorem Th23:
theorem Th24:
:: deftheorem Def4 defines finite-period BCIALG_6:def 4 :
for X being BCI-algebra
for x being Element of X holds
( x is finite-period iff ex n being Element of NAT st
( n <> 0 & x |^ n in BCK-part X ) );
theorem Th25:
:: deftheorem Def5 defines ord BCIALG_6:def 5 :
for X being BCI-algebra
for x being Element of X st x is finite-period holds
for b3 being Element of NAT holds
( b3 = ord x iff ( x |^ b3 in BCK-part X & b3 <> 0 & ( for m being Element of NAT st x |^ m in BCK-part X & m <> 0 holds
b3 <= m ) ) );
theorem Th26:
theorem
theorem Th28:
theorem Th29:
theorem
theorem
theorem
theorem
begin
theorem Th34:
:: deftheorem Def6 defines multiplicative BCIALG_6:def 6 :
for X, X9 being non empty BCIStr_0
for f being Function of X,X9 holds
( f is multiplicative iff for a, b being Element of X holds f . (a \ b) = (f . a) \ (f . b) );
:: deftheorem defines isotonic BCIALG_6:def 7 :
for X, X9 being BCI-algebra
for f being BCI-homomorphism of X,X9 holds
( f is isotonic iff for x, y being Element of X st x <= y holds
f . x <= f . y );
:: deftheorem defines Ker BCIALG_6:def 8 :
for X, X9 being BCI-algebra
for f being BCI-homomorphism of X,X9 holds Ker f = { x where x is Element of X : f . x = 0. X9 } ;
theorem Th35:
theorem
theorem
theorem
theorem
theorem
canceled;
theorem
theorem Th42:
theorem Th43:
theorem
theorem
theorem Th46:
theorem
theorem Th48:
theorem
:: deftheorem Def9 defines are_isomorphic BCIALG_6:def 9 :
for X, X9 being BCI-algebra holds
( X,X9 are_isomorphic iff ex f being BCI-homomorphism of X,X9 st f is bijective );
:: deftheorem Def10 defines nat_hom BCIALG_6:def 10 :
for X being BCI-algebra
for I being Ideal of X
for RI being I-congruence of X,I
for b4 being BCI-homomorphism of X,(X ./. RI) holds
( b4 = nat_hom RI iff for x being Element of X holds b4 . x = Class (RI,x) );
begin
theorem
theorem Th51:
theorem
theorem
Lm4:
for X9, X being BCI-algebra
for H9 being SubAlgebra of X9
for f being BCI-homomorphism of X,X9 st the carrier of H9 = rng f holds
f is BCI-homomorphism of X,H9
begin
theorem
theorem Th55:
begin
:: deftheorem defines Union BCIALG_6:def 11 :
for X being BCI-algebra
for G being SubAlgebra of X
for K being closed Ideal of X
for RK being I-congruence of X,K holds Union (G,RK) = union { (Class (RK,a)) where a is Element of G : Class (RK,a) in the carrier of (X ./. RK) } ;
Lm5:
for X being BCI-algebra
for G being SubAlgebra of X
for K being closed Ideal of X
for RK being I-congruence of X,K
for w being Element of Union (G,RK) ex a being Element of G st w in Class (RK,a)
definition
let X be
BCI-algebra;
let G be
SubAlgebra of
X;
let K be
closed Ideal of
X;
let RK be
I-congruence of
X,
K;
func HKOp (
G,
RK)
-> BinOp of
(Union (G,RK)) means :
Def12:
for
w1,
w2 being
Element of
Union (
G,
RK)
for
x,
y being
Element of
X st
w1 = x &
w2 = y holds
it . (
w1,
w2)
= x \ y;
existence
ex b1 being BinOp of (Union (G,RK)) st
for w1, w2 being Element of Union (G,RK)
for x, y being Element of X st w1 = x & w2 = y holds
b1 . (w1,w2) = x \ y
uniqueness
for b1, b2 being BinOp of (Union (G,RK)) st ( for w1, w2 being Element of Union (G,RK)
for x, y being Element of X st w1 = x & w2 = y holds
b1 . (w1,w2) = x \ y ) & ( for w1, w2 being Element of Union (G,RK)
for x, y being Element of X st w1 = x & w2 = y holds
b2 . (w1,w2) = x \ y ) holds
b1 = b2
end;
:: deftheorem Def12 defines HKOp BCIALG_6:def 12 :
for X being BCI-algebra
for G being SubAlgebra of X
for K being closed Ideal of X
for RK being I-congruence of X,K
for b5 being BinOp of (Union (G,RK)) holds
( b5 = HKOp (G,RK) iff for w1, w2 being Element of Union (G,RK)
for x, y being Element of X st w1 = x & w2 = y holds
b5 . (w1,w2) = x \ y );
:: deftheorem defines zeroHK BCIALG_6:def 13 :
for X being BCI-algebra
for G being SubAlgebra of X
for K being closed Ideal of X
for RK being I-congruence of X,K holds zeroHK (G,RK) = 0. X;
definition
let X be
BCI-algebra;
let G be
SubAlgebra of
X;
let K be
closed Ideal of
X;
let RK be
I-congruence of
X,
K;
func HK (
G,
RK)
-> BCIStr_0 equals
BCIStr_0(#
(Union (G,RK)),
(HKOp (G,RK)),
(zeroHK (G,RK)) #);
coherence
BCIStr_0(# (Union (G,RK)),(HKOp (G,RK)),(zeroHK (G,RK)) #) is BCIStr_0
;
end;
:: deftheorem defines HK BCIALG_6:def 14 :
for X being BCI-algebra
for G being SubAlgebra of X
for K being closed Ideal of X
for RK being I-congruence of X,K holds HK (G,RK) = BCIStr_0(# (Union (G,RK)),(HKOp (G,RK)),(zeroHK (G,RK)) #);
:: deftheorem defines \ BCIALG_6:def 15 :
for X being BCI-algebra
for G being SubAlgebra of X
for K being closed Ideal of X
for RK being I-congruence of X,K
for w1, w2 being Element of Union (G,RK) holds w1 \ w2 = (HKOp (G,RK)) . (w1,w2);
theorem Th56:
theorem Th57:
theorem
theorem