aboutsummaryrefslogtreecommitdiffhomepage
path: root/vernac/indschemes.ml
diff options
context:
space:
mode:
Diffstat (limited to 'vernac/indschemes.ml')
-rw-r--r--vernac/indschemes.ml3
1 files changed, 2 insertions, 1 deletions
diff --git a/vernac/indschemes.ml b/vernac/indschemes.ml
index b21e80bef..885769143 100644
--- a/vernac/indschemes.ml
+++ b/vernac/indschemes.ml
@@ -472,7 +472,8 @@ let build_combined_scheme env schemes =
let ctx, ind, nargs = find_inductive t in
(* Number of clauses, including the predicates quantification *)
let prods = nb_prod Evd.empty (EConstr.of_constr t) - (nargs + 1) (** FIXME *) in
- let coqand = Coqlib.build_coq_and () and coqconj = Coqlib.build_coq_conj () in
+ let coqand = Universes.constr_of_global @@ Coqlib.build_coq_and () in
+ let coqconj = Universes.constr_of_global @@ Coqlib.build_coq_conj () in
let relargs = rel_vect 0 prods in
let concls = List.rev_map
(fun (cst, t) -> (* FIXME *)