Documentation

Lean.Elab.Util

Equations
Instances For
    Equations
    • One or more equations did not get rendered due to their size.
    Instances For

      Two names are from the same lexical scope if their scoping information modulo MacroScopesView.name is equal.

      Instances For
        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          Instances For
            @[reducible, inline]
            Instances For

              If ref does not have position information, then try to use macroStack

              Instances For
                Equations
                Instances For
                  Equations
                  • One or more equations did not get rendered due to their size.
                  Instances For
                    @[implemented_by _private.Lean.Elab.Util.0.Lean.Elab.evalSyntaxConstantUnsafe]
                    unsafe def Lean.Elab.mkElabAttribute (γ : Type) (attrBuiltinName attrName parserNamespace typeName : Lean.Name) (kind : String) (attrDeclName : Lean.Name := by exact decl_name%) :
                    Instances For
                      @[implemented_by Lean.Elab.mkMacroAttributeUnsafe]

                      Try to expand macro at syntax tree root and return macro declaration name and new syntax if successful. Return none if all macros threw Macro.Exception.unsupportedSyntax.

                      Instances For
                        Instances
                          @[always_inline]
                          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.
                            Instances For
                              partial def Lean.Elab.mkUnusedBaseName.loop (baseName currNamespace : Lean.Name) (idx : Nat) :
                              Equations
                              Instances For

                                If x throws an exception, catch it and turn it into a log message (using logException).

                                Instances For
                                  Equations
                                  • One or more equations did not get rendered due to their size.
                                  Instances For