src/ZF/OrderType.thy
changeset 2469 b50b8c0eec01
parent 1478 2b8c2a7547ab
child 9654 9754ba005b64
equal deleted inserted replaced
2468:428efffe8599 2469:b50b8c0eec01
     6 Order types and ordinal arithmetic.
     6 Order types and ordinal arithmetic.
     7 
     7 
     8 The order type of a well-ordering is the least ordinal isomorphic to it.
     8 The order type of a well-ordering is the least ordinal isomorphic to it.
     9 *)
     9 *)
    10 
    10 
    11 OrderType = OrderArith + Ordinal + 
    11 OrderType = OrderArith + OrdQuant + 
    12 consts
    12 consts
    13   ordermap  :: [i,i]=>i
    13   ordermap  :: [i,i]=>i
    14   ordertype :: [i,i]=>i
    14   ordertype :: [i,i]=>i
    15 
    15 
    16   Ord_alt   :: i => o   
    16   Ord_alt   :: i => o