Skip to content

Commit

Permalink
update lemmas
Browse files Browse the repository at this point in the history
  • Loading branch information
HuStmpHrrr committed Nov 8, 2024
1 parent e629616 commit ebbadc6
Showing 1 changed file with 25 additions and 1 deletion.
26 changes: 25 additions & 1 deletion theories/Core/Soundness/LogicalRelation/CoreLemmas.v
Original file line number Diff line number Diff line change
Expand Up @@ -686,7 +686,7 @@ Qed.
end);
eauto; intuition.

Lemma glu_univ_elem_resp_per_univ : forall i a a' R,
Lemma glu_univ_elem_resp_per_univ_elem : forall i a a' R,
{{ DF a ≈ a' ∈ per_univ_elem i ↘ R }} ->
forall P El,
{{ DG a ∈ glu_univ_elem i ↘ P ↘ El }} ->
Expand Down Expand Up @@ -798,6 +798,30 @@ Proof.
mauto.
Qed.


Lemma glu_univ_elem_resp_per_univ : forall i a a' P El,
{{ Dom a ≈ a' ∈ per_univ i }} ->
{{ DG a ∈ glu_univ_elem i ↘ P ↘ El }} ->
{{ DG a' ∈ glu_univ_elem i ↘ P ↘ El }}.
Proof.
intros * [? H] ?.
eapply glu_univ_elem_resp_per_univ_elem in H; eauto.
intuition.
Qed.

Lemma glu_univ_elem_resp_per_elem : forall i a a' R P El Γ M A m m',
{{ DF a ≈ a' ∈ per_univ_elem i ↘ R }} ->
{{ DG a ∈ glu_univ_elem i ↘ P ↘ El }} ->
{{ Γ ⊢ M : A ® m ∈ El }} ->
{{ Dom m ≈ m' ∈ R }} ->
{{ Γ ⊢ M : A ® m' ∈ El }}.
Proof.
intros * H ?.
eapply glu_univ_elem_resp_per_univ_elem in H; eauto.
intuition.
Qed.


(** *** Morphism instances for [glu_univ_elem] *)
Add Parametric Morphism i : (glu_univ_elem i)
with signature glu_typ_pred_equivalence ==> glu_exp_pred_equivalence ==> per_univ i ==> iff as glu_univ_elem_morphism_iff.
Expand Down

0 comments on commit ebbadc6

Please sign in to comment.