aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/eauto.mli
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2016-03-21 00:26:02 +0100
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2016-03-21 00:36:57 +0100
commita581331f26d96d1a037128ae83bebd5e6c27f665 (patch)
treea45c2df2962dffd9ccdab2806f23c717d87d9fdc /tactics/eauto.mli
parentdf6132c06f9c8480b01f0a269cd1b95bbaa7f912 (diff)
Creating a dedicated ltac/ folder for Hightactics.
Diffstat (limited to 'tactics/eauto.mli')
-rw-r--r--tactics/eauto.mli33
1 files changed, 0 insertions, 33 deletions
diff --git a/tactics/eauto.mli b/tactics/eauto.mli
deleted file mode 100644
index 8812093d5..000000000
--- a/tactics/eauto.mli
+++ /dev/null
@@ -1,33 +0,0 @@
-(************************************************************************)
-(* v * The Coq Proof Assistant / The Coq Development Team *)
-(* <O___,, * INRIA - CNRS - LIX - LRI - PPS - Copyright 1999-2016 *)
-(* \VV/ **************************************************************)
-(* // * This file is distributed under the terms of the *)
-(* * GNU Lesser General Public License Version 2.1 *)
-(************************************************************************)
-
-open Term
-open Proof_type
-open Hints
-
-val e_assumption : unit Proofview.tactic
-
-val registered_e_assumption : unit Proofview.tactic
-
-val e_give_exact : ?flags:Unification.unify_flags -> constr -> unit Proofview.tactic
-
-val prolog_tac : Tacexpr.delayed_open_constr list -> int -> unit Proofview.tactic
-
-val gen_eauto : ?debug:Tacexpr.debug -> bool * int -> Tacexpr.delayed_open_constr list ->
- hint_db_name list option -> unit Proofview.tactic
-
-val eauto_with_bases :
- ?debug:Tacexpr.debug ->
- bool * int ->
- Tacexpr.delayed_open_constr list -> hint_db list -> Proof_type.tactic
-
-val autounfold : hint_db_name list -> Locus.clause -> unit Proofview.tactic
-val autounfold_tac : hint_db_name list option -> Locus.clause -> unit Proofview.tactic
-val autounfold_one : hint_db_name list -> Locus.hyp_location option -> unit Proofview.tactic
-
-val make_dimension : int option -> int option -> bool * int