aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/ftactic.ml
diff options
context:
space:
mode:
Diffstat (limited to 'tactics/ftactic.ml')
-rw-r--r--tactics/ftactic.ml10
1 files changed, 5 insertions, 5 deletions
diff --git a/tactics/ftactic.ml b/tactics/ftactic.ml
index fcc385c4e..bbc739a3b 100644
--- a/tactics/ftactic.ml
+++ b/tactics/ftactic.ml
@@ -29,7 +29,7 @@ let bind (type a) (type b) (m : a t) (f : a -> b t) : b t = m >>= function
| Uniform x ->
(** We dispatch the uniform result on each goal under focus, as we know
that the [m] argument was actually dependent. *)
- Proofview.Goal.raw_goals >>= fun l ->
+ Proofview.Goal.goals >>= fun l ->
let ans = List.map (fun _ -> x) l in
Proofview.tclUNIT ans
| Depends l -> Proofview.tclUNIT l
@@ -37,12 +37,12 @@ let bind (type a) (type b) (m : a t) (f : a -> b t) : b t = m >>= function
Proofview.tclDISPATCHL (List.map f l) >>= fun l ->
Proofview.tclUNIT (Depends (List.concat l))
-let enter f =
- bind (Proofview.Goal.goals >>= fun l -> Proofview.tclUNIT (Depends l))
+let nf_enter f =
+ bind (Proofview.Goal.nf_goals >>= fun l -> Proofview.tclUNIT (Depends l))
(fun gl -> Proofview.V82.wrap_exceptions (fun () -> f gl))
-let raw_enter f =
- bind (Proofview.Goal.raw_goals >>= fun l -> Proofview.tclUNIT (Depends l))
+let enter f =
+ bind (Proofview.Goal.goals >>= fun l -> Proofview.tclUNIT (Depends l))
(fun gl -> Proofview.V82.wrap_exceptions (fun () -> f gl))
let lift (type a) (t:a Proofview.tactic) : a t =