aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/refine.mli
blob: 50b08265f427365abdcce2f46d841f99a6975a9e (plain)
1
2
3
4
5
6
7
8

(* $Id$ *)

open Term
open Tacmach

val refine : (int * constr) list * constr -> tactic
val refine_tac : (int * constr) list * constr -> tactic