src/HOL/Library/refute.ML
changeset 61770 a20048c78891
parent 60924 610794dff23c
child 62519 a564458f94db
--- a/src/HOL/Library/refute.ML	Tue Dec 01 22:21:40 2015 +0100
+++ b/src/HOL/Library/refute.ML	Tue Dec 01 22:24:37 2015 +0100
@@ -375,7 +375,6 @@
     end
 
 val close_form = ATP_Util.close_form
-val monomorphic_term = ATP_Util.monomorphic_term
 val specialize_type = ATP_Util.specialize_type
 
 (* ------------------------------------------------------------------------- *)
@@ -451,7 +450,7 @@
             if s=s' then
               let
                 val typeSubs = Sign.typ_match thy (T', T) Vartab.empty
-                val ax'      = monomorphic_term typeSubs ax
+                val ax'      = Envir.subst_term_types typeSubs ax
                 val rhs      = norm_rhs ax'
               in
                 SOME (axname, rhs)
@@ -495,7 +494,7 @@
                   val T'' = domain_type (domain_type T')
                   val typeSubs = Sign.typ_match thy (T'', T) Vartab.empty
                 in
-                  SOME (axname, monomorphic_term typeSubs ax)
+                  SOME (axname, Envir.subst_term_types typeSubs ax)
                 end
             | NONE => get_typedef_ax axioms
           end handle ERROR _         => get_typedef_ax axioms
@@ -669,7 +668,7 @@
         val monomorphic_class_axioms = map (fn (axname, ax) =>
           (case Term.add_tvars ax [] of
             [] => (axname, ax)
-          | [(idx, S)] => (axname, monomorphic_term (Vartab.make [(idx, (S, T))]) ax)
+          | [(idx, S)] => (axname, Envir.subst_term_types (Vartab.make [(idx, (S, T))]) ax)
           | _ =>
             raise REFUTE ("collect_axioms", "class axiom " ^ axname ^ " (" ^
               Syntax.string_of_term ctxt ax ^