aboutsummaryrefslogtreecommitdiff
path: root/plugins/rtauto/refl_tauto.mli
blob: 66ce065226d85225b538bac52240596dd4d01cef (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
22
23
24
25
26
27
28
(************************************************************************)
(*         *   The Coq Proof Assistant / The Coq Development Team       *)
(*  v      *         Copyright INRIA, CNRS and contributors             *)
(* <O___,, * (see version control and CREDITS file for authors & dates) *)
(*   \VV/  **************************************************************)
(*    //   *    This file is distributed under the terms of the         *)
(*         *     GNU Lesser General Public License Version 2.1          *)
(*         *     (see LICENSE file for the text of the license)         *)
(************************************************************************)
(* raises Not_found if no proof is found *)


type atom_env=
    {mutable next:int;
     mutable env:(Constr.t*int) list}

val make_form
  :  Environ.env -> Evd.evar_map -> atom_env
  -> EConstr.types -> Proof_search.form

val make_hyps
  :  Environ.env -> Evd.evar_map
  -> atom_env
  -> EConstr.types list
  -> EConstr.named_context
  -> (Names.Id.t Context.binder_annot * Proof_search.form) list

val rtauto_tac : unit Proofview.tactic