aboutsummaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/bug_4217.v
blob: af1fe2c755434f1d82681ca1785c763beeed20cd (plain)
1
2
3
4
5
6
7
(* Checking correct index of implicit by pos in fixpoints *)

Fixpoint ith_default
         {default_A : nat}
         {As : list nat}
         {struct As} : Set.
Abort.