diff options
| author | Gaëtan Gilbert | 2020-07-21 17:04:03 +0200 |
|---|---|---|
| committer | Gaëtan Gilbert | 2020-07-21 17:04:03 +0200 |
| commit | 56fd98a932f2700a63fe701bb71533fb48d6d06b (patch) | |
| tree | da2ef1194d21f47949dba6bf3a629334d53d40b3 | |
| parent | 8f4d7ddf4c3736a190b3e073fadb844c017628d3 (diff) | |
| parent | 708869a116102fb29baa9379c103999f2e8e2dc2 (diff) | |
Merge PR #12714: [declare] Remove some dead code in declare_mutual_definition
Reviewed-by: SkySkimmer
| -rw-r--r-- | vernac/declare.ml | 10 |
1 files changed, 2 insertions, 8 deletions
diff --git a/vernac/declare.ml b/vernac/declare.ml index 12a261517f..eedbee852b 100644 --- a/vernac/declare.ml +++ b/vernac/declare.ml @@ -1152,13 +1152,6 @@ let declare_mutual_definition ~pm l = Some (List.map3 compute_possible_guardness_evidences wfl fixdefs fixtypes) | IsCoFixpoint -> None in - (* In the future we will pack all this in a proper record *) - (* XXX: info refactoring *) - let _kind = - if fixkind != IsCoFixpoint then Decls.(IsDefinition Fixpoint) - else Decls.(IsDefinition CoFixpoint) - in - let scope = first.prg_info.Info.scope in (* Declare the recursive definitions *) let kns = declare_mutually_recursive_core ~info:first.prg_info ~ntns:first.prg_notations @@ -1167,6 +1160,7 @@ let declare_mutual_definition ~pm l = in (* Only for the first constant *) let dref = List.hd kns in + let scope = first.prg_info.Info.scope in let s_hook = {Hook.S.uctx = first.prg_uctx; obls; scope; dref} in Hook.call ?hook:first.prg_info.Info.hook s_hook; (* XXX: We call the obligation hook here, by consistency with the @@ -1503,7 +1497,7 @@ let start_mutual_with_initialization ~info ~cinfo ~mutual_info sigma snl = in match cinfo with | [] -> CErrors.anomaly (Pp.str "No proof to start.") - | { CInfo.name; typ; impargs; _} :: thms -> + | { CInfo.name; typ; _} :: thms -> let pinfo = Proof_info.make ~cinfo ~info ~compute_guard () in (* start_lemma has the responsibility to add (name, impargs, typ) to thms, once Info.t is more refined this won't be necessary *) |
