aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/tacsubst.ml
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-05-21 17:08:04 +0200
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-05-21 17:38:48 +0200
commit741747c4ecb2be5f51bf5e0395f9fcb28329e86b (patch)
tree1c9595161bca3a6f2bf5f2503bb03b33b31c49f5 /tactics/tacsubst.ml
parentbf18afeefa06e972c6cb98fa8a81ec7172fdde7f (diff)
Moving left & right tactics out of the AST.
Diffstat (limited to 'tactics/tacsubst.ml')
-rw-r--r--tactics/tacsubst.ml2
1 files changed, 0 insertions, 2 deletions
diff --git a/tactics/tacsubst.ml b/tactics/tacsubst.ml
index 1b15fa8e1..bea77a0b0 100644
--- a/tactics/tacsubst.ml
+++ b/tactics/tacsubst.ml
@@ -181,8 +181,6 @@ let rec subst_atomic subst (t:glob_atomic_tactic_expr) = match t with
| TacRevert _ as x -> x
(* Constructors *)
- | TacLeft (ev,bl) -> TacLeft (ev,subst_bindings subst bl)
- | TacRight (ev,bl) -> TacRight (ev,subst_bindings subst bl)
| TacSplit (ev,b,bll) -> TacSplit (ev,b,List.map (subst_bindings subst) bll)
| TacAnyConstructor (ev,t) -> TacAnyConstructor (ev,Option.map (subst_tactic subst) t)
| TacConstructor (ev,n,bl) -> TacConstructor (ev,n,subst_bindings subst bl)