summaryrefslogtreecommitdiff
path: root/common/Memdata.v
diff options
context:
space:
mode:
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: