src/HOL/Groups.thy
changeset 48891 c0eafbd55de3
parent 48556 62a3fbf9d35b
child 49388 1ffd5a055acf
--- a/src/HOL/Groups.thy	Wed Aug 22 22:47:16 2012 +0200
+++ b/src/HOL/Groups.thy	Wed Aug 22 22:55:41 2012 +0200
@@ -6,7 +6,6 @@
 
 theory Groups
 imports Orderings
-uses ("Tools/group_cancel.ML")
 begin
 
 subsection {* Fact collections *}
@@ -830,7 +829,7 @@
 
 end
 
-use "Tools/group_cancel.ML"
+ML_file "Tools/group_cancel.ML"
 
 simproc_setup group_cancel_add ("a + b::'a::ab_group_add") =
   {* fn phi => fn ss => try Group_Cancel.cancel_add_conv *}