aboutsummaryrefslogtreecommitdiffstats
path: root/backend/RTLtyping.v
diff options
context:
space:
mode:
authorxleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2009-03-26 09:50:18 +0000
committerxleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2009-03-26 09:50:18 +0000
commit00b605a1d52696b055dd232a05dd54a312680b93 (patch)
tree7ebbd57e1d7c60e8b52e07526617c1aa30f3740f /backend/RTLtyping.v
parentc90abe06d110eb9c39b941792d896c741dc851dd (diff)
downloadcompcert-kvx-00b605a1d52696b055dd232a05dd54a312680b93.tar.gz
compcert-kvx-00b605a1d52696b055dd232a05dd54a312680b93.zip
Added tail call optimization pass
git-svn-id: https://yquem.inria.fr/compcert/svn/compcert/trunk@1015 fca1b0fc-160b-0410-b1d3-a4f43f01ea2e
Diffstat (limited to 'backend/RTLtyping.v')
-rw-r--r--backend/RTLtyping.v6
1 files changed, 0 insertions, 6 deletions
diff --git a/backend/RTLtyping.v b/backend/RTLtyping.v
index 60b1d72c..f466a90c 100644
--- a/backend/RTLtyping.v
+++ b/backend/RTLtyping.v
@@ -167,12 +167,6 @@ Section TYPECHECKING.
Variable funct: function.
Variable env: regenv.
-Lemma typ_eq: forall (t1 t2: typ), {t1=t2} + {t1<>t2}.
-Proof. decide equality. Qed.
-
-Lemma opt_typ_eq: forall (t1 t2: option typ), {t1=t2} + {t1<>t2}.
-Proof. decide equality. apply typ_eq. Qed.
-
Definition check_reg (r: reg) (ty: typ): bool :=
if typ_eq (env r) ty then true else false.