(************************************************************************) (* v * The Coq Proof Assistant / The Coq Development Team *) (* constr -> tactic val lemInvIn_gen : quantified_hypothesis -> constr -> identifier list -> tactic val lemInv_clause : quantified_hypothesis -> constr -> identifier list -> tactic val inversion_lemma_from_goal : int -> identifier -> identifier located -> sorts -> bool -> (identifier -> tactic) -> unit val add_inversion_lemma_exn : identifier -> constr_expr -> glob_sort -> bool -> (identifier -> tactic) -> unit