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.mli7
1 files changed, 2 insertions, 5 deletions
diff --git a/proofs/proof_type.mli b/proofs/proof_type.mli
index 4f7e87ea9..d6081e56c 100644
--- a/proofs/proof_type.mli
+++ b/proofs/proof_type.mli
@@ -79,11 +79,10 @@ type proof_tree = {
and rule =
| Prim of prim_rule
- | Nested of compound_rule * proof_tree
| Decl_proof of bool
| Daimon
-and compound_rule=
+type compound_rule=
(** the boolean of Tactic tells if the default tactic is used *)
| Tactic of tactic_expr * bool
@@ -123,7 +122,7 @@ and tactic_arg =
type ltac_call_kind =
| LtacNotationCall of string
| LtacNameCall of ltac_constant
- | LtacAtomCall of glob_atomic_tactic_expr * atomic_tactic_expr option ref
+ | LtacAtomCall of glob_atomic_tactic_expr
| LtacVarCall of identifier * glob_tactic_expr
| LtacConstrInterp of glob_constr *
(extended_patvar_map * (identifier * identifier option) list)
@@ -131,5 +130,3 @@ type ltac_call_kind =
type ltac_trace = (int * Loc.t * ltac_call_kind) list
exception LtacLocated of (int * ltac_call_kind * ltac_trace * Loc.t) * exn
-
-val abstract_tactic_box : atomic_tactic_expr option ref ref