TFL/tfl.ML
changeset 22578 b0eb5652f210
parent 20951 868120282837
child 22692 1e057a3f087d
--- a/TFL/tfl.ML	Wed Apr 04 00:10:59 2007 +0200
+++ b/TFL/tfl.ML	Wed Apr 04 00:11:03 2007 +0200
@@ -392,7 +392,7 @@
      val wfrec_R_M =  map_types poly_tvars
                           (wfrec $ map_types poly_tvars R)
                       $ functional
-     val def_term = mk_const_def (Theory.sign_of thy) (x, Ty, wfrec_R_M)
+     val def_term = mk_const_def thy (x, Ty, wfrec_R_M)
      val ([def], thy') = PureThy.add_defs_i false [Thm.no_attributes (def_name, def_term)] thy
  in (thy', def) end;
 end;
@@ -502,7 +502,7 @@
      val dummy =
            if !trace then
                writeln ("ORIGINAL PROTO_DEF: " ^
-                          Sign.string_of_term (Theory.sign_of thy) proto_def)
+                          Sign.string_of_term thy proto_def)
            else ()
      val R1 = S.rand WFR
      val corollary' = R.UNDISCH(R.UNDISCH WFREC_THM)
@@ -543,13 +543,12 @@
      val proto_def' = subst_free[(R1,R')] proto_def
      val dummy = if !trace then writeln ("proto_def' = " ^
                                          Sign.string_of_term
-                                         (Theory.sign_of thy) proto_def')
+                                         thy proto_def')
                            else ()
      val {lhs,rhs} = S.dest_eq proto_def'
      val (c,args) = S.strip_comb lhs
      val (name,Ty) = dest_atom c
-     val defn = mk_const_def (Theory.sign_of thy)
-                 (name, Ty, S.list_mk_abs (args,rhs))
+     val defn = mk_const_def thy (name, Ty, S.list_mk_abs (args,rhs))
      val ([def0], theory) =
        thy
        |> PureThy.add_defs_i false