aboutsummaryrefslogtreecommitdiff
path: root/src/Util/SideConditions/Autosolve.v
diff options
context:
space:
mode:
authorGravatar Jason Gross <jgross@mit.edu>2017-11-17 20:08:29 -0500
committerGravatar Jason Gross <jgross@mit.edu>2017-11-17 20:08:29 -0500
commit3d2e80e1c91fd06197236405740e6b115b4addc4 (patch)
treed1e5a64ee15d7149b60e5e7f3cb13e46ffdd154b /src/Util/SideConditions/Autosolve.v
parent0d68c007fe0ea485cc2296d52579c83bcea58a05 (diff)
Add support for custom intro tactic in ring pkg, for speed
Diffstat (limited to 'src/Util/SideConditions/Autosolve.v')
-rw-r--r--src/Util/SideConditions/Autosolve.v10
1 files changed, 6 insertions, 4 deletions
diff --git a/src/Util/SideConditions/Autosolve.v b/src/Util/SideConditions/Autosolve.v
index 9f8eb61de..840d3a592 100644
--- a/src/Util/SideConditions/Autosolve.v
+++ b/src/Util/SideConditions/Autosolve.v
@@ -5,15 +5,17 @@ Require Import Crypto.Util.SideConditions.ModInvPackage.
Require Import Crypto.Util.SideConditions.ReductionPackages.
Require Import Crypto.Util.SideConditions.RingPackage.
-Ltac autosolve_gen autosolve_tac else_tac :=
+Ltac autosolve_gen autosolve_tac ring_intros_tac else_tac :=
CorePackages.preautosolve ();
CorePackages.Internal.autosolve ltac:(fun _ =>
AdmitPackage.autosolve ltac:(fun _ =>
ModInvPackage.autosolve ltac:(fun _ =>
ReductionPackages.autosolve autosolve_tac ltac:(fun _ =>
- RingPackage.autosolve ltac:(fun _ =>
+ RingPackage.autosolve_gen_intros ring_intros_tac ltac:(fun _ =>
CorePackages.autosolve else_tac
))))).
-Ltac autosolve else_tac :=
- autosolve_gen autosolve else_tac.
+Ltac autosolve_gen_intros ring_intros_tac else_tac :=
+ autosolve_gen ltac:(autosolve_gen_intros ring_intros_tac) ring_intros_tac else_tac.
+
+Ltac autosolve else_tac := autosolve_gen_intros default_ring_intros_tac else_tac.