summaryrefslogtreecommitdiff
path: root/common/Memdata.v
diff options
context:
space:
mode:
authorGravatar xleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2012-01-14 14:23:26 +0000
committerGravatar xleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2012-01-14 14:23:26 +0000
commita82c9c0e4a0b8e37c9c3ea5ae99714982563606f (patch)
tree93b9999698a4cd47ec4cb5fcdcdfd215d62f8e9e /common/Memdata.v
parentbb8f49c419eb8205ef541edcbe17f4d14aa99564 (diff)
Merge of the nonstrict-ops branch:
- Most RTL operators now evaluate to Some Vundef instead of None when undefined behavior occurs. - More aggressive instruction selection. - "Bertotization" of pattern-matchings now implemented by a proper preprocessor. - Cast optimization moved to cfrontend/Cminorgen; removed backend/CastOptim. git-svn-id: https://yquem.inria.fr/compcert/svn/compcert/trunk@1790 fca1b0fc-160b-0410-b1d3-a4f43f01ea2e
Diffstat (limited to 'common/Memdata.v')
-rw-r--r--common/Memdata.v16
1 files changed, 0 insertions, 16 deletions
diff --git a/common/Memdata.v b/common/Memdata.v
index fde8b47..47ed79e 100644
--- a/common/Memdata.v
+++ b/common/Memdata.v
@@ -1029,22 +1029,6 @@ Proof.
apply repeat_Undef_inject_any. apply encode_val_length.
Qed.
-(** The identity injection has interesting properties. *)
-
-Definition inject_id : meminj := fun b => Some(b, 0).
-
-Lemma val_inject_id:
- forall v1 v2,
- val_inject inject_id v1 v2 <-> Val.lessdef v1 v2.
-Proof.
- intros; split; intros.
- inv H. constructor. constructor.
- unfold inject_id in H0. inv H0. rewrite Int.add_zero. constructor.
- constructor.
- inv H. destruct v2; econstructor. unfold inject_id; reflexivity. rewrite Int.add_zero; auto.
- constructor.
-Qed.
-
Definition memval_lessdef: memval -> memval -> Prop := memval_inject inject_id.
Lemma memval_lessdef_refl: