Nuprl Lemma : es-local-pred-cases-sq

[Info:Type]
  ∀es:EO+(Info). ∀e:E. ∀P:{e':E| (e' <loc e)}  ⟶ 𝔹.
    (¬↑first(e))
    ∧ (((↑(P pred(e))) ∧ (do-apply(last(P);e) pred(e)))
      ∨ ((¬↑(P pred(e))) ∧ (↑can-apply(last(P);pred(e))) ∧ (do-apply(last(P);e) do-apply(last(P);pred(e))))) 
    supposing ↑can-apply(last(P);e)


Proof




Definitions occuring in Statement :  es-local-pred: last(P) event-ordering+: EO+(Info) es-locl: (e <loc e') es-first: first(e) es-pred: pred(e) es-E: E assert: b bool: 𝔹 uimplies: supposing a uall: [x:A]. B[x] all: x:A. B[x] not: ¬A or: P ∨ Q and: P ∧ Q set: {x:A| B[x]}  apply: a function: x:A ⟶ B[x] universe: Type sqequal: t do-apply: do-apply(f;x) can-apply: can-apply(f;x)
Definitions unfolded in proof :  uall: [x:A]. B[x] all: x:A. B[x] do-apply: do-apply(f;x) can-apply: can-apply(f;x) es-local-pred: last(P) member: t ∈ T subtype_rel: A ⊆B implies:  Q bool: 𝔹 unit: Unit it: btrue: tt uiff: uiff(P;Q) and: P ∧ Q uimplies: supposing a ifthenelse: if then else fi  assert: b isl: isl(x) outl: outl(x) bfalse: ff false: False prop: exists: x:A. B[x] or: P ∨ Q sq_type: SQType(T) guard: {T} bnot: ¬bb true: True cand: c∧ B not: ¬A so_lambda: λ2x.t[x] so_apply: x[s] sq_exists: x:{A| B[x]} top: Top

Latex:
\mforall{}[Info:Type]
    \mforall{}es:EO+(Info).  \mforall{}e:E.  \mforall{}P:\{e':E|  (e'  <loc  e)\}    {}\mrightarrow{}  \mBbbB{}.
        (\mneg{}\muparrow{}first(e))
        \mwedge{}  (((\muparrow{}(P  pred(e)))  \mwedge{}  (do-apply(last(P);e)  \msim{}  pred(e)))
            \mvee{}  ((\mneg{}\muparrow{}(P  pred(e)))
                \mwedge{}  (\muparrow{}can-apply(last(P);pred(e)))
                \mwedge{}  (do-apply(last(P);e)  \msim{}  do-apply(last(P);pred(e))))) 
        supposing  \muparrow{}can-apply(last(P);e)



Date html generated: 2016_05_16-PM-11_27_43
Last ObjectModification: 2015_12_29-AM-10_43_16

Theory : event-ordering


Home Index