src/HOL/Bali/Type.thy
changeset 58249 180f1b3508ed
parent 37956 ee939247b2fb
child 58310 91ea607a34d8
equal deleted inserted replaced
58248:25af24e1f37b 58249:180f1b3508ed
    12 \item only the most important primitive types
    12 \item only the most important primitive types
    13 \item the null type is regarded as reference type
    13 \item the null type is regarded as reference type
    14 \end{itemize}
    14 \end{itemize}
    15 *}
    15 *}
    16 
    16 
    17 datatype prim_ty        --{* primitive type, cf. 4.2 *}
    17 datatype_new prim_ty        --{* primitive type, cf. 4.2 *}
    18         = Void          --{* result type of void methods *}
    18         = Void          --{* result type of void methods *}
    19         | Boolean
    19         | Boolean
    20         | Integer
    20         | Integer
    21 
    21 
    22 
    22 
    23 datatype ref_ty         --{* reference type, cf. 4.3 *}
    23 datatype_new ref_ty         --{* reference type, cf. 4.3 *}
    24         = NullT         --{* null type, cf. 4.1 *}
    24         = NullT         --{* null type, cf. 4.1 *}
    25         | IfaceT qtname --{* interface type *}
    25         | IfaceT qtname --{* interface type *}
    26         | ClassT qtname --{* class type *}
    26         | ClassT qtname --{* class type *}
    27         | ArrayT ty     --{* array type *}
    27         | ArrayT ty     --{* array type *}
    28 
    28