aboutsummaryrefslogtreecommitdiffstats
path: root/mppa_k1c/Asmaux.v
blob: 94b39f4e71e81544cfc53df5cc2dd842e3906c60 (plain)
1
2
3
4
5
Require Import Asm.
Require Import AST.

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