aboutsummaryrefslogtreecommitdiff
path: root/plugins
diff options
context:
space:
mode:
authorJason Gross2018-12-03 18:10:03 -0500
committerJason Gross2019-01-24 14:29:03 -0500
commita10076e834720c05e55397c9e26b9d7a8786298b (patch)
tree8c29f94b44247d50f16dfa9ee8469c5da362b748 /plugins
parent4e66d30ba33310dfc96f7f1e57c651db9fc53c97 (diff)
Move cleanup from the test-suite to Z.div_mod_to_quot_rem_cleanup
Also fold it into `Z.div_mod_to_quot_rem` Note that the test-suite file is a bit slow. On my machine, it is ``` real 2m32.983s user 2m32.544s sys 0m0.492s ```
Diffstat (limited to 'plugins')
-rw-r--r--plugins/omega/PreOmega.v14
1 files changed, 12 insertions, 2 deletions
diff --git a/plugins/omega/PreOmega.v b/plugins/omega/PreOmega.v
index 08bfec84bc..7ebc2fb04f 100644
--- a/plugins/omega/PreOmega.v
+++ b/plugins/omega/PreOmega.v
@@ -16,7 +16,8 @@ Local Open Scope Z_scope.
(** This tactic uses the complete specification of [Z.div] and
[Z.modulo] to remove these functions from the goal without losing
- information. *)
+ information. The [Z.div_mod_to_quot_rem_cleanup] tactic removes
+ needless hypotheses, which makes tactics like [nia] run faster. *)
Module Z.
Lemma mod_0_r_ext x y : y = 0 -> x mod y = 0.
@@ -42,7 +43,16 @@ Module Z.
| [ H : context[?x / ?y] |- _ ] => div_mod_to_quot_rem_generalize x y
| [ H : context[?x mod ?y] |- _ ] => div_mod_to_quot_rem_generalize x y
end.
- Ltac div_mod_to_quot_rem := repeat div_mod_to_quot_rem_step.
+ Ltac div_mod_to_quot_rem' := repeat div_mod_to_quot_rem_step.
+ Ltac div_mod_to_quot_rem_cleanup :=
+ repeat match goal with
+ | [ H : ?T -> _, H' : ?T |- _ ] => specialize (H H')
+ | [ H : ?T -> _, H' : ~?T |- _ ] => clear H
+ | [ H : ~?T -> _, H' : ?T |- _ ] => clear H
+ | [ H : 0 < ?x -> _, H' : ?x < 0 |- _ ] => clear H
+ | [ H : ?x < 0 -> _, H' : 0 < ?x |- _ ] => clear H
+ end.
+ Ltac div_mod_to_quot_rem := div_mod_to_quot_rem'; div_mod_to_quot_rem_cleanup.
End Z.
(** * zify: the Z-ification tactic *)