aboutsummaryrefslogtreecommitdiff
path: root/src/Util/ZUtil/AddGetCarry.v
diff options
context:
space:
mode:
authorGravatar Jason Gross <jgross@mit.edu>2017-10-19 13:57:48 -0400
committerGravatar Jason Gross <jgross@mit.edu>2017-10-19 13:57:48 -0400
commit9d16ae4ecb6f24ae7eefabd056902b00bf2fe001 (patch)
tree0ad36b87d1d6670ff7d0c5e57d818104bcdf911f /src/Util/ZUtil/AddGetCarry.v
parentb0d6dfe21d669be0b12a76d37c9bd78c20f788f9 (diff)
Update ZUtil cps definitions
This will hopefully allow the compiler to reflective-land an easier job.
Diffstat (limited to 'src/Util/ZUtil/AddGetCarry.v')
-rw-r--r--src/Util/ZUtil/AddGetCarry.v4
1 files changed, 3 insertions, 1 deletions
diff --git a/src/Util/ZUtil/AddGetCarry.v b/src/Util/ZUtil/AddGetCarry.v
index e8897431a..85e9ece74 100644
--- a/src/Util/ZUtil/AddGetCarry.v
+++ b/src/Util/ZUtil/AddGetCarry.v
@@ -5,8 +5,10 @@ Require Import Crypto.Util.ZUtil.Hints.ZArith.
Require Import Crypto.Util.Prod.
Require Import Crypto.Util.ZUtil.Tactics.PullPush.Modulo.
Require Import Crypto.Util.ZUtil.Tactics.DivModToQuotRem.
+Require Import Crypto.Util.ZUtil.Tactics.LtbToLt.
Require Import Crypto.Util.LetIn.
Require Import Crypto.Util.Tactics.BreakMatch.
+Require Import Crypto.Util.Tactics.RewriteHyp.
Local Open Scope Z_scope.
Local Notation eta x := (fst x, snd x).
@@ -55,7 +57,7 @@ Module Z.
Local Ltac easypeasy :=
repeat progress autounfold;
- break_match; autorewrite with cancel_pair zsimplify;
+ break_match; Z.ltb_to_lt; rewrite_hyp ?*; autorewrite with cancel_pair zsimplify;
solve [repeat (f_equal; try ring)].
Local Hint Unfold Z.get_carry Z.get_borrow