summaryrefslogtreecommitdiff
path: root/test-suite/output/ErrorInSection.v
blob: 505c5ce378743694a3e72fcd84ec158eb4d05be3 (plain)
1
2
3
4
(* -*- mode: coq; coq-prog-args: ("-quick") -*- *)
Section S.
  Definition foo := nonexistent.
End S.