aboutsummaryrefslogtreecommitdiffhomepage
path: root/toplevel/class.ml
diff options
context:
space:
mode:
Diffstat (limited to 'toplevel/class.ml')
-rw-r--r--toplevel/class.ml7
1 files changed, 4 insertions, 3 deletions
diff --git a/toplevel/class.ml b/toplevel/class.ml
index d3acbe66b..1a252dc13 100644
--- a/toplevel/class.ml
+++ b/toplevel/class.ml
@@ -24,6 +24,7 @@ open Classops
open Declare
open Libnames
open Nametab
+open Decl_kinds
open Safe_typing
let strength_min4 stre1 stre2 stre3 stre4 =
@@ -37,7 +38,7 @@ let id_of_varid c = match kind_of_term c with
lc liste des variable dont depend la classe source *)
let rec stre_unif_cond = function
- | ([],[]) -> NeverDischarge
+ | ([],[]) -> Global
| (v::l,[]) -> variable_strength v
| ([],v::l) -> variable_strength v
| (v1::l1,v2::l2) ->
@@ -213,7 +214,7 @@ let get_strength stre ref cls clt =
(* 01/00: Supprimé la prise en compte de la force des variables locales. Sens ?
let streunif = stre_unif_cond (s_vardep,f_vardep) in
*)
- let streunif = NeverDischarge in
+ let streunif = Global in
let stre' = strength_min4 stres stret stref streunif in
strength_min (stre,stre')
@@ -265,7 +266,7 @@ let build_id_coercion idf_opt source =
{ const_entry_body = mkCast (val_f, typ_f);
const_entry_type = Some typ_f;
const_entry_opaque = false } in
- let (_,kn) = declare_constant idf (constr_entry,NeverDischarge) in
+ let (_,kn) = declare_constant idf (constr_entry,Decl_kinds.IsDefinition) in
ConstRef kn
(*