src/ZF/Resid/Terms.ML
changeset 6046 2c8a8be36c94
parent 5527 38928c4a8eb2
child 6112 5e4871c5136b
--- a/src/ZF/Resid/Terms.ML	Mon Dec 28 16:53:24 1998 +0100
+++ b/src/ZF/Resid/Terms.ML	Mon Dec 28 16:54:01 1998 +0100
@@ -5,41 +5,14 @@
     Logic Image: ZF
 *)
 
-open Terms;
-
-(* ------------------------------------------------------------------------- *)
-(*       unmark simplifications                                              *)
-(* ------------------------------------------------------------------------- *)
-
-Goalw [unmark_def] "unmark(Var(n)) = Var(n)";
-by (Asm_simp_tac 1);
-qed "unmark_Var";
-
-Goalw [unmark_def] "unmark(Fun(t)) = Fun(unmark(t))";
-by (Asm_simp_tac 1);
-qed "unmark_Fun";
-
-Goalw [unmark_def] "unmark(App(b,n,m)) = App(0,unmark(n),unmark(m))";
-by (Asm_simp_tac 1);
-qed "unmark_App";
-
-
-(* ------------------------------------------------------------------------- *)
-(*        term simplification set                                            *)
-(* ------------------------------------------------------------------------- *)
-
-
-Addsimps ([unmark_App, unmark_Fun, unmark_Var,
-	   lambda.dom_subset RS subsetD] @ 
-	  lambda.intrs);
+Addsimps ([lambda.dom_subset RS subsetD] @ lambda.intrs);
 
 
 (* ------------------------------------------------------------------------- *)
 (*        unmark lemmas                                                      *)
 (* ------------------------------------------------------------------------- *)
 
-Goalw [unmark_def] 
-    "u:redexes ==> unmark(u):lambda";
+Goal "u:redexes ==> unmark(u):lambda";
 by (etac redexes.induct 1);
 by (ALLGOALS Asm_simp_tac);
 qed "unmark_type";
@@ -57,14 +30,13 @@
 Goal "v:lambda ==> ALL k:nat. lift_rec(v,k):lambda";
 by (etac lambda.induct 1);
 by (ALLGOALS (asm_simp_tac (simpset() addsimps [lift_rec_Var])));
-qed "liftL_typea";
-val liftL_type =liftL_typea RS bspec ;
+bind_thm ("liftL_type", result() RS bspec);
 
 Goal "v:lambda ==>  ALL n:nat. ALL u:lambda. subst_rec(u,v,n):lambda";
 by (etac lambda.induct 1);
 by (ALLGOALS (asm_simp_tac (simpset() addsimps [liftL_type,subst_Var])));
 qed "substL_typea";
-val substL_type = substL_typea RS bspec RS bspec ;
+bind_thm ("substL_type", result() RS bspec RS bspec);
 
 
 (* ------------------------------------------------------------------------- *)