aboutsummaryrefslogtreecommitdiffstats
path: root/powerpc/Asm.v
diff options
context:
space:
mode:
authorBernhard Schommer <bernhardschommer@gmail.com>2015-06-22 23:49:11 +0200
committerBernhard Schommer <bernhardschommer@gmail.com>2015-06-22 23:49:11 +0200
commitff62587774f6ca437c887cc3ff5d079895c5e214 (patch)
tree475cdf441bc9486aff6e9535f562ae0864e0cdbd /powerpc/Asm.v
parent0e9ededa8c1d194453f5113bf57c93d0803f03b1 (diff)
downloadcompcert-kvx-ff62587774f6ca437c887cc3ff5d079895c5e214.tar.gz
compcert-kvx-ff62587774f6ca437c887cc3ff5d079895c5e214.zip
Changed a minor typo: Pstwxu should be Pstwux
Diffstat (limited to 'powerpc/Asm.v')
-rw-r--r--powerpc/Asm.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/powerpc/Asm.v b/powerpc/Asm.v
index d707b2b5..3fa7af31 100644
--- a/powerpc/Asm.v
+++ b/powerpc/Asm.v
@@ -260,7 +260,7 @@ Inductive instruction : Type :=
| Pstw: ireg -> constant -> ireg -> instruction (**r store 32-bit int *)
| Pstwu: ireg -> constant -> ireg -> instruction (**r store 32-bit int with update *)
| Pstwx: ireg -> ireg -> ireg -> instruction (**r same, with 2 index regs *)
- | Pstwxu: ireg -> ireg -> ireg -> instruction (**r same, with 2 index regs and update *)
+ | Pstwux: ireg -> ireg -> ireg -> instruction (**r same, with 2 index regs and update *)
| Pstw_a: ireg -> constant -> ireg -> instruction (**r store 32-bit quantity from int reg *)
| Pstwx_a: ireg -> ireg -> ireg -> instruction (**r same, with 2 index regs *)
| Pstwbrx: ireg -> ireg -> ireg -> instruction (**r store 32-bit int with reverse endianness *)
@@ -878,7 +878,7 @@ Definition exec_instr (f: function) (i: instruction) (rs: regset) (m: mem) : out
| Pstfdu _ _ _
| Psthbrx _ _ _
| Pstwu _ _ _
- | Pstwxu _ _ _
+ | Pstwux _ _ _
| Psubfze _ _
| Psync
| Ptrap