src/Pure/simplifier.ML
changeset 67561 f0b11413f1c9
parent 67147 dea94b1aabc3
child 68046 6aba668aea78
--- a/src/Pure/simplifier.ML	Thu Feb 01 15:12:57 2018 +0100
+++ b/src/Pure/simplifier.ML	Thu Feb 01 15:31:25 2018 +0100
@@ -56,7 +56,7 @@
   val set_mkcong: (Proof.context -> thm -> thm) -> Proof.context -> Proof.context
   val set_mksym: (Proof.context -> thm -> thm option) -> Proof.context -> Proof.context
   val set_mkeqTrue: (Proof.context -> thm -> thm option) -> Proof.context -> Proof.context
-  val set_termless: (term * term -> bool) -> Proof.context -> Proof.context
+  val set_term_ord: (term * term -> order) -> Proof.context -> Proof.context
   val set_subgoaler: (Proof.context -> int -> tactic) -> Proof.context -> Proof.context
   type trace_ops
   val set_trace_ops: trace_ops -> theory -> theory