forall_elim_var(s) move here from drule.ML;
authorwenzelm
Thu, 21 Oct 1999 18:42:38 +0200
changeset 7899 58c91ff28c3d
parent 7898 d7e65a52acf9
child 7900 e62973fccc97
forall_elim_var(s) move here from drule.ML; add_axioms/defs: forall_elim_vars on result;
src/Pure/pure_thy.ML
--- a/src/Pure/pure_thy.ML	Thu Oct 21 18:41:51 1999 +0200
+++ b/src/Pure/pure_thy.ML	Thu Oct 21 18:42:38 1999 +0200
@@ -28,6 +28,8 @@
   val thms_containing: theory -> string list -> (string * thm) list
   val store_thm: (bstring * thm) * theory attribute list -> theory -> theory * thm
   val smart_store_thms: (bstring * thm list) -> thm list
+  val forall_elim_var: int -> thm -> thm
+  val forall_elim_vars: int -> thm -> thm
   val add_thms: ((bstring * thm) * theory attribute list) list -> theory -> theory
   val add_thmss: ((bstring * thm list) * theory attribute list) list -> theory -> theory
   val have_thmss: bstring -> theory attribute list ->
@@ -266,10 +268,29 @@
       in enter_thmx (Sign.deref sg_ref) name_multi (name, thms) end;
 
 
+(* forall_elim_vars (belongs to drule.ML) *)
+
+(*Replace outermost quantified variable by Var of given index.
+    Could clash with Vars already present.*)
+fun forall_elim_var i th =
+    let val {prop,sign,...} = rep_thm th
+    in case prop of
+          Const("all",_) $ Abs(a,T,_) =>
+              forall_elim (cterm_of sign (Var((a,i), T)))  th
+        | _ => raise THM("forall_elim_var", i, [th])
+    end;
+
+(*Repeat forall_elim_var until all outer quantifiers are removed*)
+fun forall_elim_vars i th =
+    forall_elim_vars i (forall_elim_var i th)
+        handle THM _ => th;
+
+
 (* store axioms as theorems *)
 
 local
-  fun get_axs thy named_axs = map (Thm.get_axiom thy o fst) named_axs;
+  fun get_axs thy named_axs =
+    map (forall_elim_vars 0 o Thm.get_axiom thy o fst) named_axs;
 
   fun add_single add ((name, ax), atts) thy =
     let