aboutsummaryrefslogtreecommitdiff
path: root/src/RewriterRules.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/RewriterRules.v')
-rw-r--r--src/RewriterRules.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/src/RewriterRules.v b/src/RewriterRules.v
index 097497d9a..8f23c1793 100644
--- a/src/RewriterRules.v
+++ b/src/RewriterRules.v
@@ -481,7 +481,7 @@ Definition arith_with_casts_rewrite_rulesT : list (bool * Prop)
].
Definition strip_literal_casts_rewrite_rulesT : list (bool * Prop)
- := [dont_do_again (forall rx x, x ∈ rx -> cstZ rx ('x) = 'x)]%Z%zrange.
+ := generalize_cast [dont_do_again (forall rx x, x ∈ rx -> cstZ rx ('x) = 'x)]%Z%zrange.
Section fancy.
Context (invert_low invert_high : Z (*log2wordmax*) -> Z -> option Z)