aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/hiddentac.ml
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-04-14 08:23:46 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-04-14 08:23:46 +0000
commit2d0513787170553e2d887c5571b2de02e790a219 (patch)
tree0a02f8a491761b8e3fcb118c6112a0108795a5e5 /tactics/hiddentac.ml
parenta5ff2b91cd406e7acdeef18d1b1ee14a331ffdaa (diff)
Removing redundant internal variants of apply tactic and simplification of ML names
(late consequences of commit r12603) git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12934 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'tactics/hiddentac.ml')
-rw-r--r--tactics/hiddentac.ml8
1 files changed, 4 insertions, 4 deletions
diff --git a/tactics/hiddentac.ml b/tactics/hiddentac.ml
index 756212f0a..4fed5d27c 100644
--- a/tactics/hiddentac.ml
+++ b/tactics/hiddentac.ml
@@ -32,7 +32,7 @@ let h_vm_cast_no_check c =
abstract_tactic (TacVmCastNoCheck c) (vm_cast_no_check c)
let h_apply simple ev cb =
abstract_tactic (TacApply (simple,ev,List.map snd cb,None))
- (apply_with_ebindings_gen simple ev cb)
+ (apply_with_bindings_gen simple ev cb)
let h_apply_in simple ev cb (id,ipat as inhyp) =
abstract_tactic (TacApply (simple,ev,List.map snd cb,Some inhyp))
(apply_in simple ev id cb ipat)
@@ -94,9 +94,9 @@ let h_rename l =
let h_revert l = abstract_tactic (TacRevert l) (revert l)
(* Constructors *)
-let h_left ev l = abstract_tactic (TacLeft (ev,l)) (left_with_ebindings ev l)
-let h_right ev l = abstract_tactic (TacRight (ev,l)) (right_with_ebindings ev l)
-let h_split ev l = abstract_tactic (TacSplit (ev,false,l)) (split_with_ebindings ev l)
+let h_left ev l = abstract_tactic (TacLeft (ev,l)) (left_with_bindings ev l)
+let h_right ev l = abstract_tactic (TacRight (ev,l)) (right_with_bindings ev l)
+let h_split ev l = abstract_tactic (TacSplit (ev,false,l)) (split_with_bindings ev l)
(* Moved to tacinterp because of dependencies in Tacinterp.interp
let h_any_constructor t =
abstract_tactic (TacAnyConstructor t) (any_constructor t)