From aab16ea645fefd71b6bd0fdb155a076640ab0d4e Mon Sep 17 00:00:00 2001 From: msozeau Date: Mon, 2 Aug 2010 21:14:19 +0000 Subject: Fix [clenv_missing] to compute a better approximation of missing dependent arguments. It breaks compatibility as some [apply with] clauses are not necessary anymore. Typically when applying [f_equal], the domain type of the function can be infered even if it does not appear directly in the conclusion of the goal. Fixes bug #2154. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@13367 85f007b7-540e-0410-9357-904b9bb8a0f7 --- plugins/rtauto/Rtauto.v | 2 +- 1 file changed, 1 insertion(+), 1 deletion(-) (limited to 'plugins/rtauto/Rtauto.v') diff --git a/plugins/rtauto/Rtauto.v b/plugins/rtauto/Rtauto.v index 63e6717a0..e80542831 100644 --- a/plugins/rtauto/Rtauto.v +++ b/plugins/rtauto/Rtauto.v @@ -41,7 +41,7 @@ end. Theorem pos_eq_refl : forall m n, pos_eq m n = true -> m = n. induction m;simpl;destruct n;congruence || -(intro e;apply f_equal with positive;auto). +(intro e;apply f_equal;auto). Qed. Fixpoint form_eq (p q:form) {struct p} :bool := -- cgit v1.2.3