src/HOL/Subst/UTerm.ML
changeset 1476 608483c2122a
parent 1465 5d7a7e439cec
child 1977 26edb2771d94
--- a/src/HOL/Subst/UTerm.ML	Mon Feb 05 21:27:16 1996 +0100
+++ b/src/HOL/Subst/UTerm.ML	Mon Feb 05 21:29:06 1996 +0100
@@ -206,8 +206,18 @@
 
 (*** UTerm_rec -- by wf recursion on pred_sexp ***)
 
-val UTerm_rec_unfold =
-    [UTerm_rec_def, wf_pred_sexp RS wf_trancl] MRS def_wfrec;
+goal UTerm.thy
+   "(%M. UTerm_rec M b c d) = wfrec (trancl pred_sexp) \
+   \ (%g. Case (%x.b(x)) (Case (%y. c(y)) (Split (%x y. d x y (g x) (g y)))))";
+by (simp_tac (HOL_ss addsimps [UTerm_rec_def]) 1);
+bind_thm("UTerm_rec_unfold", (wf_pred_sexp RS wf_trancl) RS 
+                            ((result() RS eq_reflection) RS def_wfrec));
+
+(*---------------------------------------------------------------------------
+ * Old:
+ * val UTerm_rec_unfold =
+ *   [UTerm_rec_def, wf_pred_sexp RS wf_trancl] MRS def_wfrec;
+ *---------------------------------------------------------------------------*)
 
 (** conversion rules **)