aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar Guillaume Melquiond <guillaume.melquiond@inria.fr>2016-11-22 17:48:14 +0100
committerGravatar Guillaume Melquiond <guillaume.melquiond@inria.fr>2017-06-14 07:27:39 +0200
commit376da97be60957b25e59afb5791fae665127b17b (patch)
tree33a57ac995bbaca4566440f305b53664c9381080
parent165e3000844c1e84cc5c9d1b579a0a7dab8a3684 (diff)
Remove options deprecated since 8.4.
-rw-r--r--pretyping/unification.ml13
-rw-r--r--vernac/indschemes.ml7
-rw-r--r--vernac/vernacentries.ml11
3 files changed, 1 insertions, 30 deletions
diff --git a/pretyping/unification.ml b/pretyping/unification.ml
index ef4f7f754..b4964c1f3 100644
--- a/pretyping/unification.ml
+++ b/pretyping/unification.ml
@@ -248,20 +248,9 @@ let sort_eqns = unify_r2l
let global_pattern_unification_flag = ref true
-(* Compatibility option introduced and activated in Coq 8.3 whose
- syntax is now deprecated. *)
-
open Goptions
-let _ =
- declare_bool_option
- { optdepr = true;
- optname = "pattern-unification for existential variables in tactics";
- optkey = ["Tactic";"Evars";"Pattern";"Unification"];
- optread = (fun () -> !global_pattern_unification_flag);
- optwrite = (:=) global_pattern_unification_flag }
-(* Compatibility option superseding the previous one, introduced and
- activated in Coq 8.4 *)
+(* Compatibility option introduced and activated in Coq 8.4 *)
let _ =
declare_bool_option
diff --git a/vernac/indschemes.ml b/vernac/indschemes.ml
index e90c25926..44d6f37cc 100644
--- a/vernac/indschemes.ml
+++ b/vernac/indschemes.ml
@@ -84,13 +84,6 @@ let _ =
optkey = ["Boolean";"Equality";"Schemes"];
optread = (fun () -> !eq_flag) ;
optwrite = (fun b -> eq_flag := b) }
-let _ = (* compatibility *)
- declare_bool_option
- { optdepr = true;
- optname = "automatic declaration of boolean equality";
- optkey = ["Equality";"Scheme"];
- optread = (fun () -> !eq_flag) ;
- optwrite = (fun b -> eq_flag := b) }
let is_eq_flag () = !eq_flag
diff --git a/vernac/vernacentries.ml b/vernac/vernacentries.ml
index ef16df5b7..9978848ff 100644
--- a/vernac/vernacentries.ml
+++ b/vernac/vernacentries.ml
@@ -1394,17 +1394,6 @@ let _ =
optread = (fun () -> !CClosure.share);
optwrite = (fun b -> CClosure.share := b) }
-(* No more undo limit in the new proof engine.
- The command still exists for compatibility (e.g. with ProofGeneral) *)
-
-let _ =
- declare_int_option
- { optdepr = true;
- optname = "the undo limit (OBSOLETE)";
- optkey = ["Undo"];
- optread = (fun _ -> None);
- optwrite = (fun _ -> ()) }
-
let _ =
declare_bool_option
{ optdepr = false;