aboutsummaryrefslogtreecommitdiff
path: root/plugins/funind
diff options
context:
space:
mode:
authorEmilio Jesus Gallego Arias2020-05-25 16:30:20 +0200
committerEmilio Jesus Gallego Arias2020-06-26 14:38:11 +0200
commitb143d124e140628e5974da4af1b8a70a4d534598 (patch)
tree3e105d09b0c6490cb1b9d1fe185e4eab68ef957e /plugins/funind
parenta6d663c85d71b3cce007af23419e8030b8c5ac88 (diff)
[declare] Move udecl to Info structure.
Diffstat (limited to 'plugins/funind')
-rw-r--r--plugins/funind/functional_principles_proofs.ml2
-rw-r--r--plugins/funind/gen_principle.ml5
-rw-r--r--plugins/funind/recdef.ml7
3 files changed, 6 insertions, 8 deletions
diff --git a/plugins/funind/functional_principles_proofs.ml b/plugins/funind/functional_principles_proofs.ml
index 6ec12db952..2c85ae079f 100644
--- a/plugins/funind/functional_principles_proofs.ml
+++ b/plugins/funind/functional_principles_proofs.ml
@@ -856,7 +856,7 @@ let generate_equation_lemma evd fnames f fun_num nb_params nb_args rec_args_num
let info = Declare.Info.make () in
let lemma =
Declare.start_proof ~name:(mk_equation_id f_id) ~poly:false ~info
- ~impargs:[] ~udecl:UState.default_univ_decl evd lemma_type
+ ~impargs:[] evd lemma_type
in
let lemma, _ = Declare.by (Proofview.V82.tactic prove_replacement) lemma in
let () =
diff --git a/plugins/funind/gen_principle.ml b/plugins/funind/gen_principle.ml
index 8a07c2109e..a914cef6e4 100644
--- a/plugins/funind/gen_principle.ml
+++ b/plugins/funind/gen_principle.ml
@@ -1520,8 +1520,8 @@ let derive_correctness (funs : Constr.pconstant list) (graphs : inductive list)
let typ, _ = lemmas_types_infos.(i) in
let info = Declare.Info.make () in
let lemma =
- Declare.start_proof ~name:lem_id ~poly:false ~info ~impargs:[]
- ~udecl:UState.default_univ_decl !evd typ
+ Declare.start_proof ~name:lem_id ~poly:false ~info ~impargs:[] !evd
+ typ
in
let lemma =
fst @@ Declare.by (Proofview.V82.tactic (proving_tac i)) lemma
@@ -1587,7 +1587,6 @@ let derive_correctness (funs : Constr.pconstant list) (graphs : inductive list)
let info = Declare.Info.make () in
let lemma =
Declare.start_proof ~name:lem_id ~poly:false sigma ~info ~impargs:[]
- ~udecl:UState.default_univ_decl
(fst lemmas_types_infos.(i))
in
let lemma =
diff --git a/plugins/funind/recdef.ml b/plugins/funind/recdef.ml
index 853a54592d..9f36eada45 100644
--- a/plugins/funind/recdef.ml
+++ b/plugins/funind/recdef.ml
@@ -1494,8 +1494,8 @@ let open_new_goal ~lemma build_proof sigma using_lemmas ref_ goal_name
in
let info = Declare.Info.make ~hook:(Declare.Hook.make hook) () in
let lemma =
- Declare.start_proof ~name:na ~poly:false (* FIXME *) ~info ~impargs:[]
- ~udecl:UState.default_univ_decl sigma gls_type
+ Declare.start_proof ~name:na ~poly:false (* FIXME *) ~info ~impargs:[] sigma
+ gls_type
in
let lemma =
if Indfun_common.is_strict_tcc () then
@@ -1534,7 +1534,7 @@ let com_terminate interactive_proof tcc_lemma_name tcc_lemma_ref is_mes
let info = Declare.Info.make ~hook () in
let lemma =
Declare.start_proof ~name:thm_name ~poly:false (*FIXME*) ~info ctx
- ~impargs:[] ~udecl:UState.default_univ_decl
+ ~impargs:[]
(EConstr.of_constr (compute_terminate_type nb_args fonctional_ref))
in
let lemma =
@@ -1608,7 +1608,6 @@ let com_eqn uctx nb_arg eq_name functional_ref f_ref terminate_ref
let info = Declare.Info.make () in
let lemma =
Declare.start_proof ~name:eq_name ~poly:false evd ~info ~impargs:[]
- ~udecl:UState.default_univ_decl
(EConstr.of_constr equation_lemma_type)
in
let lemma =