summaryrefslogtreecommitdiff
path: root/test-suite/output/names.v
blob: f1efd0df2aca4d0ac9dca7fb8b68fbc0b1e3e070 (plain)
1
2
3
4
5
6
7
8
9
(* Test no clash names occur *)
(* see bug #2723 *)

Parameter a : forall x, {y:nat|x=y}.
Fail Definition b y : {x:nat|x=y} := a y.

Goal (forall n m, n <= m -> m <= n -> n = m) -> True.
intro H; epose proof (H _ 3) as H.
Show.