aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/output/ErrorInSection.v
diff options
context:
space:
mode:
authorGravatar Tej Chajed <tchajed@mit.edu>2017-03-08 14:57:16 -0500
committerGravatar Tej Chajed <tchajed@mit.edu>2017-03-29 07:30:58 -0500
commitc5e6f5ee545ee24541836233a18c0c772077fbdf (patch)
treec69570c1ce215118c5cc392801078fa524dfe7bb /test-suite/output/ErrorInSection.v
parent9c80dd80feb1cc2ae6d0dc6e08985d4f51d4f329 (diff)
Run non-tactic comands without resilient_command
Diffstat (limited to 'test-suite/output/ErrorInSection.v')
-rw-r--r--test-suite/output/ErrorInSection.v4
1 files changed, 4 insertions, 0 deletions
diff --git a/test-suite/output/ErrorInSection.v b/test-suite/output/ErrorInSection.v
new file mode 100644
index 000000000..3036f8f05
--- /dev/null
+++ b/test-suite/output/ErrorInSection.v
@@ -0,0 +1,4 @@
+(* -*- mode: coq; coq-prog-args: ("-emacs" "-quick") -*- *)
+Section S.
+ Definition foo := nonexistent.
+End S.