aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/HoTT_coq_107.v
diff options
context:
space:
mode:
authorGravatar Paul Steckler <steck@stecksoft.com>2017-05-01 11:34:00 -0400
committerGravatar Paul Steckler <steck@stecksoft.com>2017-05-01 11:34:00 -0400
commitf6856c5022ef27cdc492daadd1301cfcad025b01 (patch)
treee886b9ef6667a23460c72b581481b227336b7128 /test-suite/bugs/closed/HoTT_coq_107.v
parent68fb8e13c44c5ee95dbc9256b1d74c7c83303d2d (diff)
remove unneeded -emacs flag to coq-prog-args
Diffstat (limited to 'test-suite/bugs/closed/HoTT_coq_107.v')
-rw-r--r--test-suite/bugs/closed/HoTT_coq_107.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/test-suite/bugs/closed/HoTT_coq_107.v b/test-suite/bugs/closed/HoTT_coq_107.v
index 7c1ab8dc2..fa4072a8f 100644
--- a/test-suite/bugs/closed/HoTT_coq_107.v
+++ b/test-suite/bugs/closed/HoTT_coq_107.v
@@ -1,4 +1,4 @@
-(* -*- mode: coq; coq-prog-args: ("-emacs" "-nois" "-R" "../theories" "Coq") -*- *)
+(* -*- mode: coq; coq-prog-args: ("-nois" "-R" "../theories" "Coq") -*- *)
(* File reduced by coq-bug-finder from 4897 lines to 2605 lines, then from 2297 lines to 236 lines, then from 239 lines to 137 lines, then from 118 lines to 67 lines, then from 520 lines to 76 lines. *)
(** Note: The bug here is the same as the #113, that is, HoTT_coq_113.v *)
Require Import Coq.Init.Logic.