aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs/proof_type.mli
diff options
context:
space:
mode:
Diffstat (limited to 'proofs/proof_type.mli')
-rw-r--r--proofs/proof_type.mli22
1 files changed, 11 insertions, 11 deletions
diff --git a/proofs/proof_type.mli b/proofs/proof_type.mli
index 95ca33e90..37d5c4544 100644
--- a/proofs/proof_type.mli
+++ b/proofs/proof_type.mli
@@ -23,18 +23,18 @@ open Misctypes
is used by [Proof_tree] and [Refiner] *)
type prim_rule =
- | Intro of identifier
- | Cut of bool * bool * identifier * types
- | FixRule of identifier * int * (identifier * int * constr) list * int
- | Cofix of identifier * (identifier * constr) list * int
+ | Intro of Id.t
+ | Cut of bool * bool * Id.t * types
+ | FixRule of Id.t * int * (Id.t * int * constr) list * int
+ | Cofix of Id.t * (Id.t * constr) list * int
| Refine of constr
| Convert_concl of types * cast_kind
| Convert_hyp of named_declaration
- | Thin of identifier list
- | ThinBody of identifier list
- | Move of bool * identifier * identifier move_location
- | Order of identifier list
- | Rename of identifier * identifier
+ | Thin of Id.t list
+ | ThinBody of Id.t list
+ | Move of bool * Id.t * Id.t move_location
+ | Order of Id.t list
+ | Rename of Id.t * Id.t
| Change_evars
(** Nowadays, the only rules we'll consider are the primitive rules *)
@@ -76,9 +76,9 @@ type ltac_call_kind =
| LtacNotationCall of string
| LtacNameCall of ltac_constant
| LtacAtomCall of glob_atomic_tactic_expr
- | LtacVarCall of identifier * glob_tactic_expr
+ | LtacVarCall of Id.t * glob_tactic_expr
| LtacConstrInterp of glob_constr *
- (extended_patvar_map * (identifier * identifier option) list)
+ (extended_patvar_map * (Id.t * Id.t option) list)
type ltac_trace = (int * Loc.t * ltac_call_kind) list