aboutsummaryrefslogtreecommitdiff
path: root/tactics/eauto.ml
diff options
context:
space:
mode:
authorPierre-Marie Pédrot2018-11-19 08:12:28 +0100
committerPierre-Marie Pédrot2018-11-19 13:29:55 +0100
commit733cb74a2038ff92156b7209713fc2ea741ccca6 (patch)
treeee664936850ce6160d9e3fc3219b9dba7b7ea096 /tactics/eauto.ml
parentad5aea737ecc639c31dda84322b3550a4d380b47 (diff)
Rename TranspState into TransparentState.
Diffstat (limited to 'tactics/eauto.ml')
-rw-r--r--tactics/eauto.ml6
1 files changed, 3 insertions, 3 deletions
diff --git a/tactics/eauto.ml b/tactics/eauto.ml
index c18b7bb214..9a6bdab7b9 100644
--- a/tactics/eauto.ml
+++ b/tactics/eauto.ml
@@ -29,7 +29,7 @@ open Locusops
open Hints
open Proofview.Notations
-let eauto_unif_flags = auto_flags_of_state TranspState.full
+let eauto_unif_flags = auto_flags_of_state TransparentState.full
let e_give_exact ?(flags=eauto_unif_flags) c =
Proofview.Goal.enter begin fun gl ->
@@ -307,7 +307,7 @@ module SearchProblem = struct
let gls = {Evd.it = gl; sigma = lgls.Evd.sigma } in
let hyps' = pf_hyps gls in
if hyps' == hyps then List.hd s.localdb
- else make_local_hint_db (pf_env gls) (project gls) ~ts:TranspState.full true s.local_lemmas)
+ else make_local_hint_db (pf_env gls) (project gls) ~ts:TransparentState.full true s.local_lemmas)
(List.firstn ((nbgl'-nbgl) + 1) (sig_it lgls))
in
{ depth = pred s.depth; priority = cost; tacres = lgls;
@@ -388,7 +388,7 @@ let make_initial_state dbg n gl dblist localdb lems =
}
let e_search_auto debug (in_depth,p) lems db_list gl =
- let local_db = make_local_hint_db (pf_env gl) (project gl) ~ts:TranspState.full true lems in
+ let local_db = make_local_hint_db (pf_env gl) (project gl) ~ts:TransparentState.full true lems in
let d = mk_eauto_dbg debug in
let tac = match in_depth,d with
| (true,Debug) -> Search.debug_depth_first