--- a/src/HOL/Hilbert_Choice.thy Wed Aug 22 22:47:16 2012 +0200
+++ b/src/HOL/Hilbert_Choice.thy Wed Aug 22 22:55:41 2012 +0200
@@ -8,7 +8,6 @@
theory Hilbert_Choice
imports Nat Wellfounded Plain
keywords "specification" "ax_specification" :: thy_goal
-uses ("Tools/choice_specification.ML")
begin
subsection {* Hilbert's epsilon *}
@@ -649,6 +648,6 @@
lemma exE_some: "[| Ex P ; c == Eps P |] ==> P c"
by (simp only: someI_ex)
-use "Tools/choice_specification.ML"
+ML_file "Tools/choice_specification.ML"
end