src/HOL/FunDef.thy
changeset 24162 8dfd5dd65d82
parent 23739 c5ead5df7f35
child 24194 96013f81faef
equal deleted inserted replaced
24161:09027ee4eeaa 24162:8dfd5dd65d82
     4 *)
     4 *)
     5 
     5 
     6 header {* General recursive function definitions *}
     6 header {* General recursive function definitions *}
     7 
     7 
     8 theory FunDef
     8 theory FunDef
     9 imports Datatype Accessible_Part
     9 imports Datatype Option Accessible_Part
    10 uses
    10 uses
    11   ("Tools/function_package/fundef_lib.ML")
    11   ("Tools/function_package/fundef_lib.ML")
    12   ("Tools/function_package/fundef_common.ML")
    12   ("Tools/function_package/fundef_common.ML")
    13   ("Tools/function_package/inductive_wrap.ML")
    13   ("Tools/function_package/inductive_wrap.ML")
    14   ("Tools/function_package/context_tree.ML")
    14   ("Tools/function_package/context_tree.ML")