summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/4670.v
blob: 611399295393d1f4b2ad254c11b33795b23c38a3 (plain)
1
2
3
4
5
6
7
Require Import Coq.Vectors.Vector.
Module Bar.
  Definition foo A n (l : Vector.t A n) : True.
  Proof.
    induction l ; exact I.
  Defined.
End Bar.