Loogle!
Result
Found 28 declarations mentioning Std.DTreeMap.Raw.Const.getD.
- Std.DTreeMap.Raw.Const.getD 📋 Std.Data.DTreeMap.Raw.Basic
{α : Type u} {cmp : α → α → Ordering} {β : Type v} (t : Std.DTreeMap.Raw α (fun x => β) cmp) (a : α) (fallback : β) : β - Std.DTreeMap.Raw.Const.getD_unitOfList 📋 Std.Data.DTreeMap.Raw.Lemmas
{α : Type u} {cmp : α → α → Ordering} {l : List α} {k : α} {fallback : Unit} : Std.DTreeMap.Raw.Const.getD (Std.DTreeMap.Raw.Const.unitOfList l cmp) k fallback = () - Std.DTreeMap.Raw.Const.getD_emptyc 📋 Std.Data.DTreeMap.Raw.Lemmas
{α : Type u} {cmp : α → α → Ordering} {β : Type v} [Std.TransCmp cmp] {a : α} {fallback : β} : Std.DTreeMap.Raw.Const.getD ∅ a fallback = fallback - Std.DTreeMap.Raw.Const.getD_erase_self 📋 Std.Data.DTreeMap.Raw.Lemmas
{α : Type u} {cmp : α → α → Ordering} {β : Type v} {t : Std.DTreeMap.Raw α (fun x => β) cmp} [Std.TransCmp cmp] (h : t.WF) {k : α} {fallback : β} : Std.DTreeMap.Raw.Const.getD (t.erase k) k fallback = fallback - Std.DTreeMap.Raw.Const.getD_eq_getD_get? 📋 Std.Data.DTreeMap.Raw.Lemmas
{α : Type u} {cmp : α → α → Ordering} {β : Type v} {t : Std.DTreeMap.Raw α (fun x => β) cmp} [Std.TransCmp cmp] (h : t.WF) {a : α} {fallback : β} : Std.DTreeMap.Raw.Const.getD t a fallback = (Std.DTreeMap.Raw.Const.get? t a).getD fallback - Std.DTreeMap.Raw.Const.getD_insert_self 📋 Std.Data.DTreeMap.Raw.Lemmas
{α : Type u} {cmp : α → α → Ordering} {β : Type v} {t : Std.DTreeMap.Raw α (fun x => β) cmp} [Std.TransCmp cmp] (h : t.WF) {k : α} {fallback v : β} : Std.DTreeMap.Raw.Const.getD (t.insert k v) k fallback = v - Std.DTreeMap.Raw.Const.get!_eq_getD_default 📋 Std.Data.DTreeMap.Raw.Lemmas
{α : Type u} {cmp : α → α → Ordering} {β : Type v} {t : Std.DTreeMap.Raw α (fun x => β) cmp} [Std.TransCmp cmp] [Inhabited β] (h : t.WF) {a : α} : Std.DTreeMap.Raw.Const.get! t a = Std.DTreeMap.Raw.Const.getD t a default - Std.DTreeMap.Raw.Const.getD_of_isEmpty 📋 Std.Data.DTreeMap.Raw.Lemmas
{α : Type u} {cmp : α → α → Ordering} {β : Type v} {t : Std.DTreeMap.Raw α (fun x => β) cmp} [Std.TransCmp cmp] (h : t.WF) {a : α} {fallback : β} : t.isEmpty = true → Std.DTreeMap.Raw.Const.getD t a fallback = fallback - Std.DTreeMap.Raw.Const.getD_eq_fallback_of_contains_eq_false 📋 Std.Data.DTreeMap.Raw.Lemmas
{α : Type u} {cmp : α → α → Ordering} {β : Type v} {t : Std.DTreeMap.Raw α (fun x => β) cmp} [Std.TransCmp cmp] (h : t.WF) {a : α} {fallback : β} : t.contains a = false → Std.DTreeMap.Raw.Const.getD t a fallback = fallback - Std.DTreeMap.Raw.Const.getD_eq_getD 📋 Std.Data.DTreeMap.Raw.Lemmas
{α : Type u} {cmp : α → α → Ordering} {β : Type v} {t : Std.DTreeMap.Raw α (fun x => β) cmp} [Std.TransCmp cmp] [Std.LawfulEqCmp cmp] (h : t.WF) {a : α} {fallback : β} : Std.DTreeMap.Raw.Const.getD t a fallback = t.getD a fallback - Std.DTreeMap.Raw.Const.getD_congr 📋 Std.Data.DTreeMap.Raw.Lemmas
{α : Type u} {cmp : α → α → Ordering} {β : Type v} {t : Std.DTreeMap.Raw α (fun x => β) cmp} [Std.TransCmp cmp] (h : t.WF) {a b : α} {fallback : β} (hab : cmp a b = Ordering.eq) : Std.DTreeMap.Raw.Const.getD t a fallback = Std.DTreeMap.Raw.Const.getD t b fallback - Std.DTreeMap.Raw.Const.getD_insertManyIfNewUnit_list 📋 Std.Data.DTreeMap.Raw.Lemmas
{α : Type u} {cmp : α → α → Ordering} {t : Std.DTreeMap.Raw α (fun x => Unit) cmp} {l : List α} {k : α} {fallback : Unit} : Std.DTreeMap.Raw.Const.getD (Std.DTreeMap.Raw.Const.insertManyIfNewUnit t l) k fallback = () - Std.DTreeMap.Raw.Const.getD_eq_fallback 📋 Std.Data.DTreeMap.Raw.Lemmas
{α : Type u} {cmp : α → α → Ordering} {β : Type v} {t : Std.DTreeMap.Raw α (fun x => β) cmp} [Std.TransCmp cmp] (h : t.WF) {a : α} {fallback : β} : a ∉ t → Std.DTreeMap.Raw.Const.getD t a fallback = fallback - Std.DTreeMap.Raw.Const.get?_eq_some_getD_of_contains 📋 Std.Data.DTreeMap.Raw.Lemmas
{α : Type u} {cmp : α → α → Ordering} {β : Type v} {t : Std.DTreeMap.Raw α (fun x => β) cmp} [Std.TransCmp cmp] (h : t.WF) {a : α} {fallback : β} : t.contains a = true → Std.DTreeMap.Raw.Const.get? t a = some (Std.DTreeMap.Raw.Const.getD t a fallback) - Std.DTreeMap.Raw.Const.getD_alter_self 📋 Std.Data.DTreeMap.Raw.Lemmas
{α : Type u} {cmp : α → α → Ordering} {β : Type v} {t : Std.DTreeMap.Raw α (fun x => β) cmp} [Std.TransCmp cmp] (h : t.WF) {k : α} {fallback : β} {f : Option β → Option β} : Std.DTreeMap.Raw.Const.getD (Std.DTreeMap.Raw.Const.alter t k f) k fallback = (f (Std.DTreeMap.Raw.Const.get? t k)).getD fallback - Std.DTreeMap.Raw.Const.getD_ofList_of_contains_eq_false 📋 Std.Data.DTreeMap.Raw.Lemmas
{α : Type u} {cmp : α → α → Ordering} {β : Type v} [Std.TransCmp cmp] [BEq α] [Std.LawfulBEqCmp cmp] {l : List (α × β)} {k : α} {fallback : β} (contains_eq_false : (List.map Prod.fst l).contains k = false) : Std.DTreeMap.Raw.Const.getD (Std.DTreeMap.Raw.Const.ofList l cmp) k fallback = fallback - Std.DTreeMap.Raw.Const.getD_modify_self 📋 Std.Data.DTreeMap.Raw.Lemmas
{α : Type u} {cmp : α → α → Ordering} [Std.TransCmp cmp] {β : Type v} {t : Std.DTreeMap.Raw α (fun x => β) cmp} (h : t.WF) {k : α} {fallback : β} {f : β → β} : Std.DTreeMap.Raw.Const.getD (Std.DTreeMap.Raw.Const.modify t k f) k fallback = (Option.map f (Std.DTreeMap.Raw.Const.get? t k)).getD fallback - Std.DTreeMap.Raw.Const.get_eq_getD 📋 Std.Data.DTreeMap.Raw.Lemmas
{α : Type u} {cmp : α → α → Ordering} {β : Type v} {t : Std.DTreeMap.Raw α (fun x => β) cmp} [Std.TransCmp cmp] (h : t.WF) {a : α} {fallback : β} {h' : a ∈ t} : Std.DTreeMap.Raw.Const.get t a h' = Std.DTreeMap.Raw.Const.getD t a fallback - Std.DTreeMap.Raw.Const.get?_eq_some_getD 📋 Std.Data.DTreeMap.Raw.Lemmas
{α : Type u} {cmp : α → α → Ordering} {β : Type v} {t : Std.DTreeMap.Raw α (fun x => β) cmp} [Std.TransCmp cmp] (h : t.WF) {a : α} {fallback : β} : a ∈ t → Std.DTreeMap.Raw.Const.get? t a = some (Std.DTreeMap.Raw.Const.getD t a fallback) - Std.DTreeMap.Raw.Const.getD_erase 📋 Std.Data.DTreeMap.Raw.Lemmas
{α : Type u} {cmp : α → α → Ordering} {β : Type v} {t : Std.DTreeMap.Raw α (fun x => β) cmp} [Std.TransCmp cmp] (h : t.WF) {k a : α} {fallback : β} : Std.DTreeMap.Raw.Const.getD (t.erase k) a fallback = if cmp k a = Ordering.eq then fallback else Std.DTreeMap.Raw.Const.getD t a fallback - Std.DTreeMap.Raw.Const.getD_insert 📋 Std.Data.DTreeMap.Raw.Lemmas
{α : Type u} {cmp : α → α → Ordering} {β : Type v} {t : Std.DTreeMap.Raw α (fun x => β) cmp} [Std.TransCmp cmp] (h : t.WF) {k a : α} {fallback v : β} : Std.DTreeMap.Raw.Const.getD (t.insert k v) a fallback = if cmp k a = Ordering.eq then v else Std.DTreeMap.Raw.Const.getD t a fallback - Std.DTreeMap.Raw.Const.getD_alter 📋 Std.Data.DTreeMap.Raw.Lemmas
{α : Type u} {cmp : α → α → Ordering} {β : Type v} {t : Std.DTreeMap.Raw α (fun x => β) cmp} [Std.TransCmp cmp] (h : t.WF) {k k' : α} {fallback : β} {f : Option β → Option β} : Std.DTreeMap.Raw.Const.getD (Std.DTreeMap.Raw.Const.alter t k f) k' fallback = if cmp k k' = Ordering.eq then (f (Std.DTreeMap.Raw.Const.get? t k)).getD fallback else Std.DTreeMap.Raw.Const.getD t k' fallback - Std.DTreeMap.Raw.Const.getD_modify 📋 Std.Data.DTreeMap.Raw.Lemmas
{α : Type u} {cmp : α → α → Ordering} [Std.TransCmp cmp] {β : Type v} {t : Std.DTreeMap.Raw α (fun x => β) cmp} (h : t.WF) {k k' : α} {fallback : β} {f : β → β} : Std.DTreeMap.Raw.Const.getD (Std.DTreeMap.Raw.Const.modify t k f) k' fallback = if cmp k k' = Ordering.eq then (Option.map f (Std.DTreeMap.Raw.Const.get? t k)).getD fallback else Std.DTreeMap.Raw.Const.getD t k' fallback - Std.DTreeMap.Raw.Const.getD_ofList_of_mem 📋 Std.Data.DTreeMap.Raw.Lemmas
{α : Type u} {cmp : α → α → Ordering} {β : Type v} [Std.TransCmp cmp] {l : List (α × β)} {k k' : α} (k_eq : cmp k k' = Ordering.eq) {v fallback : β} (distinct : List.Pairwise (fun a b => ¬cmp a.1 b.1 = Ordering.eq) l) (mem : (k, v) ∈ l) : Std.DTreeMap.Raw.Const.getD (Std.DTreeMap.Raw.Const.ofList l cmp) k' fallback = v - Std.DTreeMap.Raw.Const.getD_insertMany_list_of_contains_eq_false 📋 Std.Data.DTreeMap.Raw.Lemmas
{α : Type u} {cmp : α → α → Ordering} {β : Type v} {t : Std.DTreeMap.Raw α (fun x => β) cmp} [Std.TransCmp cmp] [BEq α] [Std.LawfulBEqCmp cmp] (h : t.WF) {l : List (α × β)} {k : α} {fallback : β} (contains_eq_false : (List.map Prod.fst l).contains k = false) : Std.DTreeMap.Raw.Const.getD (Std.DTreeMap.Raw.Const.insertMany t l) k fallback = Std.DTreeMap.Raw.Const.getD t k fallback - Std.DTreeMap.Raw.Const.getD_insertIfNew 📋 Std.Data.DTreeMap.Raw.Lemmas
{α : Type u} {cmp : α → α → Ordering} {β : Type v} {t : Std.DTreeMap.Raw α (fun x => β) cmp} [Std.TransCmp cmp] (h : t.WF) {k a : α} {fallback v : β} : Std.DTreeMap.Raw.Const.getD (t.insertIfNew k v) a fallback = if cmp k a = Ordering.eq ∧ k ∉ t then v else Std.DTreeMap.Raw.Const.getD t a fallback - Std.DTreeMap.Raw.Const.getD_insertMany_list_of_mem 📋 Std.Data.DTreeMap.Raw.Lemmas
{α : Type u} {cmp : α → α → Ordering} {β : Type v} {t : Std.DTreeMap.Raw α (fun x => β) cmp} [Std.TransCmp cmp] (h : t.WF) {l : List (α × β)} {k k' : α} (k_eq : cmp k k' = Ordering.eq) {v fallback : β} (distinct : List.Pairwise (fun a b => ¬cmp a.1 b.1 = Ordering.eq) l) (mem : (k, v) ∈ l) : Std.DTreeMap.Raw.Const.getD (Std.DTreeMap.Raw.Const.insertMany t l) k' fallback = v - Std.DTreeMap.Raw.Const.getD_insertMany_list 📋 Std.Data.DTreeMap.Raw.Lemmas
{α : Type u} {cmp : α → α → Ordering} {β : Type v} {t : Std.DTreeMap.Raw α (fun x => β) cmp} [Std.TransCmp cmp] [BEq α] [Std.LawfulBEqCmp cmp] (h : t.WF) {l : List (α × β)} {k : α} {fallback : β} : Std.DTreeMap.Raw.Const.getD (Std.DTreeMap.Raw.Const.insertMany t l) k fallback = (List.findSomeRev? (fun x => match x with | (a, b) => if cmp a k = Ordering.eq then some b else none) l).getD (Std.DTreeMap.Raw.Const.getD t k fallback)
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:
By constant:
🔍Real.sin
finds all lemmas whose statement somehow mentions the sine function.By lemma name substring:
🔍"differ"
finds all lemmas that have"differ"
somewhere in their lemma name.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
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 findtsum_lt_tsum
even though the hypothesisf 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 19971e9
serving mathlib revision bce1d65