blob: ba3acd088d4a5c4fda5a371a9561b05415d58254 (
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 *)
|