definition
existence
ex b1 being Function of [:REALPLUS,REALPLUS:],REALPLUS st
for x being Element of [:REALPLUS,REALPLUS:] ex y, z being Element of REALPLUS st
( x = [y,z] & b1 . x = REAL_ratio (y,z) )
uniqueness
for b1, b2 being Function of [:REALPLUS,REALPLUS:],REALPLUS st ( for x being Element of [:REALPLUS,REALPLUS:] ex y, z being Element of REALPLUS st
( x = [y,z] & b1 . x = REAL_ratio (y,z) ) ) & ( for x being Element of [:REALPLUS,REALPLUS:] ex y, z being Element of REALPLUS st
( x = [y,z] & b2 . x = REAL_ratio (y,z) ) ) holds
b1 = b2
end;
definition
func EQUIV_REAL_ratio -> Relation of
[:REALPLUS,REALPLUS:],
[:REALPLUS,REALPLUS:] means :
Def03:
for
x,
y being
Element of
[:REALPLUS,REALPLUS:] holds
(
[x,y] in it iff ex
a,
b,
c,
d being
Element of
REALPLUS st
(
x = [a,b] &
y = [c,d] &
REAL_ratio (
a,
b)
= REAL_ratio (
c,
d) ) );
existence
ex b1 being Relation of [:REALPLUS,REALPLUS:],[:REALPLUS,REALPLUS:] st
for x, y being Element of [:REALPLUS,REALPLUS:] holds
( [x,y] in b1 iff ex a, b, c, d being Element of REALPLUS st
( x = [a,b] & y = [c,d] & REAL_ratio (a,b) = REAL_ratio (c,d) ) )
uniqueness
for b1, b2 being Relation of [:REALPLUS,REALPLUS:],[:REALPLUS,REALPLUS:] st ( for x, y being Element of [:REALPLUS,REALPLUS:] holds
( [x,y] in b1 iff ex a, b, c, d being Element of REALPLUS st
( x = [a,b] & y = [c,d] & REAL_ratio (a,b) = REAL_ratio (c,d) ) ) ) & ( for x, y being Element of [:REALPLUS,REALPLUS:] holds
( [x,y] in b2 iff ex a, b, c, d being Element of REALPLUS st
( x = [a,b] & y = [c,d] & REAL_ratio (a,b) = REAL_ratio (c,d) ) ) ) holds
b1 = b2
end;
::
deftheorem Def03 defines
EQUIV_REAL_ratio MUSIC_S1:def 6 :
for b1 being Relation of [:REALPLUS,REALPLUS:],[:REALPLUS,REALPLUS:] holds
( b1 = EQUIV_REAL_ratio iff for x, y being Element of [:REALPLUS,REALPLUS:] holds
( [x,y] in b1 iff ex a, b, c, d being Element of REALPLUS st
( x = [a,b] & y = [c,d] & REAL_ratio (a,b) = REAL_ratio (c,d) ) ) );
definition
existence
ex b1 being Function of [:RATPLUS,RATPLUS:],RATPLUS st
for x being Element of [:RATPLUS,RATPLUS:] ex y, z being Element of RATPLUS st
( x = [y,z] & b1 . x = RAT_ratio (y,z) )
uniqueness
for b1, b2 being Function of [:RATPLUS,RATPLUS:],RATPLUS st ( for x being Element of [:RATPLUS,RATPLUS:] ex y, z being Element of RATPLUS st
( x = [y,z] & b1 . x = RAT_ratio (y,z) ) ) & ( for x being Element of [:RATPLUS,RATPLUS:] ex y, z being Element of RATPLUS st
( x = [y,z] & b2 . x = RAT_ratio (y,z) ) ) holds
b1 = b2
end;
definition
func EQUIV_RAT_ratio -> Relation of
[:RATPLUS,RATPLUS:],
[:RATPLUS,RATPLUS:] means :
Def06:
for
x,
y being
Element of
[:RATPLUS,RATPLUS:] holds
(
[x,y] in it iff ex
a,
b,
c,
d being
Element of
RATPLUS st
(
x = [a,b] &
y = [c,d] &
RAT_ratio (
a,
b)
= RAT_ratio (
c,
d) ) );
existence
ex b1 being Relation of [:RATPLUS,RATPLUS:],[:RATPLUS,RATPLUS:] st
for x, y being Element of [:RATPLUS,RATPLUS:] holds
( [x,y] in b1 iff ex a, b, c, d being Element of RATPLUS st
( x = [a,b] & y = [c,d] & RAT_ratio (a,b) = RAT_ratio (c,d) ) )
uniqueness
for b1, b2 being Relation of [:RATPLUS,RATPLUS:],[:RATPLUS,RATPLUS:] st ( for x, y being Element of [:RATPLUS,RATPLUS:] holds
( [x,y] in b1 iff ex a, b, c, d being Element of RATPLUS st
( x = [a,b] & y = [c,d] & RAT_ratio (a,b) = RAT_ratio (c,d) ) ) ) & ( for x, y being Element of [:RATPLUS,RATPLUS:] holds
( [x,y] in b2 iff ex a, b, c, d being Element of RATPLUS st
( x = [a,b] & y = [c,d] & RAT_ratio (a,b) = RAT_ratio (c,d) ) ) ) holds
b1 = b2
end;
::
deftheorem Def06 defines
EQUIV_RAT_ratio MUSIC_S1:def 10 :
for b1 being Relation of [:RATPLUS,RATPLUS:],[:RATPLUS,RATPLUS:] holds
( b1 = EQUIV_RAT_ratio iff for x, y being Element of [:RATPLUS,RATPLUS:] holds
( [x,y] in b1 iff ex a, b, c, d being Element of RATPLUS st
( x = [a,b] & y = [c,d] & RAT_ratio (a,b) = RAT_ratio (c,d) ) ) );
theorem Th23:
for
MS being
satisfying_equiv MusicStruct for
a,
b,
c,
d,
e,
f being
Element of
MS st
a,
b equiv c,
d &
c,
d equiv e,
f holds
a,
b equiv e,
f
definition
let S be
satisfying_equiv satisfying_interval satisfying_Nat satisfying_harmonic_closed MusicStruct ;
let frequency be
Element of
S;
let n be non
zero Nat;
existence
ex b1 being Element of S st [frequency,b1] in Class ( the Equidistance of S,[1,n])
by Def13a;
uniqueness
for b1, b2 being Element of S st [frequency,b1] in Class ( the Equidistance of S,[1,n]) & [frequency,b2] in Class ( the Equidistance of S,[1,n]) holds
b1 = b2
end;
definition
let MS be
satisfying_equiv satisfying_interval satisfying_Nat satisfying_harmonic_closed MusicStruct ;
let frequency be
Element of
MS;
coherence
Class ( the Equidistance of MS,[(1 -harmonique (MS,frequency)),(1 -harmonique (MS,frequency))]) is Subset of [: the carrier of MS, the carrier of MS:]
;
coherence
Class ( the Equidistance of MS,[(1 -harmonique (MS,frequency)),(2 -harmonique (MS,frequency))]) is Subset of [: the carrier of MS, the carrier of MS:]
;
coherence
Class ( the Equidistance of MS,[(2 -harmonique (MS,frequency)),(3 -harmonique (MS,frequency))]) is Subset of [: the carrier of MS, the carrier of MS:]
;
coherence
Class ( the Equidistance of MS,[(3 -harmonique (MS,frequency)),(4 -harmonique (MS,frequency))]) is Subset of [: the carrier of MS, the carrier of MS:]
;
coherence
Class ( the Equidistance of MS,[(3 -harmonique (MS,frequency)),(5 -harmonique (MS,frequency))]) is Subset of [: the carrier of MS, the carrier of MS:]
;
coherence
Class ( the Equidistance of MS,[(4 -harmonique (MS,frequency)),(5 -harmonique (MS,frequency))]) is Subset of [: the carrier of MS, the carrier of MS:]
;
coherence
Class ( the Equidistance of MS,[(5 -harmonique (MS,frequency)),(6 -harmonique (MS,frequency))]) is Subset of [: the carrier of MS, the carrier of MS:]
;
coherence
Class ( the Equidistance of MS,[(5 -harmonique (MS,frequency)),(8 -harmonique (MS,frequency))]) is Subset of [: the carrier of MS, the carrier of MS:]
;
coherence
Class ( the Equidistance of MS,[(8 -harmonique (MS,frequency)),(9 -harmonique (MS,frequency))]) is Subset of [: the carrier of MS, the carrier of MS:]
;
coherence
Class ( the Equidistance of MS,[(9 -harmonique (MS,frequency)),(10 -harmonique (MS,frequency))]) is Subset of [: the carrier of MS, the carrier of MS:]
;
end;
definition
let MS be
satisfying_equiv satisfying_interval satisfying_Nat satisfying_harmonic_closed MusicStruct ;
coherence
Class ( the Equidistance of MS,[1,1]) is Subset of [: the carrier of MS, the carrier of MS:]
;
coherence
Class ( the Equidistance of MS,[1,2]) is Subset of [: the carrier of MS, the carrier of MS:]
;
coherence
Class ( the Equidistance of MS,[2,3]) is Subset of [: the carrier of MS, the carrier of MS:]
;
coherence
Class ( the Equidistance of MS,[3,4]) is Subset of [: the carrier of MS, the carrier of MS:]
;
coherence
Class ( the Equidistance of MS,[3,5]) is Subset of [: the carrier of MS, the carrier of MS:]
;
coherence
Class ( the Equidistance of MS,[4,5]) is Subset of [: the carrier of MS, the carrier of MS:]
;
coherence
Class ( the Equidistance of MS,[5,6]) is Subset of [: the carrier of MS, the carrier of MS:]
;
coherence
Class ( the Equidistance of MS,[5,8]) is Subset of [: the carrier of MS, the carrier of MS:]
;
coherence
Class ( the Equidistance of MS,[8,9]) is Subset of [: the carrier of MS, the carrier of MS:]
;
coherence
Class ( the Equidistance of MS,[9,10]) is Subset of [: the carrier of MS, the carrier of MS:]
;
end;
definition
let MS be
satisfying_equiv satisfying_interval satisfying_commutativity satisfying_Nat satisfying_harmonic_closed satisfying_fifth_constructible satisfying_octave_constructible satisfying_octave_descendent_constructible MusicStruct ;
let fondamentale,
frequency be
Element of
MS;
correctness
coherence
( ( Fifth (MS,frequency) is_Between fondamentale, Octave (MS,fondamentale) implies Fifth (MS,frequency) is Element of MS ) & ( not Fifth (MS,frequency) is_Between fondamentale, Octave (MS,fondamentale) implies Octave_descendent (MS,(Fifth (MS,frequency))) is Element of MS ) );
consistency
for b1 being Element of MS holds verum;
;
end;
::
deftheorem Def18 defines
Fifth_reduct MUSIC_S1:def 52 :
for MS being satisfying_equiv satisfying_interval satisfying_commutativity satisfying_Nat satisfying_harmonic_closed satisfying_fifth_constructible satisfying_octave_constructible satisfying_octave_descendent_constructible MusicStruct
for fondamentale, frequency being Element of MS holds
( ( Fifth (MS,frequency) is_Between fondamentale, Octave (MS,fondamentale) implies Fifth_reduct (MS,fondamentale,frequency) = Fifth (MS,frequency) ) & ( not Fifth (MS,frequency) is_Between fondamentale, Octave (MS,fondamentale) implies Fifth_reduct (MS,fondamentale,frequency) = Octave_descendent (MS,(Fifth (MS,frequency))) ) );
definition
let MS be
MusicSpace;
let frequency be
Element of
MS;
func pentatonic_pythagorean_scale (
MS,
frequency)
-> Element of 6
-tuples_on the
carrier of
MS means :
Def20:
(
it . 1
= frequency &
it . 2
= (spiral_of_fifths (MS,frequency,frequency)) . 2 &
it . 3
= (spiral_of_fifths (MS,frequency,frequency)) . 4 &
it . 4
= (spiral_of_fifths (MS,frequency,frequency)) . 1 &
it . 5
= (spiral_of_fifths (MS,frequency,frequency)) . 3 &
it . 6
= Octave (
MS,
frequency) );
existence
ex b1 being Element of 6 -tuples_on the carrier of MS st
( b1 . 1 = frequency & b1 . 2 = (spiral_of_fifths (MS,frequency,frequency)) . 2 & b1 . 3 = (spiral_of_fifths (MS,frequency,frequency)) . 4 & b1 . 4 = (spiral_of_fifths (MS,frequency,frequency)) . 1 & b1 . 5 = (spiral_of_fifths (MS,frequency,frequency)) . 3 & b1 . 6 = Octave (MS,frequency) )
uniqueness
for b1, b2 being Element of 6 -tuples_on the carrier of MS st b1 . 1 = frequency & b1 . 2 = (spiral_of_fifths (MS,frequency,frequency)) . 2 & b1 . 3 = (spiral_of_fifths (MS,frequency,frequency)) . 4 & b1 . 4 = (spiral_of_fifths (MS,frequency,frequency)) . 1 & b1 . 5 = (spiral_of_fifths (MS,frequency,frequency)) . 3 & b1 . 6 = Octave (MS,frequency) & b2 . 1 = frequency & b2 . 2 = (spiral_of_fifths (MS,frequency,frequency)) . 2 & b2 . 3 = (spiral_of_fifths (MS,frequency,frequency)) . 4 & b2 . 4 = (spiral_of_fifths (MS,frequency,frequency)) . 1 & b2 . 5 = (spiral_of_fifths (MS,frequency,frequency)) . 3 & b2 . 6 = Octave (MS,frequency) holds
b1 = b2
end;
::
deftheorem Def20 defines
pentatonic_pythagorean_scale MUSIC_S1:def 62 :
for MS being MusicSpace
for frequency being Element of MS
for b3 being Element of 6 -tuples_on the carrier of MS holds
( b3 = pentatonic_pythagorean_scale (MS,frequency) iff ( b3 . 1 = frequency & b3 . 2 = (spiral_of_fifths (MS,frequency,frequency)) . 2 & b3 . 3 = (spiral_of_fifths (MS,frequency,frequency)) . 4 & b3 . 4 = (spiral_of_fifths (MS,frequency,frequency)) . 1 & b3 . 5 = (spiral_of_fifths (MS,frequency,frequency)) . 3 & b3 . 6 = Octave (MS,frequency) ) );
theorem Th68:
for
MS being
MusicSpace for
frequency being
Element of
MS for
r1,
r2,
r3,
r4,
r5,
r6 being
positive Real st
(pentatonic_pythagorean_scale (MS,frequency)) . 1
= r1 &
(pentatonic_pythagorean_scale (MS,frequency)) . 2
= r2 &
(pentatonic_pythagorean_scale (MS,frequency)) . 3
= r3 &
(pentatonic_pythagorean_scale (MS,frequency)) . 4
= r4 &
(pentatonic_pythagorean_scale (MS,frequency)) . 5
= r5 &
(pentatonic_pythagorean_scale (MS,frequency)) . 6
= r6 holds
(
r2 / r1 = 9
/ 8 &
r3 / r2 = 9
/ 8 &
r4 / r3 = 32
/ 27 &
r5 / r4 = 9
/ 8 &
r6 / r5 = 32
/ 27 )
theorem Th69:
for
MS being
MusicSpace for
frequency being
Element of
MS ex
r1,
r2,
r3,
r4,
r5,
r6 being
positive Real st
(
(pentatonic_pythagorean_scale (MS,frequency)) . 1
= r1 &
(pentatonic_pythagorean_scale (MS,frequency)) . 2
= r2 &
(pentatonic_pythagorean_scale (MS,frequency)) . 3
= r3 &
(pentatonic_pythagorean_scale (MS,frequency)) . 4
= r4 &
(pentatonic_pythagorean_scale (MS,frequency)) . 5
= r5 &
(pentatonic_pythagorean_scale (MS,frequency)) . 6
= r6 &
r2 / r1 = 9
/ 8 &
r3 / r2 = 9
/ 8 &
r4 / r3 = 32
/ 27 &
r5 / r4 = 9
/ 8 &
r6 / r5 = 32
/ 27 )
theorem
for
MS being
MusicSpace for
frequency being
Element of
MS holds
(
intrval (
(penta_fondamentale (MS,frequency)),
(penta_1 (MS,frequency)))
= pythagorean_tone &
intrval (
(penta_1 (MS,frequency)),
(penta_2 (MS,frequency)))
= pythagorean_tone &
intrval (
(penta_2 (MS,frequency)),
(penta_3 (MS,frequency)))
= pentatonic_pythagorean_semiditone &
intrval (
(penta_3 (MS,frequency)),
(penta_4 (MS,frequency)))
= pythagorean_tone &
intrval (
(penta_4 (MS,frequency)),
(penta_octave (MS,frequency)))
= pentatonic_pythagorean_semiditone )
theorem Th71:
for
MS being
MusicSpace for
fondamentale,
f1,
f2 being
Element of
MS for
r1,
r2 being
positive Real st
f1 = r1 &
f2 = r2 &
r2 = (4 / 3) * r1 holds
( (
Fifth (
MS,
f2)
is_Between fondamentale,
Octave (
MS,
fondamentale) implies
Octave_descendent (
MS,
(Fifth_reduct (MS,fondamentale,f2)))
= f1 ) & ( not
Fifth (
MS,
f2)
is_Between fondamentale,
Octave (
MS,
fondamentale) implies
Fifth_reduct (
MS,
fondamentale,
f2)
= f1 ) )
definition
let HPS be
Heptatonic_Pythagorean_Score;
let frequency be
Element of
HPS;
func heptatonic_pythagorean_scale (
HPS,
frequency)
-> Element of 8
-tuples_on the
carrier of
HPS means :
Def26:
(
it . 1
= (spiral_of_fifths (HPS,frequency,(Fourth (HPS,frequency)))) . 1 &
it . 2
= (spiral_of_fifths (HPS,frequency,(Fourth (HPS,frequency)))) . 3 &
it . 3
= (spiral_of_fifths (HPS,frequency,(Fourth (HPS,frequency)))) . 5 &
it . 4
= Fourth (
HPS,
frequency) &
it . 5
= (spiral_of_fifths (HPS,frequency,(Fourth (HPS,frequency)))) . 2 &
it . 6
= (spiral_of_fifths (HPS,frequency,(Fourth (HPS,frequency)))) . 4 &
it . 7
= (spiral_of_fifths (HPS,frequency,(Fourth (HPS,frequency)))) . 6 &
it . 8
= Octave (
HPS,
((spiral_of_fifths (HPS,frequency,(Fourth (HPS,frequency)))) . 1)) );
existence
ex b1 being Element of 8 -tuples_on the carrier of HPS st
( b1 . 1 = (spiral_of_fifths (HPS,frequency,(Fourth (HPS,frequency)))) . 1 & b1 . 2 = (spiral_of_fifths (HPS,frequency,(Fourth (HPS,frequency)))) . 3 & b1 . 3 = (spiral_of_fifths (HPS,frequency,(Fourth (HPS,frequency)))) . 5 & b1 . 4 = Fourth (HPS,frequency) & b1 . 5 = (spiral_of_fifths (HPS,frequency,(Fourth (HPS,frequency)))) . 2 & b1 . 6 = (spiral_of_fifths (HPS,frequency,(Fourth (HPS,frequency)))) . 4 & b1 . 7 = (spiral_of_fifths (HPS,frequency,(Fourth (HPS,frequency)))) . 6 & b1 . 8 = Octave (HPS,((spiral_of_fifths (HPS,frequency,(Fourth (HPS,frequency)))) . 1)) )
uniqueness
for b1, b2 being Element of 8 -tuples_on the carrier of HPS st b1 . 1 = (spiral_of_fifths (HPS,frequency,(Fourth (HPS,frequency)))) . 1 & b1 . 2 = (spiral_of_fifths (HPS,frequency,(Fourth (HPS,frequency)))) . 3 & b1 . 3 = (spiral_of_fifths (HPS,frequency,(Fourth (HPS,frequency)))) . 5 & b1 . 4 = Fourth (HPS,frequency) & b1 . 5 = (spiral_of_fifths (HPS,frequency,(Fourth (HPS,frequency)))) . 2 & b1 . 6 = (spiral_of_fifths (HPS,frequency,(Fourth (HPS,frequency)))) . 4 & b1 . 7 = (spiral_of_fifths (HPS,frequency,(Fourth (HPS,frequency)))) . 6 & b1 . 8 = Octave (HPS,((spiral_of_fifths (HPS,frequency,(Fourth (HPS,frequency)))) . 1)) & b2 . 1 = (spiral_of_fifths (HPS,frequency,(Fourth (HPS,frequency)))) . 1 & b2 . 2 = (spiral_of_fifths (HPS,frequency,(Fourth (HPS,frequency)))) . 3 & b2 . 3 = (spiral_of_fifths (HPS,frequency,(Fourth (HPS,frequency)))) . 5 & b2 . 4 = Fourth (HPS,frequency) & b2 . 5 = (spiral_of_fifths (HPS,frequency,(Fourth (HPS,frequency)))) . 2 & b2 . 6 = (spiral_of_fifths (HPS,frequency,(Fourth (HPS,frequency)))) . 4 & b2 . 7 = (spiral_of_fifths (HPS,frequency,(Fourth (HPS,frequency)))) . 6 & b2 . 8 = Octave (HPS,((spiral_of_fifths (HPS,frequency,(Fourth (HPS,frequency)))) . 1)) holds
b1 = b2
end;
::
deftheorem Def26 defines
heptatonic_pythagorean_scale MUSIC_S1:def 79 :
for HPS being Heptatonic_Pythagorean_Score
for frequency being Element of HPS
for b3 being Element of 8 -tuples_on the carrier of HPS holds
( b3 = heptatonic_pythagorean_scale (HPS,frequency) iff ( b3 . 1 = (spiral_of_fifths (HPS,frequency,(Fourth (HPS,frequency)))) . 1 & b3 . 2 = (spiral_of_fifths (HPS,frequency,(Fourth (HPS,frequency)))) . 3 & b3 . 3 = (spiral_of_fifths (HPS,frequency,(Fourth (HPS,frequency)))) . 5 & b3 . 4 = Fourth (HPS,frequency) & b3 . 5 = (spiral_of_fifths (HPS,frequency,(Fourth (HPS,frequency)))) . 2 & b3 . 6 = (spiral_of_fifths (HPS,frequency,(Fourth (HPS,frequency)))) . 4 & b3 . 7 = (spiral_of_fifths (HPS,frequency,(Fourth (HPS,frequency)))) . 6 & b3 . 8 = Octave (HPS,((spiral_of_fifths (HPS,frequency,(Fourth (HPS,frequency)))) . 1)) ) );
Lem89:
for HPS being Heptatonic_Pythagorean_Score
for frequency being Element of HPS
for r1, r2, r3, r4, r5, r6, r7, r8 being positive Real st (heptatonic_pythagorean_scale (HPS,frequency)) . 1 = r1 & (heptatonic_pythagorean_scale (HPS,frequency)) . 2 = r2 & (heptatonic_pythagorean_scale (HPS,frequency)) . 3 = r3 & (heptatonic_pythagorean_scale (HPS,frequency)) . 4 = r4 & (heptatonic_pythagorean_scale (HPS,frequency)) . 5 = r5 & (heptatonic_pythagorean_scale (HPS,frequency)) . 6 = r6 & (heptatonic_pythagorean_scale (HPS,frequency)) . 7 = r7 & (heptatonic_pythagorean_scale (HPS,frequency)) . 8 = r8 holds
( r2 / r1 = 9 / 8 & r3 / r2 = 9 / 8 & r4 / r3 = 256 / 243 & r5 / r4 = 9 / 8 & r6 / r5 = 9 / 8 & r7 / r6 = 9 / 8 & r8 / r7 = 256 / 243 )
Lem90:
for HPS being Heptatonic_Pythagorean_Score
for frequency being Element of HPS ex r1, r2, r3, r4, r5, r6, r7, r8 being positive Real st
( (heptatonic_pythagorean_scale (HPS,frequency)) . 1 = r1 & (heptatonic_pythagorean_scale (HPS,frequency)) . 2 = r2 & (heptatonic_pythagorean_scale (HPS,frequency)) . 3 = r3 & (heptatonic_pythagorean_scale (HPS,frequency)) . 4 = r4 & (heptatonic_pythagorean_scale (HPS,frequency)) . 5 = r5 & (heptatonic_pythagorean_scale (HPS,frequency)) . 6 = r6 & (heptatonic_pythagorean_scale (HPS,frequency)) . 7 = r7 & (heptatonic_pythagorean_scale (HPS,frequency)) . 8 = r8 & r2 / r1 = 9 / 8 & r3 / r2 = 9 / 8 & r4 / r3 = 256 / 243 & r5 / r4 = 9 / 8 & r6 / r5 = 9 / 8 & r7 / r6 = 9 / 8 & r8 / r7 = 256 / 243 )
theorem Th90:
for
HPS being
Heptatonic_Pythagorean_Score for
frequency being
Element of
HPS holds
(
intrval (
(hepta_fondamental (HPS,frequency)),
(hepta_1 (HPS,frequency)))
= pythagorean_tone &
intrval (
(hepta_1 (HPS,frequency)),
(hepta_2 (HPS,frequency)))
= pythagorean_tone &
intrval (
(hepta_2 (HPS,frequency)),
(hepta_3 (HPS,frequency)))
= heptatonic_pythagorean_semitone &
intrval (
(hepta_3 (HPS,frequency)),
(hepta_4 (HPS,frequency)))
= pythagorean_tone &
intrval (
(hepta_4 (HPS,frequency)),
(hepta_5 (HPS,frequency)))
= pythagorean_tone &
intrval (
(hepta_5 (HPS,frequency)),
(hepta_6 (HPS,frequency)))
= pythagorean_tone &
intrval (
(hepta_6 (HPS,frequency)),
(hepta_octave (HPS,frequency)))
= heptatonic_pythagorean_semitone )
theorem Th92:
for
HPS being
Heptatonic_Pythagorean_Score for
frequency being
Element of
HPS holds
(
intrval (
(hepta_4 (HPS,frequency)),
(hepta_1 (HPS,(Octave (HPS,frequency)))))
= 3
/ 2 &
intrval (
(hepta_5 (HPS,frequency)),
(hepta_2 (HPS,(Octave (HPS,frequency)))))
= 3
/ 2 &
intrval (
(hepta_6 (HPS,frequency)),
(hepta_3 (HPS,(Octave (HPS,frequency)))))
<> 3
/ 2 &
intrval (
(hepta_octave (HPS,frequency)),
(hepta_4 (HPS,(Octave (HPS,frequency)))))
= 3
/ 2 )
definition
let HPS be
MusicSpace;
let n be
natural non
zero Number ;
let scale be
Element of
n -tuples_on the
carrier of
HPS;
assume
scale is
heptatonic
;
attr scale is
dorian means
ex
t1,
t2 being
positive Real st
(
(((((t1 * t1) * t1) * t1) * t1) * t2) * t2 = 2 &
intrval (
(# (scale,1)),
(# (scale,2)))
= t1 &
intrval (
(# (scale,2)),
(# (scale,3)))
= t2 &
intrval (
(# (scale,3)),
(# (scale,4)))
= t1 &
intrval (
(# (scale,4)),
(# (scale,5)))
= t1 &
intrval (
(# (scale,5)),
(# (scale,6)))
= t1 &
intrval (
(# (scale,6)),
(# (scale,7)))
= t2 &
intrval (
(# (scale,7)),
(# (scale,8)))
= t1 );
end;
::
deftheorem defines
dorian MUSIC_S1:def 92 :
for HPS being MusicSpace
for n being natural non zero Number
for scale being Element of n -tuples_on the carrier of HPS st scale is heptatonic holds
( scale is dorian iff ex t1, t2 being positive Real st
( (((((t1 * t1) * t1) * t1) * t1) * t2) * t2 = 2 & intrval ((# (scale,1)),(# (scale,2))) = t1 & intrval ((# (scale,2)),(# (scale,3))) = t2 & intrval ((# (scale,3)),(# (scale,4))) = t1 & intrval ((# (scale,4)),(# (scale,5))) = t1 & intrval ((# (scale,5)),(# (scale,6))) = t1 & intrval ((# (scale,6)),(# (scale,7))) = t2 & intrval ((# (scale,7)),(# (scale,8))) = t1 ) );
definition
let HPS be
MusicSpace;
let n be
natural non
zero Number ;
let scale be
Element of
n -tuples_on the
carrier of
HPS;
assume
scale is
heptatonic
;
attr scale is
hypodorian means
ex
t1,
t2 being
positive Real st
(
(((((t1 * t1) * t1) * t1) * t1) * t2) * t2 = 2 &
intrval (
(# (scale,1)),
(# (scale,2)))
= t1 &
intrval (
(# (scale,2)),
(# (scale,3)))
= t2 &
intrval (
(# (scale,3)),
(# (scale,4)))
= t1 &
intrval (
(# (scale,4)),
(# (scale,5)))
= t1 &
intrval (
(# (scale,5)),
(# (scale,6)))
= t2 &
intrval (
(# (scale,6)),
(# (scale,7)))
= t1 &
intrval (
(# (scale,7)),
(# (scale,8)))
= t1 );
end;
::
deftheorem defines
hypodorian MUSIC_S1:def 93 :
for HPS being MusicSpace
for n being natural non zero Number
for scale being Element of n -tuples_on the carrier of HPS st scale is heptatonic holds
( scale is hypodorian iff ex t1, t2 being positive Real st
( (((((t1 * t1) * t1) * t1) * t1) * t2) * t2 = 2 & intrval ((# (scale,1)),(# (scale,2))) = t1 & intrval ((# (scale,2)),(# (scale,3))) = t2 & intrval ((# (scale,3)),(# (scale,4))) = t1 & intrval ((# (scale,4)),(# (scale,5))) = t1 & intrval ((# (scale,5)),(# (scale,6))) = t2 & intrval ((# (scale,6)),(# (scale,7))) = t1 & intrval ((# (scale,7)),(# (scale,8))) = t1 ) );
definition
let HPS be
MusicSpace;
let n be
natural non
zero Number ;
let scale be
Element of
n -tuples_on the
carrier of
HPS;
assume
scale is
heptatonic
;
attr scale is
phrygian means
ex
t1,
t2 being
positive Real st
(
(((((t1 * t1) * t1) * t1) * t1) * t2) * t2 = 2 &
intrval (
(# (scale,1)),
(# (scale,2)))
= t1 &
intrval (
(# (scale,2)),
(# (scale,3)))
= t2 &
intrval (
(# (scale,3)),
(# (scale,4)))
= t1 &
intrval (
(# (scale,4)),
(# (scale,5)))
= t2 &
intrval (
(# (scale,5)),
(# (scale,6)))
= t1 &
intrval (
(# (scale,6)),
(# (scale,7)))
= t1 &
intrval (
(# (scale,7)),
(# (scale,8)))
= t1 );
end;
::
deftheorem defines
phrygian MUSIC_S1:def 94 :
for HPS being MusicSpace
for n being natural non zero Number
for scale being Element of n -tuples_on the carrier of HPS st scale is heptatonic holds
( scale is phrygian iff ex t1, t2 being positive Real st
( (((((t1 * t1) * t1) * t1) * t1) * t2) * t2 = 2 & intrval ((# (scale,1)),(# (scale,2))) = t1 & intrval ((# (scale,2)),(# (scale,3))) = t2 & intrval ((# (scale,3)),(# (scale,4))) = t1 & intrval ((# (scale,4)),(# (scale,5))) = t2 & intrval ((# (scale,5)),(# (scale,6))) = t1 & intrval ((# (scale,6)),(# (scale,7))) = t1 & intrval ((# (scale,7)),(# (scale,8))) = t1 ) );
definition
let HPS be
MusicSpace;
let n be
natural non
zero Number ;
let scale be
Element of
n -tuples_on the
carrier of
HPS;
assume
scale is
heptatonic
;
attr scale is
hypophrygian means
ex
t1,
t2 being
positive Real st
(
(((((t1 * t1) * t1) * t1) * t1) * t2) * t2 = 2 &
intrval (
(# (scale,1)),
(# (scale,2)))
= t2 &
intrval (
(# (scale,2)),
(# (scale,3)))
= t1 &
intrval (
(# (scale,3)),
(# (scale,4)))
= t1 &
intrval (
(# (scale,4)),
(# (scale,5)))
= t2 &
intrval (
(# (scale,5)),
(# (scale,6)))
= t1 &
intrval (
(# (scale,6)),
(# (scale,7)))
= t1 &
intrval (
(# (scale,7)),
(# (scale,8)))
= t1 );
end;
::
deftheorem defines
hypophrygian MUSIC_S1:def 95 :
for HPS being MusicSpace
for n being natural non zero Number
for scale being Element of n -tuples_on the carrier of HPS st scale is heptatonic holds
( scale is hypophrygian iff ex t1, t2 being positive Real st
( (((((t1 * t1) * t1) * t1) * t1) * t2) * t2 = 2 & intrval ((# (scale,1)),(# (scale,2))) = t2 & intrval ((# (scale,2)),(# (scale,3))) = t1 & intrval ((# (scale,3)),(# (scale,4))) = t1 & intrval ((# (scale,4)),(# (scale,5))) = t2 & intrval ((# (scale,5)),(# (scale,6))) = t1 & intrval ((# (scale,6)),(# (scale,7))) = t1 & intrval ((# (scale,7)),(# (scale,8))) = t1 ) );
definition
let HPS be
MusicSpace;
let n be
natural non
zero Number ;
let scale be
Element of
n -tuples_on the
carrier of
HPS;
assume
scale is
heptatonic
;
attr scale is
lydian means
ex
t1,
t2 being
positive Real st
(
(((((t1 * t1) * t1) * t1) * t1) * t2) * t2 = 2 &
intrval (
(# (scale,1)),
(# (scale,2)))
= t1 &
intrval (
(# (scale,2)),
(# (scale,3)))
= t1 &
intrval (
(# (scale,3)),
(# (scale,4)))
= t2 &
intrval (
(# (scale,4)),
(# (scale,5)))
= t1 &
intrval (
(# (scale,5)),
(# (scale,6)))
= t1 &
intrval (
(# (scale,6)),
(# (scale,7)))
= t2 &
intrval (
(# (scale,7)),
(# (scale,8)))
= t1 );
end;
::
deftheorem defines
lydian MUSIC_S1:def 96 :
for HPS being MusicSpace
for n being natural non zero Number
for scale being Element of n -tuples_on the carrier of HPS st scale is heptatonic holds
( scale is lydian iff ex t1, t2 being positive Real st
( (((((t1 * t1) * t1) * t1) * t1) * t2) * t2 = 2 & intrval ((# (scale,1)),(# (scale,2))) = t1 & intrval ((# (scale,2)),(# (scale,3))) = t1 & intrval ((# (scale,3)),(# (scale,4))) = t2 & intrval ((# (scale,4)),(# (scale,5))) = t1 & intrval ((# (scale,5)),(# (scale,6))) = t1 & intrval ((# (scale,6)),(# (scale,7))) = t2 & intrval ((# (scale,7)),(# (scale,8))) = t1 ) );
definition
let HPS be
MusicSpace;
let n be
natural non
zero Number ;
let scale be
Element of
n -tuples_on the
carrier of
HPS;
assume
scale is
heptatonic
;
attr scale is
hypolydian means
ex
t1,
t2 being
positive Real st
(
(((((t1 * t1) * t1) * t1) * t1) * t2) * t2 = 2 &
intrval (
(# (scale,1)),
(# (scale,2)))
= t1 &
intrval (
(# (scale,2)),
(# (scale,3)))
= t1 &
intrval (
(# (scale,3)),
(# (scale,4)))
= t2 &
intrval (
(# (scale,4)),
(# (scale,5)))
= t1 &
intrval (
(# (scale,5)),
(# (scale,6)))
= t1 &
intrval (
(# (scale,6)),
(# (scale,7)))
= t1 &
intrval (
(# (scale,7)),
(# (scale,8)))
= t2 );
end;
::
deftheorem defines
hypolydian MUSIC_S1:def 97 :
for HPS being MusicSpace
for n being natural non zero Number
for scale being Element of n -tuples_on the carrier of HPS st scale is heptatonic holds
( scale is hypolydian iff ex t1, t2 being positive Real st
( (((((t1 * t1) * t1) * t1) * t1) * t2) * t2 = 2 & intrval ((# (scale,1)),(# (scale,2))) = t1 & intrval ((# (scale,2)),(# (scale,3))) = t1 & intrval ((# (scale,3)),(# (scale,4))) = t2 & intrval ((# (scale,4)),(# (scale,5))) = t1 & intrval ((# (scale,5)),(# (scale,6))) = t1 & intrval ((# (scale,6)),(# (scale,7))) = t1 & intrval ((# (scale,7)),(# (scale,8))) = t2 ) );
definition
let HPS be
MusicSpace;
let n be
natural non
zero Number ;
let scale be
Element of
n -tuples_on the
carrier of
HPS;
assume
scale is
heptatonic
;
attr scale is
mixolydian means
ex
t1,
t2 being
positive Real st
(
(((((t1 * t1) * t1) * t1) * t1) * t2) * t2 = 2 &
intrval (
(# (scale,1)),
(# (scale,2)))
= t1 &
intrval (
(# (scale,2)),
(# (scale,3)))
= t1 &
intrval (
(# (scale,3)),
(# (scale,4)))
= t2 &
intrval (
(# (scale,4)),
(# (scale,5)))
= t1 &
intrval (
(# (scale,5)),
(# (scale,6)))
= t1 &
intrval (
(# (scale,6)),
(# (scale,7)))
= t2 &
intrval (
(# (scale,7)),
(# (scale,8)))
= t1 );
end;
::
deftheorem defines
mixolydian MUSIC_S1:def 98 :
for HPS being MusicSpace
for n being natural non zero Number
for scale being Element of n -tuples_on the carrier of HPS st scale is heptatonic holds
( scale is mixolydian iff ex t1, t2 being positive Real st
( (((((t1 * t1) * t1) * t1) * t1) * t2) * t2 = 2 & intrval ((# (scale,1)),(# (scale,2))) = t1 & intrval ((# (scale,2)),(# (scale,3))) = t1 & intrval ((# (scale,3)),(# (scale,4))) = t2 & intrval ((# (scale,4)),(# (scale,5))) = t1 & intrval ((# (scale,5)),(# (scale,6))) = t1 & intrval ((# (scale,6)),(# (scale,7))) = t2 & intrval ((# (scale,7)),(# (scale,8))) = t1 ) );
definition
let HPS be
MusicSpace;
let n be
natural non
zero Number ;
let scale be
Element of
n -tuples_on the
carrier of
HPS;
assume
scale is
heptatonic
;
attr scale is
hypomixolydian means
ex
t1,
t2 being
positive Real st
(
(((((t1 * t1) * t1) * t1) * t1) * t2) * t2 = 2 &
intrval (
(# (scale,1)),
(# (scale,2)))
= t1 &
intrval (
(# (scale,2)),
(# (scale,3)))
= t2 &
intrval (
(# (scale,3)),
(# (scale,4)))
= t1 &
intrval (
(# (scale,4)),
(# (scale,5)))
= t1 &
intrval (
(# (scale,5)),
(# (scale,6)))
= t1 &
intrval (
(# (scale,6)),
(# (scale,7)))
= t2 &
intrval (
(# (scale,7)),
(# (scale,8)))
= t1 );
end;
::
deftheorem defines
hypomixolydian MUSIC_S1:def 99 :
for HPS being MusicSpace
for n being natural non zero Number
for scale being Element of n -tuples_on the carrier of HPS st scale is heptatonic holds
( scale is hypomixolydian iff ex t1, t2 being positive Real st
( (((((t1 * t1) * t1) * t1) * t1) * t2) * t2 = 2 & intrval ((# (scale,1)),(# (scale,2))) = t1 & intrval ((# (scale,2)),(# (scale,3))) = t2 & intrval ((# (scale,3)),(# (scale,4))) = t1 & intrval ((# (scale,4)),(# (scale,5))) = t1 & intrval ((# (scale,5)),(# (scale,6))) = t1 & intrval ((# (scale,6)),(# (scale,7))) = t2 & intrval ((# (scale,7)),(# (scale,8))) = t1 ) );
definition
let HPS be
MusicSpace;
let n be
natural non
zero Number ;
let scale be
Element of
n -tuples_on the
carrier of
HPS;
assume
scale is
heptatonic
;
attr scale is
eolian means
ex
t1,
t2 being
positive Real st
(
(((((t1 * t1) * t1) * t1) * t1) * t2) * t2 = 2 &
intrval (
(# (scale,1)),
(# (scale,2)))
= t1 &
intrval (
(# (scale,2)),
(# (scale,3)))
= t2 &
intrval (
(# (scale,3)),
(# (scale,4)))
= t1 &
intrval (
(# (scale,4)),
(# (scale,5)))
= t1 &
intrval (
(# (scale,5)),
(# (scale,6)))
= t2 &
intrval (
(# (scale,6)),
(# (scale,7)))
= t1 &
intrval (
(# (scale,7)),
(# (scale,8)))
= t1 );
end;
::
deftheorem defines
eolian MUSIC_S1:def 100 :
for HPS being MusicSpace
for n being natural non zero Number
for scale being Element of n -tuples_on the carrier of HPS st scale is heptatonic holds
( scale is eolian iff ex t1, t2 being positive Real st
( (((((t1 * t1) * t1) * t1) * t1) * t2) * t2 = 2 & intrval ((# (scale,1)),(# (scale,2))) = t1 & intrval ((# (scale,2)),(# (scale,3))) = t2 & intrval ((# (scale,3)),(# (scale,4))) = t1 & intrval ((# (scale,4)),(# (scale,5))) = t1 & intrval ((# (scale,5)),(# (scale,6))) = t2 & intrval ((# (scale,6)),(# (scale,7))) = t1 & intrval ((# (scale,7)),(# (scale,8))) = t1 ) );
definition
let HPS be
MusicSpace;
let n be
natural non
zero Number ;
let scale be
Element of
n -tuples_on the
carrier of
HPS;
assume
scale is
heptatonic
;
attr scale is
hypoeolian means
ex
t1,
t2 being
positive Real st
(
(((((t1 * t1) * t1) * t1) * t1) * t2) * t2 = 2 &
intrval (
(# (scale,1)),
(# (scale,2)))
= t2 &
intrval (
(# (scale,2)),
(# (scale,3)))
= t1 &
intrval (
(# (scale,3)),
(# (scale,4)))
= t1 &
intrval (
(# (scale,4)),
(# (scale,5)))
= t1 &
intrval (
(# (scale,5)),
(# (scale,6)))
= t2 &
intrval (
(# (scale,6)),
(# (scale,7)))
= t1 &
intrval (
(# (scale,7)),
(# (scale,8)))
= t1 );
end;
::
deftheorem defines
hypoeolian MUSIC_S1:def 101 :
for HPS being MusicSpace
for n being natural non zero Number
for scale being Element of n -tuples_on the carrier of HPS st scale is heptatonic holds
( scale is hypoeolian iff ex t1, t2 being positive Real st
( (((((t1 * t1) * t1) * t1) * t1) * t2) * t2 = 2 & intrval ((# (scale,1)),(# (scale,2))) = t2 & intrval ((# (scale,2)),(# (scale,3))) = t1 & intrval ((# (scale,3)),(# (scale,4))) = t1 & intrval ((# (scale,4)),(# (scale,5))) = t1 & intrval ((# (scale,5)),(# (scale,6))) = t2 & intrval ((# (scale,6)),(# (scale,7))) = t1 & intrval ((# (scale,7)),(# (scale,8))) = t1 ) );
definition
let HPS be
MusicSpace;
let n be
natural non
zero Number ;
let scale be
Element of
n -tuples_on the
carrier of
HPS;
assume
scale is
heptatonic
;
attr scale is
ionan means :
Def29:
ex
t1,
t2 being
positive Real st
(
(((((t1 * t1) * t1) * t1) * t1) * t2) * t2 = 2 &
intrval (
(# (scale,1)),
(# (scale,2)))
= t1 &
intrval (
(# (scale,2)),
(# (scale,3)))
= t1 &
intrval (
(# (scale,3)),
(# (scale,4)))
= t2 &
intrval (
(# (scale,4)),
(# (scale,5)))
= t1 &
intrval (
(# (scale,5)),
(# (scale,6)))
= t1 &
intrval (
(# (scale,6)),
(# (scale,7)))
= t1 &
intrval (
(# (scale,7)),
(# (scale,8)))
= t2 );
end;
::
deftheorem Def29 defines
ionan MUSIC_S1:def 102 :
for HPS being MusicSpace
for n being natural non zero Number
for scale being Element of n -tuples_on the carrier of HPS st scale is heptatonic holds
( scale is ionan iff ex t1, t2 being positive Real st
( (((((t1 * t1) * t1) * t1) * t1) * t2) * t2 = 2 & intrval ((# (scale,1)),(# (scale,2))) = t1 & intrval ((# (scale,2)),(# (scale,3))) = t1 & intrval ((# (scale,3)),(# (scale,4))) = t2 & intrval ((# (scale,4)),(# (scale,5))) = t1 & intrval ((# (scale,5)),(# (scale,6))) = t1 & intrval ((# (scale,6)),(# (scale,7))) = t1 & intrval ((# (scale,7)),(# (scale,8))) = t2 ) );
definition
let HPS be
MusicSpace;
let n be
natural non
zero Number ;
let scale be
Element of
n -tuples_on the
carrier of
HPS;
assume
scale is
heptatonic
;
attr scale is
hypoionan means
ex
t1,
t2 being
positive Real st
(
(((((t1 * t1) * t1) * t1) * t1) * t2) * t2 = 2 &
intrval (
(# (scale,1)),
(# (scale,2)))
= t1 &
intrval (
(# (scale,2)),
(# (scale,3)))
= t1 &
intrval (
(# (scale,3)),
(# (scale,4)))
= t2 &
intrval (
(# (scale,4)),
(# (scale,5)))
= t1 &
intrval (
(# (scale,5)),
(# (scale,6)))
= t1 &
intrval (
(# (scale,6)),
(# (scale,7)))
= t2 &
intrval (
(# (scale,7)),
(# (scale,8)))
= t1 );
end;
::
deftheorem defines
hypoionan MUSIC_S1:def 103 :
for HPS being MusicSpace
for n being natural non zero Number
for scale being Element of n -tuples_on the carrier of HPS st scale is heptatonic holds
( scale is hypoionan iff ex t1, t2 being positive Real st
( (((((t1 * t1) * t1) * t1) * t1) * t2) * t2 = 2 & intrval ((# (scale,1)),(# (scale,2))) = t1 & intrval ((# (scale,2)),(# (scale,3))) = t1 & intrval ((# (scale,3)),(# (scale,4))) = t2 & intrval ((# (scale,4)),(# (scale,5))) = t1 & intrval ((# (scale,5)),(# (scale,6))) = t1 & intrval ((# (scale,6)),(# (scale,7))) = t2 & intrval ((# (scale,7)),(# (scale,8))) = t1 ) );