src/HOL/Fun_Def.thy
changeset 59141 9a5c2e9b001e
parent 58889 5b7a9633cfa8
child 59953 3d207f8f40dd
--- a/src/HOL/Fun_Def.thy	Fri Dec 12 14:42:37 2014 +0100
+++ b/src/HOL/Fun_Def.thy	Mon Dec 15 07:20:48 2014 +0100
@@ -5,7 +5,7 @@
 section {* Function Definitions and Termination Proofs *}
 
 theory Fun_Def
-imports Basic_BNF_Least_Fixpoints Partial_Function SAT
+imports Basic_BNF_LFPs Partial_Function SAT
 keywords "function" "termination" :: thy_goal and "fun" "fun_cases" :: thy_decl
 begin