diff options
author | herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2010-09-17 16:02:50 +0000 |
---|---|---|
committer | herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2010-09-17 16:02:50 +0000 |
commit | 84aaa74ff9537dfdfc214ab60f8acf42466878b1 (patch) | |
tree | 6fe6ad11a592f51385f4f82c747c9e08b2929584 /test-suite/success | |
parent | 2a35022f6e0ed8b5a2b2fce5077104cfa6cea1b3 (diff) |
In the computation of missing arguments for apply, accept that the
user either gives all missing arguments not dependent in the concl or
all missing arguments not *recursively* dependent in the concl (as
introduced by commit 13367). In practice, this means that "apply
f_equal with A" remains allowed even though the new, recursive,
analysis detects that all arguments of f_equal are inferable,
including the first type argument (which is inferable from the
knowledge of the function).
Sized the opportunity to better explain the behavior of clenv_dependent.
Also made minor code simplification.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@13426 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/success')
-rw-r--r-- | test-suite/success/auto.v | 18 |
1 files changed, 18 insertions, 0 deletions
diff --git a/test-suite/success/auto.v b/test-suite/success/auto.v new file mode 100644 index 000000000..a2701f8bb --- /dev/null +++ b/test-suite/success/auto.v @@ -0,0 +1,18 @@ +(* Wish #2154 by E. van der Weegen *) + +(* auto was not using f_equal-style lemmas with metavariables occuring + only in the type of an evar of the concl, but not directly in the + concl itself *) + +Parameters + (F: Prop -> Prop) + (G: forall T, (T -> Prop) -> Type) + (L: forall A (P: A -> Prop), G A P -> forall x, F (P x)) + (Q: unit -> Prop). + +Hint Resolve L. + +Goal G unit Q -> F (Q tt). + intro. + auto. +Qed. |