author | blanchet |
Mon, 01 Sep 2014 16:34:40 +0200 | |
changeset 58128 | 43a1ba26a8cb |
parent 57959 | 1bfed12a7646 |
child 58816 | aab139c0003f |
permissions | -rw-r--r-- |
(* Title: HOL/Fun_Def_Base.thy Author: Alexander Krauss, TU Muenchen *) header {* Function Definition Base *} theory Fun_Def_Base imports Ctr_Sugar Set Wellfounded begin ML_file "Tools/Function/function_lib.ML" named_theorems termination_simp "simplification rules for termination proofs" ML_file "Tools/Function/function_common.ML" ML_file "Tools/Function/context_tree.ML" setup Function_Ctx_Tree.setup ML_file "Tools/Function/sum_tree.ML" end