src/ZF/ex/Term.ML
changeset 760 f0200e91b272
parent 529 f0d16216e394
child 782 200a16083201
--- a/src/ZF/ex/Term.ML	Wed Dec 07 12:34:47 1994 +0100
+++ b/src/ZF/ex/Term.ML	Wed Dec 07 13:12:04 1994 +0100
@@ -38,7 +38,7 @@
 by (rtac (major RS term.induct) 1);
 by (resolve_tac prems 1);
 by (REPEAT (eresolve_tac [asm_rl, map_list_Collect, list_CollectD] 1));
-val term_induct_eqn = result();
+qed "term_induct_eqn";
 
 (**  Lemmas to justify using "term" in other recursive type definitions **)
 
@@ -86,7 +86,7 @@
 by (rewrite_goals_tac term.con_defs);
 val term_rec_ss = ZF_ss addsimps [Ord_rank, rank_pair2, prem RS map_lemma];
 by (simp_tac term_rec_ss 1);
-val term_rec = result();
+qed "term_rec";
 
 (*Slightly odd typing condition on r in the second premise!*)
 val major::prems = goal Term.thy
@@ -110,7 +110,7 @@
 \    j(Apply(a,ts)) = d(a, ts, map(%Z.j(Z), ts))";
 by (rewtac rew);
 by (rtac (tslist RS term_rec) 1);
-val def_term_rec = result();
+qed "def_term_rec";
 
 val prems = goal Term.thy
     "[| t: term(A);					     \
@@ -119,7 +119,7 @@
 \    |] ==> term_rec(t,d) : C";
 by (REPEAT (ares_tac (term_rec_type::prems) 1));
 by (etac (subset_refl RS UN_least RS list_mono RS subsetD) 1);
-val term_rec_simple_type = result();
+qed "term_rec_simple_type";
 
 
 (** term_map **)
@@ -129,13 +129,13 @@
 val prems = goalw Term.thy [term_map_def]
     "[| t: term(A);  !!x. x: A ==> f(x): B |] ==> term_map(f,t) : term(B)";
 by (REPEAT (ares_tac ([term_rec_simple_type, term.Apply_I] @ prems) 1));
-val term_map_type = result();
+qed "term_map_type";
 
 val [major] = goal Term.thy
     "t: term(A) ==> term_map(f,t) : term({f(u). u:A})";
 by (rtac (major RS term_map_type) 1);
 by (etac RepFunI 1);
-val term_map_type2 = result();
+qed "term_map_type2";
 
 
 (** term_size **)