aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite
diff options
context:
space:
mode:
Diffstat (limited to 'test-suite')
-rw-r--r--test-suite/success/induct.v11
1 files changed, 11 insertions, 0 deletions
diff --git a/test-suite/success/induct.v b/test-suite/success/induct.v
index f15bcce8a..4e20a5077 100644
--- a/test-suite/success/induct.v
+++ b/test-suite/success/induct.v
@@ -64,3 +64,14 @@ Undo 2.
Fail induction (S _) in |- * at 4.
Abort.
+(* Check use of "as" clause *)
+
+Inductive I := C : forall x, x<0 -> I -> I.
+
+Goal forall x:I, x=x.
+intros.
+induction x as [y * IHx].
+change (x = x) in IHx. (* We should have IHx:x=x *)
+Abort.
+
+