summaryrefslogtreecommitdiff
path: root/common/Memdata.v
diff options
context:
space:
mode:
authorGravatar xleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2011-08-19 09:13:09 +0000
committerGravatar xleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2011-08-19 09:13:09 +0000
commit7ea8a55692e2a2d32efa0c84e19c37a3b56a0fd1 (patch)
treee324aff1a958e0a5d83f805ff3ca1d9eb07939f4 /common/Memdata.v
parent5b73a4f223a0cadb7df3f1320fed86cde0d67d6e (diff)
Cleaned up old commented-out parts
git-svn-id: https://yquem.inria.fr/compcert/svn/compcert/trunk@1719 fca1b0fc-160b-0410-b1d3-a4f43f01ea2e
Diffstat (limited to 'common/Memdata.v')
-rw-r--r--common/Memdata.v8
1 files changed, 0 insertions, 8 deletions
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.