aboutsummaryrefslogtreecommitdiff
path: root/src/Assembly/HighLevel.v
blob: bae67f31298bb65fccfbd014c003e5bded5b0068 (plain)
1
2
3
4
5
6
7
8
9

Inductive Const32 : Set = | const32: word 32 -> Const32.

Inductive HL :=
  | Input: Const32 -> HL
  | Variable: Const32 -> HL
  | Let: forall m, nat -> HL -> HL -> HL
  | Lift1: (Const32 -> Const32) -> HL -> HL
  | Lift2: (Const32 -> Const32 -> Const32) -> HL -> HL -> HL.