src/ZF/CardinalArith.thy
changeset 9683 f87c8c449018
parent 9654 9754ba005b64
child 9964 7966a2902266
equal deleted inserted replaced
9682:00f8be1b7209 9683:f87c8c449018
    37          UN X:Pow(K). {z. r: Pow(K*K), well_ord(X,r) & z = ordertype(X,r)}"
    37          UN X:Pow(K). {z. r: Pow(K*K), well_ord(X,r) & z = ordertype(X,r)}"
    38 
    38 
    39   (*needed because jump_cardinal(K) might not be the successor of K*)
    39   (*needed because jump_cardinal(K) might not be the successor of K*)
    40   csucc_def "csucc(K) == LEAST L. Card(L) & K<L"
    40   csucc_def "csucc(K) == LEAST L. Card(L) & K<L"
    41 
    41 
    42 syntax (symbols)
    42 syntax (xsymbols)
    43   "op |*|"     :: [i,i] => i          (infixr "|\\<times>|" 70)
    43   "op |+|"     :: [i,i] => i          (infixl "\\<oplus>" 65)
       
    44   "op |*|"     :: [i,i] => i          (infixl "\\<otimes>" 70)
    44 
    45 
    45 end
    46 end