aboutsummaryrefslogtreecommitdiffstats
path: root/mppa_k1c/ExtValues.v
diff options
context:
space:
mode:
authorDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2019-05-11 07:59:11 +0200
committerDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2019-05-11 07:59:11 +0200
commitae22df3c5ef0a60527ea85b83bb71e8c95a6ab9c (patch)
treec9a29a001c7ca63d607c335a4b767b54736b8744 /mppa_k1c/ExtValues.v
parent428af5f71a063962e53e4ab58eaa372ccc926394 (diff)
downloadcompcert-kvx-ae22df3c5ef0a60527ea85b83bb71e8c95a6ab9c.tar.gz
compcert-kvx-ae22df3c5ef0a60527ea85b83bb71e8c95a6ab9c.zip
Pmsub compiled
Diffstat (limited to 'mppa_k1c/ExtValues.v')
-rw-r--r--mppa_k1c/ExtValues.v16
1 files changed, 16 insertions, 0 deletions
diff --git a/mppa_k1c/ExtValues.v b/mppa_k1c/ExtValues.v
index 1aa17458..0d56fd1c 100644
--- a/mppa_k1c/ExtValues.v
+++ b/mppa_k1c/ExtValues.v
@@ -131,3 +131,19 @@ Definition val_shrxl (v1 v2: val): val :=
else Vundef
| _, _ => Vundef
end.
+
+Lemma sub_add_neg :
+ forall x y, Val.sub x y = Val.add x (Val.neg y).
+Proof.
+ destruct x; destruct y; simpl; trivial.
+ f_equal.
+ apply Int.sub_add_opp.
+Qed.
+
+Lemma neg_mul_distr_r :
+ forall x y, Val.neg (Val.mul x y) = Val.mul x (Val.neg y).
+Proof.
+ destruct x; destruct y; simpl; trivial.
+ f_equal.
+ apply Int.neg_mul_distr_r.
+Qed. \ No newline at end of file