aboutsummaryrefslogtreecommitdiff
path: root/vernac/comFixpoint.ml
diff options
context:
space:
mode:
authorEmilio Jesus Gallego Arias2020-06-18 20:14:19 +0200
committerEmilio Jesus Gallego Arias2020-06-26 14:38:12 +0200
commitc7a62d0ee0205dfe5bef4bb874c04f1978d4b5c3 (patch)
treebbd20c6801c5d7e885759ef31df51a3eaa030027 /vernac/comFixpoint.ml
parent22bb101bae56a56a7bcdad2562daf5150ee9408b (diff)
[declare] Refactor analysis and construction of mutual lemmas
When declaring a lemma, the code path is quite different depending on whether the lemma is inferred to be a mutually-defined lemma or not. We refactor the code path in declare to reflect that; this will allow to better organize constant information and to reuse the `Recthm.t` type in particular.
Diffstat (limited to 'vernac/comFixpoint.ml')
-rw-r--r--vernac/comFixpoint.ml4
1 files changed, 2 insertions, 2 deletions
diff --git a/vernac/comFixpoint.ml b/vernac/comFixpoint.ml
index 99db8df803..304df6fe93 100644
--- a/vernac/comFixpoint.ml
+++ b/vernac/comFixpoint.ml
@@ -271,8 +271,8 @@ let declare_fixpoint_interactive_generic ?indexes ~scope ~poly ((fixnames,_fixrs
let init_terms = Some fixdefs in
let evd = Evd.from_ctx ctx in
let lemma =
- Declare.Proof.start_with_initialization ~poly ~scope ~kind:(Decls.IsDefinition fix_kind) ~udecl
- evd (Some(cofix,indexes,init_terms)) thms None in
+ Declare.Proof.start_mutual_with_initialization ~poly ~scope ~kind:(Decls.IsDefinition fix_kind) ~udecl
+ evd ~mutual_info:(cofix,indexes,init_terms) thms None in
(* Declare notations *)
List.iter (Metasyntax.add_notation_interpretation (Global.env())) ntns;
lemma