Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
partial def
Std.Do.SPred.Notation.unpack
{m : Type → Type}
[Monad m]
[Lean.MonadRef m]
[Lean.MonadQuotation m]
:
Remove an spred
layer from a term
syntax object.
Idiom notation #
Embedding of pure Lean values into SVal
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
‹t› in SVal
idiom notation. Accesses the state of type t
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Use getter t : SVal σs σ
in SVal
idiom notation; sugar for SVal.uncurry t (by assumption)
.
Equations
- Std.Do.«term#_» = Lean.ParserDescr.node `Std.Do.«term#_» 1024 (Lean.ParserDescr.binary `andthen (Lean.ParserDescr.symbol "#") (Lean.ParserDescr.cat `term 1024))
Instances For
Sugar for SPred
#
Entailment in SPred
; sugar for SPred.entails
.
Equations
- Std.Do.«term_⊢ₛ_» = Lean.ParserDescr.trailingNode `Std.Do.«term_⊢ₛ_» 25 26 (Lean.ParserDescr.binary `andthen (Lean.ParserDescr.symbol " ⊢ₛ ") (Lean.ParserDescr.cat `term 25))
Instances For
Tautology in SPred
; sugar for SPred.entails ⌜True⌝
.
Equations
- Std.Do.«term⊢ₛ_» = Lean.ParserDescr.node `Std.Do.«term⊢ₛ_» 25 (Lean.ParserDescr.binary `andthen (Lean.ParserDescr.symbol "⊢ₛ ") (Lean.ParserDescr.cat `term 25))
Instances For
Bi-entailment in SPred
; sugar for SPred.bientails
.
Equations
- Std.Do.«term_⊣⊢ₛ_» = Lean.ParserDescr.trailingNode `Std.Do.«term_⊣⊢ₛ_» 25 25 (Lean.ParserDescr.binary `andthen (Lean.ParserDescr.symbol " ⊣⊢ₛ ") (Lean.ParserDescr.cat `term 25))