aboutsummaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/bug_4859.v
blob: 7be0bedcfc3123db0577e8ef34fcd12f502bc4ce (plain)
1
2
3
4
5
6
7
(* Not supported but check at least that it does not raise an anomaly *)

Inductive Fin{n : nat} : Set :=
| F1{i : nat}{e : n = S i}
| FS{i : nat}(f : @ Fin i){e : n = S i}.

Fail Scheme Equality for Fin.