aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/ftactic.mli
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2015-10-20 14:45:31 +0200
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2015-10-20 16:05:46 +0200
commit4cc1714ac9b0944b6203c23af8c46145e7239ad3 (patch)
tree5793c3cc93b435c86373855b9bb782f70ae052a6 /tactics/ftactic.mli
parentcc42541eeaaec0371940e07efdb009a4ee74e468 (diff)
Indexing Proofview.goals with a stage.
This is not perfect though, some primitives are unsound, and some higher-order API should use polymorphic functions so as not to depend on a given level.
Diffstat (limited to 'tactics/ftactic.mli')
-rw-r--r--tactics/ftactic.mli6
1 files changed, 4 insertions, 2 deletions
diff --git a/tactics/ftactic.mli b/tactics/ftactic.mli
index 483515674..449649922 100644
--- a/tactics/ftactic.mli
+++ b/tactics/ftactic.mli
@@ -37,12 +37,14 @@ val run : 'a t -> ('a -> unit Proofview.tactic) -> unit Proofview.tactic
(** {5 Focussing} *)
-val nf_enter : ([ `NF ] Proofview.Goal.t -> 'a t) -> 'a t
+val nf_enter : (([ `NF ], 'r) Proofview.Goal.t -> 'a t) -> 'a t
(** Enter a goal. The resulting tactic is focussed. *)
+(** FIXME: Should be polymorphic over the stage. *)
-val enter : ([ `LZ ] Proofview.Goal.t -> 'a t) -> 'a t
+val enter : (([ `LZ ], 'r) Proofview.Goal.t -> 'a t) -> 'a t
(** Enter a goal, without evar normalization. The resulting tactic is
focussed. *)
+(** FIXME: Should be polymorphic over the stage. *)
val with_env : 'a t -> (Environ.env*'a) t
(** [with_env t] returns, in addition to the return type of [t], an