aboutsummaryrefslogtreecommitdiffhomepage
path: root/pretyping/coercion.ml
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2016-02-15 13:31:54 +0100
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2016-02-15 13:41:16 +0100
commit1a8c37ca352c95b4cd530efbbf47f0e7671d1fb3 (patch)
tree15aadd829fe3e8c3ee0a747de34a9b96614bfdba /pretyping/coercion.ml
parent968dfdb15cc11d48783017b2a91147b25c854ad6 (diff)
Renaming functions in Typing to stick to the standard e_* scheme.
Diffstat (limited to 'pretyping/coercion.ml')
-rw-r--r--pretyping/coercion.ml2
1 files changed, 1 insertions, 1 deletions
diff --git a/pretyping/coercion.ml b/pretyping/coercion.ml
index 489a311bc..8dae311a9 100644
--- a/pretyping/coercion.ml
+++ b/pretyping/coercion.ml
@@ -187,7 +187,7 @@ and coerce loc env evdref (x : Term.constr) (y : Term.constr)
(subst1 hdy restT') (succ i) (fun x -> eq_app (co x))
else Some (fun x ->
let term = co x in
- Typing.solve_evars env evdref term)
+ Typing.e_solve_evars env evdref term)
in
if isEvar c || isEvar c' then
(* Second-order unification needed. *)