equal
deleted
inserted
replaced
592 in |
592 in |
593 map_index (prep_typ binds) annos |
593 map_index (prep_typ binds) annos |
594 end |
594 end |
595 |
595 |
596 in |
596 in |
597 map (map (map (map (fn (a, b, c) => (a, b, c, !alpha_type))))) |
597 map (map (map (map (fn (a, b, c) => (a, b, c, if !alpha_type=AlphaLst andalso a = NONE then AlphaGen else !alpha_type))))) |
598 (map (map prep_binds) (extract_annos_binds (get_cnstrs dt_strs))) |
598 (map (map prep_binds) (extract_annos_binds (get_cnstrs dt_strs))) |
599 end |
599 end |
600 *} |
600 *} |
601 |
601 |
602 ML {* |
602 ML {* |