Step
*
2
1
of Lemma
do-apply-p-first-disjoint
.....assertion..... 
1. A : Type
2. B : Type
3. L : (A ⟶ (B + Top)) List
4. x : A
5. (∀f,g∈L.  p-disjoint(A;f;g))
6. f : A ⟶ (B + Top)
7. (f ∈ L)
8. ↑can-apply(f;x)
⊢ hd(filter(λf.can-apply(f;x);L)) = f ∈ (A ⟶ (B + Top))
BY
{ xxx(Lemmaize [-1;-2;-4] THEN InductionOnList)xxx }
1
1. A : Type
2. B : Type
⊢ ∀x:A. ∀f:A ⟶ (B + Top).
    ((∀f,g∈[].  p-disjoint(A;f;g))
    
⇒ (f ∈ [])
    
⇒ (↑can-apply(f;x))
    
⇒ (hd(filter(λf.can-apply(f;x);[])) = f ∈ (A ⟶ (B + Top))))
2
1. A : Type
2. B : Type
3. u : A ⟶ (B + Top)
4. v : (A ⟶ (B + Top)) List
5. ∀x:A. ∀f:A ⟶ (B + Top).
     ((∀f,g∈v.  p-disjoint(A;f;g))
     
⇒ (f ∈ v)
     
⇒ (↑can-apply(f;x))
     
⇒ (hd(filter(λf.can-apply(f;x);v)) = f ∈ (A ⟶ (B + Top))))
⊢ ∀x:A. ∀f:A ⟶ (B + Top).
    ((∀f,g∈[u / v].  p-disjoint(A;f;g))
    
⇒ (f ∈ [u / v])
    
⇒ (↑can-apply(f;x))
    
⇒ (hd(filter(λf.can-apply(f;x);[u / v])) = f ∈ (A ⟶ (B + Top))))
Latex:
Latex:
.....assertion..... 
1.  A  :  Type
2.  B  :  Type
3.  L  :  (A  {}\mrightarrow{}  (B  +  Top))  List
4.  x  :  A
5.  (\mforall{}f,g\mmember{}L.    p-disjoint(A;f;g))
6.  f  :  A  {}\mrightarrow{}  (B  +  Top)
7.  (f  \mmember{}  L)
8.  \muparrow{}can-apply(f;x)
\mvdash{}  hd(filter(\mlambda{}f.can-apply(f;x);L))  =  f
By
Latex:
xxx(Lemmaize  [-1;-2;-4]  THEN  InductionOnList)xxx
Home
Index