aboutsummaryrefslogtreecommitdiff
path: root/plugins
diff options
context:
space:
mode:
authorErik Martin-Dorel2019-03-01 16:06:14 +0100
committerErik Martin-Dorel2019-04-23 12:54:43 +0200
commit01b5e6e64b2af828b18fa6ee7037a7b7055f026e (patch)
tree6029fc25ce24811dd3314b7ea0127731ae3a081b /plugins
parentf294fe1684e03f63871864def0f82190da087ebe (diff)
[ssr] Remove the unify_helper tactic that appears unnecessary
It was only required in the (not realistic) test case "test_over_2_2", which happened to introduce evars after the context variables.
Diffstat (limited to 'plugins')
-rw-r--r--plugins/ssr/ssreflect.v23
1 files changed, 0 insertions, 23 deletions
diff --git a/plugins/ssr/ssreflect.v b/plugins/ssr/ssreflect.v
index c78381d3cc..e1e4d25ced 100644
--- a/plugins/ssr/ssreflect.v
+++ b/plugins/ssr/ssreflect.v
@@ -528,28 +528,6 @@ Parameter under_done :
forall (T : Type) (x : T), @Under T x x.
Notation "''Under[' x ]" := (@Under _ x _)
(at level 8, format "''Under[' x ]").
-
-Ltac beta_expand c e :=
- match e with
- | ?G ?z =>
- let T := type of z in
- match c with
- | context f [z] =>
- let b := constr:(fun x : T => ltac:(let r := context f [x] in refine r)) in
- rewrite -{1}[c]/(b z); beta_expand b G
- | (* constante *) _ =>
- let b := constr:(fun x : T => ltac:(exact c)) in
- rewrite -{1}[c]/(b z); beta_expand b G
- end
- | ?G => idtac
- end.
-
-Ltac unify_helper :=
- move=> *;
- lazymatch goal with
- | [ |- @Under _ ?c ?e ] =>
- beta_expand c e
- end.
End UNDER.
Module Export Under : UNDER.
@@ -575,7 +553,6 @@ Register Under_from_eq as plugins.ssreflect.Under_from_eq.
Ltac over :=
solve [ apply Under.under_done
| by rewrite over
- | unify_helper; eapply Under.under_done
].
(* The 2 variants below wouldn't work on [test-suite/ssr/over.v:test_over_2_1]