Skip to content

Commit 777f0ac

Browse files
committed
Removing dead code.
1 parent db293d1 commit 777f0ac

Some content is hidden

Large Commits have some content hidden by default. Use the searchbox below for content that may be hidden.

73 files changed

+3
-164
lines changed

dev/top_printers.ml

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -22,7 +22,6 @@ open Evd
2222
open Goptions
2323
open Genarg
2424
open Clenv
25-
open Universes
2625

2726
let _ = Detyping.print_evar_arguments := true
2827
let _ = Detyping.print_universes := true

intf/tacexpr.mli

Lines changed: 0 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -10,12 +10,10 @@ open Loc
1010
open Names
1111
open Constrexpr
1212
open Libnames
13-
open Globnames
1413
open Nametab
1514
open Genredexpr
1615
open Genarg
1716
open Pattern
18-
open Decl_kinds
1917
open Misctypes
2018
open Locus
2119

kernel/cbytegen.mli

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1,4 +1,3 @@
1-
open Names
21
open Cbytecodes
32
open Cemitcodes
43
open Term

kernel/cemitcodes.ml

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -10,7 +10,6 @@
1010
machine, Oct 2004 *)
1111
(* Extension: Arnaud Spiwack (support for native arithmetic), May 2005 *)
1212

13-
open Names
1413
open Term
1514
open Cbytecodes
1615
open Copcodes

kernel/closure.ml

Lines changed: 0 additions & 18 deletions
Original file line numberDiff line numberDiff line change
@@ -771,24 +771,6 @@ let drop_parameters depth n argstk =
771771
(* we know that n < stack_args_size(argstk) (if well-typed term) *)
772772
anomaly (Pp.str "ill-typed term: found a match on a partially applied constructor")
773773

774-
775-
let rec get_parameters depth n argstk =
776-
match argstk with
777-
Zapp args::s ->
778-
let q = Array.length args in
779-
if n > q then Array.append args (get_parameters depth (n-q) s)
780-
else if Int.equal n q then [||]
781-
else Array.sub args 0 n
782-
| Zshift(k)::s ->
783-
get_parameters (depth-k) n s
784-
| [] -> (* we know that n < stack_args_size(argstk) (if well-typed term) *)
785-
if Int.equal n 0 then [||]
786-
else raise Not_found (* Trying to eta-expand a partial application..., should do
787-
eta expansion first? *)
788-
| _ -> assert false
789-
(* strip_update_shift_app only produces Zapp and Zshift items *)
790-
791-
792774
(** [eta_expand_ind_stack env ind c s t] computes stacks correspoding
793775
to the conversion of the eta expansion of t, considered as an inhabitant
794776
of ind, and the Constructor c of this inductive type applied to arguments

kernel/declareops.mli

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -9,7 +9,6 @@
99
open Declarations
1010
open Mod_subst
1111
open Univ
12-
open Context
1312

1413
(** Operations concerning types in [Declarations] :
1514
[constant_body], [mutual_inductive_body], [module_body] ... *)

kernel/fast_typeops.mli

Lines changed: 0 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -6,13 +6,8 @@
66
(* * GNU Lesser General Public License Version 2.1 *)
77
(************************************************************************)
88

9-
open Names
10-
open Univ
119
open Term
12-
open Context
1310
open Environ
14-
open Entries
15-
open Declarations
1611

1712
(** {6 Typing functions (not yet tagged as safe) }
1813

kernel/indtypes.ml

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -654,7 +654,6 @@ let used_section_variables env inds =
654654
keep_hyps env ids
655655

656656
let rel_vect n m = Array.init m (fun i -> mkRel(n+m-i))
657-
let rel_appvect n m = rel_vect n (List.length m)
658657

659658
exception UndefinableExpansion
660659

kernel/inductive.ml

Lines changed: 0 additions & 7 deletions
Original file line numberDiff line numberDiff line change
@@ -447,13 +447,6 @@ type subterm_spec =
447447

448448
let eq_wf_paths = Rtree.equal Declareops.eq_recarg
449449

450-
let pp_recarg = function
451-
| Norec -> Pp.str "Norec"
452-
| Mrec i -> Pp.str ("Mrec "^MutInd.to_string (fst i))
453-
| Imbr i -> Pp.str ("Imbr "^MutInd.to_string (fst i))
454-
455-
let pp_wf_paths = Rtree.pp_tree pp_recarg
456-
457450
let inter_recarg r1 r2 = match r1, r2 with
458451
| Norec, Norec -> Some r1
459452
| Mrec i1, Mrec i2

kernel/names.ml

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -571,7 +571,6 @@ let constr_modpath (ind,_) = ind_modpath ind
571571

572572
let ith_mutual_inductive (mind, _) i = (mind, i)
573573
let ith_constructor_of_inductive ind i = (ind, i)
574-
let ith_constructor_of_pinductive (ind,u) i = ((ind,i),u)
575574
let inductive_of_constructor (ind, i) = ind
576575
let index_of_constructor (ind, i) = i
577576

0 commit comments

Comments
 (0)