aboutsummaryrefslogtreecommitdiffstats
path: root/aarch64/Asmgen.v
blob: f81f37d678df2ccff212474bb05b8de99104cd5f (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
22
23
24
25
26
27
28
29
30
31
32
33
(* *************************************************************)
(*                                                             *)
(*             The Compcert verified compiler                  *)
(*                                                             *)
(*           Sylvain Boulmé     Grenoble-INP, VERIMAG          *)
(*           Justus Fasse       UGA, VERIMAG                   *)
(*           Xavier Leroy       INRIA Paris-Rocquencourt       *)
(*           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 Recdef Coqlib Zwf Zbits.
Require Import Errors AST Integers Floats Op.
Require Import Locations Asmblock Asm.

(** * Translation from Asmblock to assembly language 
      Inspired from the KVX backend. *)

(* STUB *)

Definition transf_function (f: Asmblock.function) : res Asm.function :=
  Error (msg "Asmgen not yet implmented").

Definition transf_fundef (f: Asmblock.fundef) : res Asm.fundef :=
  transf_partial_fundef transf_function f.

Definition transf_program (p: Asmblock.program) : res Asm.program :=
  transform_partial_program transf_fundef p.