aboutsummaryrefslogtreecommitdiff
path: root/src/Compilers/Z/Inline.v
blob: cbe6dbfde1ba540716e31e41bd23032ca599c1f9 (plain)
1
2
3
4
5
6
7
8
9
10
Require Import Crypto.Compilers.Syntax.
Require Import Crypto.Compilers.Inline.
Require Import Crypto.Compilers.Z.Syntax.
Require Import Crypto.Compilers.Z.Syntax.Util.

Definition InlineConstAndOpp {t} (e : Expr t) : Expr t
  := @InlineConst base_type op (is_const_or_opp) t e.

Definition InlineConst {t} (e : Expr t) : Expr t
  := @InlineConst base_type op (is_const) t e.