src/HOL/Types_To_Sets/Types_To_Sets.thy
changeset 68428 46beee72fb66
parent 68224 1f7308050349
child 69605 a96320074298
equal deleted inserted replaced
68427:f75d765a281f 68428:46beee72fb66
    22 ML_file "unoverloading.ML"
    22 ML_file "unoverloading.ML"
    23 
    23 
    24 text\<open>The following file implements a derived rule that internalizes type class annotations.\<close>
    24 text\<open>The following file implements a derived rule that internalizes type class annotations.\<close>
    25 ML_file "internalize_sort.ML"
    25 ML_file "internalize_sort.ML"
    26 
    26 
       
    27 text\<open>The following file provides some automation to unoverload and internalize the parameters o
       
    28   the sort constraints of a type variable.\<close>
       
    29 ML_file \<open>unoverload_type.ML\<close>
       
    30 
    27 end
    31 end