aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/unification.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-09-12 08:34:51 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-09-12 08:34:51 +0000
commit56b8bf5bdada4a09ace234c96304b4898def9664 (patch)
treecf583273e4a28924302d7cfb117e252bdbdbe655 /test-suite/success/unification.v
parent3b8a00ab56de51d59cc14ef548929403365269e8 (diff)
Ajout unification pattern dans l'algorithme d'unification des
tactiques (unification.ml) + renommages (evarconv.ml) + exemple (unification.v) git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@9131 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/success/unification.v')
-rw-r--r--test-suite/success/unification.v15
1 files changed, 15 insertions, 0 deletions
diff --git a/test-suite/success/unification.v b/test-suite/success/unification.v
index 60c03831a..688696215 100644
--- a/test-suite/success/unification.v
+++ b/test-suite/success/unification.v
@@ -48,3 +48,18 @@ Parameter t: L (unit + unit).
Check (f (fun x : unit + unit =>
sum_rec (fun _ : unit + unit => L unit)
(fun y => c y) (fun y => c y) x) t).
+
+
+(* Test patterns unification in apply *)
+
+Require Import Arith.
+Parameter x y : nat.
+Parameter G:x=y->x=y->Prop.
+Parameter K:x<>y->x<>y->Prop.
+Lemma l3 : (forall f:x=y->Prop, forall g:x<>y->Prop,
+ match eq_nat_dec x y with left a => f a | right a => g a end)
+ -> match eq_nat_dec x y with left a => G a a | right a => K a a end.
+Proof.
+intros.
+apply H.
+Qed.