src/HOL/Tools/Function/function_common.ML
changeset 36521 73ed9f18fdd3
parent 34232 36a2a3029fd3
child 36692 54b64d4ad524
equal deleted inserted replaced
36520:772ed73e1d61 36521:73ed9f18fdd3
   170 
   170 
   171 (* Default Termination Prover *)
   171 (* Default Termination Prover *)
   172 
   172 
   173 structure TerminationProver = Generic_Data
   173 structure TerminationProver = Generic_Data
   174 (
   174 (
   175   type T = Proof.context -> Proof.method
   175   type T = Proof.context -> tactic
   176   val empty = (fn _ => error "Termination prover not configured")
   176   val empty = (fn _ => error "Termination prover not configured")
   177   val extend = I
   177   val extend = I
   178   fun merge (a, b) = b  (* FIXME ? *)
   178   fun merge (a, b) = b  (* FIXME ? *)
   179 )
   179 )
   180 
   180