From 65f30c5524280b5639a94674828986f0635b2477 Mon Sep 17 00:00:00 2001 From: Yann Herklotz Date: Sun, 29 Mar 2020 16:41:09 +0100 Subject: Remove unnecessary examples from HTL --- src/translation/HTLgen.v | 7 +------ 1 file changed, 1 insertion(+), 6 deletions(-) (limited to 'src/translation/HTLgen.v') diff --git a/src/translation/HTLgen.v b/src/translation/HTLgen.v index 9c2e168..d7f88c1 100644 --- a/src/translation/HTLgen.v +++ b/src/translation/HTLgen.v @@ -17,8 +17,8 @@ *) From coqup Require Import HTL Coquplib. -From compcert Require Import Maps. +From compcert Require Import Maps. From compcert Require Errors. From compcert Require Import AST RTL. @@ -179,11 +179,6 @@ 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. -- cgit