Step
*
of Lemma
tf-apply_wf
∀[A:Type]. ∀[a:A]. ∀[B:type-function{i:l}(A)].  (tf-apply(B;a) ∈ Type)
BY
{ (At ⌜𝕌'⌝Intros⋅ THEN Try (Complete (Auto)) THEN Unfold `type-function` 3 THEN Unfold `tf-apply` 0) }
1
1. [A] : Type
2. [a] : A
3. [B] : per-function(A;a.Type)
⊢ B a ∈ Type
Latex:
Latex:
\mforall{}[A:Type].  \mforall{}[a:A].  \mforall{}[B:type-function\{i:l\}(A)].    (tf-apply(B;a)  \mmember{}  Type)
By
Latex:
(At  \mkleeneopen{}\mBbbU{}'\mkleeneclose{}Intros\mcdot{}  THEN  Try  (Complete  (Auto))  THEN  Unfold  `type-function`  3  THEN  Unfold  `tf-apply`  0)
Home
Index