aboutsummaryrefslogtreecommitdiffstats
path: root/mppa_k1c/Asmaux.v
blob: 891d10683489f4eb4ce07ed0cbbf94028df53765 (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 |}.