aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/eauto.mli
diff options
context:
space:
mode:
authorGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-04-21 13:57:03 +0000
committerGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-04-21 13:57:03 +0000
commit880a83169c1d1df8726d301a9f8a9fc845cc7d1e (patch)
tree11f101429c8d8759b11a5b6589ec28e70585abcd /tactics/eauto.mli
parent6a8e2a2e13978b40f246563d7cfda0ec58370006 (diff)
- Parameterize unification by two sets of transparent_state, one for open
term unification (for constant and variable delta unfolding) and one to parameterize closed-term conversion. Most of the time conversion uses full delta and unification does no delta. This fine-grain is used in rewrite/setoid_rewrite, where only closed-term delta on global constants is allowed. - Interpret Hint Unfold as a directive for delta conversion in auto/eauto when applying lemmas (i.e., for Resolve and Immediate hints). - Remove ad-hoc support for this in typeclasses. Now setoid_rewrite works correctly w.r.t. the old version regarding local definitions. - Fix closed bugs which needed updating due to syntax modifications. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10824 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'tactics/eauto.mli')
-rw-r--r--tactics/eauto.mli2
1 files changed, 1 insertions, 1 deletions
diff --git a/tactics/eauto.mli b/tactics/eauto.mli
index d1883aa66..1c6f9920f 100644
--- a/tactics/eauto.mli
+++ b/tactics/eauto.mli
@@ -34,4 +34,4 @@ val gen_eauto : bool -> bool * int -> constr list ->
val eauto_with_bases :
bool ->
bool * int ->
- Term.constr list -> Auto.Hint_db.t list -> Proof_type.tactic
+ Term.constr list -> Auto.hint_db list -> Proof_type.tactic