aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success
diff options
context:
space:
mode:
Diffstat (limited to 'test-suite/success')
-rw-r--r--test-suite/success/induct.v8
1 files changed, 8 insertions, 0 deletions
diff --git a/test-suite/success/induct.v b/test-suite/success/induct.v
index b78651c91..aae55ec7a 100644
--- a/test-suite/success/induct.v
+++ b/test-suite/success/induct.v
@@ -32,3 +32,11 @@ Check
Inductive eq2 (A:Type) (a:A)
: forall B C:Type, let D:=(A*B*C)%type in D -> Prop :=
refl2 : eq2 A a unit bool (a,tt,true).
+
+(* Check that induction variables are cleared even with in clause *)
+
+Lemma foo : forall n m : nat, n + m = n + m.
+Proof.
+ intros; induction m as [|m] in n |- *.
+ auto.
+Qed.