aboutsummaryrefslogtreecommitdiffstats
path: root/src/translation/HTLgen.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/translation/HTLgen.v')
-rw-r--r--src/translation/HTLgen.v5
1 files changed, 5 insertions, 0 deletions
diff --git a/src/translation/HTLgen.v b/src/translation/HTLgen.v
index 705f9ad..9c2e168 100644
--- a/src/translation/HTLgen.v
+++ b/src/translation/HTLgen.v
@@ -179,6 +179,11 @@ Definition transf_function (f: function) : Errors.res module :=
| Error err => Errors.Error err
end.
+Definition example : mon HTL.code := PTree.traverse transf_instr
+ (PTree.set 2%positive (RTL.Icall sig ros args res n) (PTree.set 1%positive (RTL.Iop (Op.Omove) nil 1%positive 2%positive) (PTree.empty RTL.instruction))).
+
+Compute example.
+
Definition transf_fundef (fd: fundef) : Errors.res moddecl :=
transf_partial_fundef transf_function fd.