aboutsummaryrefslogtreecommitdiff
path: root/engine
diff options
context:
space:
mode:
authorGaëtan Gilbert2017-10-12 13:55:08 +0200
committerGaëtan Gilbert2019-03-14 13:27:38 +0100
commita0e16c9e5c3f88a8b72935dd4877f13388640f69 (patch)
treeb177cc86b2742893adf0b181e53c03b8897b48cc /engine
parent6c447d7a7190857b03bb2992f443f1b818618a94 (diff)
Make Sorts.t private
Diffstat (limited to 'engine')
-rw-r--r--engine/eConstr.ml2
-rw-r--r--engine/evarutil.ml2
-rw-r--r--engine/evd.ml4
-rw-r--r--engine/univGen.ml4
4 files changed, 6 insertions, 6 deletions
diff --git a/engine/eConstr.ml b/engine/eConstr.ml
index 8756ebfdf2..c7b092b114 100644
--- a/engine/eConstr.ml
+++ b/engine/eConstr.ml
@@ -50,7 +50,7 @@ let in_punivs a = (a, EInstance.empty)
let mkProp = of_kind (Sort (ESorts.make Sorts.prop))
let mkSet = of_kind (Sort (ESorts.make Sorts.set))
-let mkType u = of_kind (Sort (ESorts.make (Sorts.Type u)))
+let mkType u = of_kind (Sort (ESorts.make (Sorts.sort_of_univ u)))
let mkRel n = of_kind (Rel n)
let mkVar id = of_kind (Var id)
let mkMeta n = of_kind (Meta n)
diff --git a/engine/evarutil.ml b/engine/evarutil.ml
index 840c14b241..5c2b480db4 100644
--- a/engine/evarutil.ml
+++ b/engine/evarutil.ml
@@ -836,7 +836,7 @@ let occur_evar_upto sigma n c =
let judge_of_new_Type evd =
let open EConstr in
let (evd', s) = new_univ_variable univ_rigid evd in
- (evd', { uj_val = mkSort (Sorts.Type s); uj_type = mkSort (Sorts.Type (Univ.super s)) })
+ (evd', { uj_val = mkType s; uj_type = mkType (Univ.super s) })
let subterm_source evk ?where (loc,k) =
let evk = match k with
diff --git a/engine/evd.ml b/engine/evd.ml
index dd2be29bd9..b8c52b27df 100644
--- a/engine/evd.ml
+++ b/engine/evd.ml
@@ -898,7 +898,7 @@ let new_univ_variable ?loc ?name rigid evd =
let new_sort_variable ?loc ?name rigid d =
let (d', u) = new_univ_variable ?loc rigid ?name d in
- (d', Type u)
+ (d', Sorts.sort_of_univ u)
let add_global_univ d u =
{ d with universes = UState.add_global_univ d.universes u }
@@ -965,7 +965,7 @@ let normalize_sort evars s =
| Prop | Set -> s
| Type u ->
let u' = normalize_universe evars u in
- if u' == u then s else Type u'
+ if u' == u then s else Sorts.sort_of_univ u'
(* FIXME inefficient *)
let set_eq_sort env d s1 s2 =
diff --git a/engine/univGen.ml b/engine/univGen.ml
index 40c4c909fe..4ad7fccb3a 100644
--- a/engine/univGen.ml
+++ b/engine/univGen.ml
@@ -28,7 +28,7 @@ let fresh_level () =
(* TODO: remove *)
let new_univ () = Univ.Universe.make (fresh_level ())
let new_Type () = mkType (new_univ ())
-let new_Type_sort () = Type (new_univ ())
+let new_Type_sort () = sort_of_univ (new_univ ())
let fresh_instance auctx =
let inst = Array.init (AUContext.size auctx) (fun _ -> fresh_level()) in
@@ -132,7 +132,7 @@ let fresh_sort_in_family = function
| InSet -> Sorts.set, ContextSet.empty
| InType ->
let u = fresh_level () in
- Type (Univ.Universe.make u), ContextSet.singleton u
+ sort_of_univ (Univ.Universe.make u), ContextSet.singleton u
let new_sort_in_family sf =
fst (fresh_sort_in_family sf)