aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/hipattern.mli
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <mattam@mattam.org>2017-05-29 18:34:47 +0200
committerGravatar Matthieu Sozeau <mattam@mattam.org>2017-05-29 18:35:10 +0200
commitef8cf82668a794f116ae714749f434e3505880d1 (patch)
tree7534ef1a657c1618b1b0497c1db1c2d1a8e77872 /tactics/hipattern.mli
parent22014c3fd400446556d3c2d7548d4638a7ed96ee (diff)
tactics cleanup: remove constr_of_global calls
Diffstat (limited to 'tactics/hipattern.mli')
-rw-r--r--tactics/hipattern.mli2
1 files changed, 1 insertions, 1 deletions
diff --git a/tactics/hipattern.mli b/tactics/hipattern.mli
index 82a3d47b5..9110830aa 100644
--- a/tactics/hipattern.mli
+++ b/tactics/hipattern.mli
@@ -142,7 +142,7 @@ val is_matching_sigma : evar_map -> constr -> bool
(** Match a decidable equality judgement (e.g [{t=u:>T}+{~t=u}]), returns
[t,u,T] and a boolean telling if equality is on the left side *)
-val match_eqdec : evar_map -> constr -> bool * constr * constr * constr * constr
+val match_eqdec : evar_map -> constr -> bool * Globnames.global_reference * constr * constr * constr
(** Match an equality up to conversion; returns [(eq,t1,t2)] in normal form *)
val dest_nf_eq : ('a, 'r) Proofview.Goal.t -> constr -> (constr * constr * constr)