aboutsummaryrefslogtreecommitdiffstats
path: root/backend/Asmaux.v
blob: 1167c34c482c406067ed65b2067002680cb741c7 (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
(* *************************************************************)
(*                                                             *)
(*             The Compcert verified compiler                  *)
(*                                                             *)
(*           Sylvain Boulmé     Grenoble-INP, VERIMAG          *)
(*           David Monniaux     CNRS, VERIMAG                  *)
(*           Cyril Six          Kalray                         *)
(*                                                             *)
(*  Copyright Kalray. Copyright VERIMAG. All rights reserved.  *)
(*  This file is distributed under the terms of the INRIA      *)
(*  Non-Commercial License Agreement.                          *)
(*                                                             *)
(* *************************************************************)

Require Import Asm.
Require Import AST.

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