aboutsummaryrefslogtreecommitdiffhomepage
path: root/lib
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2013-04-23 18:15:43 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2013-04-23 18:15:43 +0000
commitd8324290e855b2d36e906599c7598fe5ebedb299 (patch)
treec32b263e2a281ac1befd2ee7a19e6853b42dd9e2 /lib
parentc9917c210da30521673e843b626359f4a1051e74 (diff)
Remove deprecated option -no-hash-consing (currently doing nothing)
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@16442 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'lib')
-rw-r--r--lib/flags.ml2
-rw-r--r--lib/flags.mli2
2 files changed, 0 insertions, 4 deletions
diff --git a/lib/flags.ml b/lib/flags.ml
index 6c67cb237..c6b1cdd7d 100644
--- a/lib/flags.ml
+++ b/lib/flags.ml
@@ -87,8 +87,6 @@ let is_auto_intros () = version_strictly_greater V8_2 && !auto_intros
let program_mode = ref false
let is_program_mode () = !program_mode
-let hash_cons_proofs = ref true
-
let warn = ref true
let make_warn flag = warn := flag; ()
let if_warn f x = if !warn then f x
diff --git a/lib/flags.mli b/lib/flags.mli
index 6325d7cd4..797ee3875 100644
--- a/lib/flags.mli
+++ b/lib/flags.mli
@@ -58,8 +58,6 @@ val is_program_mode : unit -> bool
val make_warn : bool -> unit
val if_warn : ('a -> unit) -> 'a -> unit
-val hash_cons_proofs : bool ref
-
(** Temporary activate an option (to activate option [o] on [f x y z],
use [with_option o (f x y) z]) *)
val with_option : bool ref -> ('a -> 'b) -> 'a -> 'b