aboutsummaryrefslogtreecommitdiffstats
path: root/backend/Asmaux.v
blob: 51e94f6b108593ec518419b95ea8534bd1d1e26e (plain)
1
2
3
4
5
Require Import Asm.
Require Import AST.

(* Constant only needed by Asmexpandaux.ml *)
Definition dummy_function := {| fn_code := nil; fn_sig := signature_main |}.