package coq

  1. Overview
  2. Docs
Legend:
Library
Module
Module type
Parameter
Class
Class type
val pr_constr : (Environ.env -> Evd.evar_map -> Constr.constr -> Pp.t) Hook.t
val refine : typecheck:bool -> (Evd.evar_map -> Evd.evar_map * EConstr.t) -> unit Proofview.tactic
val refine_one : typecheck:bool -> (Evd.evar_map -> Evd.evar_map * ('a * EConstr.t)) -> 'a Proofview.tactic
val generic_refine : typecheck:bool -> ('a * EConstr.t) Proofview.tactic -> Proofview.Goal.t -> 'a Proofview.tactic
val refine_casted : typecheck:bool -> (Evd.evar_map -> Evd.evar_map * EConstr.t) -> unit Proofview.tactic
val solve_constraints : unit Proofview.tactic