Documentation

Lean.Compiler.LCNF.FVarUtil

Instances
    partial def Lean.Compiler.LCNF.Expr.mapFVarM {m : TypeType u_1} [MonadLiftT CompilerM m] [Monad m] (f : FVarIdm FVarId) (e : Expr) :
    partial def Lean.Compiler.LCNF.Expr.forFVarM {m : TypeType u_1} [Monad m] (f : FVarIdm Unit) (e : Expr) :
    Equations
    • One or more equations did not get rendered due to their size.
    Equations
    • One or more equations did not get rendered due to their size.
    Equations
    • One or more equations did not get rendered due to their size.
    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.
      def Lean.Compiler.LCNF.Param.mapFVarM {m : TypeType u_1} [MonadLiftT CompilerM m] [Monad m] (f : FVarIdm FVarId) (param : Param) :
      Equations
      Instances For
        def Lean.Compiler.LCNF.Param.forFVarM {m : TypeType u_1} [Monad m] (f : FVarIdm Unit) (param : Param) :
        Equations
        Instances For
          Equations
          • One or more equations did not get rendered due to their size.
          partial def Lean.Compiler.LCNF.Code.mapFVarM {m : TypeType} [MonadLiftT CompilerM m] [Monad m] (f : FVarIdm FVarId) (c : Code) :
          partial def Lean.Compiler.LCNF.Code.forFVarM {m : TypeType} [Monad m] (f : FVarIdm Unit) (c : Code) :
          Equations
          • One or more equations did not get rendered due to their size.
          Equations
          • One or more equations did not get rendered due to their size.
          Instances For
            def Lean.Compiler.LCNF.FunDecl.forFVarM {m : TypeType} [Monad m] (f : FVarIdm Unit) (decl : FunDecl) :
            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.
              Equations
              • One or more equations did not get rendered due to their size.
              Equations
              • One or more equations did not get rendered due to their size.
              def Lean.Compiler.LCNF.anyFVarM {m : TypeType} {α : Type} [Monad m] [TraverseFVar α] (f : FVarIdm Bool) (x : α) :
              Equations
              • One or more equations did not get rendered due to their size.
              Instances For
                def Lean.Compiler.LCNF.anyFVarM.go {m : TypeType} [Monad m] (f : FVarIdm Bool) (fvar : FVarId) :
                Equations
                Instances For
                  def Lean.Compiler.LCNF.allFVarM {m : TypeType} {α : Type} [Monad m] [TraverseFVar α] (f : FVarIdm Bool) (x : α) :
                  Equations
                  • One or more equations did not get rendered due to their size.
                  Instances For
                    def Lean.Compiler.LCNF.allFVarM.go {m : TypeType} [Monad m] (f : FVarIdm Bool) (fvar : FVarId) :
                    Equations
                    Instances For
                      def Lean.Compiler.LCNF.anyFVar {α : Type} [TraverseFVar α] (f : FVarIdBool) (x : α) :
                      Equations
                      Instances For
                        def Lean.Compiler.LCNF.allFVar {α : Type} [TraverseFVar α] (f : FVarIdBool) (x : α) :
                        Equations
                        Instances For