summaryrefslogtreecommitdiff
path: root/test-suite/output/ShowProof.v
blob: 73ecaf2200000686da4e907fb37f750d83184674 (plain)
1
2
3
4
5
6
(* Was #4524 *)
Definition foo (x : Type) : True /\ True.
Proof.
split.
- exact I.
  Show Proof. (* Was not finding an evar name at some time *)