Documentation

Init.Meta

@[extern lean_get_githash]
@[extern lean_version_get_is_release]
@[extern lean_version_get_special_desc]

Additional version description like "nightly-2018-03-11"

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
      Equations
      Instances For
        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          @[extern lean_internal_is_stage0]
          @[extern lean_internal_has_llvm_backend]

          This function can be used to detect whether the compiler has support for generating LLVM instead of C. It is used by lake instead of the --features flag in order to avoid having to run a compiler for this every time on startup. See #2572.

          @[inline]

          Valid identifier names

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

                                Creates a round-trippable string name component if possible, otherwise returns none. Names that are valid identifiers are not escaped, and otherwise, if they do not contain », they are escaped.

                                • If force is true, then even valid identifiers are escaped.
                                Equations
                                • One or more equations did not get rendered due to their size.
                                Instances For
                                  def Lean.Name.toStringWithSep (sep : String) (escape : Bool) (n : Name) (isToken : StringBool := fun (x : String) => Bool.false) :

                                  Uses the separator sep (usually ".") to combine the components of the Name into a string. See the documentation for Name.toString for an explanation of escape and isToken.

                                  Instances For
                                    Equations
                                    Instances For
                                      def Lean.Name.toString (n : Name) (escape : Bool := Bool.true) (isToken : StringBool := fun (x : String) => Bool.false) :

                                      Converts a name to a string.

                                      • If escape is true, then escapes name components using « and » to ensure that those names that can appear in source files round trip. Names with number components, anonymous names, and names containing » might not round trip. Furthermore, "pseudo-syntax" produced by the delaborator, such as _, #0 or ?u, is not escaped.
                                      • The optional isToken function is used when escape is true to determine whether more escaping is necessary to avoid parser tokens. The insertion algorithm works so long as parser tokens do not themselves contain « or ».
                                      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
                                          Equations
                                          Instances For
                                            Equations
                                            • One or more equations did not get rendered due to their size.
                                            Instances For
                                              Equations
                                              Instances For
                                                Equations
                                                Instances For
                                                  Instances For

                                                    eraseSuffix? n s return n' if n is of the form n == n' ++ s.

                                                    Instances For
                                                      @[inline]
                                                      def Lean.Name.modifyBase (n : Name) (f : NameName) :

                                                      Remove macros scopes, apply f, and put them back

                                                      Equations
                                                      • One or more equations did not get rendered due to their size.
                                                      Instances For
                                                        @[export lean_name_append_after]
                                                        def Lean.Name.appendAfter (n : Name) (suffix : String) :
                                                        Equations
                                                        • One or more equations did not get rendered due to their size.
                                                        Instances For
                                                          @[export lean_name_append_index_after]
                                                          Equations
                                                          • One or more equations did not get rendered due to their size.
                                                          Instances For
                                                            @[export lean_name_append_before]
                                                            Equations
                                                            • One or more equations did not get rendered due to their size.
                                                            Instances For
                                                              theorem Lean.Name.beq_iff_eq {m n : Name} :
                                                              Iff (Eq (BEq.beq m n) Bool.true) (Eq m n)
                                                              @[inline]
                                                              Equations
                                                              Instances For
                                                                @[inline]
                                                                Equations
                                                                Instances For
                                                                  @[inline]
                                                                  Equations
                                                                  Instances For
                                                                    structure Lean.MonadNameGenerator (m : TypeType) :
                                                                    Instances For
                                                                      @[reducible, inline]

                                                                      Syntax that represents a Lean term.

                                                                      Equations
                                                                      Instances For
                                                                        @[reducible, inline]

                                                                        Syntax that represents a command.

                                                                        Equations
                                                                        Instances For
                                                                          @[reducible, inline]

                                                                          Syntax that represents a universe level.

                                                                          Equations
                                                                          Instances For
                                                                            @[reducible, inline]

                                                                            Syntax that represents a tactic.

                                                                            Equations
                                                                            Instances For
                                                                              @[reducible, inline]

                                                                              Syntax that represents a precedence (e.g. for an operator).

                                                                              Equations
                                                                              Instances For
                                                                                @[reducible, inline]

                                                                                Syntax that represents a priority (e.g. for an instance declaration).

                                                                                Equations
                                                                                Instances For
                                                                                  @[reducible, inline]

                                                                                  Syntax that represents an identifier.

                                                                                  Equations
                                                                                  Instances For
                                                                                    @[reducible, inline]

                                                                                    Syntax that represents a string literal.

                                                                                    Equations
                                                                                    Instances For
                                                                                      @[reducible, inline]

                                                                                      Syntax that represents a character literal.

                                                                                      Equations
                                                                                      Instances For
                                                                                        @[reducible, inline]

                                                                                        Syntax that represents a quoted name literal that begins with a back-tick.

                                                                                        Equations
                                                                                        Instances For
                                                                                          @[reducible, inline]

                                                                                          Syntax that represents a scientific numeric literal that may have decimal and exponential parts.

                                                                                          Equations
                                                                                          Instances For
                                                                                            @[reducible, inline]

                                                                                            Syntax that represents a numeric literal.

                                                                                            Equations
                                                                                            Instances For
                                                                                              @[reducible, inline]

                                                                                              Syntax that represents macro hygiene info.

                                                                                              Equations
                                                                                              Instances For
                                                                                                Equations
                                                                                                Instances For
                                                                                                  Equations
                                                                                                  Instances For
                                                                                                    partial def Lean.Syntax.structEq :

                                                                                                    Compare syntax structures modulo source info.

                                                                                                    Equations
                                                                                                    Instances For

                                                                                                      Finds the first SourceInfo from the back of stx or none if no SourceInfo can be found.

                                                                                                      Finds the first SourceInfo from the back of stx or SourceInfo.none if no SourceInfo can be found.

                                                                                                      Equations
                                                                                                      Instances For

                                                                                                        Finds the trailing size of the first SourceInfo from the back of stx. If no SourceInfo can be found or the first SourceInfo from the back of stx contains no trailing whitespace, the result is 0.

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

                                                                                                          Finds the trailing whitespace substring of the first SourceInfo from the back of stx. If no SourceInfo can be found or the first SourceInfo from the back of stx contains no trailing whitespace, the result is none.

                                                                                                          Equations
                                                                                                          Instances For

                                                                                                            Finds the tail position of the trailing whitespace of the first SourceInfo from the back of stx. If no SourceInfo can be found or the first SourceInfo from the back of stx contains no trailing whitespace and lacks a tail position, the result is none.

                                                                                                            Equations
                                                                                                            Instances For
                                                                                                              def Lean.Syntax.getSubstring? (stx : Syntax) (withLeading withTrailing : Bool := Bool.true) :

                                                                                                              Return substring of original input covering stx. Result is meaningful only if all involved SourceInfo.originals refer to the same string (as is the case after parsing).

                                                                                                              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

                                                                                                                  Replaces the trailing whitespace in stx, if any, with an empty substring.

                                                                                                                  The trailing substring's startPos and str are preserved in order to ensure that the result could have been produced by the parser, in case any syntax consumers rely on such an assumption.

                                                                                                                  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
                                                                                                                      Equations
                                                                                                                      • One or more equations did not get rendered due to their size.
                                                                                                                      Instances For

                                                                                                                        Return the first atom/identifier that has position information

                                                                                                                        Equations
                                                                                                                        Instances For

                                                                                                                          Ensure head position is synthetic. The server regards syntax as "original" only if both head and tail info are original.

                                                                                                                          Equations
                                                                                                                          Instances For
                                                                                                                            @[inline]
                                                                                                                            def Lean.withHeadRefOnly {m : TypeType} [Monad m] [MonadRef m] {α : Type} (x : m α) :
                                                                                                                            m α

                                                                                                                            Use the head atom/identifier of the current ref as the ref

                                                                                                                            Equations
                                                                                                                            • One or more equations did not get rendered due to their size.
                                                                                                                            Instances For
                                                                                                                              partial def Lean.expandMacros (stx : Syntax) (p : SyntaxNodeKindBool := fun (k : SyntaxNodeKind) => bne k `Lean.Parser.Term.byTactic) :

                                                                                                                              Expand macros in the given syntax. A node with kind k is visited only if p k is true.

                                                                                                                              Note that the default value for p returns false for by ... nodes. This is a "hack". The tactic framework abuses the macro system to implement extensible tactics. For example, one can define

                                                                                                                              syntax "my_trivial" : tactic -- extensible tactic
                                                                                                                              
                                                                                                                              macro_rules | `(tactic| my_trivial) => `(tactic| decide)
                                                                                                                              macro_rules | `(tactic| my_trivial) => `(tactic| assumption)
                                                                                                                              

                                                                                                                              When the tactic evaluator finds the tactic my_trivial, it tries to evaluate the macro_rule expansions until one "works", i.e., the macro expansion is evaluated without producing an exception. We say this solution is a bit hackish because the term elaborator may invoke expandMacros with (p := fun _ => true), and expand the tactic macros as just macros. In the example above, my_trivial would be replaced with assumption, decide would not be tried if assumption fails at tactic evaluation time.

                                                                                                                              We are considering two possible solutions for this issue: 1- A proper extensible tactic feature that does not rely on the macro system.

                                                                                                                              2- Typed macros that know the syntax categories they're working in. Then, we would be able to select which syntactic categories are expanded by expandMacros.

                                                                                                                              Helper functions for processing Syntax programmatically #

                                                                                                                              def Lean.mkIdentFrom (src : Syntax) (val : Name) (canonical : Bool := Bool.false) :

                                                                                                                              Create an identifier copying the position from src. To refer to a specific constant, use mkCIdentFrom instead.

                                                                                                                              Equations
                                                                                                                              Instances For
                                                                                                                                def Lean.mkIdentFromRef {m : TypeType} [Monad m] [MonadRef m] (val : Name) (canonical : Bool := Bool.false) :
                                                                                                                                Equations
                                                                                                                                Instances For
                                                                                                                                  def Lean.mkCIdentFrom (src : Syntax) (c : Name) (canonical : Bool := Bool.false) :

                                                                                                                                  Create an identifier referring to a constant c copying the position from src. This variant of mkIdentFrom makes sure that the identifier cannot accidentally be captured.

                                                                                                                                  Equations
                                                                                                                                  • One or more equations did not get rendered due to their size.
                                                                                                                                  Instances For
                                                                                                                                    def Lean.mkCIdentFromRef {m : TypeType} [Monad m] [MonadRef m] (c : Name) (canonical : Bool := Bool.false) :
                                                                                                                                    Equations
                                                                                                                                    Instances For
                                                                                                                                      @[export lean_mk_syntax_ident]
                                                                                                                                      Equations
                                                                                                                                      Instances For
                                                                                                                                        @[inline]
                                                                                                                                        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
                                                                                                                                              def Lean.mkHole (ref : Syntax) (canonical : Bool := Bool.false) :
                                                                                                                                              Equations
                                                                                                                                              Instances For
                                                                                                                                                Equations
                                                                                                                                                Instances For
                                                                                                                                                  Equations
                                                                                                                                                  Instances For
                                                                                                                                                    def Lean.Syntax.SepArray.ofElemsUsingRef {m : TypeType} [Monad m] [MonadRef m] {sep : String} (elems : Array Syntax) :
                                                                                                                                                    m (SepArray sep)
                                                                                                                                                    Equations
                                                                                                                                                    • One or more equations did not get rendered due to their size.
                                                                                                                                                    Instances For

                                                                                                                                                      Constructs a typed separated array from elements. The given array does not include the separators.

                                                                                                                                                      Like Syntax.SepArray.ofElems but for typed syntax.

                                                                                                                                                      Equations
                                                                                                                                                      Instances For

                                                                                                                                                        Create syntax representing a Lean term application, but avoid degenerate empty applications.

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

                                                                                                                                                              Recall that we don't have special Syntax constructors for storing numeric and string atoms. The idea is to have an extensible approach where embedded DSLs may have new kind of atoms and/or different ways of representing them. So, our atoms contain just the parsed string. The main Lean parser uses the kind numLitKind for storing natural numbers that can be encoded in binary, octal, decimal and hexadecimal format. isNatLit implements a "decoder" for Syntax objects representing these numerals.

                                                                                                                                                              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

                                                                                                                                                                  Decodes a 'scientific number' string which is consumed by the OfScientific class. Takes as input a string such as 123, 123.456e7 and returns a triple (n, sign, e) with value given by n * 10^-e if sign else n * 10^e.

                                                                                                                                                                  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
                                                                                                                                                                      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
                                                                                                                                                                          Equations
                                                                                                                                                                          Instances For
                                                                                                                                                                            Equations
                                                                                                                                                                            • One or more equations did not get rendered due to their size.
                                                                                                                                                                            Instances For

                                                                                                                                                                              Decodes a valid string gap after the \. Note that this function matches "\" whitespace+ rather than the more restrictive "\" newline whitespace* since this simplifies the implementation. Justification: this does not overlap with any other sequences beginning with \.

                                                                                                                                                                              Equations
                                                                                                                                                                              Instances For
                                                                                                                                                                                partial def Lean.Syntax.decodeRawStrLitAux (s : String) (i : String.Pos) (num : Nat) :

                                                                                                                                                                                Takes a raw string literal, counts the number of #'s after the r, and interprets it as a string. The position i should start at 1, which is the character after the leading r. The algorithm is simple: we are given r##...#"...string..."##...# with zero or more #s. By counting the number of leading #'s, we can extract the ...string....

                                                                                                                                                                                Takes the string literal lexical syntax parsed by the parser and interprets it as a string. This is where escape sequences are processed for example. The string s is either a plain string literal or a raw string literal.

                                                                                                                                                                                If it returns none then the string literal is ill-formed, which indicates a bug in the parser. The function is not required to return none if the string literal is ill-formed.

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

                                                                                                                                                                                  If the provided Syntax is a string literal, returns the string it represents.

                                                                                                                                                                                  Even if the Syntax is a str node, the function may return none if its internally ill-formed. The parser should always create well-formed str nodes.

                                                                                                                                                                                  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
                                                                                                                                                                                      Equations
                                                                                                                                                                                      • One or more equations did not get rendered due to their size.
                                                                                                                                                                                      Instances For

                                                                                                                                                                                        Split a name literal (without the backtick) into its dot-separated components. For example, foo.bla.«bo.o»["foo", "bla", "«bo.o»"]. If the literal cannot be parsed, return [].

                                                                                                                                                                                        Equations
                                                                                                                                                                                        Instances For

                                                                                                                                                                                          Converts a substring to the Lean compiler's representation of names. The resulting name is hierarchical, and the string is split at the dots ('.').

                                                                                                                                                                                          "a.b".toSubstring.toName is the name a.b, not «a.b». For the latter, use Name.mkSimple ∘ Substring.toString.

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

                                                                                                                                                                                            Converts a string to the Lean compiler's representation of names. The resulting name is hierarchical, and the string is split at the dots ('.').

                                                                                                                                                                                            "a.b".toName is the name a.b, not «a.b». For the latter, use Name.mkSimple.

                                                                                                                                                                                            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
                                                                                                                                                                                                  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
                                                                                                                                                                                                          Equations
                                                                                                                                                                                                          • One or more equations did not get rendered due to their size.
                                                                                                                                                                                                          Instances For
                                                                                                                                                                                                            Equations
                                                                                                                                                                                                            Instances For

                                                                                                                                                                                                              Interprets a numeric literal as a natural number.

                                                                                                                                                                                                              Returns 0 if the syntax is malformed.

                                                                                                                                                                                                              Equations
                                                                                                                                                                                                              Instances For

                                                                                                                                                                                                                Extracts the parsed name from the syntax of an identifier.

                                                                                                                                                                                                                Returns Name.anonymous if the syntax is malformed.

                                                                                                                                                                                                                Equations
                                                                                                                                                                                                                Instances For

                                                                                                                                                                                                                  Extracts the components of a scientific numeric literal.

                                                                                                                                                                                                                  Returns a triple (n, sign, e) : Nat × Bool × Nat; the number's value is given by:

                                                                                                                                                                                                                  if sign then n * 10 ^ (-e) else n * 10 ^ e
                                                                                                                                                                                                                  

                                                                                                                                                                                                                  Returns (0, false, 0) if the syntax is malformed.

                                                                                                                                                                                                                  Equations
                                                                                                                                                                                                                  Instances For

                                                                                                                                                                                                                    Decodes a string literal, removing quotation marks and unescaping escaped characters.

                                                                                                                                                                                                                    Returns "" if the syntax is malformed.

                                                                                                                                                                                                                    Equations
                                                                                                                                                                                                                    Instances For

                                                                                                                                                                                                                      Decodes a character literal.

                                                                                                                                                                                                                      Returns (default : Char) if the syntax is malformed.

                                                                                                                                                                                                                      Equations
                                                                                                                                                                                                                      Instances For

                                                                                                                                                                                                                        Decodes a quoted name literal, returning the name.

                                                                                                                                                                                                                        Returns Lean.Name.anonymous if the syntax is malformed.

                                                                                                                                                                                                                        Equations
                                                                                                                                                                                                                        Instances For

                                                                                                                                                                                                                          Decodes macro hygiene information.

                                                                                                                                                                                                                          Equations
                                                                                                                                                                                                                          Instances For
                                                                                                                                                                                                                            Equations
                                                                                                                                                                                                                            • One or more equations did not get rendered due to their size.
                                                                                                                                                                                                                            Instances For
                                                                                                                                                                                                                              structure Lean.Quote (α : Type) (k : SyntaxNodeKind := `term) :

                                                                                                                                                                                                                              Reflect a runtime datum back to surface syntax (best-effort).

                                                                                                                                                                                                                              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
                                                                                                                                                                                                                                    Equations
                                                                                                                                                                                                                                    • One or more equations did not get rendered due to their size.
                                                                                                                                                                                                                                    Instances For
                                                                                                                                                                                                                                      def Lean.instQuoteProdMkStr1 {α β : Type} [Quote α] [Quote β] :
                                                                                                                                                                                                                                      Quote (Prod α β)
                                                                                                                                                                                                                                      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

                                                                                                                                                                                                                                            Evaluator for prec DSL

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

                                                                                                                                                                                                                                                Evaluator for prio DSL

                                                                                                                                                                                                                                                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
                                                                                                                                                                                                                                                      @[reducible, inline]
                                                                                                                                                                                                                                                      abbrev Array.getSepElems {α : Type u_1} (as : Array α) :
                                                                                                                                                                                                                                                      Equations
                                                                                                                                                                                                                                                      Instances For

                                                                                                                                                                                                                                                        Filters an array of syntax, treating every other element as a separator rather than an element to test with the monadic predicate p. The resulting array contains the tested elements for which p returns true, separated by the corresponding separator elements.

                                                                                                                                                                                                                                                        Equations
                                                                                                                                                                                                                                                        Instances For

                                                                                                                                                                                                                                                          Filters an array of syntax, treating every other element as a separator rather than an element to test with the predicate p. The resulting array contains the tested elements for which p returns true, separated by the corresponding separator elements.

                                                                                                                                                                                                                                                          Equations
                                                                                                                                                                                                                                                          Instances For
                                                                                                                                                                                                                                                            def Lean.Syntax.TSepArray.push {k : SyntaxNodeKinds} {sep : String} (sa : TSepArray k sep) (e : TSyntax k) :
                                                                                                                                                                                                                                                            TSepArray k sep
                                                                                                                                                                                                                                                            Equations
                                                                                                                                                                                                                                                            Instances For
                                                                                                                                                                                                                                                              Equations
                                                                                                                                                                                                                                                              • One or more equations did not get rendered due to their size.
                                                                                                                                                                                                                                                              Instances For

                                                                                                                                                                                                                                                                Helper functions for manipulating interpolated strings #

                                                                                                                                                                                                                                                                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
                                                                                                                                                                                                                                                                    Equations
                                                                                                                                                                                                                                                                    • One or more equations did not get rendered due to their size.
                                                                                                                                                                                                                                                                    Instances For
                                                                                                                                                                                                                                                                      def Lean.TSyntax.getDocString (stx : TSyntax (List.cons `Lean.Parser.Command.docComment List.nil)) :
                                                                                                                                                                                                                                                                      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

                                                                                                                                                                                                                                                                          Controls which new mvars are turned in to goals by the apply tactic.

                                                                                                                                                                                                                                                                          • nonDependentFirst mvars that don't depend on other goals appear first in the goal list.
                                                                                                                                                                                                                                                                          • nonDependentOnly only mvars that don't depend on other goals are added to goal list.
                                                                                                                                                                                                                                                                          • all all unassigned mvars are added to the goal list.
                                                                                                                                                                                                                                                                          Instances For

                                                                                                                                                                                                                                                                            Configures the behaviour of the apply tactic.

                                                                                                                                                                                                                                                                            • newGoals : ApplyNewGoals
                                                                                                                                                                                                                                                                            • synthAssignedInstances : Bool

                                                                                                                                                                                                                                                                              If synthAssignedInstances is true, then apply will synthesize instance implicit arguments even if they have assigned by isDefEq, and then check whether the synthesized value matches the one inferred. The congr tactic sets this flag to false.

                                                                                                                                                                                                                                                                            • allowSynthFailures : Bool

                                                                                                                                                                                                                                                                              If allowSynthFailures is true, then apply will return instance implicit arguments for which typeclass search failed as new goals.

                                                                                                                                                                                                                                                                            • approx : Bool

                                                                                                                                                                                                                                                                              If approx := true, then we turn on isDefEq approximations. That is, we use the approxDefEq combinator.

                                                                                                                                                                                                                                                                            Instances For
                                                                                                                                                                                                                                                                              @[reducible, inline]

                                                                                                                                                                                                                                                                              Controls which new mvars are turned in to goals by the apply tactic.

                                                                                                                                                                                                                                                                              • nonDependentFirst mvars that don't depend on other goals appear first in the goal list.
                                                                                                                                                                                                                                                                              • nonDependentOnly only mvars that don't depend on other goals are added to goal list.
                                                                                                                                                                                                                                                                              • all all unassigned mvars are added to the goal list.
                                                                                                                                                                                                                                                                              Equations
                                                                                                                                                                                                                                                                              Instances For

                                                                                                                                                                                                                                                                                Configures the behavior of the rewrite and rw tactics.

                                                                                                                                                                                                                                                                                • transparency : TransparencyMode

                                                                                                                                                                                                                                                                                  The transparency mode to use for unfolding

                                                                                                                                                                                                                                                                                • offsetCnstrs : Bool

                                                                                                                                                                                                                                                                                  Whether to support offset constraints such as ?x + 1 =?= e

                                                                                                                                                                                                                                                                                • Which occurrences to rewrite

                                                                                                                                                                                                                                                                                • newGoals : NewGoals

                                                                                                                                                                                                                                                                                  How to convert the resulting metavariables into new goals

                                                                                                                                                                                                                                                                                Instances For

                                                                                                                                                                                                                                                                                  Configures the behaviour of the omega tactic.

                                                                                                                                                                                                                                                                                  • splitDisjunctions : Bool

                                                                                                                                                                                                                                                                                    Split disjunctions in the context.

                                                                                                                                                                                                                                                                                    Note that with splitDisjunctions := false omega will not be able to solve x = y goals as these are usually handled by introducing ¬ x = y as a hypothesis, then replacing this with x < y ∨ x > y.

                                                                                                                                                                                                                                                                                    On the other hand, omega does not currently detect disjunctions which, when split, introduce no new useful information, so the presence of irrelevant disjunctions in the context can significantly increase run time.

                                                                                                                                                                                                                                                                                  • splitNatSub : Bool

                                                                                                                                                                                                                                                                                    Whenever ((a - b : Nat) : Int) is found, register the disjunction b ≤ a ∧ ((a - b : Nat) : Int) = a - b ∨ a < b ∧ ((a - b : Nat) : Int) = 0 for later splitting.

                                                                                                                                                                                                                                                                                  • splitNatAbs : Bool

                                                                                                                                                                                                                                                                                    Whenever Int.natAbs a is found, register the disjunction 0 ≤ a ∧ Int.natAbs a = a ∨ a < 0 ∧ Int.natAbs a = - a for later splitting.

                                                                                                                                                                                                                                                                                  • splitMinMax : Bool

                                                                                                                                                                                                                                                                                    Whenever min a b or max a b is found, rewrite in terms of the definition if a ≤ b ..., for later case splitting.

                                                                                                                                                                                                                                                                                  Instances For
                                                                                                                                                                                                                                                                                    inductive Lean.Meta.CheckTactic.CheckGoalType {α : Sort u} (val : α) :

                                                                                                                                                                                                                                                                                    Type used to lift an arbitrary value into a type parameter so it can appear in a proof goal.

                                                                                                                                                                                                                                                                                    It is used by the #check_tactic command.

                                                                                                                                                                                                                                                                                    Instances For
                                                                                                                                                                                                                                                                                      partial def Lean.Parser.Tactic.getConfigItems (c : Syntax) :
                                                                                                                                                                                                                                                                                      TSyntaxArray (List.cons `Lean.Parser.Tactic.configItem List.nil)

                                                                                                                                                                                                                                                                                      Extracts the items from a tactic configuration, either a Lean.Parser.Tactic.optConfig, Lean.Parser.Tactic.config, or these wrapped in null nodes.

                                                                                                                                                                                                                                                                                      def Lean.Parser.Tactic.mkOptConfig (items : TSyntaxArray (List.cons `Lean.Parser.Tactic.configItem List.nil)) :
                                                                                                                                                                                                                                                                                      TSyntax (List.cons `Lean.Parser.Tactic.optConfig List.nil)
                                                                                                                                                                                                                                                                                      Equations
                                                                                                                                                                                                                                                                                      Instances For
                                                                                                                                                                                                                                                                                        def Lean.Parser.Tactic.appendConfig (cfg cfg' : Syntax) :
                                                                                                                                                                                                                                                                                        TSyntax (List.cons `Lean.Parser.Tactic.optConfig List.nil)

                                                                                                                                                                                                                                                                                        Appends two tactic configurations. The configurations can be Lean.Parser.Tactic.optConfig, Lean.Parser.Tactic.config, or these wrapped in null nodes (for example because the syntax is (config)?).

                                                                                                                                                                                                                                                                                        Equations
                                                                                                                                                                                                                                                                                        Instances For

                                                                                                                                                                                                                                                                                          erw [rules] is a shorthand for rw (transparency := .default) [rules]. This does rewriting up to unfolding of regular definitions (by comparison to regular rw which only unfolds @[reducible] definitions).

                                                                                                                                                                                                                                                                                          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
                                                                                                                                                                                                                                                                                              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

                                                                                                                                                                                                                                                                                                  simp! is shorthand for simp with autoUnfold := true. This will rewrite with all equation lemmas, which can be used to partially evaluate many definitions.

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

                                                                                                                                                                                                                                                                                                    simp_arith has been deprecated. It was a shorthand for simp +arith +decide. Note that +decide is not needed for reducing arithmetic terms since simprocs have been added to Lean.

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

                                                                                                                                                                                                                                                                                                      simp_arith! has been deprecated. It was a shorthand for simp! +arith +decide. Note that +decide is not needed for reducing arithmetic terms since simprocs have been added to Lean.

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

                                                                                                                                                                                                                                                                                                        simp_all! is shorthand for simp_all with autoUnfold := true. This will rewrite with all equation lemmas, which can be used to partially evaluate many definitions.

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

                                                                                                                                                                                                                                                                                                          simp_all_arith has been deprecated. It was a shorthand for simp_all +arith +decide. Note that +decide is not needed for reducing arithmetic terms since simprocs have been added to Lean.

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

                                                                                                                                                                                                                                                                                                            simp_all_arith! has been deprecated. It was a shorthand for simp_all! +arith +decide. Note that +decide is not needed for reducing arithmetic terms since simprocs have been added to Lean.

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

                                                                                                                                                                                                                                                                                                              dsimp! is shorthand for dsimp with autoUnfold := true. This will rewrite with all equation lemmas, which can be used to partially evaluate many definitions.

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