aboutsummaryrefslogtreecommitdiff
path: root/interp
diff options
context:
space:
mode:
authorGaëtan Gilbert2018-10-26 18:25:34 +0200
committerGaëtan Gilbert2018-10-26 18:25:34 +0200
commitbe144dcaa1d1d8ff22e9e39f49fd247e813ac1f8 (patch)
tree075437b5eefd1b526acdf13d00b25fdec3765213 /interp
parent27266c1f79e565a6a19da4c79fc1ce83f748e31c (diff)
parentec80d04cfb4075922386dc8517577fd4819f1912 (diff)
Merge PR #8684: Remove a few circumvolutions around parameters of inductive entries
Diffstat (limited to 'interp')
-rw-r--r--interp/discharge.ml11
1 files changed, 1 insertions, 10 deletions
diff --git a/interp/discharge.ml b/interp/discharge.ml
index 0e44a8b467..21b2e85e8f 100644
--- a/interp/discharge.ml
+++ b/interp/discharge.ml
@@ -8,8 +8,6 @@
(* * (see LICENSE file for the text of the license) *)
(************************************************************************)
-open Names
-open CErrors
open Util
open Term
open Constr
@@ -17,17 +15,10 @@ open Vars
open Declarations
open Cooking
open Entries
-open Context.Rel.Declaration
(********************************)
(* Discharging mutual inductive *)
-let detype_param =
- function
- | LocalAssum (Name id, p) -> id, LocalAssumEntry p
- | LocalDef (Name id, p,_) -> id, LocalDefEntry p
- | _ -> anomaly (Pp.str "Unnamed inductive local variable.")
-
(* Replace
Var(y1)..Var(yq):C1..Cq |- Ij:Bj
@@ -57,7 +48,7 @@ let abstract_inductive decls nparamdecls inds =
(* To be sure to be the same as before, should probably be moved to process_inductive *)
let params' = let (_,arity,_,_,_) = List.hd inds' in
let (params,_) = decompose_prod_n_assum nparamdecls' arity in
- List.map detype_param params
+ params
in
let ind'' =
List.map