Documentation

Batteries.Lean.Syntax

Helper functions for working with typed syntaxes. #

def Lean.TSyntax.replaceM {M : TypeType} {k : SyntaxNodeKinds} [Monad M] (f : SyntaxM (Option Syntax)) (stx : TSyntax k) :
M (TSyntax k)

Applies the given function to every subsyntax.

Like Syntax.replaceM but for typed syntax. (Note there are no guarantees of type correctness here.)

Equations
Instances For