:: FUNCT_7 semantic presentation
theorem Th1: :: FUNCT_7:1
theorem Th2: :: FUNCT_7:2
theorem Th3: :: FUNCT_7:3
theorem Th4: :: FUNCT_7:4
theorem Th5: :: FUNCT_7:5
theorem Th6: :: FUNCT_7:6
theorem Th7: :: FUNCT_7:7
theorem Th8: :: FUNCT_7:8
theorem Th9: :: FUNCT_7:9
canceled;
theorem Th10: :: FUNCT_7:10
theorem Th11: :: FUNCT_7:11
theorem Th12: :: FUNCT_7:12
theorem Th13: :: FUNCT_7:13
theorem Th14: :: FUNCT_7:14
theorem Th15: :: FUNCT_7:15
theorem Th16: :: FUNCT_7:16
theorem Th17: :: FUNCT_7:17
canceled;
theorem Th18: :: FUNCT_7:18
theorem Th19: :: FUNCT_7:19
theorem Th20: :: FUNCT_7:20
theorem Th21: :: FUNCT_7:21
for
A,
B being
set st
A * c= B * holds
A c= B
theorem Th22: :: FUNCT_7:22
theorem Th23: :: FUNCT_7:23
theorem Th24: :: FUNCT_7:24
theorem Th25: :: FUNCT_7:25
:: deftheorem Def1 defines In FUNCT_7:def 1 :
for
x,
y being
set st
x in y holds
In x,
y = x;
theorem Th26: :: FUNCT_7:26
:: deftheorem Def2 defines equal_outside FUNCT_7:def 2 :
theorem Th27: :: FUNCT_7:27
theorem Th28: :: FUNCT_7:28
theorem Th29: :: FUNCT_7:29
theorem Th30: :: FUNCT_7:30
theorem Th31: :: FUNCT_7:31
:: deftheorem Def3 defines +* FUNCT_7:def 3 :
theorem Th32: :: FUNCT_7:32
theorem Th33: :: FUNCT_7:33
theorem Th34: :: FUNCT_7:34
theorem Th35: :: FUNCT_7:35
theorem Th36: :: FUNCT_7:36
theorem Th37: :: FUNCT_7:37
theorem Th38: :: FUNCT_7:38
theorem Th39: :: FUNCT_7:39
theorem Th40: :: FUNCT_7:40
:: deftheorem Def4 defines compose FUNCT_7:def 4 :
:: deftheorem Def5 defines apply FUNCT_7:def 5 :
theorem Th41: :: FUNCT_7:41
theorem Th42: :: FUNCT_7:42
theorem Th43: :: FUNCT_7:43
theorem Th44: :: FUNCT_7:44
theorem Th45: :: FUNCT_7:45
theorem Th46: :: FUNCT_7:46
theorem Th47: :: FUNCT_7:47
theorem Th48: :: FUNCT_7:48
theorem Th49: :: FUNCT_7:49
theorem Th50: :: FUNCT_7:50
theorem Th51: :: FUNCT_7:51
theorem Th52: :: FUNCT_7:52
theorem Th53: :: FUNCT_7:53
theorem Th54: :: FUNCT_7:54
theorem Th55: :: FUNCT_7:55
theorem Th56: :: FUNCT_7:56
theorem Th57: :: FUNCT_7:57
theorem Th58: :: FUNCT_7:58
:: deftheorem Def6 defines firstdom FUNCT_7:def 6 :
:: deftheorem Def7 defines lastrng FUNCT_7:def 7 :
theorem Th59: :: FUNCT_7:59
theorem Th60: :: FUNCT_7:60
theorem Th61: :: FUNCT_7:61
:: deftheorem Def8 defines FuncSeq-like FUNCT_7:def 8 :
theorem Th62: :: FUNCT_7:62
theorem Th63: :: FUNCT_7:63
theorem Th64: :: FUNCT_7:64
theorem Th65: :: FUNCT_7:65
theorem Th66: :: FUNCT_7:66
theorem Th67: :: FUNCT_7:67
:: deftheorem Def9 defines FuncSequence FUNCT_7:def 9 :
:: deftheorem Def10 defines FuncSequence FUNCT_7:def 10 :
theorem Th68: :: FUNCT_7:68
theorem Th69: :: FUNCT_7:69
Lemma133:
for X being set
for f being Function of X,X holds rng f c= dom f
Lemma134:
for f being Function
for n being Element of NAT
for p1, p2 being Function of NAT , PFuncs ((dom f) \/ (rng f)),((dom f) \/ (rng f)) st p1 . 0 = id ((dom f) \/ (rng f)) & ( for k being Element of NAT ex g being Function st
( g = p1 . k & p1 . (k + 1) = g * f ) ) & p2 . 0 = id ((dom f) \/ (rng f)) & ( for k being Element of NAT ex g being Function st
( g = p2 . k & p2 . (k + 1) = g * f ) ) holds
p1 = p2
definition
let f be
Function;
let n be
Nat;
func iter c1,
c2 -> Function means :
Def11:
:: FUNCT_7:def 11
ex
p being
Function of
NAT ,
PFuncs ((dom f) \/ (rng f)),
((dom f) \/ (rng f)) st
(
it = p . n &
p . 0
= id ((dom f) \/ (rng f)) & ( for
k being
Element of
NAT ex
g being
Function st
(
g = p . k &
p . (k + 1) = g * f ) ) );
existence
ex b1 being Function ex p being Function of NAT , PFuncs ((dom f) \/ (rng f)),((dom f) \/ (rng f)) st
( b1 = p . n & p . 0 = id ((dom f) \/ (rng f)) & ( for k being Element of NAT ex g being Function st
( g = p . k & p . (k + 1) = g * f ) ) )
uniqueness
for b1, b2 being Function st ex p being Function of NAT , PFuncs ((dom f) \/ (rng f)),((dom f) \/ (rng f)) st
( b1 = p . n & p . 0 = id ((dom f) \/ (rng f)) & ( for k being Element of NAT ex g being Function st
( g = p . k & p . (k + 1) = g * f ) ) ) & ex p being Function of NAT , PFuncs ((dom f) \/ (rng f)),((dom f) \/ (rng f)) st
( b2 = p . n & p . 0 = id ((dom f) \/ (rng f)) & ( for k being Element of NAT ex g being Function st
( g = p . k & p . (k + 1) = g * f ) ) ) holds
b1 = b2
by ;
end;
:: deftheorem Def11 defines iter FUNCT_7:def 11 :
Lemma140:
for f being Function holds
( (id ((dom f) \/ (rng f))) * f = f & f * (id ((dom f) \/ (rng f))) = f )
theorem Th70: :: FUNCT_7:70
Lemma142:
for f being Function st rng f c= dom f holds
iter f,0 = id (dom f)
theorem Th71: :: FUNCT_7:71
theorem Th72: :: FUNCT_7:72
theorem Th73: :: FUNCT_7:73
theorem Th74: :: FUNCT_7:74
theorem Th75: :: FUNCT_7:75
theorem Th76: :: FUNCT_7:76
theorem Th77: :: FUNCT_7:77
theorem Th78: :: FUNCT_7:78
theorem Th79: :: FUNCT_7:79
Lemma150:
for f being Function
for m, k being Element of NAT st iter (iter f,m),k = iter f,(m * k) holds
iter (iter f,m),(k + 1) = iter f,(m * (k + 1))
theorem Th80: :: FUNCT_7:80
theorem Th81: :: FUNCT_7:81
theorem Th82: :: FUNCT_7:82
theorem Th83: :: FUNCT_7:83
theorem Th84: :: FUNCT_7:84
theorem Th85: :: FUNCT_7:85
theorem Th86: :: FUNCT_7:86
theorem Th87: :: FUNCT_7:87
theorem Th88: :: FUNCT_7:88
theorem Th89: :: FUNCT_7:89
theorem Th90: :: FUNCT_7:90
theorem Th91: :: FUNCT_7:91
theorem Th92: :: FUNCT_7:92
theorem Th93: :: FUNCT_7:93
theorem Th94: :: FUNCT_7:94
theorem Th95: :: FUNCT_7:95
theorem Th96: :: FUNCT_7:96
theorem Th97: :: FUNCT_7:97
theorem Th98: :: FUNCT_7:98