aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar Emilio Jesus Gallego Arias <e+git@x80.org>2017-11-20 03:09:43 +0100
committerGravatar Emilio Jesus Gallego Arias <e+git@x80.org>2017-11-22 11:33:58 +0100
commit9f47342d890dc3ef7f4950004513a47d940af5ca (patch)
treecfcd56e7e022fd2b416a815af5635296c6cd78c5
parentbf1e64fc3a79e2eff49aaeeaa966516b11f1cd9f (diff)
[api] A few more minor deprecation notices.
Note the problem with `create_evar_defs`.
-rw-r--r--engine/evarutil.mli5
-rw-r--r--engine/evd.mli13
-rw-r--r--engine/universes.mli1
-rw-r--r--library/lib.ml1
-rw-r--r--pretyping/cases.mli4
-rw-r--r--pretyping/pretyping.mli2
6 files changed, 16 insertions, 10 deletions
diff --git a/engine/evarutil.mli b/engine/evarutil.mli
index 62288ced4..42f2d5f25 100644
--- a/engine/evarutil.mli
+++ b/engine/evarutil.mli
@@ -238,7 +238,8 @@ val subterm_source : existential_key -> Evar_kinds.t Loc.located ->
val meta_counter_summary_name : string
-(** Deprecater *)
-
+(** Deprecated *)
type type_constraint = types option
+[@@ocaml.deprecated "use the version in Evardefine"]
type val_constraint = constr option
+[@@ocaml.deprecated "use the version in Evardefine"]
diff --git a/engine/evd.mli b/engine/evd.mli
index af5373582..17fa15045 100644
--- a/engine/evd.mli
+++ b/engine/evd.mli
@@ -599,11 +599,16 @@ type open_constr = evar_map * constr (* Special case when before is empty *)
type unsolvability_explanation = SeveralInstancesFound of int
(** Failure explanation. *)
+(** {5 Summary names} *)
+
+(* This stuff is internal and should not be used. Currently a hack in
+ the STM relies on it. *)
+val evar_counter_summary_name : string
+
(** {5 Deprecated functions} *)
+val create_evar_defs : evar_map -> evar_map
+(* XXX: This is supposed to be deprecated by used by ssrmatching, what
+ should the replacement be? *)
-val create_evar_defs : evar_map -> evar_map
(** Create an [evar_map] with empty meta map: *)
-(** {5 Summary names} *)
-
-val evar_counter_summary_name : string
diff --git a/engine/universes.mli b/engine/universes.mli
index 24613c4b9..a960099ed 100644
--- a/engine/universes.mli
+++ b/engine/universes.mli
@@ -169,6 +169,7 @@ val constr_of_global : Globnames.global_reference -> constr
(** ** DEPRECATED ** synonym of [constr_of_global] *)
val constr_of_reference : Globnames.global_reference -> constr
+[@@ocaml.deprecated "synonym of [constr_of_global]"]
(** Returns the type of the global reference, by creating a fresh instance of polymorphic
references and computing their instantiated universe context. (side-effect on the
diff --git a/library/lib.ml b/library/lib.ml
index 6abbf7ef9..3dbb16c7b 100644
--- a/library/lib.ml
+++ b/library/lib.ml
@@ -12,7 +12,6 @@ open Util
open Names
open Libnames
open Globnames
-(* open Nameops *)
open Libobject
open Context.Named.Declaration
diff --git a/pretyping/cases.mli b/pretyping/cases.mli
index 3a139b7b0..43dbc3105 100644
--- a/pretyping/cases.mli
+++ b/pretyping/cases.mli
@@ -13,8 +13,8 @@ open Environ
open EConstr
open Inductiveops
open Glob_term
-open Evarutil
open Ltac_pretype
+open Evardefine
(** {5 Compilation of pattern-matching } *)
@@ -116,7 +116,7 @@ type 'a pattern_matching_problem =
val compile : 'a pattern_matching_problem -> unsafe_judgment
val prepare_predicate : ?loc:Loc.t ->
- (Evarutil.type_constraint ->
+ (type_constraint ->
Environ.env -> Evd.evar_map ref -> ltac_var_map -> glob_constr -> unsafe_judgment) ->
Environ.env ->
Evd.evar_map ->
diff --git a/pretyping/pretyping.mli b/pretyping/pretyping.mli
index eb2b435bf..b2735ee22 100644
--- a/pretyping/pretyping.mli
+++ b/pretyping/pretyping.mli
@@ -17,8 +17,8 @@ open Environ
open Evd
open EConstr
open Glob_term
-open Evarutil
open Ltac_pretype
+open Evardefine
(** An auxiliary function for searching for fixpoint guard indexes *)