summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/2995.v
blob: b6c5b6df448034de3ad9014cf26452f1129d1917 (plain)
1
2
3
4
5
6
7
8
9
Module Type Interface.
  Parameter error: nat.
End Interface.

Module Implementation <: Interface.
  Definition t := bool.
  Definition error: t := false.
Fail End Implementation.
(* A UserError here is expected, not an uncaught Not_found *)