LogRel.Substitution.Reflexivity

From LogRel.AutoSubst Require Import core unscoped Ast Extra.
From LogRel Require Import Utils BasicAst Notations Context NormalForms Weakening GenericTyping LogicalRelation Validity.
From LogRel.LogicalRelation Require Import Irrelevance Escape Reflexivity Weakening Neutral.

Set Universe Polymorphism.

Section Reflexivity.
Context `{GenericTypingProperties}.

Lemma reflValidTy {Γ A l} ( : [||-v Γ])
  (VA : [Γ ||-v<l> A | ]) :
  [Γ ||-v<l> A A | | VA].
Proof.
  constructor; intros; apply reflLRTyEq.
Qed.

Lemma reflValidTm {Γ t A l} ( : [||-v Γ])
  (VA : [Γ ||-v<l> A | ])
  (Vt : [Γ ||-v<l> t : A | | VA]) :
  [Γ ||-v<l> t t : A | | VA].
Proof.
  constructor; intros; apply reflLRTmEq; now eapply validTm.
Qed.

End Reflexivity.