aboutsummaryrefslogtreecommitdiff
path: root/engine/univProblem.ml
diff options
context:
space:
mode:
authorGaëtan Gilbert2021-04-06 13:30:13 +0200
committerGaëtan Gilbert2021-04-06 13:30:13 +0200
commite7c29762b995827288f09f7ad736185fb090d39c (patch)
treefc48b9b8c813f2c84a7147d9c7e1b7914637e10f /engine/univProblem.ml
parentdc565f2898145536cc6d3cf4346b6a60726bb8a9 (diff)
Remove unused UnivProblem.Set.subst_univs
Diffstat (limited to 'engine/univProblem.ml')
-rw-r--r--engine/univProblem.ml24
1 files changed, 0 insertions, 24 deletions
diff --git a/engine/univProblem.ml b/engine/univProblem.ml
index 7ac6ca1180..10ee601f3f 100644
--- a/engine/univProblem.ml
+++ b/engine/univProblem.ml
@@ -9,7 +9,6 @@
(************************************************************************)
open Univ
-open UnivSubst
type t =
| ULe of Universe.t * Universe.t
@@ -22,24 +21,6 @@ let is_trivial = function
| ULe (u, v) | UEq (u, v) -> Universe.equal u v
| ULub (u, v) | UWeak (u, v) -> Level.equal u v
-let subst_univs fn = function
- | ULe (u, v) ->
- let u' = subst_univs_universe fn u and v' = subst_univs_universe fn v in
- if Universe.equal u' v' then None
- else Some (ULe (u',v'))
- | UEq (u, v) ->
- let u' = subst_univs_universe fn u and v' = subst_univs_universe fn v in
- if Universe.equal u' v' then None
- else Some (UEq (u',v'))
- | ULub (u, v) ->
- let u' = level_subst_of fn u and v' = level_subst_of fn v in
- if Level.equal u' v' then None
- else Some (ULub (u',v'))
- | UWeak (u, v) ->
- let u' = level_subst_of fn u and v' = level_subst_of fn v in
- if Level.equal u' v' then None
- else Some (UWeak (u',v'))
-
module Set = struct
module S = Set.Make(
struct
@@ -88,11 +69,6 @@ module Set = struct
let equal x y =
x == y || equal x y
-
- let subst_univs subst csts =
- fold
- (fun c -> Option.fold_right add (subst_univs subst c))
- csts empty
end
type 'a accumulator = Set.t -> 'a -> 'a option