diff options
author | herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2007-05-24 12:16:09 +0000 |
---|---|---|
committer | herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2007-05-24 12:16:09 +0000 |
commit | a11acc8e5008d988451ffec989be6be07bdc43b9 (patch) | |
tree | a5095420b4046d36a029d07e85cd334c30291021 /test-suite | |
parent | 9b4967f77498f83c0ad37598a0338947c4f276ab (diff) |
Unification suite: petits affinements pour préserver la compatibilité
(en particulier, la décision de quelle instance garder quand une méta
a plusieurs solutions importe; comment trouver une critère objectif ?
la compatibilité demande à donner préférence aux instances trouvées
par with-bindings).
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@9855 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite')
-rw-r--r-- | test-suite/success/apply.v | 27 |
1 files changed, 23 insertions, 4 deletions
diff --git a/test-suite/success/apply.v b/test-suite/success/apply.v index fb6250d50..adb55cf2c 100644 --- a/test-suite/success/apply.v +++ b/test-suite/success/apply.v @@ -7,8 +7,7 @@ assumption. Qed. Require Import ZArith. -Open Scope Z_scope. -Goal forall x y z, ~ z <= 0 -> x * z < y * z -> x <= y. +Goal (forall x y z, ~ z <= 0 -> x * z < y * z -> x <= y)%Z. intros; apply Znot_le_gt, Zgt_lt in H. apply Zmult_lt_reg_r, Zlt_le_weak in H0; auto. Qed. @@ -28,6 +27,7 @@ Notation S':=S (only parsing). Goal (forall S, S = S' S) -> (forall S, S = S' S). intros. apply H with (S0 := S). +Qed. (* Check inference of implicit arguments in bindings *) @@ -44,7 +44,6 @@ exists Prop. trivial. Qed. -Definition E := Type. Variable Eq : Prop = (Prop -> Prop) :> E. Goal Prop. rewrite Eq. @@ -69,7 +68,7 @@ Abort. Reset P. (* Two examples that show that hnf_constr is used when unifying types - of bindings *) + of bindings (a simplification of a script from Field_Theory) *) Require Import List. Open Scope list_scope. @@ -91,5 +90,25 @@ intros. apply L with (1:=H). Qed. +(* The following call to auto fails if the type of the clause + associated to the H is not beta-reduced [but apply H works] + (a simplification of a script from FSetAVL) *) + +Definition apply (f:nat->Prop) := forall x, f x. +Goal apply (fun n => n=0) -> 1=0. +intro H. +auto. +Qed. +(* The following fails if the coercion Zpos is not introduced around p + before trying a subterm that matches the left-hand-side of the equality + (a simplication of an example taken from Nijmegen/QArith) *) +Require Import ZArith. +Coercion Zpos : positive >-> Z. +Variable f : Z -> Z -> Z. +Variable g : forall q1 q2 p : Z, f (f q1 p) (f q2 p) = Z0. +Goal forall p q1 q2, f (f q1 (Zpos p)) (f q2 (Zpos p)) = Z0. +intros; rewrite g with (p:=p). +reflexivity. +Qed. |