aboutsummaryrefslogtreecommitdiffhomepage
path: root/plugins
diff options
context:
space:
mode:
Diffstat (limited to 'plugins')
-rw-r--r--plugins/funind/functional_principles_types.ml17
-rw-r--r--plugins/funind/recdef.ml4
-rw-r--r--plugins/setoid_ring/newring.ml44
3 files changed, 14 insertions, 11 deletions
diff --git a/plugins/funind/functional_principles_types.ml b/plugins/funind/functional_principles_types.ml
index 2661a78a5..56b1a3f1c 100644
--- a/plugins/funind/functional_principles_types.ml
+++ b/plugins/funind/functional_principles_types.ml
@@ -339,15 +339,14 @@ let generate_functional_principle
let name = Indrec.make_elimination_ident base_new_princ_name fam_sort in
let value = change_property_sort s new_principle_type new_princ_name in
(* Pp.msgnl (str "new principle := " ++ pr_lconstr value); *)
- let ce =
- { const_entry_body =
- Future.from_val (value,Declareops.no_seff);
- const_entry_secctx = None;
- const_entry_type = None;
- const_entry_opaque = false;
- const_entry_inline_code = false
- }
- in
+ let ce = {
+ const_entry_body = Future.from_val (value,Declareops.no_seff);
+ const_entry_secctx = None;
+ const_entry_type = None;
+ const_entry_opaque = false;
+ const_entry_inline_code = false;
+ const_entry_feedback = None;
+ } in
ignore(
Declare.declare_constant
name
diff --git a/plugins/funind/recdef.ml b/plugins/funind/recdef.ml
index 082d7ad51..26e1011ba 100644
--- a/plugins/funind/recdef.ml
+++ b/plugins/funind/recdef.ml
@@ -61,7 +61,9 @@ let (declare_fun : Id.t -> logical_kind -> constr -> global_reference) =
const_entry_secctx = None;
const_entry_type = None;
const_entry_opaque = false;
- const_entry_inline_code = false} in
+ const_entry_inline_code = false;
+ const_entry_feedback = None;
+ } in
ConstRef(declare_constant f_id (DefinitionEntry ce, kind));;
let defined () = Lemmas.save_proof (Vernacexpr.Proved (false,None))
diff --git a/plugins/setoid_ring/newring.ml4 b/plugins/setoid_ring/newring.ml4
index aee7efb76..b8507041f 100644
--- a/plugins/setoid_ring/newring.ml4
+++ b/plugins/setoid_ring/newring.ml4
@@ -152,7 +152,9 @@ let decl_constant na c =
const_entry_secctx = None;
const_entry_type = None;
const_entry_opaque = true;
- const_entry_inline_code = false},
+ const_entry_inline_code = false;
+ const_entry_feedback = None;
+ },
IsProof Lemma))
(* Calling a global tactic *)