Documentation

Lean.Meta.Instances

@[reducible, inline]
Equations
Instances For
    Instances For
      Equations
      Equations
      Equations
      Instances For
        Equations
        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          Equations
          Instances For
            def Lean.Meta.Instances.erase {m : TypeType} [Monad m] [MonadError m] (d : Instances) (declName : Name) :
            Equations
            • One or more equations did not get rendered due to their size.
            Instances For
              def Lean.Meta.addInstance (declName : Name) (attrKind : AttributeKind) (prio : Nat) :
              Equations
              • One or more equations did not get rendered due to their size.
              Instances For
                Equations
                Instances For
                  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

                      Default instance support #

                      Instances For
                        @[reducible, inline]
                        Equations
                        Instances For
                          Instances For
                            Equations
                            • One or more equations did not get rendered due to their size.
                            Instances For
                              def Lean.Meta.addDefaultInstance (declName : Name) (prio : Nat := 0) :
                              Equations
                              • One or more equations did not get rendered due to their size.
                              Instances For
                                def Lean.Meta.getDefaultInstances {m : TypeType} [Monad m] [MonadEnv m] (className : Name) :
                                m (List (Name × Nat))
                                Equations
                                Instances For