aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/setoid_replace.ml
diff options
context:
space:
mode:
Diffstat (limited to 'tactics/setoid_replace.ml')
-rw-r--r--tactics/setoid_replace.ml10
1 files changed, 5 insertions, 5 deletions
diff --git a/tactics/setoid_replace.ml b/tactics/setoid_replace.ml
index 8c2077f46..3a4ae8e13 100644
--- a/tactics/setoid_replace.ml
+++ b/tactics/setoid_replace.ml
@@ -30,6 +30,7 @@ open Tacticals
open Vernacexpr
open Safe_typing
open Nametab
+open Decl_kinds
type setoid =
{ set_a : constr;
@@ -297,12 +298,12 @@ let add_setoid a aeq th =
((DefinitionEntry {const_entry_body = eq_morph;
const_entry_type = Some eq_morph_typ;
const_entry_opaque = true}),
- Libnames.NeverDischarge) in
+ IsProof Lemma) in
let _ = Declare.declare_constant eq_ext_name2
((DefinitionEntry {const_entry_body = eq_morph2;
const_entry_type = Some eq_morph2_typ;
const_entry_opaque = true}),
- Libnames.NeverDischarge) in
+ IsProof Lemma) in
let eqmorph = (current_constant eq_ext_name) in
let eqmorph2 = (current_constant eq_ext_name2) in
(Lib.add_anonymous_leaf
@@ -415,8 +416,7 @@ let new_morphism m id hook =
let lem = (gen_compat_lemma env m body args_t poss) in
let lemast = (ast_of_constr true env lem) in
new_edited id m poss;
- start_proof_com (Some id) (false,Libnames.NeverDischarge)
- ([],lemast) hook;
+ start_proof_com (Some id) (IsGlobal DefinitionBody) ([],lemast) hook;
(Options.if_verbose Vernacentries.show_open_subgoals ()))
let rec sub_bool l1 n = function
@@ -511,7 +511,7 @@ let add_morphism lem_name (m,profil) =
((DefinitionEntry {const_entry_body = lem_2;
const_entry_type = None;
const_entry_opaque = true}),
- Libnames.NeverDischarge) in
+ IsProof Lemma) in
let lem2 = (current_constant lem2_name) in
(Lib.add_anonymous_leaf
(morphism_to_obj (m,