Loogle!

_ * (_ ^ _)

Result

Found 3381 declarations mentioning HMul.hMul and HPow.hPow. Of these, 1541 match your pattern(s). Of these, only the first 200 are shown.

About

Loogle searches Lean and Mathlib definitions and theorems.

You can use Loogle from within the Lean4 VSCode language extension using (by default) Ctrl-K Ctrl-S. You can also try the #loogle command from LeanSearchClient, the CLI version, the Loogle VS Code extension, the lean.nvim integration or the Zulip bot.

Usage

Loogle finds definitions and lemmas in various ways:

  1. By constant:
    πŸ” Real.sin
    finds all lemmas whose statement somehow mentions the sine function.

  2. By lemma name substring:
    πŸ” "differ"
    finds all lemmas that have "differ" somewhere in their lemma name.

  3. By subexpression:
    πŸ” _ * (_ ^ _)
    finds all lemmas whose statements somewhere include a product where the second argument is raised to some power.

    The pattern can also be non-linear, as in
    πŸ” Real.sqrt ?a * Real.sqrt ?a

    If the pattern has parameters, they are matched in any order. Both of these will find List.map:
    πŸ” (?a -> ?b) -> List ?a -> List ?b
    πŸ” List ?a -> (?a -> ?b) -> List ?b

  4. By main conclusion:
    πŸ” |- tsum _ = _ * tsum _
    finds all lemmas where the conclusion (the subexpression to the right of all β†’ and βˆ€) has the given shape.

    As before, if the pattern has parameters, they are matched against the hypotheses of the lemma in any order; for example,
    πŸ” |- _ < _ β†’ tsum _ < tsum _
    will find tsum_lt_tsum even though the hypothesis f i < g i is not the last.

If you pass more than one such search filter, separated by commas Loogle will return lemmas which match all of them. The search
πŸ” Real.sin, "two", tsum, _ * _, _ ^ _, |- _ < _ β†’ _
would find all lemmas which mention the constants Real.sin and tsum, have "two" as a substring of the lemma name, include a product and a power somewhere in the type, and have a hypothesis of the form _ < _ (if there were any such lemmas). Metavariables (?a) are assigned independently in each filter.

The #lucky button will directly send you to the documentation of the first hit.

Source code

You can find the source code for this service at https://github.com/nomeata/loogle. The https://loogle.lean-lang.org/ service is provided by the Lean FRO.

This is Loogle revision ad0d2bb serving mathlib revision dc82ad5