aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/4527.v
diff options
context:
space:
mode:
Diffstat (limited to 'test-suite/bugs/closed/4527.v')
-rw-r--r--test-suite/bugs/closed/4527.v1
1 files changed, 1 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/4527.v b/test-suite/bugs/closed/4527.v
index 08628377f..c6fcc24b6 100644
--- a/test-suite/bugs/closed/4527.v
+++ b/test-suite/bugs/closed/4527.v
@@ -5,6 +5,7 @@ then from 269 lines to 255 lines *)
(* coqc version 8.5 (January 2016) compiled on Jan 23 2016 16:15:22 with OCaml
4.01.0
coqtop version 8.5 (January 2016) *)
+Declare ML Module "ltac_plugin".
Inductive False := .
Axiom proof_admitted : False.
Tactic Notation "admit" := case proof_admitted.