aboutsummaryrefslogtreecommitdiff
path: root/engine
diff options
context:
space:
mode:
authorGaëtan Gilbert2017-06-13 21:43:59 +0200
committerGaëtan Gilbert2017-06-20 12:23:19 +0200
commita2bc4d3be684ad24ea7888df4dd0cf35d9733c64 (patch)
tree054f4dac6eed0adbc86aa4a608d8d28493afdf22 /engine
parentd30ed5fe0694466f70eed51bc689cd0fa8c00da5 (diff)
Remove dead code [Universes.simplify_universe_context]
Dead since 23f4804b50307766219392229757e75da9aa41d9
Diffstat (limited to 'engine')
-rw-r--r--engine/universes.ml28
-rw-r--r--engine/universes.mli3
2 files changed, 0 insertions, 31 deletions
diff --git a/engine/universes.ml b/engine/universes.ml
index bd4d75930c..dd6a69d9f9 100644
--- a/engine/universes.ml
+++ b/engine/universes.ml
@@ -1015,34 +1015,6 @@ let normalize_context_set ctx us algs =
(* let normalize_conkey = Profile.declare_profile "normalize_context_set" *)
(* let normalize_context_set a b c = Profile.profile3 normalize_conkey normalize_context_set a b c *)
-let simplify_universe_context (univs,csts) =
- let uf = UF.create () in
- let noneqs =
- Constraint.fold (fun (l,d,r) noneqs ->
- if d == Eq && (LSet.mem l univs || LSet.mem r univs) then
- (UF.union l r uf; noneqs)
- else Constraint.add (l,d,r) noneqs)
- csts Constraint.empty
- in
- let partition = UF.partition uf in
- let flex x = LSet.mem x univs in
- let subst, univs', csts' = List.fold_left (fun (subst, univs, cstrs) s ->
- let canon, (global, rigid, flexible) = choose_canonical univs flex LSet.empty s in
- (* Add equalities for globals which can't be merged anymore. *)
- let cstrs = LSet.fold (fun g cst ->
- Constraint.add (canon, Univ.Eq, g) cst) (LSet.union global rigid)
- cstrs
- in
- let subst = LSet.fold (fun f -> LMap.add f canon)
- flexible subst
- in (subst, LSet.diff univs flexible, cstrs))
- (LMap.empty, univs, noneqs) partition
- in
- (* Noneqs is now in canonical form w.r.t. equality constraints,
- and contains only inequality constraints. *)
- let csts' = subst_univs_level_constraints subst csts' in
- (univs', csts'), subst
-
let is_trivial_leq (l,d,r) =
Univ.Level.is_prop l && (d == Univ.Le || (d == Univ.Lt && Univ.Level.is_set r))
diff --git a/engine/universes.mli b/engine/universes.mli
index 5ce5e4a42a..6c2cee485c 100644
--- a/engine/universes.mli
+++ b/engine/universes.mli
@@ -210,9 +210,6 @@ val unsafe_type_of_global : Globnames.global_reference -> types
val nf_evars_and_universes_opt_subst : (existential -> constr option) ->
universe_opt_subst -> constr -> constr
-val simplify_universe_context : universe_context_set ->
- universe_context_set * universe_level_subst
-
val refresh_constraints : UGraph.t -> universe_context_set -> universe_context_set * UGraph.t
(** Pretty-printing *)