From 4dc76691537c57cb8344e82d6bb493360ae12aaa Mon Sep 17 00:00:00 2001 From: herbelin Date: Fri, 21 Sep 2007 09:42:04 +0000 Subject: - Fixing bug 1703 ("intros until n" falls back on the variable name when the latter is bound to a var which is not a quantified one - this led to remove a line marked "temporary compatibility" ... ; made a distinction between quantified hypothesis as for "intros until" and binding names as in "apply with"; in both cases, we now expect that a identifier not used as a variable, as in "apply f_equal with f:=g" where "f" is a true binder name in f_equal, must not be used as a variable elsewhere [see corresponding change in Ints/Tactic.v]) - Fixing bug 1643 (bug in the algorithm used to possibly reuse a global name in the recursive calls of a coinductive term) - Fixing bug 1699 (bug in contracting nested patterns at printing time when the return clause of the subpatterns is dependent) - Fixing bug 1697 (bug in the TacAssert clause of Tacinterp.subst_tactic) - Fixing bug 1678 (bug in converting constr_pattern to constr in Constrextern) git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10131 85f007b7-540e-0410-9357-904b9bb8a0f7 --- test-suite/output/Cases.out | 13 +++++++++++++ 1 file changed, 13 insertions(+) (limited to 'test-suite/output/Cases.out') diff --git a/test-suite/output/Cases.out b/test-suite/output/Cases.out index a3033e94f..3c440b9d0 100644 --- a/test-suite/output/Cases.out +++ b/test-suite/output/Cases.out @@ -7,3 +7,16 @@ fix F (t : t) : P t := : forall P : t -> Type, (let x := t in forall x0 : x, P x0 -> P (k x0)) -> forall t : t, P t +proj = +fun (x y : nat) (P : nat -> Type) (def : P x) (prf : P y) => +match eq_nat_dec x y with +| left eqprf => + match eqprf in (_ = z) return (P z) with + | refl_equal => def + end +| right _ => prf +end + : forall (x y : nat) (P : nat -> Type), P x -> P y -> P y + + +Argument scopes are [nat_scope nat_scope _ _ _] -- cgit v1.2.3