LogRel.Validity.Introductions.Universe

From LogRel Require Import Utils Syntax.All GenericTyping LogicalRelation.
From LogRel.LogicalRelation Require Import Properties.
From LogRel.LogicalRelation.Introductions Require Import Universe.
From LogRel.Validity Require Import Validity Irrelevance Properties.

Set Universe Polymorphism.
Set Printing Primitive Projection Parameters.

Section Universe.
Context `{GenericTypingProperties} {Γ Γ' : context}.

Lemma UValid ( : [||-v Γ Γ' ]) : [Γ ||-v<one> U | ].
Proof. unshelve econstructor; intros; now eapply LRU_, redUOneCtx. Defined.

Lemma univValid {A A' l} l' { : [||-v Γ Γ']}
  {VU : [Γ ||-v<l> U | ]}
  (VA : [Γ ||-v<l> A A' : U | | VU]) :
  [Γ ||-v<l'> A A' | ].
Proof. constructor; intros ???? Vσ ; eapply UnivEq; exact (validTmExt VA _ Vσ). Qed.

End Universe.