Step
*
of Lemma
can-apply-p-filter
∀[T:Type]. ∀[P:T ⟶ ℙ].  ∀f:∀x:T. Dec(P[x]). ∀x:T.  (↑can-apply(p-filter(f);x) 
⇐⇒ P[x])
BY
{ ((UnivCD THENA Auto) THEN RepUR ``can-apply p-filter`` 0) }
1
1. [T] : Type
2. [P] : T ⟶ ℙ
3. f : ∀x:T. Dec(P[x])@i
4. x : T@i
⊢ ↑isl(case f x of inl(p) => inl x | inr(p) => inr p ) 
⇐⇒ P[x]
Latex:
Latex:
\mforall{}[T:Type].  \mforall{}[P:T  {}\mrightarrow{}  \mBbbP{}].    \mforall{}f:\mforall{}x:T.  Dec(P[x]).  \mforall{}x:T.    (\muparrow{}can-apply(p-filter(f);x)  \mLeftarrow{}{}\mRightarrow{}  P[x])
By
Latex:
((UnivCD  THENA  Auto)  THEN  RepUR  ``can-apply  p-filter``  0)
Home
Index