From 7ea8a55692e2a2d32efa0c84e19c37a3b56a0fd1 Mon Sep 17 00:00:00 2001 From: xleroy Date: Fri, 19 Aug 2011 09:13:09 +0000 Subject: Cleaned up old commented-out parts git-svn-id: https://yquem.inria.fr/compcert/svn/compcert/trunk@1719 fca1b0fc-160b-0410-b1d3-a4f43f01ea2e --- common/Memdata.v | 8 -------- 1 file changed, 8 deletions(-) (limited to 'common/Memdata.v') diff --git a/common/Memdata.v b/common/Memdata.v index 16adb23..fde8b47 100644 --- a/common/Memdata.v +++ b/common/Memdata.v @@ -534,14 +534,6 @@ Definition decode_val (chunk: memory_chunk) (vl: list memval) : val := end end. -(* -Lemma inj_pointer_length: - forall b ofs n, List.length(inj_pointer n b ofs) = n. -Proof. - induction n; simpl; congruence. -Qed. -*) - Lemma encode_val_length: forall chunk v, length(encode_val chunk v) = size_chunk_nat chunk. Proof. -- cgit v1.2.3