Documentation

LeanStlc.Progress

Equations
Instances For
    inductive Value :
    Instances For
      theorem value_sound {t : Term} :
      Value t∀ (t' : Term), ¬t ~> t'
      inductive VarSpine :
      Instances For
        theorem lam_value {Γ : List Ty} {t : Term} {A B : Ty} :
        Γ t : (A -t> B) → Value t → ( (b : Term), t = :λ[A] b) VarSpine t
        theorem progress (t : Term) :
        Value t (t' : Term), t ~> t'