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

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