aboutsummaryrefslogtreecommitdiffstats
path: root/backend/Injectproof.v
diff options
context:
space:
mode:
authorDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2020-03-30 18:46:50 +0200
committerDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2020-03-30 18:46:50 +0200
commit27c8e10f4e0a3eee6bf9feb03d0f12990f74badd (patch)
tree7761f2d1e53a8d4bd0c47d0b40411c46c1bfe3ad /backend/Injectproof.v
parentb937a4c10226930b7109ae6c9707255e53a0dd2b (diff)
downloadcompcert-kvx-27c8e10f4e0a3eee6bf9feb03d0f12990f74badd.tar.gz
compcert-kvx-27c8e10f4e0a3eee6bf9feb03d0f12990f74badd.zip
use inject_l
Diffstat (limited to 'backend/Injectproof.v')
-rw-r--r--backend/Injectproof.v21
1 files changed, 3 insertions, 18 deletions
diff --git a/backend/Injectproof.v b/backend/Injectproof.v
index b0dcfad5..80b217bc 100644
--- a/backend/Injectproof.v
+++ b/backend/Injectproof.v
@@ -81,7 +81,7 @@ Proof.
Qed.
Program Definition bounded_nth_S_statement : Prop :=
- forall {T : Type} (k : nat) (h : T) (l : list T) (BOUND : (k < List.length l)%nat),
+ forall (T : Type) (k : nat) (h : T) (l : list T) (BOUND : (k < List.length l)%nat),
bounded_nth (S k) (h::l) _ = bounded_nth k l BOUND.
Obligation 1.
lia.
@@ -231,23 +231,6 @@ Definition inject_l (prog : code) extra_pc injections :=
injections
(extra_pc, prog).
-(*
-Lemma inject_l_position_ok:
- forall injections prog extra_pc,
- (fst (inject_l prog extra_pc injections)) =
- inject_l_position extra_pc injections.
-Proof.
- induction injections; intros; simpl; trivial.
- destruct a as [pc l].
- unfold inject_l. simpl.
- rewrite (pair_expand (inject_at prog pc extra_pc l)).
- fold (inject_l (snd (inject_at prog pc extra_pc l)) (fst (inject_at prog pc extra_pc l)) injections).
- rewrite IHinjections.
- f_equal.
- rewrite inject_at_increases.
- reflexivity.
-Qed.
-*)
Lemma inject_l_preserves :
forall injections prog extra_pc pc0,
pc0 < extra_pc ->
@@ -507,6 +490,7 @@ Proof.
}
Qed.
+(*
Lemma inject'_preserves :
forall injections prog extra_pc pc0,
pc0 < extra_pc ->
@@ -538,3 +522,4 @@ Proof.
unfold inject'.
apply inject'_preserves.
Qed.
+*)