aboutsummaryrefslogtreecommitdiffstats
path: root/mppa_k1c/Asm.v
diff options
context:
space:
mode:
authorDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2019-04-02 09:03:25 +0200
committerDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2019-04-02 09:03:25 +0200
commit8fb2d1a49443767ce353520ea045383430a2655e (patch)
treefc3f737acca869af517f213214f19f8bc78d50d3 /mppa_k1c/Asm.v
parentff67146a6e1c7ee9c202b5e770706415f45a674d (diff)
parent629252b160fd4b909231bcad6edcf6f254aca0d6 (diff)
downloadcompcert-kvx-8fb2d1a49443767ce353520ea045383430a2655e.tar.gz
compcert-kvx-8fb2d1a49443767ce353520ea045383430a2655e.zip
Merge branch 'mppa-ternary' of gricad-gitlab.univ-grenoble-alpes.fr:sixcy/CompCert into mppa-ternary
Diffstat (limited to 'mppa_k1c/Asm.v')
-rw-r--r--mppa_k1c/Asm.v6
1 files changed, 3 insertions, 3 deletions
diff --git a/mppa_k1c/Asm.v b/mppa_k1c/Asm.v
index 1e022218..245804f3 100644
--- a/mppa_k1c/Asm.v
+++ b/mppa_k1c/Asm.v
@@ -30,7 +30,7 @@ Require Import Smallstep.
Require Import Locations.
Require Stacklayout.
Require Import Conventions.
-Require Import Asmblock.
+Require Import Asmvliw.
Require Import Linking.
Require Import Errors.
@@ -477,7 +477,7 @@ Definition program_proj (p: program) : Asmblock.program :=
End RELSEM.
-Definition semantics (p: program) := Asmblock.semantics (program_proj p).
+Definition semantics (p: program) := Asmvliw.semantics (program_proj p).
(** Determinacy of the [Asm] semantics. *)
@@ -608,7 +608,7 @@ Proof (Genv.senv_match TRANSF).
Theorem transf_program_correct:
- forward_simulation (Asmblock.semantics prog) (semantics tprog).
+ forward_simulation (Asmvliw.semantics prog) (semantics tprog).
Proof.
pose proof (match_program_transf prog tprog TRANSF) as TR.
subst. unfold semantics. rewrite transf_program_proj.