aboutsummaryrefslogtreecommitdiffhomepage
path: root/pretyping/unification.ml
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-09-30 17:38:31 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-09-30 17:38:31 +0000
commit77e3ca28bbac9d973fbf0c5cd36de58159356710 (patch)
tree29a85b47d1fb380204b6638202fa038e79fd8936 /pretyping/unification.ml
parent0373800479dfeefbe6dabccaa476c42a368f6d46 (diff)
Improve handling of metas as evars in unification (patch by Hugo)
Pratical situation: simple eapply foo on a goal ?123, while foo is a (forall f, exists ...). git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@13479 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'pretyping/unification.ml')
-rw-r--r--pretyping/unification.ml3
1 files changed, 2 insertions, 1 deletions
diff --git a/pretyping/unification.ml b/pretyping/unification.ml
index b45d23098..38cf59bc0 100644
--- a/pretyping/unification.ml
+++ b/pretyping/unification.ml
@@ -673,7 +673,8 @@ let w_merge env with_types flags (evd,metas,evars) =
metas evars' eqns
| _ ->
- w_merge_rec (solve_simple_evar_eqn env evd ev rhs')
+ let evd', rhs'' = pose_all_metas_as_evars env evd rhs' in
+ w_merge_rec (solve_simple_evar_eqn env evd' ev rhs'')
metas evars' eqns
end
| [] ->