| author | paulson <lp15@cam.ac.uk> |
| Wed, 02 Apr 2014 16:45:31 +0100 | |
| changeset 56366 | 0362c3bb4d02 |
| parent 55968 | 94242fa87638 |
| child 57959 | 1bfed12a7646 |
| 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" 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