src/HOL/Sledgehammer.thy
changeset 37399 34f080a12063
parent 36569 3a29eb7606c3
child 37410 2bf7e6136047
--- a/src/HOL/Sledgehammer.thy	Fri Jun 11 17:07:27 2010 +0200
+++ b/src/HOL/Sledgehammer.thy	Fri Jun 11 17:10:23 2010 +0200
@@ -25,6 +25,12 @@
   ("Tools/Sledgehammer/metis_tactics.ML")
 begin
 
+definition skolem_Eps :: "('a \<Rightarrow> bool) \<Rightarrow> 'a" where
+[no_atp]: "skolem_Eps = Eps"
+
+lemma skolem_someI_ex [no_atp]: "\<exists>x. P x \<Longrightarrow> P (skolem_Eps (\<lambda>x. P x))"
+unfolding skolem_Eps_def by (rule someI_ex)
+
 definition COMBI :: "'a \<Rightarrow> 'a" where
 [no_atp]: "COMBI P \<equiv> P"