From c5e6f5ee545ee24541836233a18c0c772077fbdf Mon Sep 17 00:00:00 2001 From: Tej Chajed Date: Wed, 8 Mar 2017 14:57:16 -0500 Subject: Run non-tactic comands without resilient_command --- test-suite/output/ErrorInModule.v | 4 ++++ 1 file changed, 4 insertions(+) create mode 100644 test-suite/output/ErrorInModule.v (limited to 'test-suite/output/ErrorInModule.v') diff --git a/test-suite/output/ErrorInModule.v b/test-suite/output/ErrorInModule.v new file mode 100644 index 0000000000..e69e23276b --- /dev/null +++ b/test-suite/output/ErrorInModule.v @@ -0,0 +1,4 @@ +(* -*- mode: coq; coq-prog-args: ("-emacs" "-quick") -*- *) +Module M. + Definition foo := nonexistent. +End M. -- cgit v1.2.3