begin
:: deftheorem defines permutations CAYLEY:def 1 :
for X being set holds permutations X = { f where f is Permutation of X : verum } ;
theorem Th1:
theorem Th2:
theorem Th3:
theorem Th4:
:: deftheorem Def2 defines SymGroup CAYLEY:def 2 :
for X being set
for b2 being strict constituted-Functions multMagma holds
( b2 = SymGroup X iff ( the carrier of b2 = permutations X & ( for x, y being Element of b2 holds x * y = y * x ) ) );
theorem Th5:
theorem Th6:
theorem
theorem
theorem Th9:
:: deftheorem Def3 defines SymGroupsIso CAYLEY:def 3 :
for X, Y being set
for p being Function of X,Y st X <> {} & Y <> {} & p is bijective holds
for b4 being Function of (SymGroup X),(SymGroup Y) holds
( b4 = SymGroupsIso p iff for x being Element of (SymGroup X) holds b4 . x = (p * x) * (p ") );
theorem Th10:
theorem Th11:
theorem Th12:
theorem
:: deftheorem Def4 defines CayleyIso CAYLEY:def 4 :
for G being Group
for b2 being Function of G,(SymGroup the carrier of G) holds
( b2 = CayleyIso G iff for g being Element of G holds b2 . g = * g );
theorem