aboutsummaryrefslogtreecommitdiffhomepage
path: root/pretyping/evd.ml
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-10-27 13:58:11 +0100
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-10-27 13:58:11 +0100
commit0b83f3f96d6320847bd55a6dbbff109b95f3d039 (patch)
tree4c36c93b469b787b793a711855e407fe927cf010 /pretyping/evd.ml
parent324d0b06a777018fc7441e8aeaae8e3e85a48671 (diff)
Removing dead code from Evd.
Diffstat (limited to 'pretyping/evd.ml')
-rw-r--r--pretyping/evd.ml24
1 files changed, 0 insertions, 24 deletions
diff --git a/pretyping/evd.ml b/pretyping/evd.ml
index e1d5c5a98..a3c9e3963 100644
--- a/pretyping/evd.ml
+++ b/pretyping/evd.ml
@@ -16,7 +16,6 @@ open Vars
open Termops
open Environ
open Globnames
-open Mod_subst
(** Generic filters *)
module Filter :
@@ -730,29 +729,6 @@ let is_empty d =
List.is_empty d.conv_pbs &&
Metamap.is_empty d.metas
-let subst_named_context_val s = map_named_val (subst_mps s)
-
-let subst_evar_info s evi =
- let subst_evb = function
- | Evar_empty -> Evar_empty
- | Evar_defined c -> Evar_defined (subst_mps s c)
- in
- { evi with
- evar_concl = subst_mps s evi.evar_concl;
- evar_hyps = subst_named_context_val s evi.evar_hyps;
- evar_body = subst_evb evi.evar_body }
-
-let subst_evar_defs_light sub evd =
- assert (Univ.is_initial_universes evd.universes.uctx_universes);
- assert (List.is_empty evd.conv_pbs);
- let map_info i = subst_evar_info sub i in
- { evd with
- undf_evars = EvMap.smartmap map_info evd.undf_evars;
- defn_evars = EvMap.smartmap map_info evd.defn_evars;
- metas = Metamap.smartmap (map_clb (subst_mps sub)) evd.metas; }
-
-let subst_evar_map = subst_evar_defs_light
-
let cmap f evd =
{ evd with
metas = Metamap.map (map_clb f) evd.metas;