aboutsummaryrefslogtreecommitdiff
diff options
context:
space:
mode:
authorGravatar Jason Gross <jgross@mit.edu>2018-10-23 19:55:14 -0400
committerGravatar Jason Gross <jgross@mit.edu>2018-10-23 19:55:14 -0400
commit4ad320a862e34e6a831e0f05c148c6abb54889d4 (patch)
treede4bde4cf442997298fa6c1cf922157f5234cd1a
parent2cb0107e5f587c79e11b3e0e27d9a5dca799f24c (diff)
Add under_with_unification_resultT'_relation1_gen_always
-rw-r--r--src/Experiments/NewPipeline/RewriterWf1.v18
1 files changed, 18 insertions, 0 deletions
diff --git a/src/Experiments/NewPipeline/RewriterWf1.v b/src/Experiments/NewPipeline/RewriterWf1.v
index a24510fb7..df99b78a6 100644
--- a/src/Experiments/NewPipeline/RewriterWf1.v
+++ b/src/Experiments/NewPipeline/RewriterWf1.v
@@ -711,6 +711,24 @@ Module Compilers.
induction ls as [|l ls IHls]; cbn in *; [ tauto | ].
setoid_rewrite IHls; split; intro H; intros; first [ apply H | apply (H (_, _)) ].
Qed.
+
+ Lemma under_type_of_list_relation1_cps_always {A1 ls F v}
+ (F_always : forall v, F v : Prop)
+ : @under_type_of_list_relation1_cps A1 ls F v.
+ Proof using Type.
+ cbv [under_type_of_list_relation1_cps] in *.
+ induction ls; cbn in *; eauto.
+ Qed.
+
+ Lemma under_with_unification_resultT'_relation1_gen_always
+ {t p evm K1 FH F v}
+ (F_always : forall v, F v : Prop)
+ : @under_with_unification_resultT'_relation1_gen
+ ident var pident pident_arg_types t p evm K1 FH F v.
+ Proof using Type.
+ revert evm K1 F v F_always.
+ induction p; intros; cbn in *; eauto using @under_type_of_list_relation1_cps_always.
+ Qed.
End with_var1.
Section with_var2.