aboutsummaryrefslogtreecommitdiff
path: root/vernac/comProgramFixpoint.ml
diff options
context:
space:
mode:
authorEnrico Tassi2020-10-13 15:32:54 +0200
committerEnrico Tassi2020-11-02 10:05:17 +0100
commit7de7fe612ffc5a598311f9542e57e50803ff2007 (patch)
tree282e882f6f9b8ebd99ee627d0c1c26a728148104 /vernac/comProgramFixpoint.ml
parentbd4d20106589562b12186ac2d02a665cf7b49dbe (diff)
[doc] attribute #[using]
Diffstat (limited to 'vernac/comProgramFixpoint.ml')
-rw-r--r--vernac/comProgramFixpoint.ml6
1 files changed, 4 insertions, 2 deletions
diff --git a/vernac/comProgramFixpoint.ml b/vernac/comProgramFixpoint.ml
index c2e07c4fd5..9623317ddf 100644
--- a/vernac/comProgramFixpoint.ml
+++ b/vernac/comProgramFixpoint.ml
@@ -262,7 +262,8 @@ let build_wellfounded pm (recname,pl,bl,arityc,body) poly ?using r measure notat
let using = using |> Option.map (fun expr ->
let terms = List.map EConstr.of_constr [evars_def; evars_typ] in
let l = Proof_using.process_expr env sigma expr terms in
- Names.Id.Set.(List.fold_right add l empty)) in
+ Names.Id.Set.(List.fold_right add l empty))
+ in
let uctx = Evd.evar_universe_context sigma in
let cinfo = Declare.CInfo.make ~name:recname ~typ:evars_typ ?using () in
let info = Declare.Info.make ~udecl ~poly ~hook () in
@@ -294,7 +295,8 @@ let do_program_recursive ~pm ~scope ~poly ?using fixkind fixl =
let using = using |> Option.map (fun expr ->
let terms = [def; typ] in
let l = Proof_using.process_expr env evd expr terms in
- Names.Id.Set.(List.fold_right add l empty)) in
+ Names.Id.Set.(List.fold_right add l empty))
+ in
let def = nf_evar evd (Termops.it_mkNamedLambda_or_LetIn def rec_sign) in
let typ = nf_evar evd (Termops.it_mkNamedProd_or_LetIn typ rec_sign) in
let evm = collect_evars_of_term evd def typ in