From 6911995ddd9d3b54d1c627b0000b65dad02cfce1 Mon Sep 17 00:00:00 2001 From: herbelin Date: Wed, 5 Mar 2008 19:55:36 +0000 Subject: Correction d'une typo restant du commit 10557 et cause d'échec de contribs telles que Godel MIME-Version: 1.0 Content-Type: text/plain; charset=UTF-8 Content-Transfer-Encoding: 8bit git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10622 85f007b7-540e-0410-9357-904b9bb8a0f7 --- pretyping/unification.ml | 3 ++- test-suite/success/unification.v | 7 +++++++ 2 files changed, 9 insertions(+), 1 deletion(-) diff --git a/pretyping/unification.ml b/pretyping/unification.ml index 95cef9745..890f0bd78 100644 --- a/pretyping/unification.ml +++ b/pretyping/unification.ml @@ -230,7 +230,8 @@ let unify_0_with_initial_metas metas is_subterm env sigma cv_pb flags m n = in if (not(occur_meta m)) && - (if flags.modulo_conv then is_fconv (conv_pb_of cv_pb) env sigma m n + (if flags.modulo_conv_on_closed_terms + then is_fconv (conv_pb_of cv_pb) env sigma m n else eq_constr m n) then (metas,[]) diff --git a/test-suite/success/unification.v b/test-suite/success/unification.v index 4ddaab710..6a4d92851 100644 --- a/test-suite/success/unification.v +++ b/test-suite/success/unification.v @@ -89,3 +89,10 @@ Proof. intros. apply H. Qed. + +(* Test instanciation of evars by unification *) + +Goal (forall x, 0 * x = 0 -> True) -> True. +intros; eapply H. +rewrite <- plus_n_Sm. (* should refine ?x with S ?x' *) +Abort. -- cgit v1.2.3