aboutsummaryrefslogtreecommitdiffhomepage
path: root/pretyping/evd.ml
diff options
context:
space:
mode:
Diffstat (limited to 'pretyping/evd.ml')
-rw-r--r--pretyping/evd.ml11
1 files changed, 3 insertions, 8 deletions
diff --git a/pretyping/evd.ml b/pretyping/evd.ml
index 0776988d7..ae16fbebe 100644
--- a/pretyping/evd.ml
+++ b/pretyping/evd.ml
@@ -1005,14 +1005,6 @@ let fresh_constructor_instance env evd c =
with_context_set univ_flexible evd (Universes.fresh_constructor_instance env c)
let fresh_global ?(rigid=univ_flexible) env evd gr =
- (* match gr with *)
- (* | ConstructRef c -> let evd, c = fresh_constructor_instance env evd c in *)
- (* evd, mkConstructU c *)
- (* | IndRef c -> let evd, c = fresh_inductive_instance env evd c in *)
- (* evd, mkIndU c *)
- (* | ConstRef c -> let evd, c = fresh_constant_instance env evd c in *)
- (* evd, mkConstU c *)
- (* | VarRef i -> evd, mkVar i *)
with_context_set rigid evd (Universes.fresh_global_instance env gr)
let whd_sort_variable evd t = t
@@ -1420,6 +1412,9 @@ type 'a sigma = {
let sig_it x = x.it
let sig_sig x = x.sigma
+let on_sig s f =
+ let sigma', v = f s.sigma in
+ { s with sigma = sigma' }, v
(*******************************************************************)
(* The state monad with state an evar map. *)