src/HOL/Codatatype/BNF_Def.thy
changeset 49284 5f39b7940b49
parent 49283 97809ae5f7bb
child 49286 dde4967c9233
--- a/src/HOL/Codatatype/BNF_Def.thy	Tue Sep 11 17:14:49 2012 +0200
+++ b/src/HOL/Codatatype/BNF_Def.thy	Tue Sep 11 17:36:09 2012 +0200
@@ -14,6 +14,7 @@
 and
   "bnf_def" :: thy_goal
 uses
+  "Tools/bnf_def_tactics.ML"
   "Tools/bnf_def.ML"
 begin