begin
theorem Th1:
theorem Th2:
for
r being
Real st
r > 0 holds
(
ln . r <= r - 1 & (
r = 1 implies
ln . r = r - 1 ) & (
ln . r = r - 1 implies
r = 1 ) & (
r <> 1 implies
ln . r < r - 1 ) & (
ln . r < r - 1 implies
r <> 1 ) )
theorem Th3:
theorem Th4:
for
a,
b being
Real st
a > 1 &
b > 1 holds
log (
a,
b)
> 0
theorem Th5:
theorem Th6:
theorem Th7:
theorem Th8:
theorem Th9:
:: deftheorem Def1 defines nonnegative ENTROPY1:def 1 :
for p being FinSequence of REAL holds
( p is nonnegative iff for i being Element of NAT st i in dom p holds
p . i >= 0 );
theorem Th10:
:: deftheorem Def2 defines has_onlyone_value_in ENTROPY1:def 2 :
for p being FinSequence of REAL
for k being Element of NAT holds
( p has_onlyone_value_in k iff ( k in dom p & ( for i being Element of NAT st i in dom p & i <> k holds
p . i = 0 ) ) );
theorem
theorem Th12:
theorem Th13:
theorem Th14:
theorem Th15:
theorem Th16:
theorem
theorem Th18:
theorem Th19:
begin
theorem Th20:
theorem Th21:
theorem Th22:
theorem Th23:
:: deftheorem Def3 defines diagonal ENTROPY1:def 3 :
for n being Nat
for MR being Matrix of n, REAL holds
( MR is diagonal iff for i, j being Element of NAT st [i,j] in Indices MR & MR * (i,j) <> 0 holds
i = j );
theorem Th24:
:: deftheorem Def4 defines Vec2DiagMx ENTROPY1:def 4 :
for p being FinSequence of REAL
for b2 being diagonal Matrix of len p, REAL holds
( b2 = Vec2DiagMx p iff for j being Element of NAT st j in dom p holds
b2 * (j,j) = p . j );
theorem Th25:
theorem Th26:
theorem Th27:
theorem Th28:
theorem Th29:
theorem Th30:
theorem Th31:
theorem Th32:
theorem Th33:
theorem Th34:
theorem Th35:
theorem Th36:
theorem Th37:
theorem Th38:
:: deftheorem Def5 defines Mx2FinS ENTROPY1:def 5 :
for D being non empty set
for M being Matrix of D
for b3 being FinSequence of D holds
( ( len M = 0 implies ( b3 = Mx2FinS M iff b3 = {} ) ) & ( not len M = 0 implies ( b3 = Mx2FinS M iff ex p being FinSequence of D * st
( b3 = p . (len M) & len p = len M & p . 1 = M . 1 & ( for k being Element of NAT st k >= 1 & k < len M holds
p . (k + 1) = (p . k) ^ (M . (k + 1)) ) ) ) ) );
theorem Th39:
theorem Th40:
theorem Th41:
theorem Th42:
theorem Th43:
theorem Th44:
theorem Th45:
theorem
begin
:: deftheorem Def6 defines FinSeq_log ENTROPY1:def 6 :
for a being Real
for p being FinSequence of REAL st p is nonnegative holds
for b3 being FinSequence of REAL holds
( b3 = FinSeq_log (a,p) iff ( len b3 = len p & ( for k being Nat st k in dom b3 holds
( ( p . k > 0 implies b3 . k = log (a,(p . k)) ) & ( p . k = 0 implies b3 . k = 0 ) ) ) ) );
:: deftheorem defines Infor_FinSeq_of ENTROPY1:def 7 :
for p being FinSequence of REAL holds Infor_FinSeq_of p = mlt (p,(FinSeq_log (2,p)));
theorem Th47:
theorem Th48:
theorem
theorem Th50:
theorem Th51:
theorem Th52:
definition
let MR be
Matrix of
REAL;
assume A1:
MR is
m-nonnegative
;
func Infor_FinSeq_of MR -> Matrix of
REAL means :
Def8:
(
len it = len MR &
width it = width MR & ( for
k being
Element of
NAT st
k in dom it holds
it . k = mlt (
(Line (MR,k)),
(FinSeq_log (2,(Line (MR,k))))) ) );
existence
ex b1 being Matrix of REAL st
( len b1 = len MR & width b1 = width MR & ( for k being Element of NAT st k in dom b1 holds
b1 . k = mlt ((Line (MR,k)),(FinSeq_log (2,(Line (MR,k))))) ) )
uniqueness
for b1, b2 being Matrix of REAL st len b1 = len MR & width b1 = width MR & ( for k being Element of NAT st k in dom b1 holds
b1 . k = mlt ((Line (MR,k)),(FinSeq_log (2,(Line (MR,k))))) ) & len b2 = len MR & width b2 = width MR & ( for k being Element of NAT st k in dom b2 holds
b2 . k = mlt ((Line (MR,k)),(FinSeq_log (2,(Line (MR,k))))) ) holds
b1 = b2
end;
:: deftheorem Def8 defines Infor_FinSeq_of ENTROPY1:def 8 :
for MR being Matrix of REAL st MR is m-nonnegative holds
for b2 being Matrix of REAL holds
( b2 = Infor_FinSeq_of MR iff ( len b2 = len MR & width b2 = width MR & ( for k being Element of NAT st k in dom b2 holds
b2 . k = mlt ((Line (MR,k)),(FinSeq_log (2,(Line (MR,k))))) ) ) );
theorem Th53:
theorem Th54:
:: deftheorem defines Entropy ENTROPY1:def 9 :
for p being FinSequence of REAL holds Entropy p = - (Sum (Infor_FinSeq_of p));
theorem
theorem
theorem Th57:
theorem
theorem Th59:
theorem Th60:
:: deftheorem defines Entropy_of_Joint_Prob ENTROPY1:def 10 :
for MR being Matrix of REAL holds Entropy_of_Joint_Prob MR = Entropy (Mx2FinS MR);
theorem
:: deftheorem Def11 defines Entropy_of_Cond_Prob ENTROPY1:def 11 :
for MR being Matrix of REAL
for b2 being FinSequence of REAL holds
( b2 = Entropy_of_Cond_Prob MR iff ( len b2 = len MR & ( for k being Element of NAT st k in dom b2 holds
b2 . k = Entropy (Line (MR,k)) ) ) );
theorem Th62:
theorem Th63:
theorem Th64:
theorem