| author | wenzelm | 
| Sun, 16 Feb 2014 21:09:47 +0100 | |
| changeset 55522 | 23d2cbac6dce | 
| parent 55085 | 0e8e4dc55866 | 
| child 55968 | 94242fa87638 | 
| 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 end