aboutsummaryrefslogtreecommitdiff
path: root/src/Arithmetic/Saturated/Freeze.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/Arithmetic/Saturated/Freeze.v')
-rw-r--r--src/Arithmetic/Saturated/Freeze.v2
1 files changed, 2 insertions, 0 deletions
diff --git a/src/Arithmetic/Saturated/Freeze.v b/src/Arithmetic/Saturated/Freeze.v
index 65b8ee55d..b56a69a3d 100644
--- a/src/Arithmetic/Saturated/Freeze.v
+++ b/src/Arithmetic/Saturated/Freeze.v
@@ -7,6 +7,7 @@ Require Import Crypto.Arithmetic.Saturated.Core.
Require Import Crypto.Arithmetic.Saturated.Wrappers.
Require Import Crypto.Util.ZUtil.AddGetCarry.
Require Import Crypto.Util.ZUtil.Definitions.
+Require Import Crypto.Util.ZUtil.CPS.
Require Import Crypto.Util.Tactics.BreakMatch.
Require Import Crypto.Util.Decidable Crypto.Util.ZUtil.
Require Import Crypto.Util.Tuple Crypto.Util.LetIn.
@@ -101,6 +102,7 @@ Section Freeze.
pose proof Z.add_get_carry_full_mod.
pose proof Z.add_get_carry_full_div.
pose proof div_correct. pose proof modulo_correct.
+ pose proof @Z.add_get_carry_full_cps_correct.
autorewrite with uncps push_id push_basesystem_eval.
pose proof (weight_nonzero n).