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