src/HOL/FunDef.thy
changeset 46950 d0181abdbdac
parent 46526 c4cf9d03c352
child 47432 e1576d13e933
equal deleted inserted replaced
46949:94aa7b81bcf6 46950:d0181abdbdac
     4 
     4 
     5 header {* Function Definitions and Termination Proofs *}
     5 header {* Function Definitions and Termination Proofs *}
     6 
     6 
     7 theory FunDef
     7 theory FunDef
     8 imports Partial_Function Wellfounded
     8 imports Partial_Function Wellfounded
       
     9 keywords "function" "termination" :: thy_goal and "fun" :: thy_decl
     9 uses
    10 uses
    10   "Tools/prop_logic.ML"
    11   "Tools/prop_logic.ML"
    11   "Tools/sat_solver.ML"
    12   "Tools/sat_solver.ML"
    12   ("Tools/Function/function_common.ML")
    13   ("Tools/Function/function_common.ML")
    13   ("Tools/Function/context_tree.ML")
    14   ("Tools/Function/context_tree.ML")