Skip to content

Commit

Permalink
fixup! wip generic typing lemmas
Browse files Browse the repository at this point in the history
  • Loading branch information
jpoiret committed Nov 17, 2023
1 parent 7f0f113 commit 410f1cc
Showing 1 changed file with 5 additions and 5 deletions.
10 changes: 5 additions & 5 deletions theories/GenericTyping.v
Original file line number Diff line number Diff line change
Expand Up @@ -918,17 +918,17 @@ Section GenericConsequences.

(** *** Derived typing, reduction and conversion judgements *)

Lemma ty_var0 {Γ A} :
[Γ |- A] ->
Lemma ty_var0 {Γ A s} :
[Γ |- A @ s] ->
[Γ ,, A |- tRel 0 : A⟨↑⟩].
Proof.
intros; refine (ty_var _ (in_here _ _)); gen_typing.
Qed.

Lemma wft_simple_arr {Γ A B} :
[Γ |- A] ->
[Γ |- B] ->
[Γ |- arr A B].
[Γ |- A @ set] ->
[Γ |- B @ set] ->
[Γ |- arr A B @ set].
Proof.
intros. eapply wft_prod; renToWk; tea.
eapply wft_wk; gen_typing.
Expand Down

0 comments on commit 410f1cc

Please sign in to comment.