src/CCL/Term.thy
changeset 56199 8e8d28ed7529
parent 52143 36ffe23b25f8
child 58889 5b7a9633cfa8
--- a/src/CCL/Term.thy	Tue Mar 18 10:00:23 2014 +0100
+++ b/src/CCL/Term.thy	Tue Mar 18 11:07:47 2014 +0100
@@ -286,7 +286,7 @@
 subsection {* Constructors are distinct *}
 
 ML {*
-bind_thms ("term_dstncts",
+ML_Thms.bind_thms ("term_dstncts",
   mkall_dstnct_thms @{context} @{thms data_defs} (@{thms ccl_injs} @ @{thms term_injs})
     [["bot","inl","inr"], ["bot","zero","succ"], ["bot","nil","cons"]]);
 *}
@@ -305,7 +305,7 @@
 subsection {* Rewriting and Proving *}
 
 ML {*
-  bind_thms ("term_injDs", XH_to_Ds @{thms term_injs});
+  ML_Thms.bind_thms ("term_injDs", XH_to_Ds @{thms term_injs});
 *}
 
 lemmas term_rews = termBs term_injs term_dstncts ccl_porews term_porews