--- a/src/HOL/Tools/function_package/fundef_datatype.ML Wed Jan 07 20:27:23 2009 +0100
+++ b/src/HOL/Tools/function_package/fundef_datatype.ML Wed Jan 07 20:27:55 2009 +0100
@@ -199,13 +199,13 @@
fun pat_completeness ctxt = Method.SIMPLE_METHOD' (pat_complete_tac ctxt)
val by_pat_completeness_simp =
- Proof.future_terminal_proof
+ Proof.global_future_terminal_proof
(Method.Basic (pat_completeness, Position.none),
SOME (Method.Source_i (Args.src (("HOL.auto", []), Position.none))))
fun termination_by method int =
FundefPackage.setup_termination_proof NONE
- #> Proof.future_terminal_proof
+ #> Proof.global_future_terminal_proof
(Method.Basic (method, Position.none), NONE) int
fun mk_catchall fixes arities =