path
stringlengths
12
84
imports
sequencelengths
0
4.45k
premises
listlengths
0
625
Mathlib/Data/Rbtree/Find.lean
[ "Mathlib/Mathport/Rename.lean", ".lake/packages/lean4/src/lean/Init.lean" ]
[]
Mathlib/Combinatorics/SimpleGraph/StronglyRegular.lean
[ "Mathlib/Combinatorics/Enumerative/DoubleCounting.lean", "Mathlib/Combinatorics/SimpleGraph/Basic.lean", ".lake/packages/lean4/src/lean/Init.lean", "Mathlib/Data/Set/Finite.lean", "Mathlib/Combinatorics/SimpleGraph/AdjMatrix.lean" ]
[ { "full_name": "SimpleGraph.IsSRGWith", "code": "structure IsSRGWith (n k β„“ ΞΌ : β„•) : Prop where\n card : Fintype.card V = n\n regular : G.IsRegularOfDegree k\n of_adj : βˆ€ v w : V, G.Adj v w β†’ Fintype.card (G.commonNeighbors v w) = β„“\n of_not_adj : Pairwise fun v w => Β¬G.Adj v w β†’ Fintype.card (G.commonNeighbors v w) = ΞΌ", "start": [ 43, 1 ], "end": [ 53, 89 ], "kind": "commanddeclaration" }, { "full_name": "SimpleGraph.bot_strongly_regular", "code": "theorem bot_strongly_regular : (βŠ₯ : SimpleGraph V).IsSRGWith (Fintype.card V) 0 β„“ 0 where", "start": [ 59, 1 ], "end": [ 68, 31 ], "kind": "commanddeclaration" }, { "full_name": "SimpleGraph.IsSRGWith.top", "code": "theorem IsSRGWith.top :\n (⊀ : SimpleGraph V).IsSRGWith (Fintype.card V) (Fintype.card V - 1) (Fintype.card V - 2) ΞΌ where", "start": [ 71, 1 ], "end": [ 80, 68 ], "kind": "commanddeclaration" }, { "full_name": "SimpleGraph.IsSRGWith.card_neighborFinset_union_eq", "code": "theorem IsSRGWith.card_neighborFinset_union_eq {v w : V} (h : G.IsSRGWith n k β„“ ΞΌ) :\n (G.neighborFinset v βˆͺ G.neighborFinset w).card =\n 2 * k - Fintype.card (G.commonNeighbors v w)", "start": [ 84, 1 ], "end": [ 95, 40 ], "kind": "commanddeclaration" }, { "full_name": "SimpleGraph.IsSRGWith.card_neighborFinset_union_of_not_adj", "code": "theorem IsSRGWith.card_neighborFinset_union_of_not_adj {v w : V} (h : G.IsSRGWith n k β„“ ΞΌ)\n (hne : v β‰  w) (ha : Β¬G.Adj v w) :\n (G.neighborFinset v βˆͺ G.neighborFinset w).card = 2 * k - ΞΌ", "start": [ 99, 1 ], "end": [ 106, 39 ], "kind": "commanddeclaration" }, { "full_name": "SimpleGraph.IsSRGWith.card_neighborFinset_union_of_adj", "code": "theorem IsSRGWith.card_neighborFinset_union_of_adj {v w : V} (h : G.IsSRGWith n k β„“ ΞΌ)\n (ha : G.Adj v w) : (G.neighborFinset v βˆͺ G.neighborFinset w).card = 2 * k - β„“", "start": [ 110, 1 ], "end": [ 113, 39 ], "kind": "commanddeclaration" }, { "full_name": "SimpleGraph.compl_neighborFinset_sdiff_inter_eq", "code": "theorem compl_neighborFinset_sdiff_inter_eq {v w : V} :\n (G.neighborFinset v)ᢜ \\ {v} ∩ ((G.neighborFinset w)ᢜ \\ {w}) =\n ((G.neighborFinset v)ᢜ ∩ (G.neighborFinset w)ᢜ) \\ ({w} βˆͺ {v})", "start": [ 117, 1 ], "end": [ 122, 57 ], "kind": "commanddeclaration" }, { "full_name": "SimpleGraph.sdiff_compl_neighborFinset_inter_eq", "code": "theorem sdiff_compl_neighborFinset_inter_eq {v w : V} (h : G.Adj v w) :\n ((G.neighborFinset v)ᢜ ∩ (G.neighborFinset w)ᢜ) \\ ({w} βˆͺ {v}) =\n (G.neighborFinset v)ᢜ ∩ (G.neighborFinset w)ᢜ", "start": [ 125, 1 ], "end": [ 134, 19 ], "kind": "commanddeclaration" }, { "full_name": "SimpleGraph.IsSRGWith.compl_is_regular", "code": "theorem IsSRGWith.compl_is_regular (h : G.IsSRGWith n k β„“ ΞΌ) :\n Gᢜ.IsRegularOfDegree (n - k - 1)", "start": [ 137, 1 ], "end": [ 140, 24 ], "kind": "commanddeclaration" }, { "full_name": "SimpleGraph.IsSRGWith.card_commonNeighbors_eq_of_adj_compl", "code": "theorem IsSRGWith.card_commonNeighbors_eq_of_adj_compl (h : G.IsSRGWith n k β„“ ΞΌ) {v w : V}\n (ha : Gᢜ.Adj v w) : Fintype.card (Gᢜ.commonNeighbors v w) = n - (2 * k - ΞΌ) - 2", "start": [ 144, 1 ], "end": [ 156, 55 ], "kind": "commanddeclaration" }, { "full_name": "SimpleGraph.IsSRGWith.card_commonNeighbors_eq_of_not_adj_compl", "code": "theorem IsSRGWith.card_commonNeighbors_eq_of_not_adj_compl (h : G.IsSRGWith n k β„“ ΞΌ) {v w : V}\n (hn : v β‰  w) (hna : Β¬Gᢜ.Adj v w) :\n Fintype.card (Gᢜ.commonNeighbors v w) = n - (2 * k - β„“)", "start": [ 160, 1 ], "end": [ 168, 87 ], "kind": "commanddeclaration" }, { "full_name": "SimpleGraph.IsSRGWith.compl", "code": "theorem IsSRGWith.compl (h : G.IsSRGWith n k β„“ ΞΌ) :\n Gᢜ.IsSRGWith n (n - k - 1) (n - (2 * k - ΞΌ) - 2) (n - (2 * k - β„“)) where", "start": [ 172, 1 ], "end": [ 178, 86 ], "kind": "commanddeclaration" }, { "full_name": "SimpleGraph.IsSRGWith.param_eq", "code": "theorem IsSRGWith.param_eq (h : G.IsSRGWith n k β„“ ΞΌ) (hn : 0 < n) :\n k * (k - β„“ - 1) = (n - k - 1) * ΞΌ", "start": [ 182, 1 ], "end": [ 215, 11 ], "kind": "commanddeclaration" }, { "full_name": "SimpleGraph.IsSRGWith.matrix_eq", "code": "theorem IsSRGWith.matrix_eq {Ξ± : Type*} [Semiring Ξ±] (h : G.IsSRGWith n k β„“ ΞΌ) :\n G.adjMatrix Ξ± ^ 2 = k β€’ (1 : Matrix V V Ξ±) + β„“ β€’ G.adjMatrix Ξ± + ΞΌ β€’ Gᢜ.adjMatrix Ξ±", "start": [ 217, 1 ], "end": [ 235, 30 ], "kind": "commanddeclaration" } ]
Mathlib/LinearAlgebra/TensorProduct/DirectLimit.lean
[ ".lake/packages/lean4/src/lean/Init.lean", "Mathlib/Algebra/DirectLimit.lean" ]
[ { "full_name": "TensorProduct.fromDirectLimit", "code": "noncomputable def fromDirectLimit :\n DirectLimit (G Β· βŠ—[R] M) (f β–· M) β†’β‚—[R] DirectLimit G f βŠ—[R] M :=\n DirectLimit.lift _ _ _ _ (fun _ ↦ (of _ _ _ _ _).rTensor M)\n fun _ _ _ x ↦ by refine x.induction_on ?_ ?_ ?_ <;> aesop", "start": [ 39, 1 ], "end": [ 46, 62 ], "kind": "commanddeclaration" }, { "full_name": "TensorProduct.fromDirectLimit_of_tmul", "code": "@[simp] lemma fromDirectLimit_of_tmul {i : ΞΉ} (g : G i) (m : M) :\n fromDirectLimit f M (of _ _ _ _ i (g βŠ—β‚œ m)) = (of _ _ _ f i g) βŠ—β‚œ m :=\n lift_of (G := (G Β· βŠ—[R] M)) _ _ (g βŠ—β‚œ m)", "start": [ 49, 1 ], "end": [ 51, 43 ], "kind": "lemma" }, { "full_name": "TensorProduct.toDirectLimit", "code": "noncomputable def toDirectLimit : DirectLimit G f βŠ—[R] M β†’β‚—[R] DirectLimit (G Β· βŠ—[R] M) (f β–· M) :=\n TensorProduct.lift <| DirectLimit.lift _ _ _ _\n (fun i ↦\n (TensorProduct.mk R _ _).comprβ‚‚ (of R ΞΉ _ (fun _i _j h ↦ (f _ _ h).rTensor M) i))\n fun _ _ _ g ↦ DFunLike.ext _ _ (of_f (G := (G Β· βŠ—[R] M)) (x := g βŠ—β‚œ Β·))", "start": [ 53, 1 ], "end": [ 62, 76 ], "kind": "commanddeclaration" }, { "full_name": "TensorProduct.toDirectLimit_tmul_of", "code": "@[simp] lemma toDirectLimit_tmul_of\n {i : ΞΉ} (g : G i) (m : M) :\n (toDirectLimit f M <| (of _ _ G f i g) βŠ—β‚œ m) = (of _ _ _ _ i (g βŠ—β‚œ m)) := by\n rw [toDirectLimit, lift.tmul, lift_of]\n rfl", "start": [ 65, 1 ], "end": [ 69, 6 ], "kind": "lemma" }, { "full_name": "TensorProduct.directLimitLeft", "code": "noncomputable def directLimitLeft :\n DirectLimit G f βŠ—[R] M ≃ₗ[R] DirectLimit (G Β· βŠ—[R] M) (f β–· M) := by\n refine LinearEquiv.ofLinear (toDirectLimit f M) (fromDirectLimit f M) ?_ ?_\n <;> cases isEmpty_or_nonempty ΞΉ\n Β· ext; apply Subsingleton.elim\n Β· refine DFunLike.ext _ _ fun x ↦ x.induction_on fun i g ↦ g.induction_on ?_ ?_ ?_ <;> aesop\n Β· ext; apply Subsingleton.elim\n Β· exact ext (DFunLike.ext _ _ fun g ↦ DFunLike.ext _ _ fun _ ↦ g.induction_on <| by aesop)", "start": [ 73, 1 ], "end": [ 83, 93 ], "kind": "commanddeclaration" }, { "full_name": "TensorProduct.directLimitLeft_tmul_of", "code": "@[simp] lemma directLimitLeft_tmul_of {i : ΞΉ} (g : G i) (m : M) :\n directLimitLeft f M (of _ _ _ _ _ g βŠ—β‚œ m) = of _ _ _ (f β–· M) _ (g βŠ—β‚œ m) :=\n toDirectLimit_tmul_of f g m", "start": [ 85, 1 ], "end": [ 87, 30 ], "kind": "lemma" }, { "full_name": "TensorProduct.directLimitLeft_symm_of_tmul", "code": "@[simp] lemma directLimitLeft_symm_of_tmul {i : ΞΉ} (g : G i) (m : M) :\n (directLimitLeft f M).symm (of _ _ _ _ _ (g βŠ—β‚œ m)) = of _ _ _ f _ g βŠ—β‚œ m :=\n fromDirectLimit_of_tmul f g m", "start": [ 89, 1 ], "end": [ 91, 32 ], "kind": "lemma" }, { "full_name": "TensorProduct.directLimitRight", "code": "noncomputable def directLimitRight :\n M βŠ—[R] DirectLimit G f ≃ₗ[R] DirectLimit (M βŠ—[R] G Β·) (M ◁ f) :=\n TensorProduct.comm _ _ _ β‰ͺ≫ₗ directLimitLeft f M β‰ͺ≫ₗ\n Module.DirectLimit.congr (fun i ↦ TensorProduct.comm _ _ _)\n (fun i j h ↦ TensorProduct.ext <| DFunLike.ext _ _ <| by aesop)", "start": [ 93, 1 ], "end": [ 100, 70 ], "kind": "commanddeclaration" }, { "full_name": "TensorProduct.directLimitRight_tmul_of", "code": "@[simp] lemma directLimitRight_tmul_of {i : ΞΉ} (m : M) (g : G i):\n directLimitRight f M (m βŠ—β‚œ of _ _ _ _ _ g) = of _ _ _ _ i (m βŠ—β‚œ g) := by\n simp [directLimitRight, congr_apply_of]", "start": [ 102, 1 ], "end": [ 104, 42 ], "kind": "lemma" }, { "full_name": "TensorProduct.directLimitRight_symm_of_tmul", "code": "@[simp] lemma directLimitRight_symm_of_tmul {i : ΞΉ} (m : M) (g : G i) :\n (directLimitRight f M).symm (of _ _ _ _ _ (m βŠ—β‚œ g)) = m βŠ—β‚œ of _ _ _ f _ g := by\n simp [directLimitRight, congr_symm_apply_of]", "start": [ 106, 1 ], "end": [ 108, 47 ], "kind": "lemma" } ]
Mathlib/Analysis/Convex/Quasiconvex.lean
[ ".lake/packages/lean4/src/lean/Init.lean", "Mathlib/Analysis/Convex/Function.lean" ]
[ { "full_name": "QuasiconvexOn", "code": "def QuasiconvexOn : Prop :=\n βˆ€ r, Convex π•œ ({ x ∈ s | f x ≀ r })", "start": [ 48, 1 ], "end": [ 51, 38 ], "kind": "commanddeclaration" }, { "full_name": "QuasiconcaveOn", "code": "def QuasiconcaveOn : Prop :=\n βˆ€ r, Convex π•œ ({ x ∈ s | r ≀ f x })", "start": [ 54, 1 ], "end": [ 57, 38 ], "kind": "commanddeclaration" }, { "full_name": "QuasilinearOn", "code": "def QuasilinearOn : Prop :=\n QuasiconvexOn π•œ s f ∧ QuasiconcaveOn π•œ s f", "start": [ 60, 1 ], "end": [ 64, 45 ], "kind": "commanddeclaration" }, { "full_name": "QuasiconvexOn.dual", "code": "theorem QuasiconvexOn.dual : QuasiconvexOn π•œ s f β†’ QuasiconcaveOn π•œ s (toDual ∘ f)", "start": [ 69, 1 ], "end": [ 70, 5 ], "kind": "commanddeclaration" }, { "full_name": "QuasiconcaveOn.dual", "code": "theorem QuasiconcaveOn.dual : QuasiconcaveOn π•œ s f β†’ QuasiconvexOn π•œ s (toDual ∘ f)", "start": [ 73, 1 ], "end": [ 74, 5 ], "kind": "commanddeclaration" }, { "full_name": "QuasilinearOn.dual", "code": "theorem QuasilinearOn.dual : QuasilinearOn π•œ s f β†’ QuasilinearOn π•œ s (toDual ∘ f)", "start": [ 77, 1 ], "end": [ 78, 11 ], "kind": "commanddeclaration" }, { "full_name": "Convex.quasiconvexOn_of_convex_le", "code": "theorem Convex.quasiconvexOn_of_convex_le (hs : Convex π•œ s) (h : βˆ€ r, Convex π•œ { x | f x ≀ r }) :\n QuasiconvexOn π•œ s f", "start": [ 81, 1 ], "end": [ 82, 51 ], "kind": "commanddeclaration" }, { "full_name": "Convex.quasiconcaveOn_of_convex_ge", "code": "theorem Convex.quasiconcaveOn_of_convex_ge (hs : Convex π•œ s) (h : βˆ€ r, Convex π•œ { x | r ≀ f x }) :\n QuasiconcaveOn π•œ s f", "start": [ 85, 1 ], "end": [ 87, 62 ], "kind": "commanddeclaration" }, { "full_name": "QuasiconvexOn.convex", "code": "theorem QuasiconvexOn.convex [IsDirected Ξ² (Β· ≀ Β·)] (hf : QuasiconvexOn π•œ s f) : Convex π•œ s", "start": [ 90, 1 ], "end": [ 93, 41 ], "kind": "commanddeclaration" }, { "full_name": "QuasiconcaveOn.convex", "code": "theorem QuasiconcaveOn.convex [IsDirected Ξ² (Β· β‰₯ Β·)] (hf : QuasiconcaveOn π•œ s f) : Convex π•œ s", "start": [ 96, 1 ], "end": [ 97, 17 ], "kind": "commanddeclaration" }, { "full_name": "QuasiconvexOn.sup", "code": "theorem QuasiconvexOn.sup [SemilatticeSup Ξ²] (hf : QuasiconvexOn π•œ s f)\n (hg : QuasiconvexOn π•œ s g) : QuasiconvexOn π•œ s (f βŠ” g)", "start": [ 106, 1 ], "end": [ 110, 28 ], "kind": "commanddeclaration" }, { "full_name": "QuasiconcaveOn.inf", "code": "theorem QuasiconcaveOn.inf [SemilatticeInf Ξ²] (hf : QuasiconcaveOn π•œ s f)\n (hg : QuasiconcaveOn π•œ s g) : QuasiconcaveOn π•œ s (f βŠ“ g)", "start": [ 113, 1 ], "end": [ 115, 17 ], "kind": "commanddeclaration" }, { "full_name": "quasiconvexOn_iff_le_max", "code": "theorem quasiconvexOn_iff_le_max : QuasiconvexOn π•œ s f ↔ Convex π•œ s ∧ βˆ€ ⦃x⦄, x ∈ s β†’ βˆ€ ⦃y⦄,\n y ∈ s β†’ βˆ€ ⦃a b : π•œβ¦„, 0 ≀ a β†’ 0 ≀ b β†’ a + b = 1 β†’ f (a β€’ x + b β€’ y) ≀ max (f x) (f y)", "start": [ 124, 1 ], "end": [ 130, 86 ], "kind": "commanddeclaration" }, { "full_name": "quasiconcaveOn_iff_min_le", "code": "theorem quasiconcaveOn_iff_min_le : QuasiconcaveOn π•œ s f ↔ Convex π•œ s ∧ βˆ€ ⦃x⦄, x ∈ s β†’ βˆ€ ⦃y⦄,\n y ∈ s β†’ βˆ€ ⦃a b : π•œβ¦„, 0 ≀ a β†’ 0 ≀ b β†’ a + b = 1 β†’ min (f x) (f y) ≀ f (a β€’ x + b β€’ y)", "start": [ 133, 1 ], "end": [ 135, 48 ], "kind": "commanddeclaration" }, { "full_name": "quasilinearOn_iff_mem_uIcc", "code": "theorem quasilinearOn_iff_mem_uIcc : QuasilinearOn π•œ s f ↔ Convex π•œ s ∧ βˆ€ ⦃x⦄, x ∈ s β†’ βˆ€ ⦃y⦄,\n y ∈ s β†’ βˆ€ ⦃a b : π•œβ¦„, 0 ≀ a β†’ 0 ≀ b β†’ a + b = 1 β†’ f (a β€’ x + b β€’ y) ∈ uIcc (f x) (f y)", "start": [ 138, 1 ], "end": [ 143, 59 ], "kind": "commanddeclaration" }, { "full_name": "QuasiconvexOn.convex_lt", "code": "theorem QuasiconvexOn.convex_lt (hf : QuasiconvexOn π•œ s f) (r : Ξ²) :\n Convex π•œ ({ x ∈ s | f x < r })", "start": [ 146, 1 ], "end": [ 150, 48 ], "kind": "commanddeclaration" }, { "full_name": "QuasiconcaveOn.convex_gt", "code": "theorem QuasiconcaveOn.convex_gt (hf : QuasiconcaveOn π•œ s f) (r : Ξ²) :\n Convex π•œ ({ x ∈ s | r < f x })", "start": [ 153, 1 ], "end": [ 155, 22 ], "kind": "commanddeclaration" }, { "full_name": "ConvexOn.quasiconvexOn", "code": "theorem ConvexOn.quasiconvexOn (hf : ConvexOn π•œ s f) : QuasiconvexOn π•œ s f", "start": [ 165, 1 ], "end": [ 166, 15 ], "kind": "commanddeclaration" }, { "full_name": "ConcaveOn.quasiconcaveOn", "code": "theorem ConcaveOn.quasiconcaveOn (hf : ConcaveOn π•œ s f) : QuasiconcaveOn π•œ s f", "start": [ 169, 1 ], "end": [ 170, 15 ], "kind": "commanddeclaration" }, { "full_name": "MonotoneOn.quasiconvexOn", "code": "theorem MonotoneOn.quasiconvexOn (hf : MonotoneOn f s) (hs : Convex π•œ s) : QuasiconvexOn π•œ s f", "start": [ 182, 1 ], "end": [ 183, 18 ], "kind": "commanddeclaration" }, { "full_name": "MonotoneOn.quasiconcaveOn", "code": "theorem MonotoneOn.quasiconcaveOn (hf : MonotoneOn f s) (hs : Convex π•œ s) : QuasiconcaveOn π•œ s f", "start": [ 186, 1 ], "end": [ 187, 18 ], "kind": "commanddeclaration" }, { "full_name": "MonotoneOn.quasilinearOn", "code": "theorem MonotoneOn.quasilinearOn (hf : MonotoneOn f s) (hs : Convex π•œ s) : QuasilinearOn π•œ s f", "start": [ 190, 1 ], "end": [ 191, 46 ], "kind": "commanddeclaration" }, { "full_name": "AntitoneOn.quasiconvexOn", "code": "theorem AntitoneOn.quasiconvexOn (hf : AntitoneOn f s) (hs : Convex π•œ s) : QuasiconvexOn π•œ s f", "start": [ 194, 1 ], "end": [ 195, 18 ], "kind": "commanddeclaration" }, { "full_name": "AntitoneOn.quasiconcaveOn", "code": "theorem AntitoneOn.quasiconcaveOn (hf : AntitoneOn f s) (hs : Convex π•œ s) : QuasiconcaveOn π•œ s f", "start": [ 198, 1 ], "end": [ 199, 18 ], "kind": "commanddeclaration" }, { "full_name": "AntitoneOn.quasilinearOn", "code": "theorem AntitoneOn.quasilinearOn (hf : AntitoneOn f s) (hs : Convex π•œ s) : QuasilinearOn π•œ s f", "start": [ 202, 1 ], "end": [ 203, 46 ], "kind": "commanddeclaration" }, { "full_name": "Monotone.quasiconvexOn", "code": "theorem Monotone.quasiconvexOn (hf : Monotone f) : QuasiconvexOn π•œ univ f", "start": [ 206, 1 ], "end": [ 207, 46 ], "kind": "commanddeclaration" }, { "full_name": "Monotone.quasiconcaveOn", "code": "theorem Monotone.quasiconcaveOn (hf : Monotone f) : QuasiconcaveOn π•œ univ f", "start": [ 210, 1 ], "end": [ 211, 47 ], "kind": "commanddeclaration" }, { "full_name": "Monotone.quasilinearOn", "code": "theorem Monotone.quasilinearOn (hf : Monotone f) : QuasilinearOn π•œ univ f", "start": [ 214, 1 ], "end": [ 215, 40 ], "kind": "commanddeclaration" }, { "full_name": "Antitone.quasiconvexOn", "code": "theorem Antitone.quasiconvexOn (hf : Antitone f) : QuasiconvexOn π•œ univ f", "start": [ 218, 1 ], "end": [ 219, 46 ], "kind": "commanddeclaration" }, { "full_name": "Antitone.quasiconcaveOn", "code": "theorem Antitone.quasiconcaveOn (hf : Antitone f) : QuasiconcaveOn π•œ univ f", "start": [ 222, 1 ], "end": [ 223, 47 ], "kind": "commanddeclaration" }, { "full_name": "Antitone.quasilinearOn", "code": "theorem Antitone.quasilinearOn (hf : Antitone f) : QuasilinearOn π•œ univ f", "start": [ 226, 1 ], "end": [ 227, 40 ], "kind": "commanddeclaration" }, { "full_name": "QuasilinearOn.monotoneOn_or_antitoneOn", "code": "theorem QuasilinearOn.monotoneOn_or_antitoneOn [LinearOrder Ξ²] (hf : QuasilinearOn π•œ s f) :\n MonotoneOn f s ∨ AntitoneOn f s", "start": [ 238, 1 ], "end": [ 242, 97 ], "kind": "commanddeclaration" }, { "full_name": "quasilinearOn_iff_monotoneOn_or_antitoneOn", "code": "theorem quasilinearOn_iff_monotoneOn_or_antitoneOn [LinearOrderedAddCommMonoid Ξ²]\n (hs : Convex π•œ s) : QuasilinearOn π•œ s f ↔ MonotoneOn f s ∨ AntitoneOn f s", "start": [ 245, 1 ], "end": [ 248, 70 ], "kind": "commanddeclaration" } ]
Mathlib/Algebra/AddConstMap/Basic.lean
[ "Mathlib/Algebra/Module/Defs.lean", "Mathlib/Algebra/Order/Group/Instances.lean", "Mathlib/Logic/Function/Iterate.lean", "Mathlib/Algebra/GroupPower/IterateHom.lean", "Mathlib/GroupTheory/GroupAction/Pi.lean", ".lake/packages/lean4/src/lean/Init.lean", "Mathlib/Algebra/Order/Archimedean.lean" ]
[ { "full_name": "AddConstMap", "code": "structure AddConstMap (G H : Type*) [Add G] [Add H] (a : G) (b : H) where\n \n protected toFun : G β†’ H\n \n map_add_const' (x : G) : toFun (x + a) = toFun x + b", "start": [ 33, 1 ], "end": [ 41, 55 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMapClass", "code": "class AddConstMapClass (F : Type*) (G H : outParam Type*) [Add G] [Add H]\n (a : outParam G) (b : outParam H) [FunLike F G H] : Prop where\n \n map_add_const (f : F) (x : G) : f (x + a) = f x + b", "start": [ 46, 1 ], "end": [ 55, 54 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMapClass.semiconj", "code": "protected theorem semiconj [Add G] [Add H] [AddConstMapClass F G H a b] (f : F) :\n Semiconj f (Β· + a) (Β· + b)", "start": [ 69, 1 ], "end": [ 71, 18 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMapClass.map_add_nsmul", "code": "@[scoped simp]\ntheorem map_add_nsmul [AddMonoid G] [AddMonoid H] [AddConstMapClass F G H a b]\n (f : F) (x : G) (n : β„•) : f (x + n β€’ a) = f x + n β€’ b", "start": [ 73, 1 ], "end": [ 76, 62 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMapClass.map_add_nat'", "code": "@[scoped simp]\ntheorem map_add_nat' [AddMonoidWithOne G] [AddMonoid H] [AddConstMapClass F G H 1 b]\n (f : F) (x : G) (n : β„•) : f (x + n) = f x + n β€’ b", "start": [ 78, 1 ], "end": [ 80, 83 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMapClass.map_add_one", "code": "theorem map_add_one [AddMonoidWithOne G] [Add H] [AddConstMapClass F G H 1 b]\n (f : F) (x : G) : f (x + 1) = f x + b", "start": [ 82, 1 ], "end": [ 83, 63 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMapClass.map_add_ofNat'", "code": "@[scoped simp]\ntheorem map_add_ofNat' [AddMonoidWithOne G] [AddMonoid H] [AddConstMapClass F G H 1 b]\n (f : F) (x : G) (n : β„•) [n.AtLeastTwo] :\n f (x + no_index (OfNat.ofNat n)) = f x + (OfNat.ofNat n : β„•) β€’ b", "start": [ 85, 1 ], "end": [ 89, 21 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMapClass.map_add_nat", "code": "theorem map_add_nat [AddMonoidWithOne G] [AddMonoidWithOne H] [AddConstMapClass F G H 1 1]\n (f : F) (x : G) (n : β„•) : f (x + n) = f x + n", "start": [ 91, 1 ], "end": [ 92, 61 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMapClass.map_add_ofNat", "code": "theorem map_add_ofNat [AddMonoidWithOne G] [AddMonoidWithOne H] [AddConstMapClass F G H 1 1]\n (f : F) (x : G) (n : β„•) [n.AtLeastTwo] :\n f (x + OfNat.ofNat n) = f x + OfNat.ofNat n", "start": [ 94, 1 ], "end": [ 96, 69 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMapClass.map_const", "code": "@[scoped simp]\ntheorem map_const [AddZeroClass G] [Add H] [AddConstMapClass F G H a b] (f : F) :\n f a = f 0 + b", "start": [ 98, 1 ], "end": [ 101, 32 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMapClass.map_one", "code": "theorem map_one [AddZeroClass G] [One G] [Add H] [AddConstMapClass F G H 1 b] (f : F) :\n f 1 = f 0 + b", "start": [ 103, 1 ], "end": [ 105, 14 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMapClass.map_nsmul_const", "code": "@[scoped simp]\ntheorem map_nsmul_const [AddMonoid G] [AddMonoid H] [AddConstMapClass F G H a b]\n (f : F) (n : β„•) : f (n β€’ a) = f 0 + n β€’ b", "start": [ 107, 1 ], "end": [ 110, 34 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMapClass.map_nat'", "code": "@[scoped simp]\ntheorem map_nat' [AddMonoidWithOne G] [AddMonoid H] [AddConstMapClass F G H 1 b]\n (f : F) (n : β„•) : f n = f 0 + n β€’ b", "start": [ 112, 1 ], "end": [ 115, 33 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMapClass.map_ofNat'", "code": "theorem map_ofNat' [AddMonoidWithOne G] [AddMonoid H] [AddConstMapClass F G H 1 b]\n (f : F) (n : β„•) [n.AtLeastTwo] :\n f (OfNat.ofNat n) = f 0 + (OfNat.ofNat n : β„•) β€’ b", "start": [ 117, 1 ], "end": [ 120, 15 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMapClass.map_nat", "code": "theorem map_nat [AddMonoidWithOne G] [AddMonoidWithOne H] [AddConstMapClass F G H 1 1]\n (f : F) (n : β„•) : f n = f 0 + n", "start": [ 122, 1 ], "end": [ 123, 47 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMapClass.map_ofNat", "code": "theorem map_ofNat [AddMonoidWithOne G] [AddMonoidWithOne H] [AddConstMapClass F G H 1 1]\n (f : F) (n : β„•) [n.AtLeastTwo] :\n f (OfNat.ofNat n) = f 0 + OfNat.ofNat n", "start": [ 125, 1 ], "end": [ 127, 59 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMapClass.map_const_add", "code": "@[scoped simp]\ntheorem map_const_add [AddCommSemigroup G] [Add H] [AddConstMapClass F G H a b]\n (f : F) (x : G) : f (a + x) = f x + b", "start": [ 129, 1 ], "end": [ 132, 31 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMapClass.map_one_add", "code": "theorem map_one_add [AddCommMonoidWithOne G] [Add H] [AddConstMapClass F G H 1 b]\n (f : F) (x : G) : f (1 + x) = f x + b", "start": [ 134, 1 ], "end": [ 135, 63 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMapClass.map_nsmul_add", "code": "@[scoped simp]\ntheorem map_nsmul_add [AddCommMonoid G] [AddMonoid H] [AddConstMapClass F G H a b]\n (f : F) (n : β„•) (x : G) : f (n β€’ a + x) = f x + n β€’ b", "start": [ 137, 1 ], "end": [ 140, 31 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMapClass.map_nat_add'", "code": "@[scoped simp]\ntheorem map_nat_add' [AddCommMonoidWithOne G] [AddMonoid H] [AddConstMapClass F G H 1 b]\n (f : F) (n : β„•) (x : G) : f (↑n + x) = f x + n β€’ b", "start": [ 142, 1 ], "end": [ 145, 34 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMapClass.map_ofNat_add'", "code": "theorem map_ofNat_add' [AddCommMonoidWithOne G] [AddMonoid H] [AddConstMapClass F G H 1 b]\n (f : F) (n : β„•) [n.AtLeastTwo] (x : G) :\n f (OfNat.ofNat n + x) = f x + OfNat.ofNat n β€’ b", "start": [ 147, 1 ], "end": [ 150, 21 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMapClass.map_nat_add", "code": "theorem map_nat_add [AddCommMonoidWithOne G] [AddMonoidWithOne H] [AddConstMapClass F G H 1 1]\n (f : F) (n : β„•) (x : G) : f (↑n + x) = f x + n", "start": [ 152, 1 ], "end": [ 153, 62 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMapClass.map_ofNat_add", "code": "theorem map_ofNat_add [AddCommMonoidWithOne G] [AddMonoidWithOne H] [AddConstMapClass F G H 1 1]\n (f : F) (n : β„•) [n.AtLeastTwo] (x : G) :\n f (OfNat.ofNat n + x) = f x + OfNat.ofNat n", "start": [ 155, 1 ], "end": [ 158, 20 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMapClass.map_sub_nsmul", "code": "@[scoped simp]\ntheorem map_sub_nsmul [AddGroup G] [AddGroup H] [AddConstMapClass F G H a b]\n (f : F) (x : G) (n : β„•) : f (x - n β€’ a) = f x - n β€’ b", "start": [ 160, 1 ], "end": [ 163, 83 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMapClass.map_sub_const", "code": "@[scoped simp]\ntheorem map_sub_const [AddGroup G] [AddGroup H] [AddConstMapClass F G H a b]\n (f : F) (x : G) : f (x - a) = f x - b", "start": [ 165, 1 ], "end": [ 168, 34 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMapClass.map_sub_one", "code": "theorem map_sub_one [AddGroup G] [One G] [AddGroup H] [AddConstMapClass F G H 1 b]\n (f : F) (x : G) : f (x - 1) = f x - b", "start": [ 170, 1 ], "end": [ 172, 20 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMapClass.map_sub_nat'", "code": "@[scoped simp]\ntheorem map_sub_nat' [AddGroupWithOne G] [AddGroup H] [AddConstMapClass F G H 1 b]\n (f : F) (x : G) (n : β„•) : f (x - n) = f x - n β€’ b", "start": [ 174, 1 ], "end": [ 177, 34 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMapClass.map_sub_ofNat'", "code": "@[scoped simp]\ntheorem map_sub_ofNat' [AddGroupWithOne G] [AddGroup H] [AddConstMapClass F G H 1 b]\n (f : F) (x : G) (n : β„•) [n.AtLeastTwo] :\n f (x - no_index (OfNat.ofNat n)) = f x - OfNat.ofNat n β€’ b", "start": [ 179, 1 ], "end": [ 183, 21 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMapClass.map_add_zsmul", "code": "@[scoped simp]\ntheorem map_add_zsmul [AddGroup G] [AddGroup H] [AddConstMapClass F G H a b]\n (f : F) (x : G) : βˆ€ n : β„€, f (x + n β€’ a) = f x + n β€’ b", "start": [ 185, 1 ], "end": [ 189, 45 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMapClass.map_zsmul_const", "code": "@[scoped simp]\ntheorem map_zsmul_const [AddGroup G] [AddGroup H] [AddConstMapClass F G H a b]\n (f : F) (n : β„€) : f (n β€’ a) = f 0 + n β€’ b", "start": [ 191, 1 ], "end": [ 194, 34 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMapClass.map_add_int'", "code": "@[scoped simp]\ntheorem map_add_int' [AddGroupWithOne G] [AddGroup H] [AddConstMapClass F G H 1 b]\n (f : F) (x : G) (n : β„€) : f (x + n) = f x + n β€’ b", "start": [ 196, 1 ], "end": [ 199, 40 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMapClass.map_add_int", "code": "theorem map_add_int [AddGroupWithOne G] [AddGroupWithOne H] [AddConstMapClass F G H 1 1]\n (f : F) (x : G) (n : β„€) : f (x + n) = f x + n", "start": [ 201, 1 ], "end": [ 202, 61 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMapClass.map_sub_zsmul", "code": "@[scoped simp]\ntheorem map_sub_zsmul [AddGroup G] [AddGroup H] [AddConstMapClass F G H a b]\n (f : F) (x : G) (n : β„€) : f (x - n β€’ a) = f x - n β€’ b", "start": [ 204, 1 ], "end": [ 207, 54 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMapClass.map_sub_int'", "code": "@[scoped simp]\ntheorem map_sub_int' [AddGroupWithOne G] [AddGroup H] [AddConstMapClass F G H 1 b]\n (f : F) (x : G) (n : β„€) : f (x - n) = f x - n β€’ b", "start": [ 209, 1 ], "end": [ 212, 34 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMapClass.map_sub_int", "code": "theorem map_sub_int [AddGroupWithOne G] [AddGroupWithOne H] [AddConstMapClass F G H 1 1]\n (f : F) (x : G) (n : β„€) : f (x - n) = f x - n", "start": [ 214, 1 ], "end": [ 215, 61 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMapClass.map_zsmul_add", "code": "@[scoped simp]\ntheorem map_zsmul_add [AddCommGroup G] [AddGroup H] [AddConstMapClass F G H a b]\n (f : F) (n : β„€) (x : G) : f (n β€’ a + x) = f x + n β€’ b", "start": [ 217, 1 ], "end": [ 220, 31 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMapClass.map_int_add'", "code": "@[scoped simp]\ntheorem map_int_add' [AddCommGroupWithOne G] [AddGroup H] [AddConstMapClass F G H 1 b]\n (f : F) (n : β„€) (x : G) : f (↑n + x) = f x + n β€’ b", "start": [ 222, 1 ], "end": [ 225, 34 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMapClass.map_int_add", "code": "theorem map_int_add [AddCommGroupWithOne G] [AddGroupWithOne H] [AddConstMapClass F G H 1 1]\n (f : F) (n : β„€) (x : G) : f (↑n + x) = f x + n", "start": [ 227, 1 ], "end": [ 228, 62 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMapClass.map_fract", "code": "theorem map_fract {R : Type*} [LinearOrderedRing R] [FloorRing R] [AddGroup H]\n [FunLike F R H] [AddConstMapClass F R H 1 b] (f : F) (x : R) :\n f (Int.fract x) = f x - ⌊xβŒ‹ β€’ b", "start": [ 230, 1 ], "end": [ 233, 18 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMapClass.rel_map_of_Icc", "code": "protected theorem rel_map_of_Icc [LinearOrderedAddCommGroup G] [Archimedean G] [AddGroup H]\n [AddConstMapClass F G H a b] {f : F} {R : H β†’ H β†’ Prop} [IsTrans H R]\n [hR : CovariantClass H H (fun x y ↦ y + x) R] (ha : 0 < a) {l : G}\n (hf : βˆ€ x ∈ Icc l (l + a), βˆ€ y ∈ Icc l (l + a), x < y β†’ R (f x) (f y)) :\n ((Β· < Β·) β‡’ R) f f", "start": [ 235, 1 ], "end": [ 276, 19 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMapClass.monotone_iff_Icc", "code": "theorem monotone_iff_Icc [LinearOrderedAddCommGroup G] [Archimedean G] [OrderedAddCommGroup H]\n [AddConstMapClass F G H a b] {f : F} (ha : 0 < a) (l : G) :\n Monotone f ↔ MonotoneOn f (Icc l (l + a))", "start": [ 278, 1 ], "end": [ 282, 78 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMapClass.antitone_iff_Icc", "code": "theorem antitone_iff_Icc [LinearOrderedAddCommGroup G] [Archimedean G] [OrderedAddCommGroup H]\n [AddConstMapClass F G H a b] {f : F} (ha : 0 < a) (l : G) :\n Antitone f ↔ AntitoneOn f (Icc l (l + a))", "start": [ 284, 1 ], "end": [ 287, 35 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMapClass.strictMono_iff_Icc", "code": "theorem strictMono_iff_Icc [LinearOrderedAddCommGroup G] [Archimedean G] [OrderedAddCommGroup H]\n [AddConstMapClass F G H a b] {f : F} (ha : 0 < a) (l : G) :\n StrictMono f ↔ StrictMonoOn f (Icc l (l + a))", "start": [ 289, 1 ], "end": [ 292, 70 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMapClass.strictAnti_iff_Icc", "code": "theorem strictAnti_iff_Icc [LinearOrderedAddCommGroup G] [Archimedean G] [OrderedAddCommGroup H]\n [AddConstMapClass F G H a b] {f : F} (ha : 0 < a) (l : G) :\n StrictAnti f ↔ StrictAntiOn f (Icc l (l + a))", "start": [ 294, 1 ], "end": [ 297, 37 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMap.coe_mk", "code": "@[scoped simp] theorem coe_mk (f : G β†’ H) (hf) : ⇑(mk f hf : G β†’+c[a, b] H) = f", "start": [ 317, 1 ], "end": [ 317, 87 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMap.mk_coe", "code": "@[scoped simp] theorem mk_coe (f : G β†’+c[a, b] H) : mk f f.2 = f", "start": [ 318, 1 ], "end": [ 318, 72 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMap.toFun_eq_coe", "code": "@[scoped simp] theorem toFun_eq_coe (f : G β†’+c[a, b] H) : f.toFun = f", "start": [ 319, 1 ], "end": [ 319, 77 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMap.ext", "code": "@[ext] protected theorem ext {f g : G β†’+c[a, b] H} (h : βˆ€ x, f x = g x) : f = g", "start": [ 324, 1 ], "end": [ 325, 21 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMap.id", "code": "@[simps (config := .asFn)]\nprotected def id : G β†’+c[a, a] G := ⟨id, fun _ ↦ rfl⟩", "start": [ 333, 1 ], "end": [ 335, 54 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMap.comp", "code": "@[simps (config := .asFn)]\ndef comp {K : Type*} [Add K] {c : K} (g : H β†’+c[b, c] K) (f : G β†’+c[a, b] H) :\n G β†’+c[a, c] K :=\n ⟨g ∘ f, by simp⟩", "start": [ 339, 1 ], "end": [ 343, 19 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMap.comp_id", "code": "@[scoped simp] theorem comp_id (f : G β†’+c[a, b] H) : f.comp .id = f", "start": [ 345, 1 ], "end": [ 345, 75 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMap.id_comp", "code": "@[scoped simp] theorem id_comp (f : G β†’+c[a, b] H) : .comp .id f = f", "start": [ 346, 1 ], "end": [ 346, 76 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMap.replaceConsts", "code": "@[simps (config := .asFn)]\ndef replaceConsts (f : G β†’+c[a, b] H) (a' b') (ha : a = a') (hb : b = b') :\n G β†’+c[a', b'] H where\n toFun := f\n map_add_const' := ha β–Έ hb β–Έ f.map_add_const'", "start": [ 348, 1 ], "end": [ 353, 47 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMap.coe_vadd", "code": "@[scoped simp]\ntheorem coe_vadd {K : Type*} [VAdd K H] [VAddAssocClass K H H] (c : K) (f : G β†’+c[a, b] H) :\n ⇑(c +α΅₯ f) = c +α΅₯ ⇑f", "start": [ 363, 1 ], "end": [ 366, 6 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMap.mul_def", "code": "theorem mul_def (f g : G β†’+c[a, a] G) : f * g = f.comp g", "start": [ 385, 1 ], "end": [ 385, 64 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMap.coe_mul", "code": "@[scoped simp] theorem coe_mul (f g : G β†’+c[a, a] G) : ⇑(f * g) = f ∘ g", "start": [ 386, 1 ], "end": [ 386, 79 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMap.one_def", "code": "theorem one_def : (1 : G β†’+c[a, a] G) = .id", "start": [ 388, 1 ], "end": [ 388, 51 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMap.coe_one", "code": "@[scoped simp] theorem coe_one : ⇑(1 : G β†’+c[a, a] G) = id", "start": [ 389, 1 ], "end": [ 389, 66 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMap.coe_pow", "code": "@[scoped simp] theorem coe_pow (f : G β†’+c[a, a] G) (n : β„•) : ⇑(f ^ n) = f^[n]", "start": [ 391, 1 ], "end": [ 391, 85 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMap.pow_apply", "code": "theorem pow_apply (f : G β†’+c[a, a] G) (n : β„•) (x : G) : (f ^ n) x = f^[n] x", "start": [ 393, 1 ], "end": [ 393, 83 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMap.smul", "code": "@[simps (config := .asFn)]\ndef smul [DistribSMul K H] (c : K) (f : G β†’+c[a, b] H) : G β†’+c[a, c β€’ b] H where\n toFun := c β€’ ⇑f\n map_add_const' x := by simp [smul_add]", "start": [ 411, 1 ], "end": [ 415, 41 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMap.addLeftHom", "code": "@[simps! (config := .asFn)]\ndef addLeftHom : Multiplicative G β†’* (G β†’+c[a, a] G) where\n toFun c := Multiplicative.toAdd c +α΅₯ .id\n map_one' := by ext; apply zero_add\n map_mul' _ _ := by ext; apply add_assoc", "start": [ 423, 1 ], "end": [ 429, 42 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMap.conjNeg", "code": "@[simps! apply_coe]\ndef conjNeg : (G β†’+c[a, b] H) ≃ (G β†’+c[a, b] H) :=\n Involutive.toPerm (fun f ↦ ⟨fun x ↦ - f (-x), fun _ ↦ by simp [neg_add_eq_sub]⟩) fun _ ↦\n AddConstMap.ext fun _ ↦ by simp", "start": [ 437, 1 ], "end": [ 441, 36 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMap.conjNeg_symm", "code": "@[scoped simp] theorem conjNeg_symm : (conjNeg (a := a) (b := b)).symm = conjNeg", "start": [ 443, 1 ], "end": [ 443, 88 ], "kind": "commanddeclaration" }, { "full_name": "AddConstMap.mkFract", "code": "def mkFract : (Ico (0 : R) 1 β†’ G) ≃ (R β†’+c[1, a] G) where\n toFun f := ⟨fun x ↦ f ⟨Int.fract x, Int.fract_nonneg _, Int.fract_lt_one _⟩ + ⌊xβŒ‹ β€’ a, fun x ↦ by\n simp [add_one_zsmul, add_assoc]⟩\n invFun f x := f x\n left_inv _ := by ext x; simp [Int.fract_eq_self.2 x.2, Int.floor_eq_zero_iff.2 x.2]\n right_inv f := by ext x; simp [map_fract]", "start": [ 451, 1 ], "end": [ 457, 44 ], "kind": "commanddeclaration" } ]
Mathlib/Probability/BorelCantelli.lean
[ "Mathlib/Probability/ConditionalExpectation.lean", ".lake/packages/lean4/src/lean/Init.lean", "Mathlib/Probability/Martingale/BorelCantelli.lean", "Mathlib/Probability/Independence/Basic.lean" ]
[ { "full_name": "ProbabilityTheory.iIndepFun.indep_comap_natural_of_lt", "code": "theorem iIndepFun.indep_comap_natural_of_lt (hf : βˆ€ i, StronglyMeasurable (f i))\n (hfi : iIndepFun (fun _ => mΞ²) f ΞΌ) (hij : i < j) :\n Indep (MeasurableSpace.comap (f j) mΞ²) (Filtration.natural f hf i) ΞΌ", "start": [ 43, 1 ], "end": [ 48, 84 ], "kind": "commanddeclaration" }, { "full_name": "ProbabilityTheory.iIndepFun.condexp_natural_ae_eq_of_lt", "code": "theorem iIndepFun.condexp_natural_ae_eq_of_lt [SecondCountableTopology Ξ²] [CompleteSpace Ξ²]\n [NormedSpace ℝ Ξ²] (hf : βˆ€ i, StronglyMeasurable (f i)) (hfi : iIndepFun (fun _ => mΞ²) f ΞΌ)\n (hij : i < j) : ΞΌ[f j|Filtration.natural f hf i] =ᡐ[ΞΌ] fun _ => ΞΌ[f j]", "start": [ 52, 1 ], "end": [ 56, 88 ], "kind": "commanddeclaration" }, { "full_name": "ProbabilityTheory.iIndepSet.condexp_indicator_filtrationOfSet_ae_eq", "code": "theorem iIndepSet.condexp_indicator_filtrationOfSet_ae_eq (hsm : βˆ€ n, MeasurableSet (s n))\n (hs : iIndepSet s ΞΌ) (hij : i < j) :\n ΞΌ[(s j).indicator (fun _ => 1 : Ξ© β†’ ℝ)|filtrationOfSet hsm i] =ᡐ[ΞΌ]\n fun _ => (ΞΌ (s j)).toReal", "start": [ 60, 1 ], "end": [ 66, 87 ], "kind": "commanddeclaration" }, { "full_name": "ProbabilityTheory.measure_limsup_eq_one", "code": "theorem measure_limsup_eq_one {s : β„• β†’ Set Ξ©} (hsm : βˆ€ n, MeasurableSet (s n)) (hs : iIndepSet s ΞΌ)\n (hs' : (βˆ‘' n, ΞΌ (s n)) = ∞) : ΞΌ (limsup s atTop) = 1", "start": [ 72, 1 ], "end": [ 105, 44 ], "kind": "commanddeclaration" } ]
Mathlib/Combinatorics/SetFamily/Compression/UV.lean
[ ".lake/packages/lean4/src/lean/Init.lean", "Mathlib/Combinatorics/SetFamily/Shadow.lean" ]
[ { "full_name": "sup_sdiff_injOn", "code": "theorem sup_sdiff_injOn [GeneralizedBooleanAlgebra Ξ±] (u v : Ξ±) :\n { x | Disjoint u x ∧ v ≀ x }.InjOn fun x => (x βŠ” u) \\ v", "start": [ 56, 1 ], "end": [ 64, 89 ], "kind": "commanddeclaration" }, { "full_name": "UV.compress", "code": "def compress (u v a : Ξ±) : Ξ± :=\n if Disjoint u a ∧ v ≀ a then (a βŠ” u) \\ v else a", "start": [ 78, 1 ], "end": [ 82, 50 ], "kind": "commanddeclaration" }, { "full_name": "UV.compress_of_disjoint_of_le", "code": "theorem compress_of_disjoint_of_le (hua : Disjoint u a) (hva : v ≀ a) :\n compress u v a = (a βŠ” u) \\ v", "start": [ 85, 1 ], "end": [ 87, 20 ], "kind": "commanddeclaration" }, { "full_name": "UV.compress_of_disjoint_of_le'", "code": "theorem compress_of_disjoint_of_le' (hva : Disjoint v a) (hua : u ≀ a) :\n compress u v ((a βŠ” v) \\ u) = a", "start": [ 90, 1 ], "end": [ 94, 79 ], "kind": "commanddeclaration" }, { "full_name": "UV.compress_self", "code": "@[simp]\ntheorem compress_self (u a : Ξ±) : compress u u a = a", "start": [ 97, 1 ], "end": [ 102, 8 ], "kind": "commanddeclaration" }, { "full_name": "UV.compress_sdiff_sdiff", "code": "@[simp]\ntheorem compress_sdiff_sdiff (a b : Ξ±) : compress (a \\ b) (b \\ a) b = a", "start": [ 105, 1 ], "end": [ 110, 23 ], "kind": "commanddeclaration" }, { "full_name": "UV.compress_idem", "code": "@[simp]\ntheorem compress_idem (u v a : Ξ±) : compress u v (compress u v a) = compress u v a", "start": [ 113, 1 ], "end": [ 120, 8 ], "kind": "commanddeclaration" }, { "full_name": "UV.compression", "code": "def compression (u v : Ξ±) (s : Finset Ξ±) :=\n (s.filter (compress u v Β· ∈ s)) βˆͺ (s.image <| compress u v).filter (Β· βˆ‰ s)", "start": [ 125, 1 ], "end": [ 128, 77 ], "kind": "commanddeclaration" }, { "full_name": "UV.IsCompressed", "code": "def IsCompressed (u v : Ξ±) (s : Finset Ξ±) :=\n 𝓒 u v s = s", "start": [ 136, 1 ], "end": [ 138, 14 ], "kind": "commanddeclaration" }, { "full_name": "UV.compress_injOn", "code": "theorem compress_injOn : Set.InjOn (compress u v) ↑(s.filter (compress u v Β· βˆ‰ s))", "start": [ 141, 1 ], "end": [ 151, 27 ], "kind": "commanddeclaration" }, { "full_name": "UV.mem_compression", "code": "theorem mem_compression :\n a ∈ 𝓒 u v s ↔ a ∈ s ∧ compress u v a ∈ s ∨ a βˆ‰ s ∧ βˆƒ b ∈ s, compress u v b = a", "start": [ 154, 1 ], "end": [ 158, 68 ], "kind": "commanddeclaration" }, { "full_name": "UV.IsCompressed.eq", "code": "protected theorem IsCompressed.eq (h : IsCompressed u v s) : 𝓒 u v s = s", "start": [ 161, 1 ], "end": [ 161, 78 ], "kind": "commanddeclaration" }, { "full_name": "UV.compression_self", "code": "@[simp]\ntheorem compression_self (u : Ξ±) (s : Finset Ξ±) : 𝓒 u u s = s", "start": [ 164, 1 ], "end": [ 173, 17 ], "kind": "commanddeclaration" }, { "full_name": "UV.isCompressed_self", "code": "theorem isCompressed_self (u : Ξ±) (s : Finset Ξ±) : IsCompressed u u s", "start": [ 176, 1 ], "end": [ 177, 94 ], "kind": "commanddeclaration" }, { "full_name": "UV.compress_disjoint", "code": "theorem compress_disjoint :\n Disjoint (s.filter (compress u v Β· ∈ s)) ((s.image <| compress u v).filter (Β· βˆ‰ s))", "start": [ 180, 1 ], "end": [ 182, 77 ], "kind": "commanddeclaration" }, { "full_name": "UV.compress_mem_compression", "code": "theorem compress_mem_compression (ha : a ∈ s) : compress u v a ∈ 𝓒 u v s", "start": [ 185, 1 ], "end": [ 190, 33 ], "kind": "commanddeclaration" }, { "full_name": "UV.compress_mem_compression_of_mem_compression", "code": "theorem compress_mem_compression_of_mem_compression (ha : a ∈ 𝓒 u v s) :\n compress u v a ∈ 𝓒 u v s", "start": [ 194, 1 ], "end": [ 200, 77 ], "kind": "commanddeclaration" }, { "full_name": "UV.compression_idem", "code": "@[simp]\ntheorem compression_idem (u v : Ξ±) (s : Finset Ξ±) : 𝓒 u v (𝓒 u v s) = 𝓒 u v s", "start": [ 203, 1 ], "end": [ 209, 57 ], "kind": "commanddeclaration" }, { "full_name": "UV.card_compression", "code": "@[simp]\ntheorem card_compression (u v : Ξ±) (s : Finset Ξ±) : (𝓒 u v s).card = s.card", "start": [ 212, 1 ], "end": [ 217, 32 ], "kind": "commanddeclaration" }, { "full_name": "UV.le_of_mem_compression_of_not_mem", "code": "theorem le_of_mem_compression_of_not_mem (h : a ∈ 𝓒 u v s) (ha : a βˆ‰ s) : u ≀ a", "start": [ 220, 1 ], "end": [ 228, 41 ], "kind": "commanddeclaration" }, { "full_name": "UV.disjoint_of_mem_compression_of_not_mem", "code": "theorem disjoint_of_mem_compression_of_not_mem (h : a ∈ 𝓒 u v s) (ha : a βˆ‰ s) : Disjoint v a", "start": [ 231, 1 ], "end": [ 239, 41 ], "kind": "commanddeclaration" }, { "full_name": "UV.sup_sdiff_mem_of_mem_compression_of_not_mem", "code": "theorem sup_sdiff_mem_of_mem_compression_of_not_mem (h : a ∈ 𝓒 u v s) (ha : a βˆ‰ s) :\n (a βŠ” v) \\ u ∈ s", "start": [ 242, 1 ], "end": [ 251, 41 ], "kind": "commanddeclaration" }, { "full_name": "UV.sup_sdiff_mem_of_mem_compression", "code": "theorem sup_sdiff_mem_of_mem_compression (ha : a ∈ 𝓒 u v s) (hva : v ≀ a) (hua : Disjoint u a) :\n (a βŠ” u) \\ v ∈ s", "start": [ 254, 1 ], "end": [ 271, 53 ], "kind": "commanddeclaration" }, { "full_name": "UV.mem_of_mem_compression", "code": "theorem mem_of_mem_compression (ha : a ∈ 𝓒 u v s) (hva : v ≀ a) (hvu : v = βŠ₯ β†’ u = βŠ₯) :\n a ∈ s", "start": [ 274, 1 ], "end": [ 285, 14 ], "kind": "commanddeclaration" }, { "full_name": "UV.card_compress", "code": "theorem card_compress (huv : u.card = v.card) (a : Finset Ξ±) : (compress u v a).card = a.card", "start": [ 296, 1 ], "end": [ 302, 8 ], "kind": "commanddeclaration" }, { "full_name": "Set.Sized.uvCompression", "code": "lemma _root_.Set.Sized.uvCompression (huv : u.card = v.card) (hπ’œ : (π’œ : Set (Finset Ξ±)).Sized r) :\n (𝓒 u v π’œ : Set (Finset Ξ±)).Sized r := by\n simp_rw [Set.Sized, mem_coe, mem_compression]\n rintro s (hs | ⟨huvt, t, ht, rfl⟩)\n Β· exact hπ’œ hs.1\n Β· rw [card_compress huv, hπ’œ ht]", "start": [ 305, 1 ], "end": [ 310, 34 ], "kind": "lemma" }, { "full_name": "UV.aux", "code": "private theorem aux (huv : βˆ€ x ∈ u, βˆƒ y ∈ v, IsCompressed (u.erase x) (v.erase y) π’œ) :\n v = βˆ… β†’ u = βˆ…", "start": [ 312, 1 ], "end": [ 314, 93 ], "kind": "commanddeclaration" }, { "full_name": "UV.shadow_compression_subset_compression_shadow", "code": "theorem shadow_compression_subset_compression_shadow (u v : Finset Ξ±)\n (huv : βˆ€ x ∈ u, βˆƒ y ∈ v, IsCompressed (u.erase x) (v.erase y) π’œ) :\n βˆ‚ (𝓒 u v π’œ) βŠ† 𝓒 u v (βˆ‚ π’œ)", "start": [ 316, 1 ], "end": [ 420, 93 ], "kind": "commanddeclaration" }, { "full_name": "UV.card_shadow_compression_le", "code": "theorem card_shadow_compression_le (u v : Finset Ξ±)\n (huv : βˆ€ x ∈ u, βˆƒ y ∈ v, IsCompressed (u.erase x) (v.erase y) π’œ) :\n (βˆ‚ (𝓒 u v π’œ)).card ≀ (βˆ‚ π’œ).card", "start": [ 423, 1 ], "end": [ 430, 32 ], "kind": "commanddeclaration" } ]
Mathlib/LinearAlgebra/AffineSpace/Pointwise.lean
[ "Mathlib/LinearAlgebra/AffineSpace/AffineSubspace.lean", ".lake/packages/lean4/src/lean/Init.lean" ]
[ { "full_name": "AffineSubspace.pointwiseAddAction", "code": "protected def pointwiseAddAction : AddAction V (AffineSubspace k P) where\n vadd x S := S.map (AffineEquiv.constVAdd k P x)\n zero_vadd p := ((congr_arg fun f => p.map f) <| AffineMap.ext <| zero_vadd _).trans p.map_id\n add_vadd _ _ p :=\n ((congr_arg fun f => p.map f) <| AffineMap.ext <| add_vadd _ _).trans (p.map_map _ _).symm", "start": [ 30, 1 ], "end": [ 37, 95 ], "kind": "commanddeclaration" }, { "full_name": "AffineSubspace.pointwise_vadd_eq_map", "code": "theorem pointwise_vadd_eq_map (v : V) (s : AffineSubspace k P) :\n v +α΅₯ s = s.map (AffineEquiv.constVAdd k P v)", "start": [ 44, 1 ], "end": [ 46, 6 ], "kind": "commanddeclaration" }, { "full_name": "AffineSubspace.coe_pointwise_vadd", "code": "@[simp]\ntheorem coe_pointwise_vadd (v : V) (s : AffineSubspace k P) :\n ((v +α΅₯ s : AffineSubspace k P) : Set P) = v +α΅₯ (s : Set P)", "start": [ 48, 1 ], "end": [ 51, 6 ], "kind": "commanddeclaration" }, { "full_name": "AffineSubspace.vadd_mem_pointwise_vadd_iff", "code": "theorem vadd_mem_pointwise_vadd_iff {v : V} {s : AffineSubspace k P} {p : P} :\n v +α΅₯ p ∈ v +α΅₯ s ↔ p ∈ s", "start": [ 54, 1 ], "end": [ 56, 24 ], "kind": "commanddeclaration" }, { "full_name": "AffineSubspace.pointwise_vadd_bot", "code": "theorem pointwise_vadd_bot (v : V) : v +α΅₯ (βŠ₯ : AffineSubspace k P) = βŠ₯", "start": [ 59, 1 ], "end": [ 60, 45 ], "kind": "commanddeclaration" }, { "full_name": "AffineSubspace.pointwise_vadd_direction", "code": "theorem pointwise_vadd_direction (v : V) (s : AffineSubspace k P) :\n (v +α΅₯ s).direction = s.direction", "start": [ 63, 1 ], "end": [ 66, 27 ], "kind": "commanddeclaration" }, { "full_name": "AffineSubspace.pointwise_vadd_span", "code": "theorem pointwise_vadd_span (v : V) (s : Set P) : v +α΅₯ affineSpan k s = affineSpan k (v +α΅₯ s)", "start": [ 69, 1 ], "end": [ 70, 15 ], "kind": "commanddeclaration" }, { "full_name": "AffineSubspace.map_pointwise_vadd", "code": "theorem map_pointwise_vadd (f : P₁ →ᡃ[k] Pβ‚‚) (v : V₁) (s : AffineSubspace k P₁) :\n (v +α΅₯ s).map f = f.linear v +α΅₯ s.map f", "start": [ 73, 1 ], "end": [ 78, 23 ], "kind": "commanddeclaration" } ]
Mathlib/Lean/CoreM.lean
[ ".lake/packages/lean4/src/lean/Init.lean", "Mathlib/Tactic/ToExpr.lean" ]
[ { "full_name": "CoreM.withImportModules", "code": "def CoreM.withImportModules (modules : Array Name) (run : CoreM Ξ±)\n (searchPath : Option SearchPath := none) (options : Options := {})\n (trustLevel : UInt32 := 0) (fileName := \"\") :\n IO Ξ± := unsafe do\n if let some sp := searchPath then searchPathRef.set sp\n Lean.withImportModules (modules.map (Import.mk Β· false)) options trustLevel fun env =>\n let ctx := {fileName, options, fileMap := default}\n let state := {env}\n Prod.fst <$> (CoreM.toIO Β· ctx state) do\n run", "start": [ 16, 1 ], "end": [ 28, 10 ], "kind": "commanddeclaration" } ]
Mathlib/Algebra/Algebra/Subalgebra/Rank.lean
[ ".lake/packages/lean4/src/lean/Init.lean", "Mathlib/LinearAlgebra/Dimension/Free.lean", "Mathlib/LinearAlgebra/FreeModule/StrongRankCondition.lean", "Mathlib/LinearAlgebra/Dimension/Finite.lean" ]
[ { "full_name": "Subalgebra.rank_sup_eq_rank_left_mul_rank_of_free", "code": "theorem rank_sup_eq_rank_left_mul_rank_of_free :\n Module.rank R β†₯(A βŠ” B) = Module.rank R A * Module.rank A (Algebra.adjoin A (B : Set S))", "start": [ 30, 1 ], "end": [ 41, 43 ], "kind": "commanddeclaration" }, { "full_name": "Subalgebra.rank_sup_eq_rank_right_mul_rank_of_free", "code": "theorem rank_sup_eq_rank_right_mul_rank_of_free :\n Module.rank R β†₯(A βŠ” B) = Module.rank R B * Module.rank B (Algebra.adjoin B (A : Set S))", "start": [ 43, 1 ], "end": [ 45, 56 ], "kind": "commanddeclaration" }, { "full_name": "Subalgebra.finrank_sup_eq_finrank_left_mul_finrank_of_free", "code": "theorem finrank_sup_eq_finrank_left_mul_finrank_of_free :\n finrank R β†₯(A βŠ” B) = finrank R A * finrank A (Algebra.adjoin A (B : Set S))", "start": [ 47, 1 ], "end": [ 49, 97 ], "kind": "commanddeclaration" }, { "full_name": "Subalgebra.finrank_sup_eq_finrank_right_mul_finrank_of_free", "code": "theorem finrank_sup_eq_finrank_right_mul_finrank_of_free :\n finrank R β†₯(A βŠ” B) = finrank R B * finrank B (Algebra.adjoin B (A : Set S))", "start": [ 51, 1 ], "end": [ 53, 65 ], "kind": "commanddeclaration" }, { "full_name": "Subalgebra.finrank_left_dvd_finrank_sup_of_free", "code": "theorem finrank_left_dvd_finrank_sup_of_free :\n finrank R A ∣ finrank R β†₯(A βŠ” B)", "start": [ 55, 1 ], "end": [ 56, 97 ], "kind": "commanddeclaration" }, { "full_name": "Subalgebra.finrank_right_dvd_finrank_sup_of_free", "code": "theorem finrank_right_dvd_finrank_sup_of_free :\n finrank R B ∣ finrank R β†₯(A βŠ” B)", "start": [ 58, 1 ], "end": [ 59, 98 ], "kind": "commanddeclaration" } ]
Mathlib/Analysis/Convex/SimplicialComplex/Basic.lean
[ "Mathlib/Analysis/Convex/Hull.lean", ".lake/packages/lean4/src/lean/Init.lean", "Mathlib/LinearAlgebra/AffineSpace/Independent.lean" ]
[ { "full_name": "Geometry.SimplicialComplex", "code": "@[ext]\nstructure SimplicialComplex where\n \n faces : Set (Finset E)\n \n not_empty_mem : βˆ… βˆ‰ faces\n \n indep : βˆ€ {s}, s ∈ faces β†’ AffineIndependent π•œ ((↑) : s β†’ E)\n \n down_closed : βˆ€ {s t}, s ∈ faces β†’ t βŠ† s β†’ t β‰  βˆ… β†’ t ∈ faces\n inter_subset_convexHull : βˆ€ {s t}, s ∈ faces β†’ t ∈ faces β†’\n convexHull π•œ ↑s ∩ convexHull π•œ ↑t βŠ† convexHull π•œ (s ∩ t : Set E)", "start": [ 53, 1 ], "end": [ 68, 69 ], "kind": "commanddeclaration" }, { "full_name": "Geometry.SimplicialComplex.space", "code": "def space (K : SimplicialComplex π•œ E) : Set E :=\n ⋃ s ∈ K.faces, convexHull π•œ (s : Set E)", "start": [ 80, 1 ], "end": [ 82, 42 ], "kind": "commanddeclaration" }, { "full_name": "Geometry.SimplicialComplex.mem_space_iff", "code": "theorem mem_space_iff : x ∈ K.space ↔ βˆƒ s ∈ K.faces, x ∈ convexHull π•œ (s : Set E)", "start": [ 86, 1 ], "end": [ 87, 15 ], "kind": "commanddeclaration" }, { "full_name": "Geometry.SimplicialComplex.convexHull_subset_space", "code": "theorem convexHull_subset_space (hs : s ∈ K.faces) : convexHull π•œ ↑s βŠ† K.space", "start": [ 91, 1 ], "end": [ 93, 6 ], "kind": "commanddeclaration" }, { "full_name": "Geometry.SimplicialComplex.subset_space", "code": "protected theorem subset_space (hs : s ∈ K.faces) : (s : Set E) βŠ† K.space", "start": [ 96, 1 ], "end": [ 97, 62 ], "kind": "commanddeclaration" }, { "full_name": "Geometry.SimplicialComplex.convexHull_inter_convexHull", "code": "theorem convexHull_inter_convexHull (hs : s ∈ K.faces) (ht : t ∈ K.faces) :\n convexHull π•œ ↑s ∩ convexHull π•œ ↑t = convexHull π•œ (s ∩ t : Set E)", "start": [ 100, 1 ], "end": [ 104, 45 ], "kind": "commanddeclaration" }, { "full_name": "Geometry.SimplicialComplex.disjoint_or_exists_inter_eq_convexHull", "code": "theorem disjoint_or_exists_inter_eq_convexHull (hs : s ∈ K.faces) (ht : t ∈ K.faces) :\n Disjoint (convexHull π•œ (s : Set E)) (convexHull π•œ ↑t) ∨\n βˆƒ u ∈ K.faces, convexHull π•œ (s : Set E) ∩ convexHull π•œ ↑t = convexHull π•œ ↑u", "start": [ 107, 1 ], "end": [ 119, 54 ], "kind": "commanddeclaration" }, { "full_name": "Geometry.SimplicialComplex.ofErase", "code": "@[simps]\ndef ofErase (faces : Set (Finset E)) (indep : βˆ€ s ∈ faces, AffineIndependent π•œ ((↑) : s β†’ E))\n (down_closed : βˆ€ s ∈ faces, βˆ€ t βŠ† s, t ∈ faces)\n (inter_subset_convexHull : βˆ€α΅‰ (s ∈ faces) (t ∈ faces),\n convexHull π•œ ↑s ∩ convexHull π•œ ↑t βŠ† convexHull π•œ (s ∩ t : Set E)) :\n SimplicialComplex π•œ E where\n faces := faces \\ {βˆ…}\n not_empty_mem h := h.2 (mem_singleton _)\n indep hs := indep _ hs.1\n down_closed hs hts ht := ⟨down_closed _ hs.1 _ hts, ht⟩\n inter_subset_convexHull hs ht := inter_subset_convexHull _ hs.1 _ ht.1", "start": [ 122, 1 ], "end": [ 133, 73 ], "kind": "commanddeclaration" }, { "full_name": "Geometry.SimplicialComplex.ofSubcomplex", "code": "@[simps]\ndef ofSubcomplex (K : SimplicialComplex π•œ E) (faces : Set (Finset E)) (subset : faces βŠ† K.faces)\n (down_closed : βˆ€ {s t}, s ∈ faces β†’ t βŠ† s β†’ t ∈ faces) : SimplicialComplex π•œ E :=\n { faces\n not_empty_mem := fun h => K.not_empty_mem (subset h)\n indep := fun hs => K.indep (subset hs)\n down_closed := fun hs hts _ => down_closed hs hts\n inter_subset_convexHull := fun hs ht => K.inter_subset_convexHull (subset hs) (subset ht) }", "start": [ 136, 1 ], "end": [ 144, 96 ], "kind": "commanddeclaration" }, { "full_name": "Geometry.SimplicialComplex.vertices", "code": "def vertices (K : SimplicialComplex π•œ E) : Set E :=\n { x | {x} ∈ K.faces }", "start": [ 150, 1 ], "end": [ 152, 24 ], "kind": "commanddeclaration" }, { "full_name": "Geometry.SimplicialComplex.mem_vertices", "code": "theorem mem_vertices : x ∈ K.vertices ↔ {x} ∈ K.faces", "start": [ 155, 1 ], "end": [ 155, 65 ], "kind": "commanddeclaration" }, { "full_name": "Geometry.SimplicialComplex.vertices_eq", "code": "theorem vertices_eq : K.vertices = ⋃ k ∈ K.faces, (k : Set E)", "start": [ 158, 1 ], "end": [ 162, 96 ], "kind": "commanddeclaration" }, { "full_name": "Geometry.SimplicialComplex.vertices_subset_space", "code": "theorem vertices_subset_space : K.vertices βŠ† K.space", "start": [ 165, 1 ], "end": [ 166, 86 ], "kind": "commanddeclaration" }, { "full_name": "Geometry.SimplicialComplex.vertex_mem_convexHull_iff", "code": "theorem vertex_mem_convexHull_iff (hx : x ∈ K.vertices) (hs : s ∈ K.faces) :\n x ∈ convexHull π•œ (s : Set E) ↔ x ∈ s", "start": [ 169, 1 ], "end": [ 176, 38 ], "kind": "commanddeclaration" }, { "full_name": "Geometry.SimplicialComplex.face_subset_face_iff", "code": "theorem face_subset_face_iff (hs : s ∈ K.faces) (ht : t ∈ K.faces) :\n convexHull π•œ (s : Set E) βŠ† convexHull π•œ ↑t ↔ s βŠ† t", "start": [ 179, 1 ], "end": [ 186, 21 ], "kind": "commanddeclaration" }, { "full_name": "Geometry.SimplicialComplex.facets", "code": "def facets (K : SimplicialComplex π•œ E) : Set (Finset E) :=\n { s ∈ K.faces | βˆ€ ⦃t⦄, t ∈ K.faces β†’ s βŠ† t β†’ s = t }", "start": [ 192, 1 ], "end": [ 194, 55 ], "kind": "commanddeclaration" }, { "full_name": "Geometry.SimplicialComplex.mem_facets", "code": "theorem mem_facets : s ∈ K.facets ↔ s ∈ K.faces ∧ βˆ€ t ∈ K.faces, s βŠ† t β†’ s = t", "start": [ 197, 1 ], "end": [ 198, 14 ], "kind": "commanddeclaration" }, { "full_name": "Geometry.SimplicialComplex.facets_subset", "code": "theorem facets_subset : K.facets βŠ† K.faces", "start": [ 201, 1 ], "end": [ 201, 63 ], "kind": "commanddeclaration" }, { "full_name": "Geometry.SimplicialComplex.not_facet_iff_subface", "code": "theorem not_facet_iff_subface (hs : s ∈ K.faces) : s βˆ‰ K.facets ↔ βˆƒ t, t ∈ K.faces ∧ s βŠ‚ t", "start": [ 204, 1 ], "end": [ 212, 33 ], "kind": "commanddeclaration" }, { "full_name": "Geometry.SimplicialComplex.hasBot", "code": "instance hasBot : Bot (SimplicialComplex π•œ E) :=\n ⟨{ faces := βˆ…\n not_empty_mem := Set.not_mem_empty βˆ…\n indep := fun hs => (Set.not_mem_empty _ hs).elim\n down_closed := fun hs => (Set.not_mem_empty _ hs).elim\n inter_subset_convexHull := fun hs => (Set.not_mem_empty _ hs).elim }⟩", "start": [ 241, 1 ], "end": [ 246, 76 ], "kind": "commanddeclaration" }, { "full_name": "Geometry.SimplicialComplex.faces_bot", "code": "theorem faces_bot : (βŠ₯ : SimplicialComplex π•œ E).faces = βˆ…", "start": [ 256, 1 ], "end": [ 256, 65 ], "kind": "commanddeclaration" }, { "full_name": "Geometry.SimplicialComplex.space_bot", "code": "theorem space_bot : (βŠ₯ : SimplicialComplex π•œ E).space = βˆ…", "start": [ 259, 1 ], "end": [ 260, 22 ], "kind": "commanddeclaration" }, { "full_name": "Geometry.SimplicialComplex.facets_bot", "code": "theorem facets_bot : (βŠ₯ : SimplicialComplex π•œ E).facets = βˆ…", "start": [ 263, 1 ], "end": [ 264, 41 ], "kind": "commanddeclaration" } ]
Mathlib/Analysis/Calculus/Gradient/Basic.lean
[ "Mathlib/Analysis/Calculus/FDeriv/Basic.lean", ".lake/packages/lean4/src/lean/Init.lean", "Mathlib/Analysis/InnerProductSpace/Dual.lean", "Mathlib/Analysis/Calculus/Deriv/Basic.lean" ]
[ { "full_name": "HasGradientAtFilter", "code": "def HasGradientAtFilter (f : F β†’ π•œ) (f' x : F) (L : Filter F) :=\n HasFDerivAtFilter f (toDual π•œ F f') x L", "start": [ 48, 1 ], "end": [ 51, 42 ], "kind": "commanddeclaration" }, { "full_name": "HasGradientWithinAt", "code": "def HasGradientWithinAt (f : F β†’ π•œ) (f' : F) (s : Set F) (x : F) :=\n HasGradientAtFilter f f' x (𝓝[s] x)", "start": [ 53, 1 ], "end": [ 56, 38 ], "kind": "commanddeclaration" }, { "full_name": "HasGradientAt", "code": "def HasGradientAt (f : F β†’ π•œ) (f' x : F) :=\n HasGradientAtFilter f f' x (𝓝 x)", "start": [ 58, 1 ], "end": [ 61, 35 ], "kind": "commanddeclaration" }, { "full_name": "gradientWithin", "code": "def gradientWithin (f : F β†’ π•œ) (s : Set F) (x : F) : F :=\n (toDual π•œ F).symm (fderivWithin π•œ f s x)", "start": [ 63, 1 ], "end": [ 68, 43 ], "kind": "commanddeclaration" }, { "full_name": "gradient", "code": "def gradient (f : F β†’ π•œ) (x : F) : F :=\n (toDual π•œ F).symm (fderiv π•œ f x)", "start": [ 70, 1 ], "end": [ 75, 35 ], "kind": "commanddeclaration" }, { "full_name": "hasGradientWithinAt_iff_hasFDerivWithinAt", "code": "theorem hasGradientWithinAt_iff_hasFDerivWithinAt {s : Set F} :\n HasGradientWithinAt f f' s x ↔ HasFDerivWithinAt f (toDual π•œ F f') s x", "start": [ 86, 1 ], "end": [ 88, 10 ], "kind": "commanddeclaration" }, { "full_name": "hasFDerivWithinAt_iff_hasGradientWithinAt", "code": "theorem hasFDerivWithinAt_iff_hasGradientWithinAt {frechet : F β†’L[π•œ] π•œ} {s : Set F} :\n HasFDerivWithinAt f frechet s x ↔ HasGradientWithinAt f ((toDual π•œ F).symm frechet) s x", "start": [ 90, 1 ], "end": [ 92, 88 ], "kind": "commanddeclaration" }, { "full_name": "hasGradientAt_iff_hasFDerivAt", "code": "theorem hasGradientAt_iff_hasFDerivAt :\n HasGradientAt f f' x ↔ HasFDerivAt f (toDual π•œ F f') x", "start": [ 94, 1 ], "end": [ 96, 10 ], "kind": "commanddeclaration" }, { "full_name": "hasFDerivAt_iff_hasGradientAt", "code": "theorem hasFDerivAt_iff_hasGradientAt {frechet : F β†’L[π•œ] π•œ} :\n HasFDerivAt f frechet x ↔ HasGradientAt f ((toDual π•œ F).symm frechet) x", "start": [ 98, 1 ], "end": [ 100, 76 ], "kind": "commanddeclaration" }, { "full_name": "gradient_eq_zero_of_not_differentiableAt", "code": "theorem gradient_eq_zero_of_not_differentiableAt (h : Β¬DifferentiableAt π•œ f x) : βˆ‡ f x = 0", "start": [ 110, 1 ], "end": [ 111, 65 ], "kind": "commanddeclaration" }, { "full_name": "HasGradientAt.unique", "code": "theorem HasGradientAt.unique {gradf gradg : F}\n (hf : HasGradientAt f gradf x) (hg : HasGradientAt f gradg x) :\n gradf = gradg", "start": [ 113, 1 ], "end": [ 116, 64 ], "kind": "commanddeclaration" }, { "full_name": "DifferentiableAt.hasGradientAt", "code": "theorem DifferentiableAt.hasGradientAt (h : DifferentiableAt π•œ f x) :\n HasGradientAt f (βˆ‡ f x) x", "start": [ 118, 1 ], "end": [ 121, 22 ], "kind": "commanddeclaration" }, { "full_name": "HasGradientAt.differentiableAt", "code": "theorem HasGradientAt.differentiableAt (h : HasGradientAt f f' x) :\n DifferentiableAt π•œ f x", "start": [ 123, 1 ], "end": [ 125, 33 ], "kind": "commanddeclaration" }, { "full_name": "DifferentiableWithinAt.hasGradientWithinAt", "code": "theorem DifferentiableWithinAt.hasGradientWithinAt (h : DifferentiableWithinAt π•œ f s x) :\n HasGradientWithinAt f (gradientWithin f s x) s x", "start": [ 127, 1 ], "end": [ 131, 28 ], "kind": "commanddeclaration" }, { "full_name": "HasGradientWithinAt.differentiableWithinAt", "code": "theorem HasGradientWithinAt.differentiableWithinAt (h : HasGradientWithinAt f f' s x) :\n DifferentiableWithinAt π•œ f s x", "start": [ 133, 1 ], "end": [ 135, 45 ], "kind": "commanddeclaration" }, { "full_name": "hasGradientWithinAt_univ", "code": "@[simp]\ntheorem hasGradientWithinAt_univ : HasGradientWithinAt f f' univ x ↔ HasGradientAt f f' x", "start": [ 137, 1 ], "end": [ 140, 31 ], "kind": "commanddeclaration" }, { "full_name": "DifferentiableOn.hasGradientAt", "code": "theorem DifferentiableOn.hasGradientAt (h : DifferentiableOn π•œ f s) (hs : s ∈ 𝓝 x) :\n HasGradientAt f (βˆ‡ f x) x", "start": [ 142, 1 ], "end": [ 144, 35 ], "kind": "commanddeclaration" }, { "full_name": "HasGradientAt.gradient", "code": "theorem HasGradientAt.gradient (h : HasGradientAt f f' x) : βˆ‡ f x = f'", "start": [ 146, 1 ], "end": [ 147, 44 ], "kind": "commanddeclaration" }, { "full_name": "gradient_eq", "code": "theorem gradient_eq {f' : F β†’ F} (h : βˆ€ x, HasGradientAt f (f' x) x) : βˆ‡ f = f'", "start": [ 149, 1 ], "end": [ 150, 33 ], "kind": "commanddeclaration" }, { "full_name": "HasGradientAtFilter.hasDerivAtFilter", "code": "theorem HasGradientAtFilter.hasDerivAtFilter (h : HasGradientAtFilter g g' u L') :\n HasDerivAtFilter g (starRingEnd π•œ g') u L'", "start": [ 156, 1 ], "end": [ 160, 31 ], "kind": "commanddeclaration" }, { "full_name": "HasDerivAtFilter.hasGradientAtFilter", "code": "theorem HasDerivAtFilter.hasGradientAtFilter (h : HasDerivAtFilter g g' u L') :\n HasGradientAtFilter g (starRingEnd π•œ g') u L'", "start": [ 162, 1 ], "end": [ 166, 36 ], "kind": "commanddeclaration" }, { "full_name": "HasGradientAt.hasDerivAt", "code": "theorem HasGradientAt.hasDerivAt (h : HasGradientAt g g' u) :\n HasDerivAt g (starRingEnd π•œ g') u", "start": [ 168, 1 ], "end": [ 171, 16 ], "kind": "commanddeclaration" }, { "full_name": "HasDerivAt.hasGradientAt", "code": "theorem HasDerivAt.hasGradientAt (h : HasDerivAt g g' u) :\n HasGradientAt g (starRingEnd π•œ g') u", "start": [ 173, 1 ], "end": [ 176, 8 ], "kind": "commanddeclaration" }, { "full_name": "gradient_eq_deriv", "code": "theorem gradient_eq_deriv : βˆ‡ g u = starRingEnd π•œ (deriv g u)", "start": [ 178, 1 ], "end": [ 181, 100 ], "kind": "commanddeclaration" }, { "full_name": "HasGradientAtFilter.hasDerivAtFilter'", "code": "theorem HasGradientAtFilter.hasDerivAtFilter' (h : HasGradientAtFilter g g' u L') :\n HasDerivAtFilter g g' u L'", "start": [ 189, 1 ], "end": [ 190, 53 ], "kind": "commanddeclaration" }, { "full_name": "HasDerivAtFilter.hasGradientAtFilter'", "code": "theorem HasDerivAtFilter.hasGradientAtFilter' (h : HasDerivAtFilter g g' u L') :\n HasGradientAtFilter g g' u L'", "start": [ 192, 1 ], "end": [ 193, 59 ], "kind": "commanddeclaration" }, { "full_name": "HasGradientAt.hasDerivAt'", "code": "theorem HasGradientAt.hasDerivAt' (h : HasGradientAt g g' u) :\n HasDerivAt g g' u", "start": [ 195, 1 ], "end": [ 196, 38 ], "kind": "commanddeclaration" }, { "full_name": "HasDerivAt.hasGradientAt'", "code": "theorem HasDerivAt.hasGradientAt' (h : HasDerivAt g g' u) :\n HasGradientAt g g' u", "start": [ 198, 1 ], "end": [ 199, 44 ], "kind": "commanddeclaration" }, { "full_name": "gradient_eq_deriv'", "code": "theorem gradient_eq_deriv' : βˆ‡ g u = deriv g u", "start": [ 201, 1 ], "end": [ 201, 68 ], "kind": "commanddeclaration" }, { "full_name": "hasGradientAtFilter_iff_isLittleO", "code": "theorem hasGradientAtFilter_iff_isLittleO :\n HasGradientAtFilter f f' x L ↔\n (fun x' : F => f x' - f x - βŸͺf', x' - x⟫) =o[L] fun x' => x' - x", "start": [ 209, 1 ], "end": [ 212, 37 ], "kind": "commanddeclaration" }, { "full_name": "hasGradientWithinAt_iff_isLittleO", "code": "theorem hasGradientWithinAt_iff_isLittleO :\n HasGradientWithinAt f f' s x ↔\n (fun x' : F => f x' - f x - βŸͺf', x' - x⟫) =o[𝓝[s] x] fun x' => x' - x", "start": [ 214, 1 ], "end": [ 217, 36 ], "kind": "commanddeclaration" }, { "full_name": "hasGradientWithinAt_iff_tendsto", "code": "theorem hasGradientWithinAt_iff_tendsto :\n HasGradientWithinAt f f' s x ↔\n Tendsto (fun x' => β€–x' - x‖⁻¹ * β€–f x' - f x - βŸͺf', x' - xβŸ«β€–) (𝓝[s] x) (𝓝 0)", "start": [ 219, 1 ], "end": [ 222, 32 ], "kind": "commanddeclaration" }, { "full_name": "hasGradientAt_iff_isLittleO", "code": "theorem hasGradientAt_iff_isLittleO : HasGradientAt f f' x ↔\n (fun x' : F => f x' - f x - βŸͺf', x' - x⟫) =o[𝓝 x] fun x' => x' - x", "start": [ 224, 1 ], "end": [ 226, 36 ], "kind": "commanddeclaration" }, { "full_name": "hasGradientAt_iff_tendsto", "code": "theorem hasGradientAt_iff_tendsto :\n HasGradientAt f f' x ↔\n Tendsto (fun x' => β€–x' - x‖⁻¹ * β€–f x' - f x - βŸͺf', x' - xβŸ«β€–) (𝓝 x) (𝓝 0)", "start": [ 228, 1 ], "end": [ 231, 32 ], "kind": "commanddeclaration" }, { "full_name": "HasGradientAtFilter.isBigO_sub", "code": "theorem HasGradientAtFilter.isBigO_sub (h : HasGradientAtFilter f f' x L) :\n (fun x' => f x' - f x) =O[L] fun x' => x' - x", "start": [ 233, 1 ], "end": [ 235, 33 ], "kind": "commanddeclaration" }, { "full_name": "hasGradientWithinAt_congr_set'", "code": "theorem hasGradientWithinAt_congr_set' {s t : Set F} (y : F) (h : s =αΆ [𝓝[{y}ᢜ] x] t) :\n HasGradientWithinAt f f' s x ↔ HasGradientWithinAt f f' t x", "start": [ 237, 1 ], "end": [ 239, 35 ], "kind": "commanddeclaration" }, { "full_name": "hasGradientWithinAt_congr_set", "code": "theorem hasGradientWithinAt_congr_set {s t : Set F} (h : s =αΆ [𝓝 x] t) :\n HasGradientWithinAt f f' s x ↔ HasGradientWithinAt f f' t x", "start": [ 241, 1 ], "end": [ 243, 32 ], "kind": "commanddeclaration" }, { "full_name": "hasGradientAt_iff_isLittleO_nhds_zero", "code": "theorem hasGradientAt_iff_isLittleO_nhds_zero : HasGradientAt f f' x ↔\n (fun h => f (x + h) - f x - βŸͺf', h⟫) =o[𝓝 0] fun h => h", "start": [ 245, 1 ], "end": [ 247, 38 ], "kind": "commanddeclaration" }, { "full_name": "Filter.EventuallyEq.hasGradientAtFilter_iff", "code": "theorem Filter.EventuallyEq.hasGradientAtFilter_iff (hβ‚€ : fβ‚€ =αΆ [L] f₁) (hx : fβ‚€ x = f₁ x)\n (h₁ : fβ‚€' = f₁') : HasGradientAtFilter fβ‚€ fβ‚€' x L ↔ HasGradientAtFilter f₁ f₁' x L", "start": [ 257, 1 ], "end": [ 259, 45 ], "kind": "commanddeclaration" }, { "full_name": "HasGradientAtFilter.congr_of_eventuallyEq", "code": "theorem HasGradientAtFilter.congr_of_eventuallyEq (h : HasGradientAtFilter f f' x L)\n (hL : f₁ =αΆ [L] f) (hx : f₁ x = f x) : HasGradientAtFilter f₁ f' x L", "start": [ 261, 1 ], "end": [ 263, 42 ], "kind": "commanddeclaration" }, { "full_name": "HasGradientWithinAt.congr_mono", "code": "theorem HasGradientWithinAt.congr_mono (h : HasGradientWithinAt f f' s x) (ht : βˆ€ x ∈ t, f₁ x = f x)\n (hx : f₁ x = f x) (h₁ : t βŠ† s) : HasGradientWithinAt f₁ f' t x", "start": [ 265, 1 ], "end": [ 267, 42 ], "kind": "commanddeclaration" }, { "full_name": "HasGradientWithinAt.congr", "code": "theorem HasGradientWithinAt.congr (h : HasGradientWithinAt f f' s x) (hs : βˆ€ x ∈ s, f₁ x = f x)\n (hx : f₁ x = f x) : HasGradientWithinAt f₁ f' s x", "start": [ 269, 1 ], "end": [ 271, 32 ], "kind": "commanddeclaration" }, { "full_name": "HasGradientWithinAt.congr_of_mem", "code": "theorem HasGradientWithinAt.congr_of_mem (h : HasGradientWithinAt f f' s x)\n (hs : βˆ€ x ∈ s, f₁ x = f x) (hx : x ∈ s) : HasGradientWithinAt f₁ f' s x", "start": [ 273, 1 ], "end": [ 275, 23 ], "kind": "commanddeclaration" }, { "full_name": "HasGradientWithinAt.congr_of_eventuallyEq", "code": "theorem HasGradientWithinAt.congr_of_eventuallyEq (h : HasGradientWithinAt f f' s x)\n (h₁ : f₁ =αΆ [𝓝[s] x] f) (hx : f₁ x = f x) : HasGradientWithinAt f₁ f' s x", "start": [ 277, 1 ], "end": [ 279, 52 ], "kind": "commanddeclaration" }, { "full_name": "HasGradientWithinAt.congr_of_eventuallyEq_of_mem", "code": "theorem HasGradientWithinAt.congr_of_eventuallyEq_of_mem (h : HasGradientWithinAt f f' s x)\n (h₁ : f₁ =αΆ [𝓝[s] x] f) (hx : x ∈ s) : HasGradientWithinAt f₁ f' s x", "start": [ 281, 1 ], "end": [ 283, 54 ], "kind": "commanddeclaration" }, { "full_name": "HasGradientAt.congr_of_eventuallyEq", "code": "theorem HasGradientAt.congr_of_eventuallyEq (h : HasGradientAt f f' x) (h₁ : f₁ =αΆ [𝓝 x] f) :\n HasGradientAt f₁ f' x", "start": [ 285, 1 ], "end": [ 287, 74 ], "kind": "commanddeclaration" }, { "full_name": "Filter.EventuallyEq.gradient_eq", "code": "theorem Filter.EventuallyEq.gradient_eq (hL : f₁ =αΆ [𝓝 x] f) : βˆ‡ f₁ x = βˆ‡ f x", "start": [ 289, 1 ], "end": [ 291, 38 ], "kind": "commanddeclaration" }, { "full_name": "Filter.EventuallyEq.gradient", "code": "protected theorem Filter.EventuallyEq.gradient (h : f₁ =αΆ [𝓝 x] f) : βˆ‡ f₁ =αΆ [𝓝 x] βˆ‡ f", "start": [ 293, 1 ], "end": [ 294, 52 ], "kind": "commanddeclaration" }, { "full_name": "hasGradientAtFilter_const", "code": "theorem hasGradientAtFilter_const : HasGradientAtFilter (fun _ => c) 0 x L", "start": [ 304, 1 ], "end": [ 305, 74 ], "kind": "commanddeclaration" }, { "full_name": "hasGradientWithinAt_const", "code": "theorem hasGradientWithinAt_const : HasGradientWithinAt (fun _ => c) 0 s x", "start": [ 307, 1 ], "end": [ 308, 34 ], "kind": "commanddeclaration" }, { "full_name": "hasGradientAt_const", "code": "theorem hasGradientAt_const : HasGradientAt (fun _ => c) 0 x", "start": [ 310, 1 ], "end": [ 311, 34 ], "kind": "commanddeclaration" }, { "full_name": "gradient_const", "code": "theorem gradient_const : βˆ‡ (fun _ => c) x = 0", "start": [ 313, 1 ], "end": [ 314, 55 ], "kind": "commanddeclaration" }, { "full_name": "gradient_const'", "code": "@[simp]\ntheorem gradient_const' : (βˆ‡ fun _ : π•œ => c) = fun _ => 0", "start": [ 316, 1 ], "end": [ 318, 37 ], "kind": "commanddeclaration" }, { "full_name": "HasGradientAtFilter.tendsto_nhds", "code": "nonrec theorem HasGradientAtFilter.tendsto_nhds (hL : L ≀ 𝓝 x) (h : HasGradientAtFilter f f' x L) :\n Tendsto f L (𝓝 (f x))", "start": [ 326, 1 ], "end": [ 328, 20 ], "kind": "commanddeclaration" }, { "full_name": "HasGradientWithinAt.continuousWithinAt", "code": "theorem HasGradientWithinAt.continuousWithinAt (h : HasGradientWithinAt f f' s x) :\n ContinuousWithinAt f s x", "start": [ 330, 1 ], "end": [ 332, 49 ], "kind": "commanddeclaration" }, { "full_name": "HasGradientAt.continuousAt", "code": "theorem HasGradientAt.continuousAt (h : HasGradientAt f f' x) : ContinuousAt f x", "start": [ 334, 1 ], "end": [ 335, 44 ], "kind": "commanddeclaration" }, { "full_name": "HasGradientAt.continuousOn", "code": "protected theorem HasGradientAt.continuousOn {f' : F β†’ F} (h : βˆ€ x ∈ s, HasGradientAt f (f' x) x) :\n ContinuousOn f s", "start": [ 337, 1 ], "end": [ 339, 55 ], "kind": "commanddeclaration" } ]
Mathlib/LinearAlgebra/TensorAlgebra/Grading.lean
[ ".lake/packages/lean4/src/lean/Init.lean", "Mathlib/RingTheory/GradedAlgebra/Basic.lean", "Mathlib/LinearAlgebra/TensorAlgebra/Basic.lean" ]
[ { "full_name": "TensorAlgebra.GradedAlgebra.ΞΉ", "code": "nonrec def GradedAlgebra.ΞΉ : M β†’β‚—[R] ⨁ i : β„•, β†₯(LinearMap.range (ΞΉ R : M β†’β‚—[_] _) ^ i) :=\n DirectSum.lof R β„• (fun i => β†₯(LinearMap.range (ΞΉ R : M β†’β‚—[_] _) ^ i)) 1 βˆ˜β‚—\n (ΞΉ R).codRestrict _ fun m => by simpa only [pow_one] using LinearMap.mem_range_self _ m", "start": [ 28, 1 ], "end": [ 32, 92 ], "kind": "commanddeclaration" }, { "full_name": "TensorAlgebra.GradedAlgebra.ΞΉ_apply", "code": "theorem GradedAlgebra.ΞΉ_apply (m : M) :\n GradedAlgebra.ΞΉ R M m =\n DirectSum.of (fun (i : β„•) => β†₯(LinearMap.range (TensorAlgebra.ΞΉ R : M β†’β‚—[_] _) ^ i)) 1\n ⟨TensorAlgebra.ΞΉ R m, by simpa only [pow_one] using LinearMap.mem_range_self _ m⟩", "start": [ 35, 1 ], "end": [ 39, 6 ], "kind": "commanddeclaration" }, { "full_name": "TensorAlgebra.gradedAlgebra", "code": "instance gradedAlgebra :\n GradedAlgebra ((LinearMap.range (ΞΉ R : M β†’β‚—[R] TensorAlgebra R M) ^ Β·) : β„• β†’ Submodule R _) :=\n GradedAlgebra.ofAlgHom _ (lift R <| GradedAlgebra.ΞΉ R M)\n (by\n ext m\n dsimp only [LinearMap.comp_apply, AlgHom.toLinearMap_apply, AlgHom.comp_apply,\n AlgHom.id_apply]\n rw [lift_ΞΉ_apply, GradedAlgebra.ΞΉ_apply R M, DirectSum.coeAlgHom_of, Subtype.coe_mk])\n fun i x => by\n cases' x with x hx\n dsimp only [Subtype.coe_mk, DirectSum.lof_eq_of]\n induction hx using Submodule.pow_induction_on_left' with\n | algebraMap r =>\n rw [AlgHom.commutes, DirectSum.algebraMap_apply]; rfl\n | add x y i hx hy ihx ihy =>\n rw [AlgHom.map_add, ihx, ihy, ← AddMonoidHom.map_add]\n rfl\n | mem_mul m hm i x hx ih =>\n obtain ⟨_, rfl⟩ := hm\n rw [AlgHom.map_mul, ih, lift_ΞΉ_apply, GradedAlgebra.ΞΉ_apply R M, DirectSum.of_mul_of]\n exact DirectSum.of_eq_of_gradedMonoid_eq (Sigma.subtype_ext (add_comm _ _) rfl)", "start": [ 44, 1 ], "end": [ 68, 86 ], "kind": "commanddeclaration" } ]
Mathlib/Data/QPF/Multivariate/Constructions/Const.lean
[ ".lake/packages/lean4/src/lean/Init.lean", "Mathlib/Control/Functor/Multivariate.lean", "Mathlib/Data/QPF/Multivariate/Basic.lean" ]
[ { "full_name": "MvQPF.Const", "code": "@[nolint unusedArguments]\ndef Const (A : Type*) (_v : TypeVec.{u} n) : Type _ := A", "start": [ 30, 1 ], "end": [ 32, 57 ], "kind": "commanddeclaration" }, { "full_name": "MvQPF.Const.inhabited", "code": "instance Const.inhabited {A Ξ±} [Inhabited A] : Inhabited (Const n A Ξ±) := ⟨(default : A)⟩", "start": [ 35, 1 ], "end": [ 35, 90 ], "kind": "commanddeclaration" }, { "full_name": "MvQPF.Const.mk", "code": "protected def mk (x : A) : Const n A Ξ± := x", "start": [ 44, 1 ], "end": [ 45, 44 ], "kind": "commanddeclaration" }, { "full_name": "MvQPF.Const.get", "code": "protected def get (x : Const n A Ξ±) : A := x", "start": [ 48, 1 ], "end": [ 49, 45 ], "kind": "commanddeclaration" }, { "full_name": "MvQPF.Const.mk_get", "code": "@[simp]\nprotected theorem mk_get (x : Const n A Ξ±) : Const.mk (Const.get x) = x", "start": [ 52, 1 ], "end": [ 53, 79 ], "kind": "commanddeclaration" }, { "full_name": "MvQPF.Const.get_mk", "code": "@[simp]\nprotected theorem get_mk (x : A) : Const.get (Const.mk x : Const n A Ξ±) = x", "start": [ 56, 1 ], "end": [ 57, 83 ], "kind": "commanddeclaration" }, { "full_name": "MvQPF.Const.map", "code": "protected def map : Const n A Ξ± β†’ Const n A Ξ² := fun x => x", "start": [ 60, 1 ], "end": [ 61, 60 ], "kind": "commanddeclaration" }, { "full_name": "MvQPF.Const.MvFunctor", "code": "instance MvFunctor : MvFunctor (Const n A) where map _f := Const.map", "start": [ 64, 1 ], "end": [ 64, 69 ], "kind": "commanddeclaration" }, { "full_name": "MvQPF.Const.map_mk", "code": "theorem map_mk (x : A) : f <$$> Const.mk x = Const.mk x", "start": [ 66, 1 ], "end": [ 66, 63 ], "kind": "commanddeclaration" }, { "full_name": "MvQPF.Const.get_map", "code": "theorem get_map (x : (Const n A) Ξ±) : Const.get (f <$$> x) = Const.get x", "start": [ 69, 1 ], "end": [ 69, 80 ], "kind": "commanddeclaration" }, { "full_name": "MvQPF.Const.mvqpf", "code": "instance mvqpf : @MvQPF _ (Const n A) where\n P := MvPFunctor.const n A\n abs x := MvPFunctor.const.get x\n repr x := MvPFunctor.const.mk n x\n abs_repr := fun _ => const.get_mk _\n abs_map := fun _ => const.get_map _", "start": [ 72, 1 ], "end": [ 77, 38 ], "kind": "commanddeclaration" } ]
Mathlib/Combinatorics/Configuration.lean
[ "Mathlib/Combinatorics/Hall/Basic.lean", "Mathlib/Data/Fintype/BigOperators.lean", "Mathlib/SetTheory/Cardinal/Finite.lean", ".lake/packages/lean4/src/lean/Init.lean", "Mathlib/Algebra/Order/BigOperators/Group/Finset.lean" ]
[ { "full_name": "Configuration.Dual", "code": "def Dual :=\n P", "start": [ 44, 1 ], "end": [ 46, 4 ], "kind": "commanddeclaration" }, { "full_name": "Configuration.Nondegenerate", "code": "class Nondegenerate : Prop where\n exists_point : βˆ€ l : L, βˆƒ p, p βˆ‰ l\n exists_line : βˆ€ p, βˆƒ l : L, p βˆ‰ l\n eq_or_eq : βˆ€ {p₁ pβ‚‚ : P} {l₁ lβ‚‚ : L}, p₁ ∈ l₁ β†’ pβ‚‚ ∈ l₁ β†’ p₁ ∈ lβ‚‚ β†’ pβ‚‚ ∈ lβ‚‚ β†’ p₁ = pβ‚‚ ∨ l₁ = lβ‚‚", "start": [ 65, 1 ], "end": [ 74, 98 ], "kind": "commanddeclaration" }, { "full_name": "Configuration.HasPoints", "code": "class HasPoints extends Nondegenerate P L where\n mkPoint : βˆ€ {l₁ lβ‚‚ : L}, l₁ β‰  lβ‚‚ β†’ P\n mkPoint_ax : βˆ€ {l₁ lβ‚‚ : L} (h : l₁ β‰  lβ‚‚), mkPoint h ∈ l₁ ∧ mkPoint h ∈ lβ‚‚", "start": [ 77, 1 ], "end": [ 80, 76 ], "kind": "commanddeclaration" }, { "full_name": "Configuration.HasLines", "code": "class HasLines extends Nondegenerate P L where\n mkLine : βˆ€ {p₁ pβ‚‚ : P}, p₁ β‰  pβ‚‚ β†’ L\n mkLine_ax : βˆ€ {p₁ pβ‚‚ : P} (h : p₁ β‰  pβ‚‚), p₁ ∈ mkLine h ∧ pβ‚‚ ∈ mkLine h", "start": [ 83, 1 ], "end": [ 86, 73 ], "kind": "commanddeclaration" }, { "full_name": "Configuration.Dual.Nondegenerate", "code": "instance Dual.Nondegenerate [Nondegenerate P L] : Nondegenerate (Dual L) (Dual P) where\n exists_point := @exists_line P L _ _\n exists_line := @exists_point P L _ _\n eq_or_eq := @fun l₁ lβ‚‚ p₁ pβ‚‚ h₁ hβ‚‚ h₃ hβ‚„ => (@eq_or_eq P L _ _ p₁ pβ‚‚ l₁ lβ‚‚ h₁ h₃ hβ‚‚ hβ‚„).symm", "start": [ 95, 1 ], "end": [ 98, 95 ], "kind": "commanddeclaration" }, { "full_name": "Configuration.Dual.hasLines", "code": "instance Dual.hasLines [HasPoints P L] : HasLines (Dual L) (Dual P) :=\n { Dual.Nondegenerate _ _ with\n mkLine := @mkPoint P L _ _\n mkLine_ax := @mkPoint_ax P L _ _ }", "start": [ 100, 1 ], "end": [ 103, 39 ], "kind": "commanddeclaration" }, { "full_name": "Configuration.Dual.hasPoints", "code": "instance Dual.hasPoints [HasLines P L] : HasPoints (Dual L) (Dual P) :=\n { Dual.Nondegenerate _ _ with\n mkPoint := @mkLine P L _ _\n mkPoint_ax := @mkLine_ax P L _ _ }", "start": [ 105, 1 ], "end": [ 108, 39 ], "kind": "commanddeclaration" }, { "full_name": "Configuration.HasPoints.existsUnique_point", "code": "theorem HasPoints.existsUnique_point [HasPoints P L] (l₁ lβ‚‚ : L) (hl : l₁ β‰  lβ‚‚) :\n βˆƒ! p, p ∈ l₁ ∧ p ∈ lβ‚‚", "start": [ 110, 1 ], "end": [ 113, 79 ], "kind": "commanddeclaration" }, { "full_name": "Configuration.HasLines.existsUnique_line", "code": "theorem HasLines.existsUnique_line [HasLines P L] (p₁ pβ‚‚ : P) (hp : p₁ β‰  pβ‚‚) :\n βˆƒ! l : L, p₁ ∈ l ∧ pβ‚‚ ∈ l", "start": [ 116, 1 ], "end": [ 118, 58 ], "kind": "commanddeclaration" }, { "full_name": "Configuration.Nondegenerate.exists_injective_of_card_le", "code": "theorem Nondegenerate.exists_injective_of_card_le [Nondegenerate P L] [Fintype P] [Fintype L]\n (h : Fintype.card L ≀ Fintype.card P) : βˆƒ f : L β†’ P, Function.Injective f ∧ βˆ€ l, f l βˆ‰ l", "start": [ 123, 1 ], "end": [ 166, 55 ], "kind": "commanddeclaration" }, { "full_name": "Configuration.lineCount", "code": "noncomputable def lineCount (p : P) : β„• :=\n Nat.card { l : L // p ∈ l }", "start": [ 172, 1 ], "end": [ 174, 30 ], "kind": "commanddeclaration" }, { "full_name": "Configuration.pointCount", "code": "noncomputable def pointCount (l : L) : β„• :=\n Nat.card { p : P // p ∈ l }", "start": [ 179, 1 ], "end": [ 181, 30 ], "kind": "commanddeclaration" }, { "full_name": "Configuration.sum_lineCount_eq_sum_pointCount", "code": "theorem sum_lineCount_eq_sum_pointCount [Fintype P] [Fintype L] :\n βˆ‘ p : P, lineCount L p = βˆ‘ l : L, pointCount P l", "start": [ 186, 1 ], "end": [ 195, 96 ], "kind": "commanddeclaration" }, { "full_name": "Configuration.HasLines.pointCount_le_lineCount", "code": "theorem HasLines.pointCount_le_lineCount [HasLines P L] {p : P} {l : L} (h : p βˆ‰ l)\n [Finite { l : L // p ∈ l }] : pointCount P l ≀ lineCount L p", "start": [ 200, 1 ], "end": [ 214, 74 ], "kind": "commanddeclaration" }, { "full_name": "Configuration.HasPoints.lineCount_le_pointCount", "code": "theorem HasPoints.lineCount_le_pointCount [HasPoints P L] {p : P} {l : L} (h : p βˆ‰ l)\n [hf : Finite { p : P // p ∈ l }] : lineCount L p ≀ pointCount P l", "start": [ 217, 1 ], "end": [ 219, 67 ], "kind": "commanddeclaration" }, { "full_name": "Configuration.HasLines.card_le", "code": "theorem HasLines.card_le [HasLines P L] [Fintype P] [Fintype L] :\n Fintype.card P ≀ Fintype.card L", "start": [ 224, 1 ], "end": [ 245, 25 ], "kind": "commanddeclaration" }, { "full_name": "Configuration.HasPoints.card_le", "code": "theorem HasPoints.card_le [HasPoints P L] [Fintype P] [Fintype L] :\n Fintype.card L ≀ Fintype.card P", "start": [ 248, 1 ], "end": [ 251, 46 ], "kind": "commanddeclaration" }, { "full_name": "Configuration.HasLines.exists_bijective_of_card_eq", "code": "theorem HasLines.exists_bijective_of_card_eq [HasLines P L] [Fintype P] [Fintype L]\n (h : Fintype.card P = Fintype.card L) :\n βˆƒ f : L β†’ P, Function.Bijective f ∧ βˆ€ l, pointCount P l = lineCount L (f l)", "start": [ 256, 1 ], "end": [ 263, 95 ], "kind": "commanddeclaration" }, { "full_name": "Configuration.HasLines.lineCount_eq_pointCount", "code": "theorem HasLines.lineCount_eq_pointCount [HasLines P L] [Fintype P] [Fintype L]\n (hPL : Fintype.card P = Fintype.card L) {p : P} {l : L} (hpl : p βˆ‰ l) :\n lineCount L p = pointCount P l", "start": [ 266, 1 ], "end": [ 290, 61 ], "kind": "commanddeclaration" }, { "full_name": "Configuration.HasPoints.lineCount_eq_pointCount", "code": "theorem HasPoints.lineCount_eq_pointCount [HasPoints P L] [Fintype P] [Fintype L]\n (hPL : Fintype.card P = Fintype.card L) {p : P} {l : L} (hpl : p βˆ‰ l) :\n lineCount L p = pointCount P l", "start": [ 293, 1 ], "end": [ 296, 86 ], "kind": "commanddeclaration" }, { "full_name": "Configuration.HasLines.hasPoints", "code": "noncomputable def HasLines.hasPoints [HasLines P L] [Fintype P] [Fintype L]\n (h : Fintype.card P = Fintype.card L) : HasPoints P L :=\n let this : βˆ€ l₁ lβ‚‚ : L, l₁ β‰  lβ‚‚ β†’ βˆƒ p : P, p ∈ l₁ ∧ p ∈ lβ‚‚ := fun l₁ lβ‚‚ hl => by\n classical\n obtain ⟨f, _, hf2⟩ := HasLines.exists_bijective_of_card_eq h\n haveI : Nontrivial L := ⟨⟨l₁, lβ‚‚, hl⟩⟩\n haveI := Fintype.one_lt_card_iff_nontrivial.mp ((congr_arg _ h).mpr Fintype.one_lt_card)\n have h₁ : βˆ€ p : P, 0 < lineCount L p := fun p =>\n Exists.elim (exists_ne p) fun q hq =>\n (congr_arg _ Nat.card_eq_fintype_card).mpr\n (Fintype.card_pos_iff.mpr ⟨⟨mkLine hq, (mkLine_ax hq).2⟩⟩)\n have hβ‚‚ : βˆ€ l : L, 0 < pointCount P l := fun l => (congr_arg _ (hf2 l)).mpr (h₁ (f l))\n obtain ⟨p, hlβ‚βŸ© := Fintype.card_pos_iff.mp ((congr_arg _ Nat.card_eq_fintype_card).mp (hβ‚‚ l₁))\n by_cases hlβ‚‚ : p ∈ lβ‚‚\n Β· exact ⟨p, hl₁, hlβ‚‚βŸ©\n have key' : Fintype.card { q : P // q ∈ lβ‚‚ } = Fintype.card { l : L // p ∈ l } :=\n ((HasLines.lineCount_eq_pointCount h hlβ‚‚).trans Nat.card_eq_fintype_card).symm.trans\n Nat.card_eq_fintype_card\n have : βˆ€ q : { q // q ∈ lβ‚‚ }, p β‰  q := fun q hq => hlβ‚‚ ((congr_arg (Β· ∈ lβ‚‚) hq).mpr q.2)\n let f : { q : P // q ∈ lβ‚‚ } β†’ { l : L // p ∈ l } := fun q =>\n ⟨mkLine (this q), (mkLine_ax (this q)).1⟩\n have hf : Function.Injective f := fun q₁ qβ‚‚ hq =>\n Subtype.ext\n ((eq_or_eq q₁.2 qβ‚‚.2 (mkLine_ax (this q₁)).2\n ((congr_arg _ (Subtype.ext_iff.mp hq)).mpr (mkLine_ax (this qβ‚‚)).2)).resolve_right\n fun h => (congr_arg (Β¬p ∈ Β·) h).mp hlβ‚‚ (mkLine_ax (this q₁)).1)\n have key' := ((Fintype.bijective_iff_injective_and_card f).mpr ⟨hf, key'⟩).2\n obtain ⟨q, hq⟩ := key' ⟨l₁, hlβ‚βŸ©\n exact ⟨q, (congr_arg _ (Subtype.ext_iff.mp hq)).mp (mkLine_ax (this q)).2, q.2⟩\n { β€ΉHasLines P Lβ€Ί with\n mkPoint := fun {l₁ lβ‚‚} hl => Classical.choose (this l₁ lβ‚‚ hl)\n mkPoint_ax := fun {l₁ lβ‚‚} hl => Classical.choose_spec (this l₁ lβ‚‚ hl) }", "start": [ 299, 1 ], "end": [ 332, 76 ], "kind": "commanddeclaration" }, { "full_name": "Configuration.HasPoints.hasLines", "code": "noncomputable def HasPoints.hasLines [HasPoints P L] [Fintype P] [Fintype L]\n (h : Fintype.card P = Fintype.card L) : HasLines P L :=\n let this := @HasLines.hasPoints (Dual L) (Dual P) _ _ _ _ h.symm\n { β€ΉHasPoints P Lβ€Ί with\n mkLine := @fun _ _ => this.mkPoint\n mkLine_ax := @fun _ _ => this.mkPoint_ax }", "start": [ 335, 1 ], "end": [ 342, 47 ], "kind": "commanddeclaration" }, { "full_name": "Configuration.ProjectivePlane", "code": "class ProjectivePlane extends HasPoints P L, HasLines P L where\n exists_config :\n βˆƒ (p₁ pβ‚‚ p₃ : P) (l₁ lβ‚‚ l₃ : L),\n p₁ βˆ‰ lβ‚‚ ∧ p₁ βˆ‰ l₃ ∧ pβ‚‚ βˆ‰ l₁ ∧ pβ‚‚ ∈ lβ‚‚ ∧ pβ‚‚ ∈ l₃ ∧ p₃ βˆ‰ l₁ ∧ p₃ ∈ lβ‚‚ ∧ p₃ βˆ‰ l₃", "start": [ 347, 1 ], "end": [ 353, 84 ], "kind": "commanddeclaration" }, { "full_name": "Configuration.ProjectivePlane.order", "code": "noncomputable def order : β„• :=\n lineCount L (Classical.choose (@exists_config P L _ _)) - 1", "start": [ 366, 1 ], "end": [ 369, 62 ], "kind": "commanddeclaration" }, { "full_name": "Configuration.ProjectivePlane.card_points_eq_card_lines", "code": "theorem card_points_eq_card_lines [Fintype P] [Fintype L] : Fintype.card P = Fintype.card L", "start": [ 372, 1 ], "end": [ 373, 61 ], "kind": "commanddeclaration" }, { "full_name": "Configuration.ProjectivePlane.lineCount_eq_lineCount", "code": "theorem lineCount_eq_lineCount [Finite P] [Finite L] (p q : P) : lineCount L p = lineCount L q", "start": [ 378, 1 ], "end": [ 395, 54 ], "kind": "commanddeclaration" }, { "full_name": "Configuration.ProjectivePlane.pointCount_eq_pointCount", "code": "theorem pointCount_eq_pointCount [Finite P] [Finite L] (l m : L) :\n pointCount P l = pointCount P m", "start": [ 400, 1 ], "end": [ 402, 40 ], "kind": "commanddeclaration" }, { "full_name": "Configuration.ProjectivePlane.lineCount_eq_pointCount", "code": "theorem lineCount_eq_pointCount [Finite P] [Finite L] (p : P) (l : L) :\n lineCount L p = pointCount P l", "start": [ 407, 1 ], "end": [ 413, 80 ], "kind": "commanddeclaration" }, { "full_name": "Configuration.ProjectivePlane.Dual.order", "code": "theorem Dual.order [Finite P] [Finite L] : order (Dual L) (Dual P) = order P L", "start": [ 418, 1 ], "end": [ 419, 59 ], "kind": "commanddeclaration" }, { "full_name": "Configuration.ProjectivePlane.lineCount_eq", "code": "theorem lineCount_eq [Finite P] [Finite L] (p : P) : lineCount L p = order P L + 1", "start": [ 424, 1 ], "end": [ 430, 44 ], "kind": "commanddeclaration" }, { "full_name": "Configuration.ProjectivePlane.pointCount_eq", "code": "theorem pointCount_eq [Finite P] [Finite L] (l : L) : pointCount P l = order P L + 1", "start": [ 435, 1 ], "end": [ 436, 80 ], "kind": "commanddeclaration" }, { "full_name": "Configuration.ProjectivePlane.one_lt_order", "code": "theorem one_lt_order [Finite P] [Finite L] : 1 < order P L", "start": [ 441, 1 ], "end": [ 450, 66 ], "kind": "commanddeclaration" }, { "full_name": "Configuration.ProjectivePlane.two_lt_lineCount", "code": "theorem two_lt_lineCount [Finite P] [Finite L] (p : P) : 2 < lineCount L p", "start": [ 455, 1 ], "end": [ 456, 77 ], "kind": "commanddeclaration" }, { "full_name": "Configuration.ProjectivePlane.two_lt_pointCount", "code": "theorem two_lt_pointCount [Finite P] [Finite L] (l : L) : 2 < pointCount P l", "start": [ 461, 1 ], "end": [ 462, 78 ], "kind": "commanddeclaration" }, { "full_name": "Configuration.ProjectivePlane.card_points", "code": "theorem card_points [Fintype P] [Finite L] : Fintype.card P = order P L ^ 2 + order P L + 1", "start": [ 467, 1 ], "end": [ 493, 94 ], "kind": "commanddeclaration" }, { "full_name": "Configuration.ProjectivePlane.card_lines", "code": "theorem card_lines [Finite P] [Fintype L] : Fintype.card L = order P L ^ 2 + order P L + 1", "start": [ 496, 1 ], "end": [ 497, 94 ], "kind": "commanddeclaration" } ]
Mathlib/FieldTheory/Laurent.lean
[ "Mathlib/Algebra/Polynomial/Taylor.lean", ".lake/packages/lean4/src/lean/Init.lean", "Mathlib/FieldTheory/RatFunc/AsPolynomial.lean" ]
[ { "full_name": "RatFunc.taylor_mem_nonZeroDivisors", "code": "theorem taylor_mem_nonZeroDivisors (hp : p ∈ R[X]⁰) : taylor r p ∈ R[X]⁰", "start": [ 39, 1 ], "end": [ 45, 60 ], "kind": "commanddeclaration" }, { "full_name": "RatFunc.laurentAux", "code": "def laurentAux : RatFunc R β†’+* RatFunc R :=\n RatFunc.mapRingHom\n ( { toFun := taylor r\n map_add' := map_add (taylor r)\n map_mul' := taylor_mul _\n map_zero' := map_zero (taylor r)\n map_one' := taylor_one r } : R[X] β†’+* R[X])\n (taylor_mem_nonZeroDivisors _)", "start": [ 48, 1 ], "end": [ 57, 35 ], "kind": "commanddeclaration" }, { "full_name": "RatFunc.laurentAux_ofFractionRing_mk", "code": "theorem laurentAux_ofFractionRing_mk (q : R[X]⁰) :\n laurentAux r (ofFractionRing (Localization.mk p q)) =\n ofFractionRing (.mk (taylor r p) ⟨taylor r q, taylor_mem_nonZeroDivisors r q q.prop⟩)", "start": [ 60, 1 ], "end": [ 63, 38 ], "kind": "commanddeclaration" }, { "full_name": "RatFunc.laurentAux_div", "code": "theorem laurentAux_div :\n laurentAux r (algebraMap _ _ p / algebraMap _ _ q) =\n algebraMap _ _ (taylor r p) / algebraMap _ _ (taylor r q)", "start": [ 66, 1 ], "end": [ 70, 62 ], "kind": "commanddeclaration" }, { "full_name": "RatFunc.laurentAux_algebraMap", "code": "@[simp]\ntheorem laurentAux_algebraMap : laurentAux r (algebraMap _ _ p) = algebraMap _ _ (taylor r p)", "start": [ 73, 1 ], "end": [ 75, 94 ], "kind": "commanddeclaration" }, { "full_name": "RatFunc.laurent", "code": "def laurent : RatFunc R →ₐ[R] RatFunc R :=\n RatFunc.mapAlgHom (.ofLinearMap (taylor r) (taylor_one _) (taylor_mul _))\n (taylor_mem_nonZeroDivisors _)", "start": [ 78, 1 ], "end": [ 81, 35 ], "kind": "commanddeclaration" }, { "full_name": "RatFunc.laurent_div", "code": "theorem laurent_div :\n laurent r (algebraMap _ _ p / algebraMap _ _ q) =\n algebraMap _ _ (taylor r p) / algebraMap _ _ (taylor r q)", "start": [ 84, 1 ], "end": [ 87, 23 ], "kind": "commanddeclaration" }, { "full_name": "RatFunc.laurent_algebraMap", "code": "@[simp]\ntheorem laurent_algebraMap : laurent r (algebraMap _ _ p) = algebraMap _ _ (taylor r p)", "start": [ 90, 1 ], "end": [ 92, 28 ], "kind": "commanddeclaration" }, { "full_name": "RatFunc.laurent_X", "code": "@[simp]\ntheorem laurent_X : laurent r X = X + C r", "start": [ 95, 1 ], "end": [ 97, 82 ], "kind": "commanddeclaration" }, { "full_name": "RatFunc.laurent_C", "code": "@[simp]\ntheorem laurent_C (x : R) : laurent r (C x) = C x", "start": [ 101, 1 ], "end": [ 103, 52 ], "kind": "commanddeclaration" }, { "full_name": "RatFunc.laurent_at_zero", "code": "@[simp]\ntheorem laurent_at_zero : laurent 0 f = f", "start": [ 107, 1 ], "end": [ 108, 93 ], "kind": "commanddeclaration" }, { "full_name": "RatFunc.laurent_laurent", "code": "theorem laurent_laurent : laurent r (laurent s f) = laurent (r + s) f", "start": [ 111, 1 ], "end": [ 113, 39 ], "kind": "commanddeclaration" }, { "full_name": "RatFunc.laurent_injective", "code": "theorem laurent_injective : Function.Injective (laurent r)", "start": [ 116, 1 ], "end": [ 117, 59 ], "kind": "commanddeclaration" } ]
Mathlib/LinearAlgebra/Matrix/Dual.lean
[ "Mathlib/LinearAlgebra/Dual.lean", ".lake/packages/lean4/src/lean/Init.lean", "Mathlib/LinearAlgebra/Matrix/ToLin.lean" ]
[ { "full_name": "LinearMap.toMatrix_transpose", "code": "@[simp]\ntheorem LinearMap.toMatrix_transpose (u : V₁ β†’β‚—[K] Vβ‚‚) :\n LinearMap.toMatrix Bβ‚‚.dualBasis B₁.dualBasis (Module.Dual.transpose (R := K) u) =\n (LinearMap.toMatrix B₁ Bβ‚‚ u)α΅€", "start": [ 31, 1 ], "end": [ 37, 70 ], "kind": "commanddeclaration" }, { "full_name": "Matrix.toLin_transpose", "code": "@[simp]\ntheorem Matrix.toLin_transpose (M : Matrix ι₁ ΞΉβ‚‚ K) : Matrix.toLin B₁.dualBasis Bβ‚‚.dualBasis Mα΅€ =\n Module.Dual.transpose (R := K) (Matrix.toLin Bβ‚‚ B₁ M)", "start": [ 40, 1 ], "end": [ 44, 88 ], "kind": "commanddeclaration" } ]
Mathlib/Geometry/Euclidean/Sphere/Ptolemy.lean
[ "Mathlib/Geometry/Euclidean/Sphere/Power.lean", ".lake/packages/lean4/src/lean/Init.lean", "Mathlib/Geometry/Euclidean/Triangle.lean" ]
[ { "full_name": "EuclideanGeometry.mul_dist_add_mul_dist_eq_mul_dist_of_cospherical", "code": "theorem mul_dist_add_mul_dist_eq_mul_dist_of_cospherical {a b c d p : P}\n (h : Cospherical ({a, b, c, d} : Set P)) (hapc : ∠ a p c = Ο€) (hbpd : ∠ b p d = Ο€) :\n dist a b * dist c d + dist b c * dist d a = dist a c * dist b d", "start": [ 52, 1 ], "end": [ 70, 51 ], "kind": "commanddeclaration" } ]
Mathlib/Topology/Order/Hom/Esakia.lean
[ ".lake/packages/lean4/src/lean/Init.lean", "Mathlib/Order/Hom/Bounded.lean", "Mathlib/Topology/Order/Hom/Basic.lean" ]
[ { "full_name": "PseudoEpimorphism", "code": "structure PseudoEpimorphism (Ξ± Ξ² : Type*) [Preorder Ξ±] [Preorder Ξ²] extends Ξ± β†’o Ξ² where\n exists_map_eq_of_map_le' ⦃a : α⦄ ⦃b : β⦄ : toFun a ≀ b β†’ βˆƒ c, a ≀ c ∧ toFun c = b", "start": [ 40, 1 ], "end": [ 42, 84 ], "kind": "commanddeclaration" }, { "full_name": "EsakiaHom", "code": "structure EsakiaHom (Ξ± Ξ² : Type*) [TopologicalSpace Ξ±] [Preorder Ξ±] [TopologicalSpace Ξ²]\n [Preorder Ξ²] extends Ξ± β†’Co Ξ² where\n exists_map_eq_of_map_le' ⦃a : α⦄ ⦃b : β⦄ : toFun a ≀ b β†’ βˆƒ c, a ≀ c ∧ toFun c = b", "start": [ 45, 1 ], "end": [ 48, 84 ], "kind": "commanddeclaration" }, { "full_name": "PseudoEpimorphismClass", "code": "class PseudoEpimorphismClass (F : Type*) (Ξ± Ξ² : outParam Type*)\n [Preorder Ξ±] [Preorder Ξ²] [FunLike F Ξ± Ξ²]\n extends RelHomClass F ((Β· ≀ Β·) : Ξ± β†’ Ξ± β†’ Prop) ((Β· ≀ Β·) : Ξ² β†’ Ξ² β†’ Prop) : Prop where\n exists_map_eq_of_map_le (f : F) ⦃a : α⦄ ⦃b : β⦄ : f a ≀ b β†’ βˆƒ c, a ≀ c ∧ f c = b", "start": [ 53, 1 ], "end": [ 59, 83 ], "kind": "commanddeclaration" }, { "full_name": "EsakiaHomClass", "code": "class EsakiaHomClass (F : Type*) (Ξ± Ξ² : outParam Type*) [TopologicalSpace Ξ±] [Preorder Ξ±]\n [TopologicalSpace Ξ²] [Preorder Ξ²] [FunLike F Ξ± Ξ²]\n extends ContinuousOrderHomClass F Ξ± Ξ² : Prop where\n exists_map_eq_of_map_le (f : F) ⦃a : α⦄ ⦃b : β⦄ : f a ≀ b β†’ βˆƒ c, a ≀ c ∧ f c = b", "start": [ 62, 1 ], "end": [ 68, 83 ], "kind": "commanddeclaration" }, { "full_name": "PseudoEpimorphismClass.toTopHomClass", "code": "instance (priority := 100) PseudoEpimorphismClass.toTopHomClass [PartialOrder Ξ±] [OrderTop Ξ±]\n [Preorder Ξ²] [OrderTop Ξ²] [PseudoEpimorphismClass F Ξ± Ξ²] : TopHomClass F Ξ± Ξ² where\n map_top f := by\n let ⟨b, h⟩ := exists_map_eq_of_map_le f (@le_top _ _ _ <| f ⊀)\n rw [← top_le_iff.1 h.1, h.2]", "start": [ 80, 1 ], "end": [ 84, 33 ], "kind": "commanddeclaration" }, { "full_name": "EsakiaHomClass.toPseudoEpimorphismClass", "code": "instance (priority := 100) EsakiaHomClass.toPseudoEpimorphismClass [TopologicalSpace Ξ±] [Preorder Ξ±]\n [TopologicalSpace Ξ²] [Preorder Ξ²] [EsakiaHomClass F Ξ± Ξ²] : PseudoEpimorphismClass F Ξ± Ξ² :=\n { β€ΉEsakiaHomClass F Ξ± Ξ²β€Ί with\n map_rel := ContinuousOrderHomClass.map_monotone }", "start": [ 88, 1 ], "end": [ 91, 54 ], "kind": "commanddeclaration" }, { "full_name": "OrderIsoClass.toPseudoEpimorphismClass", "code": "instance (priority := 100) OrderIsoClass.toPseudoEpimorphismClass [Preorder Ξ±] [Preorder Ξ²]\n [EquivLike F Ξ± Ξ²] [OrderIsoClass F Ξ± Ξ²] : PseudoEpimorphismClass F Ξ± Ξ² where\n exists_map_eq_of_map_le f _a b h :=\n ⟨EquivLike.inv f b, (le_map_inv_iff f).2 h, EquivLike.right_inv _ _⟩", "start": [ 105, 1 ], "end": [ 108, 73 ], "kind": "commanddeclaration" }, { "full_name": "PseudoEpimorphism.instFunLike", "code": "instance instFunLike : FunLike (PseudoEpimorphism Ξ± Ξ²) Ξ± Ξ² where\n coe f := f.toFun\n coe_injective' f g h := by\n obtain ⟨⟨_, _⟩, _⟩ := f\n obtain ⟨⟨_, _⟩, _⟩ := g\n congr", "start": [ 118, 1 ], "end": [ 123, 10 ], "kind": "commanddeclaration" }, { "full_name": "PseudoEpimorphism.toOrderHom_eq_coe", "code": "@[simp]\ntheorem toOrderHom_eq_coe (f : PseudoEpimorphism Ξ± Ξ²) : ⇑f.toOrderHom = f", "start": [ 129, 1 ], "end": [ 130, 81 ], "kind": "commanddeclaration" }, { "full_name": "PseudoEpimorphism.toFun_eq_coe", "code": "theorem toFun_eq_coe {f : PseudoEpimorphism Ξ± Ξ²} : f.toFun = (f : Ξ± β†’ Ξ²)", "start": [ 132, 1 ], "end": [ 132, 80 ], "kind": "commanddeclaration" }, { "full_name": "PseudoEpimorphism.ext", "code": "@[ext]\ntheorem ext {f g : PseudoEpimorphism Ξ± Ξ²} (h : βˆ€ a, f a = g a) : f = g", "start": [ 135, 1 ], "end": [ 137, 21 ], "kind": "commanddeclaration" }, { "full_name": "PseudoEpimorphism.copy", "code": "protected def copy (f : PseudoEpimorphism Ξ± Ξ²) (f' : Ξ± β†’ Ξ²) (h : f' = f) : PseudoEpimorphism Ξ± Ξ² :=\n ⟨f.toOrderHom.copy f' h, by simpa only [h.symm, toFun_eq_coe] using f.exists_map_eq_of_map_le'⟩", "start": [ 140, 1 ], "end": [ 143, 98 ], "kind": "commanddeclaration" }, { "full_name": "PseudoEpimorphism.coe_copy", "code": "@[simp]\ntheorem coe_copy (f : PseudoEpimorphism Ξ± Ξ²) (f' : Ξ± β†’ Ξ²) (h : f' = f) : ⇑(f.copy f' h) = f'", "start": [ 146, 1 ], "end": [ 147, 100 ], "kind": "commanddeclaration" }, { "full_name": "PseudoEpimorphism.copy_eq", "code": "theorem copy_eq (f : PseudoEpimorphism Ξ± Ξ²) (f' : Ξ± β†’ Ξ²) (h : f' = f) : f.copy f' h = f", "start": [ 150, 1 ], "end": [ 151, 18 ], "kind": "commanddeclaration" }, { "full_name": "PseudoEpimorphism.id", "code": "protected def id : PseudoEpimorphism Ξ± Ξ± :=\n ⟨OrderHom.id, fun _ b h => ⟨b, h, rfl⟩⟩", "start": [ 156, 1 ], "end": [ 158, 42 ], "kind": "commanddeclaration" }, { "full_name": "PseudoEpimorphism.coe_id", "code": "@[simp]\ntheorem coe_id : ⇑(PseudoEpimorphism.id Ξ±) = id", "start": [ 164, 1 ], "end": [ 165, 55 ], "kind": "commanddeclaration" }, { "full_name": "PseudoEpimorphism.coe_id_orderHom", "code": "@[simp]\ntheorem coe_id_orderHom : (PseudoEpimorphism.id Ξ± : Ξ± β†’o Ξ±) = OrderHom.id", "start": [ 168, 1 ], "end": [ 169, 81 ], "kind": "commanddeclaration" }, { "full_name": "PseudoEpimorphism.id_apply", "code": "@[simp]\ntheorem id_apply (a : Ξ±) : PseudoEpimorphism.id Ξ± a = a", "start": [ 174, 1 ], "end": [ 175, 63 ], "kind": "commanddeclaration" }, { "full_name": "PseudoEpimorphism.comp", "code": "def comp (g : PseudoEpimorphism Ξ² Ξ³) (f : PseudoEpimorphism Ξ± Ξ²) : PseudoEpimorphism Ξ± Ξ³ :=\n ⟨g.toOrderHom.comp f.toOrderHom, fun a b hβ‚€ => by\n obtain ⟨b, h₁, rfl⟩ := g.exists_map_eq_of_map_le' hβ‚€\n obtain ⟨b, hβ‚‚, rfl⟩ := f.exists_map_eq_of_map_le' h₁\n exact ⟨b, hβ‚‚, rfl⟩⟩", "start": [ 178, 1 ], "end": [ 183, 24 ], "kind": "commanddeclaration" }, { "full_name": "PseudoEpimorphism.coe_comp", "code": "@[simp]\ntheorem coe_comp (g : PseudoEpimorphism Ξ² Ξ³) (f : PseudoEpimorphism Ξ± Ξ²) :\n (g.comp f : Ξ± β†’ Ξ³) = g ∘ f", "start": [ 186, 1 ], "end": [ 188, 38 ], "kind": "commanddeclaration" }, { "full_name": "PseudoEpimorphism.coe_comp_orderHom", "code": "@[simp]\ntheorem coe_comp_orderHom (g : PseudoEpimorphism Ξ² Ξ³) (f : PseudoEpimorphism Ξ± Ξ²) :\n (g.comp f : Ξ± β†’o Ξ³) = (g : Ξ² β†’o Ξ³).comp f", "start": [ 191, 1 ], "end": [ 193, 53 ], "kind": "commanddeclaration" }, { "full_name": "PseudoEpimorphism.comp_apply", "code": "@[simp]\ntheorem comp_apply (g : PseudoEpimorphism Ξ² Ξ³) (f : PseudoEpimorphism Ξ± Ξ²) (a : Ξ±) :\n (g.comp f) a = g (f a)", "start": [ 196, 1 ], "end": [ 198, 34 ], "kind": "commanddeclaration" }, { "full_name": "PseudoEpimorphism.comp_assoc", "code": "@[simp]\ntheorem comp_assoc (h : PseudoEpimorphism Ξ³ Ξ΄) (g : PseudoEpimorphism Ξ² Ξ³)\n (f : PseudoEpimorphism Ξ± Ξ²) : (h.comp g).comp f = h.comp (g.comp f)", "start": [ 201, 1 ], "end": [ 203, 79 ], "kind": "commanddeclaration" }, { "full_name": "PseudoEpimorphism.comp_id", "code": "@[simp]\ntheorem comp_id (f : PseudoEpimorphism Ξ± Ξ²) : f.comp (PseudoEpimorphism.id Ξ±) = f", "start": [ 206, 1 ], "end": [ 208, 19 ], "kind": "commanddeclaration" }, { "full_name": "PseudoEpimorphism.id_comp", "code": "@[simp]\ntheorem id_comp (f : PseudoEpimorphism Ξ± Ξ²) : (PseudoEpimorphism.id Ξ²).comp f = f", "start": [ 211, 1 ], "end": [ 213, 19 ], "kind": "commanddeclaration" }, { "full_name": "PseudoEpimorphism.cancel_right", "code": "@[simp]\ntheorem cancel_right {g₁ gβ‚‚ : PseudoEpimorphism Ξ² Ξ³} {f : PseudoEpimorphism Ξ± Ξ²}\n (hf : Surjective f) : g₁.comp f = gβ‚‚.comp f ↔ g₁ = gβ‚‚", "start": [ 216, 1 ], "end": [ 219, 78 ], "kind": "commanddeclaration" }, { "full_name": "PseudoEpimorphism.cancel_left", "code": "@[simp]\ntheorem cancel_left {g : PseudoEpimorphism Ξ² Ξ³} {f₁ fβ‚‚ : PseudoEpimorphism Ξ± Ξ²} (hg : Injective g) :\n g.comp f₁ = g.comp fβ‚‚ ↔ f₁ = fβ‚‚", "start": [ 222, 1 ], "end": [ 225, 81 ], "kind": "commanddeclaration" }, { "full_name": "EsakiaHom.toPseudoEpimorphism", "code": "def toPseudoEpimorphism (f : EsakiaHom Ξ± Ξ²) : PseudoEpimorphism Ξ± Ξ² :=\n { f with }", "start": [ 238, 1 ], "end": [ 239, 13 ], "kind": "commanddeclaration" }, { "full_name": "EsakiaHom.instFunLike", "code": "instance instFunLike : FunLike (EsakiaHom Ξ± Ξ²) Ξ± Ξ² where\n coe f := f.toFun\n coe_injective' f g h := by\n obtain ⟨⟨⟨_, _⟩, _⟩, _⟩ := f\n obtain ⟨⟨⟨_, _⟩, _⟩, _⟩ := g\n congr", "start": [ 242, 1 ], "end": [ 247, 10 ], "kind": "commanddeclaration" }, { "full_name": "EsakiaHom.toContinuousOrderHom_coe", "code": "@[simp]\ntheorem toContinuousOrderHom_coe {f : EsakiaHom Ξ± Ξ²} :\n f.toContinuousOrderHom = (f : Ξ± β†’ Ξ²)", "start": [ 255, 1 ], "end": [ 257, 48 ], "kind": "commanddeclaration" }, { "full_name": "EsakiaHom.toFun_eq_coe", "code": "theorem toFun_eq_coe {f : EsakiaHom Ξ± Ξ²} : f.toFun = (f : Ξ± β†’ Ξ²)", "start": [ 260, 1 ], "end": [ 260, 72 ], "kind": "commanddeclaration" }, { "full_name": "EsakiaHom.ext", "code": "@[ext]\ntheorem ext {f g : EsakiaHom Ξ± Ξ²} (h : βˆ€ a, f a = g a) : f = g", "start": [ 263, 1 ], "end": [ 265, 21 ], "kind": "commanddeclaration" }, { "full_name": "EsakiaHom.copy", "code": "protected def copy (f : EsakiaHom Ξ± Ξ²) (f' : Ξ± β†’ Ξ²) (h : f' = f) : EsakiaHom Ξ± Ξ² :=\n ⟨f.toContinuousOrderHom.copy f' h, by\n simpa only [h.symm, toFun_eq_coe] using f.exists_map_eq_of_map_le'⟩", "start": [ 268, 1 ], "end": [ 272, 72 ], "kind": "commanddeclaration" }, { "full_name": "EsakiaHom.coe_copy", "code": "@[simp]\ntheorem coe_copy (f : EsakiaHom Ξ± Ξ²) (f' : Ξ± β†’ Ξ²) (h : f' = f) : ⇑(f.copy f' h) = f'", "start": [ 275, 1 ], "end": [ 276, 92 ], "kind": "commanddeclaration" }, { "full_name": "EsakiaHom.copy_eq", "code": "theorem copy_eq (f : EsakiaHom Ξ± Ξ²) (f' : Ξ± β†’ Ξ²) (h : f' = f) : f.copy f' h = f", "start": [ 279, 1 ], "end": [ 280, 18 ], "kind": "commanddeclaration" }, { "full_name": "EsakiaHom.id", "code": "protected def id : EsakiaHom Ξ± Ξ± :=\n ⟨ContinuousOrderHom.id Ξ±, fun _ b h => ⟨b, h, rfl⟩⟩", "start": [ 285, 1 ], "end": [ 287, 54 ], "kind": "commanddeclaration" }, { "full_name": "EsakiaHom.coe_id", "code": "@[simp]\ntheorem coe_id : ⇑(EsakiaHom.id Ξ±) = id", "start": [ 293, 1 ], "end": [ 294, 47 ], "kind": "commanddeclaration" }, { "full_name": "EsakiaHom.coe_id_pseudoEpimorphism", "code": "@[simp]\ntheorem coe_id_pseudoEpimorphism :\n (EsakiaHom.id Ξ± : PseudoEpimorphism Ξ± Ξ±) = PseudoEpimorphism.id Ξ±", "start": [ 297, 1 ], "end": [ 299, 77 ], "kind": "commanddeclaration" }, { "full_name": "EsakiaHom.id_apply", "code": "@[simp]\ntheorem id_apply (a : Ξ±) : EsakiaHom.id Ξ± a = a", "start": [ 304, 1 ], "end": [ 305, 55 ], "kind": "commanddeclaration" }, { "full_name": "EsakiaHom.coe_id_continuousOrderHom", "code": "@[simp]\ntheorem coe_id_continuousOrderHom : (EsakiaHom.id Ξ± : Ξ± β†’Co Ξ±) = ContinuousOrderHom.id Ξ±", "start": [ 308, 1 ], "end": [ 309, 96 ], "kind": "commanddeclaration" }, { "full_name": "EsakiaHom.comp", "code": "def comp (g : EsakiaHom Ξ² Ξ³) (f : EsakiaHom Ξ± Ξ²) : EsakiaHom Ξ± Ξ³ :=\n ⟨g.toContinuousOrderHom.comp f.toContinuousOrderHom, fun a b hβ‚€ => by\n obtain ⟨b, h₁, rfl⟩ := g.exists_map_eq_of_map_le' hβ‚€\n obtain ⟨b, hβ‚‚, rfl⟩ := f.exists_map_eq_of_map_le' h₁\n exact ⟨b, hβ‚‚, rfl⟩⟩", "start": [ 312, 1 ], "end": [ 317, 24 ], "kind": "commanddeclaration" }, { "full_name": "EsakiaHom.coe_comp_continuousOrderHom", "code": "@[simp]\ntheorem coe_comp_continuousOrderHom (g : EsakiaHom Ξ² Ξ³) (f : EsakiaHom Ξ± Ξ²) :\n (g.comp f : Ξ± β†’Co Ξ³) = (g: Ξ² β†’Co Ξ³).comp f", "start": [ 320, 1 ], "end": [ 322, 54 ], "kind": "commanddeclaration" }, { "full_name": "EsakiaHom.coe_comp_pseudoEpimorphism", "code": "@[simp]\ntheorem coe_comp_pseudoEpimorphism (g : EsakiaHom Ξ² Ξ³) (f : EsakiaHom Ξ± Ξ²) :\n (g.comp f : PseudoEpimorphism Ξ± Ξ³) = (g : PseudoEpimorphism Ξ² Ξ³).comp f", "start": [ 325, 1 ], "end": [ 327, 83 ], "kind": "commanddeclaration" }, { "full_name": "EsakiaHom.coe_comp", "code": "@[simp]\ntheorem coe_comp (g : EsakiaHom Ξ² Ξ³) (f : EsakiaHom Ξ± Ξ²) : (g.comp f : Ξ± β†’ Ξ³) = g ∘ f", "start": [ 330, 1 ], "end": [ 331, 93 ], "kind": "commanddeclaration" }, { "full_name": "EsakiaHom.comp_apply", "code": "@[simp]\ntheorem comp_apply (g : EsakiaHom Ξ² Ξ³) (f : EsakiaHom Ξ± Ξ²) (a : Ξ±) : (g.comp f) a = g (f a)", "start": [ 334, 1 ], "end": [ 335, 99 ], "kind": "commanddeclaration" }, { "full_name": "EsakiaHom.comp_assoc", "code": "@[simp]\ntheorem comp_assoc (h : EsakiaHom Ξ³ Ξ΄) (g : EsakiaHom Ξ² Ξ³) (f : EsakiaHom Ξ± Ξ²) :\n (h.comp g).comp f = h.comp (g.comp f)", "start": [ 338, 1 ], "end": [ 340, 49 ], "kind": "commanddeclaration" }, { "full_name": "EsakiaHom.comp_id", "code": "@[simp]\ntheorem comp_id (f : EsakiaHom Ξ± Ξ²) : f.comp (EsakiaHom.id Ξ±) = f", "start": [ 343, 1 ], "end": [ 345, 19 ], "kind": "commanddeclaration" }, { "full_name": "EsakiaHom.id_comp", "code": "@[simp]\ntheorem id_comp (f : EsakiaHom Ξ± Ξ²) : (EsakiaHom.id Ξ²).comp f = f", "start": [ 348, 1 ], "end": [ 350, 19 ], "kind": "commanddeclaration" }, { "full_name": "EsakiaHom.cancel_right", "code": "@[simp]\ntheorem cancel_right {g₁ gβ‚‚ : EsakiaHom Ξ² Ξ³} {f : EsakiaHom Ξ± Ξ²} (hf : Surjective f) :\n g₁.comp f = gβ‚‚.comp f ↔ g₁ = gβ‚‚", "start": [ 353, 1 ], "end": [ 356, 78 ], "kind": "commanddeclaration" }, { "full_name": "EsakiaHom.cancel_left", "code": "@[simp]\ntheorem cancel_left {g : EsakiaHom Ξ² Ξ³} {f₁ fβ‚‚ : EsakiaHom Ξ± Ξ²} (hg : Injective g) :\n g.comp f₁ = g.comp fβ‚‚ ↔ f₁ = fβ‚‚", "start": [ 359, 1 ], "end": [ 362, 81 ], "kind": "commanddeclaration" } ]
Mathlib/Analysis/Convex/EGauge.lean
[ ".lake/packages/lean4/src/lean/Init.lean", "Mathlib/Analysis/Seminorm.lean" ]
[ { "full_name": "egauge", "code": "noncomputable def egauge (π•œ : Type*) [NNNorm π•œ] {E : Type*} [SMul π•œ E] (s : Set E) (x : E) : ℝβ‰₯0∞ :=\n β¨… (c : π•œ) (_ : x ∈ c β€’ s), β€–cβ€–β‚Š", "start": [ 32, 1 ], "end": [ 43, 34 ], "kind": "commanddeclaration" }, { "full_name": "egauge_anti", "code": "@[mono, gcongr]\nlemma egauge_anti (h : s βŠ† t) (x : E) : egauge π•œ t x ≀ egauge π•œ s x :=\n iInf_mono fun _c ↦ iInf_mono' fun hc ↦ ⟨smul_set_mono h hc, le_rfl⟩", "start": [ 47, 1 ], "end": [ 49, 70 ], "kind": "lemma" }, { "full_name": "egauge_empty", "code": "@[simp] lemma egauge_empty (x : E) : egauge π•œ βˆ… x = ∞ := by simp [egauge]", "start": [ 51, 1 ], "end": [ 51, 74 ], "kind": "lemma" }, { "full_name": "egauge_le_of_mem_smul", "code": "lemma egauge_le_of_mem_smul (h : x ∈ c β€’ s) : egauge π•œ s x ≀ β€–cβ€–β‚Š := iInfβ‚‚_le c h", "start": [ 55, 1 ], "end": [ 55, 82 ], "kind": "lemma" }, { "full_name": "le_egauge_iff", "code": "lemma le_egauge_iff : r ≀ egauge π•œ s x ↔ βˆ€ c : π•œ, x ∈ c β€’ s β†’ r ≀ β€–cβ€–β‚Š := le_iInfβ‚‚_iff", "start": [ 57, 1 ], "end": [ 57, 87 ], "kind": "lemma" }, { "full_name": "egauge_eq_top", "code": "lemma egauge_eq_top : egauge π•œ s x = ∞ ↔ βˆ€ c : π•œ, x βˆ‰ c β€’ s := by simp [egauge]", "start": [ 59, 1 ], "end": [ 59, 80 ], "kind": "lemma" }, { "full_name": "egauge_lt_iff", "code": "lemma egauge_lt_iff : egauge π•œ s x < r ↔ βˆƒ c : π•œ, x ∈ c β€’ s ∧ β€–cβ€–β‚Š < r := by\n simp [egauge, iInf_lt_iff]", "start": [ 61, 1 ], "end": [ 62, 29 ], "kind": "lemma" }, { "full_name": "egauge_zero_left_eq_top", "code": "@[simp] lemma egauge_zero_left_eq_top : egauge π•œ 0 x = ∞ ↔ x β‰  0 := by\n simp [egauge_eq_top]", "start": [ 71, 1 ], "end": [ 72, 23 ], "kind": "lemma" }, { "full_name": "egauge_le_of_smul_mem_of_ne", "code": "lemma egauge_le_of_smul_mem_of_ne (h : c β€’ x ∈ s) (hc : c β‰  0) :\n egauge π•œ s x ≀ ↑(β€–cβ€–β‚Šβ»ΒΉ : ℝβ‰₯0) := by\n rw [← nnnorm_inv]\n exact egauge_le_of_mem_smul <| (mem_inv_smul_set_iffβ‚€ hc _ _).2 h", "start": [ 83, 1 ], "end": [ 89, 68 ], "kind": "lemma" }, { "full_name": "egauge_le_of_smul_mem", "code": "lemma egauge_le_of_smul_mem (h : c β€’ x ∈ s) : egauge π•œ s x ≀ (β€–cβ€–β‚Š : ℝβ‰₯0∞)⁻¹ := by\n rcases eq_or_ne c 0 with rfl | hc\n Β· simp\n Β· exact (egauge_le_of_smul_mem_of_ne h hc).trans ENNReal.coe_inv_le", "start": [ 91, 1 ], "end": [ 97, 70 ], "kind": "lemma" }, { "full_name": "mem_of_egauge_lt_one", "code": "lemma mem_of_egauge_lt_one (hs : Balanced π•œ s) (hx : egauge π•œ s x < 1) : x ∈ s :=\n let ⟨c, hxc, hc⟩ := egauge_lt_iff.1 hx\n hs c (mod_cast hc.le) hxc", "start": [ 99, 1 ], "end": [ 101, 28 ], "kind": "lemma" }, { "full_name": "egauge_zero_right", "code": "@[simp]\nlemma egauge_zero_right (hs : s.Nonempty) : egauge π•œ s 0 = 0 := by\n have : 0 ∈ (0 : π•œ) β€’ s := by simp [zero_smul_set hs]\n simpa using egauge_le_of_mem_smul this", "start": [ 105, 1 ], "end": [ 108, 41 ], "kind": "lemma" }, { "full_name": "egauge_zero_zero", "code": "@[simp]\nlemma egauge_zero_zero : egauge π•œ (0 : Set E) 0 = 0 := egauge_zero_right _ ⟨0, rfl⟩", "start": [ 110, 1 ], "end": [ 111, 84 ], "kind": "lemma" }, { "full_name": "egauge_le_one", "code": "lemma egauge_le_one (h : x ∈ s) : egauge π•œ s x ≀ 1 := by\n rw [← one_smul π•œ s] at h\n simpa using egauge_le_of_mem_smul h", "start": [ 113, 1 ], "end": [ 115, 38 ], "kind": "lemma" }, { "full_name": "le_egauge_smul_left", "code": "lemma le_egauge_smul_left (c : π•œ) (s : Set E) (x : E) :\n egauge π•œ s x / β€–cβ€–β‚Š ≀ egauge π•œ (c β€’ s) x := by\n simp_rw [le_egauge_iff, smul_smul]\n rintro a ⟨x, hx, rfl⟩\n apply ENNReal.div_le_of_le_mul\n rw [← ENNReal.coe_mul, ← nnnorm_mul]\n exact egauge_le_of_mem_smul <| smul_mem_smul_set hx", "start": [ 119, 1 ], "end": [ 125, 54 ], "kind": "lemma" }, { "full_name": "egauge_smul_left", "code": "lemma egauge_smul_left (hc : c β‰  0) (s : Set E) (x : E) :\n egauge π•œ (c β€’ s) x = egauge π•œ s x / β€–cβ€–β‚Š := by\n refine le_antisymm ?_ (le_egauge_smul_left _ _ _)\n rw [ENNReal.le_div_iff_mul_le (by simp [*]) (by simp)]\n calc\n egauge π•œ (c β€’ s) x * β€–cβ€–β‚Š = egauge π•œ (c β€’ s) x / β€–cβ»ΒΉβ€–β‚Š := by\n rw [nnnorm_inv, ENNReal.coe_inv (by simpa), div_eq_mul_inv, inv_inv]\n _ ≀ egauge π•œ (c⁻¹ β€’ c β€’ s) x := le_egauge_smul_left _ _ _\n _ = egauge π•œ s x := by rw [inv_smul_smulβ‚€ hc]", "start": [ 127, 1 ], "end": [ 135, 50 ], "kind": "lemma" }, { "full_name": "le_egauge_smul_right", "code": "lemma le_egauge_smul_right (c : π•œ) (s : Set E) (x : E) :\n β€–cβ€–β‚Š * egauge π•œ s x ≀ egauge π•œ s (c β€’ x) := by\n rw [le_egauge_iff]\n rintro a ⟨y, hy, hxy⟩\n rcases eq_or_ne c 0 with rfl | hc\n Β· simp\n Β· refine ENNReal.mul_le_of_le_div' <| le_trans ?_ ENNReal.coe_div_le\n rw [div_eq_inv_mul, ← nnnorm_inv, ← nnnorm_mul]\n refine egauge_le_of_mem_smul ⟨y, hy, ?_⟩\n simp only [mul_smul, hxy, inv_smul_smulβ‚€ hc]", "start": [ 137, 1 ], "end": [ 146, 49 ], "kind": "lemma" }, { "full_name": "egauge_smul_right", "code": "lemma egauge_smul_right (h : c = 0 β†’ s.Nonempty) (x : E) :\n egauge π•œ s (c β€’ x) = β€–cβ€–β‚Š * egauge π•œ s x := by\n refine le_antisymm ?_ (le_egauge_smul_right c s x)\n rcases eq_or_ne c 0 with rfl | hc\n Β· simp [egauge_zero_right _ (h rfl)]\n Β· rw [mul_comm, ← ENNReal.div_le_iff_le_mul (.inl <| by simpa) (.inl ENNReal.coe_ne_top),\n ENNReal.div_eq_inv_mul, ← ENNReal.coe_inv (by simpa), ← nnnorm_inv]\n refine (le_egauge_smul_right _ _ _).trans_eq ?_\n rw [inv_smul_smulβ‚€ hc]", "start": [ 148, 1 ], "end": [ 156, 27 ], "kind": "lemma" }, { "full_name": "div_le_egauge_closedBall", "code": "lemma div_le_egauge_closedBall (r : ℝβ‰₯0) (x : E) : β€–xβ€–β‚Š / r ≀ egauge π•œ (closedBall 0 r) x := by\n rw [le_egauge_iff]\n rintro c ⟨y, hy, rfl⟩\n rw [mem_closedBall_zero_iff, ← coe_nnnorm, NNReal.coe_le_coe] at hy\n simp only [nnnorm_smul, ENNReal.coe_mul]\n apply ENNReal.div_le_of_le_mul\n gcongr", "start": [ 165, 1 ], "end": [ 171, 9 ], "kind": "lemma" }, { "full_name": "le_egauge_closedBall_one", "code": "lemma le_egauge_closedBall_one (x : E) : β€–xβ€–β‚Š ≀ egauge π•œ (closedBall 0 1) x := by\n simpa using div_le_egauge_closedBall π•œ 1 x", "start": [ 173, 1 ], "end": [ 174, 45 ], "kind": "lemma" }, { "full_name": "div_le_egauge_ball", "code": "lemma div_le_egauge_ball (r : ℝβ‰₯0) (x : E) : β€–xβ€–β‚Š / r ≀ egauge π•œ (ball 0 r) x :=\n (div_le_egauge_closedBall π•œ r x).trans <| egauge_anti _ ball_subset_closedBall _", "start": [ 176, 1 ], "end": [ 177, 83 ], "kind": "lemma" }, { "full_name": "le_egauge_ball_one", "code": "lemma le_egauge_ball_one (x : E) : β€–xβ€–β‚Š ≀ egauge π•œ (ball 0 1) x := by\n simpa using div_le_egauge_ball π•œ 1 x", "start": [ 179, 1 ], "end": [ 180, 39 ], "kind": "lemma" }, { "full_name": "egauge_ball_le_of_one_lt_norm", "code": "lemma egauge_ball_le_of_one_lt_norm (hc : 1 < β€–cβ€–) (hβ‚€ : r β‰  0 ∨ x β‰  0) :\n egauge π•œ (ball 0 r) x ≀ β€–cβ€–β‚Š * β€–xβ€–β‚Š / r := by\n rcases (zero_le r).eq_or_lt with rfl | hr\n Β· rw [ENNReal.coe_zero, ENNReal.div_zero (mul_ne_zero _ _)]\n Β· apply le_top\n Β· simpa using one_pos.trans hc\n Β· simpa using hβ‚€\n Β· rcases eq_or_ne x 0 with rfl | hx\n Β· rw [egauge_zero_right] <;> simp [*]\n rcases rescale_to_shell hc hr hx with ⟨a, haβ‚€, har, -, hainv⟩\n calc\n egauge π•œ (ball 0 r) x ≀ ↑(β€–aβ€–β‚Šβ»ΒΉ) := egauge_le_of_smul_mem_of_ne (mem_ball_zero_iff.2 har) haβ‚€\n _ ≀ ↑(β€–cβ€–β‚Š * β€–xβ€–β‚Š / r) := by rwa [ENNReal.coe_le_coe, div_eq_inv_mul, ← mul_assoc]\n _ ≀ β€–cβ€–β‚Š * β€–xβ€–β‚Š / r := ENNReal.coe_div_le.trans <| by rw [ENNReal.coe_mul]", "start": [ 189, 1 ], "end": [ 202, 81 ], "kind": "lemma" }, { "full_name": "egauge_ball_one_le_of_one_lt_norm", "code": "lemma egauge_ball_one_le_of_one_lt_norm (hc : 1 < β€–cβ€–) (x : E) :\n egauge π•œ (ball 0 1) x ≀ β€–cβ€–β‚Š * β€–xβ€–β‚Š := by\n simpa using egauge_ball_le_of_one_lt_norm hc (.inl one_ne_zero)", "start": [ 204, 1 ], "end": [ 206, 66 ], "kind": "lemma" } ]
Mathlib/CategoryTheory/Localization/FiniteProducts.lean
[ "Mathlib/CategoryTheory/Localization/HasLocalization.lean", "Mathlib/CategoryTheory/Localization/Adjunction.lean", "Mathlib/CategoryTheory/MorphismProperty/Limits.lean", ".lake/packages/lean4/src/lean/Init.lean", "Mathlib/CategoryTheory/Limits/Preserves/Finite.lean", "Mathlib/CategoryTheory/Limits/ConeCategory.lean", "Mathlib/CategoryTheory/Localization/Pi.lean" ]
[ { "full_name": "CategoryTheory.Localization.HasProductsOfShapeAux.inverts", "code": "lemma inverts :\n (W.functorCategory (Discrete J)).IsInvertedBy (lim β‹™ L) :=\n fun _ _ f hf => Localization.inverts L W _ (hW.lim_map f hf)", "start": [ 38, 1 ], "end": [ 40, 63 ], "kind": "lemma" }, { "full_name": "CategoryTheory.Localization.HasProductsOfShapeAux.limitFunctor", "code": "noncomputable abbrev limitFunctor :\n (Discrete J β₯€ D) β₯€ D :=\n Localization.lift _ (inverts L hW)\n ((whiskeringRight (Discrete J) C D).obj L)", "start": [ 42, 1 ], "end": [ 47, 47 ], "kind": "commanddeclaration" }, { "full_name": "CategoryTheory.Localization.HasProductsOfShapeAux.compLimitFunctorIso", "code": "noncomputable def compLimitFunctorIso :\n ((whiskeringRight (Discrete J) C D).obj L) β‹™ limitFunctor L hW β‰…\n lim β‹™ L := by\n apply Localization.fac", "start": [ 49, 1 ], "end": [ 53, 25 ], "kind": "commanddeclaration" }, { "full_name": "CategoryTheory.Localization.HasProductsOfShapeAux.adj", "code": "noncomputable def adj :\n Functor.const _ ⊣ limitFunctor L hW :=\n constLimAdj.localization L W ((whiskeringRight (Discrete J) C D).obj L)\n (W.functorCategory (Discrete J)) (Functor.const _) (limitFunctor L hW)", "start": [ 64, 1 ], "end": [ 69, 75 ], "kind": "commanddeclaration" }, { "full_name": "CategoryTheory.Localization.HasProductsOfShapeAux.adj_counit_app", "code": "lemma adj_counit_app (F : Discrete J β₯€ C) :\n (adj L hW).counit.app (F β‹™ L) =\n (Functor.const (Discrete J)).map ((compLimitFunctorIso L hW).hom.app F) ≫\n (Functor.compConstIso (Discrete J) L).hom.app (lim.obj F) ≫\n whiskerRight (constLimAdj.counit.app F) L := by\n apply constLimAdj.localization_counit_app", "start": [ 71, 1 ], "end": [ 76, 44 ], "kind": "lemma" }, { "full_name": "CategoryTheory.Localization.HasProductsOfShapeAux.isLimitMapCone", "code": "noncomputable def isLimitMapCone (F : Discrete J β₯€ C) :\n IsLimit (L.mapCone (limit.cone F)) :=\n IsLimit.ofIsoLimit (isLimitConeOfAdj (adj L hW) (F β‹™ L))\n (Cones.ext ((compLimitFunctorIso L hW).app F) (by simp [adj_counit_app, constLimAdj]))", "start": [ 78, 1 ], "end": [ 82, 91 ], "kind": "commanddeclaration" }, { "full_name": "CategoryTheory.Localization.hasProductsOfShape", "code": "lemma hasProductsOfShape (J : Type) [Finite J] [HasProductsOfShape J C]\n (hW : W.IsStableUnderProductsOfShape J) :\n HasProductsOfShape J D :=\n hasLimitsOfShape_iff_isLeftAdjoint_const.2\n (HasProductsOfShapeAux.adj L hW).isLeftAdjoint", "start": [ 88, 1 ], "end": [ 92, 51 ], "kind": "lemma" }, { "full_name": "CategoryTheory.Localization.preservesProductsOfShape", "code": "noncomputable def preservesProductsOfShape (J : Type) [Finite J]\n [HasProductsOfShape J C] (hW : W.IsStableUnderProductsOfShape J) :\n PreservesLimitsOfShape (Discrete J) L where\n preservesLimit {F} := preservesLimitOfPreservesLimitCone (limit.isLimit F)\n (HasProductsOfShapeAux.isLimitMapCone L hW F)", "start": [ 94, 1 ], "end": [ 101, 50 ], "kind": "commanddeclaration" }, { "full_name": "CategoryTheory.Localization.hasFiniteProducts", "code": "lemma hasFiniteProducts : HasFiniteProducts D :=\n ⟨fun _ => hasProductsOfShape L W _\n (W.isStableUnderProductsOfShape_of_isStableUnderFiniteProducts _)⟩", "start": [ 105, 1 ], "end": [ 107, 71 ], "kind": "lemma" }, { "full_name": "CategoryTheory.Localization.preservesFiniteProducts", "code": "noncomputable def preservesFiniteProducts :\n PreservesFiniteProducts L where\n preserves J _ := preservesProductsOfShape L W J\n (W.isStableUnderProductsOfShape_of_isStableUnderFiniteProducts _)", "start": [ 109, 1 ], "end": [ 115, 72 ], "kind": "commanddeclaration" } ]
Mathlib/Analysis/Fourier/RiemannLebesgueLemma.lean
[ "Mathlib/MeasureTheory/Function/ContinuousMapDense.lean", "Mathlib/MeasureTheory/Integral/SetIntegral.lean", ".lake/packages/lean4/src/lean/Init.lean", "Mathlib/Analysis/Fourier/FourierTransform.lean", "Mathlib/Analysis/InnerProductSpace/Dual.lean", "Mathlib/Analysis/InnerProductSpace/EuclideanDist.lean", "Mathlib/Topology/EMetricSpace/Paracompact.lean", "Mathlib/MeasureTheory/Group/Integral.lean", "Mathlib/MeasureTheory/Measure/Haar/NormedSpace.lean", "Mathlib/MeasureTheory/Measure/Haar/Unique.lean" ]
[ { "full_name": "fourierIntegral_half_period_translate", "code": "theorem fourierIntegral_half_period_translate {w : V} (hw : w β‰  0) :\n (∫ v : V, 𝐞 (-βŸͺv, w⟫) β€’ f (v + i w)) = -∫ v : V, 𝐞 (-βŸͺv, w⟫) β€’ f v", "start": [ 67, 1 ], "end": [ 92, 37 ], "kind": "commanddeclaration" }, { "full_name": "fourierIntegral_eq_half_sub_half_period_translate", "code": "theorem fourierIntegral_eq_half_sub_half_period_translate {w : V} (hw : w β‰  0)\n (hf : Integrable f) :\n ∫ v : V, 𝐞 (-βŸͺv, w⟫) β€’ f v = (1 / (2 : β„‚)) β€’ ∫ v : V, 𝐞 (-βŸͺv, w⟫) β€’ (f v - f (v + i w))", "start": [ 95, 1 ], "end": [ 104, 69 ], "kind": "commanddeclaration" }, { "full_name": "tendsto_integral_exp_inner_smul_cocompact_of_continuous_compact_support", "code": "theorem tendsto_integral_exp_inner_smul_cocompact_of_continuous_compact_support (hf1 : Continuous f)\n (hf2 : HasCompactSupport f) :\n Tendsto (fun w : V => ∫ v : V, 𝐞 (-βŸͺv, w⟫) β€’ f v) (cocompact V) (𝓝 0)", "start": [ 107, 1 ], "end": [ 194, 74 ], "kind": "commanddeclaration" }, { "full_name": "tendsto_integral_exp_inner_smul_cocompact", "code": "theorem tendsto_integral_exp_inner_smul_cocompact :\n Tendsto (fun w : V => ∫ v, 𝐞 (-βŸͺv, w⟫) β€’ f v) (cocompact V) (𝓝 0)", "start": [ 199, 1 ], "end": [ 226, 39 ], "kind": "commanddeclaration" }, { "full_name": "Real.tendsto_integral_exp_smul_cocompact", "code": "theorem Real.tendsto_integral_exp_smul_cocompact (f : ℝ β†’ E) :\n Tendsto (fun w : ℝ => ∫ v : ℝ, 𝐞 (-(v * w)) β€’ f v) (cocompact ℝ) (𝓝 0)", "start": [ 229, 1 ], "end": [ 232, 46 ], "kind": "commanddeclaration" }, { "full_name": "Real.zero_at_infty_fourierIntegral", "code": "theorem Real.zero_at_infty_fourierIntegral (f : ℝ β†’ E) : Tendsto (𝓕 f) (cocompact ℝ) (𝓝 0)", "start": [ 235, 1 ], "end": [ 237, 46 ], "kind": "commanddeclaration" }, { "full_name": "tendsto_integral_exp_smul_cocompact_of_inner_product", "code": "theorem tendsto_integral_exp_smul_cocompact_of_inner_product (ΞΌ : Measure V) [ΞΌ.IsAddHaarMeasure] :\n Tendsto (fun w : V β†’L[ℝ] ℝ => ∫ v, 𝐞 (-w v) β€’ f v βˆ‚ΞΌ) (cocompact (V β†’L[ℝ] ℝ)) (𝓝 0)", "start": [ 240, 1 ], "end": [ 256, 55 ], "kind": "commanddeclaration" }, { "full_name": "tendsto_integral_exp_smul_cocompact", "code": "theorem tendsto_integral_exp_smul_cocompact (ΞΌ : Measure V) [ΞΌ.IsAddHaarMeasure] :\n Tendsto (fun w : V β†’L[ℝ] ℝ => ∫ v, 𝐞 (-w v) β€’ f v βˆ‚ΞΌ) (cocompact (V β†’L[ℝ] ℝ)) (𝓝 0)", "start": [ 267, 1 ], "end": [ 320, 60 ], "kind": "commanddeclaration" }, { "full_name": "Real.zero_at_infty_vector_fourierIntegral", "code": "theorem Real.zero_at_infty_vector_fourierIntegral (ΞΌ : Measure V) [ΞΌ.IsAddHaarMeasure] :\n Tendsto (VectorFourier.fourierIntegral 𝐞 ΞΌ (topDualPairing ℝ V).flip f) (cocompact (V β†’L[ℝ] ℝ))\n (𝓝 0)", "start": [ 323, 1 ], "end": [ 329, 49 ], "kind": "commanddeclaration" } ]
Mathlib/Analysis/Calculus/InverseFunctionTheorem/FiniteDimensional.lean
[ "Mathlib/Analysis/Calculus/InverseFunctionTheorem/ApproximatesLinearOn.lean", ".lake/packages/lean4/src/lean/Init.lean", "Mathlib/Analysis/NormedSpace/FiniteDimension.lean" ]
[ { "full_name": "ApproximatesLinearOn.exists_homeomorph_extension", "code": "theorem exists_homeomorph_extension {E : Type*} [NormedAddCommGroup E] [NormedSpace ℝ E]\n {F : Type*} [NormedAddCommGroup F] [NormedSpace ℝ F] [FiniteDimensional ℝ F] {s : Set E}\n {f : E β†’ F} {f' : E ≃L[ℝ] F} {c : ℝβ‰₯0} (hf : ApproximatesLinearOn f (f' : E β†’L[ℝ] F) s c)\n (hc : Subsingleton E ∨ lipschitzExtensionConstant F * c < β€–(f'.symm : F β†’L[ℝ] E)β€–β‚Šβ»ΒΉ) :\n βˆƒ g : E β‰ƒβ‚œ F, EqOn f g s", "start": [ 25, 1 ], "end": [ 47, 35 ], "kind": "commanddeclaration" } ]
Mathlib/Analysis/Convex/Radon.lean
[ ".lake/packages/lean4/src/lean/Init.lean", "Mathlib/Analysis/Convex/Combination.lean", "Mathlib/Tactic/Linarith.lean" ]
[ { "full_name": "radon_partition", "code": "theorem radon_partition (h : Β¬ AffineIndependent π•œ f) :\n βˆƒ I, (convexHull π•œ (f '' I) ∩ convexHull π•œ (f '' Iᢜ)).Nonempty", "start": [ 24, 1 ], "end": [ 50, 60 ], "kind": "commanddeclaration" } ]
Mathlib/RepresentationTheory/Character.lean
[ "Mathlib/LinearAlgebra/Trace.lean", ".lake/packages/lean4/src/lean/Init.lean", "Mathlib/RepresentationTheory/Invariants.lean", "Mathlib/RepresentationTheory/FdRep.lean" ]
[ { "full_name": "FdRep.character", "code": "def character (V : FdRep k G) (g : G) :=\n LinearMap.trace k V (V.ρ g)", "start": [ 48, 1 ], "end": [ 51, 30 ], "kind": "commanddeclaration" }, { "full_name": "FdRep.char_mul_comm", "code": "theorem char_mul_comm (V : FdRep k G) (g : G) (h : G) :\n V.character (h * g) = V.character (g * h)", "start": [ 54, 1 ], "end": [ 55, 99 ], "kind": "commanddeclaration" }, { "full_name": "FdRep.char_one", "code": "@[simp]\ntheorem char_one (V : FdRep k G) : V.character 1 = FiniteDimensional.finrank k V", "start": [ 58, 1 ], "end": [ 60, 44 ], "kind": "commanddeclaration" }, { "full_name": "FdRep.char_tensor", "code": "theorem char_tensor (V W : FdRep k G) : (V βŠ— W).character = V.character * W.character", "start": [ 63, 1 ], "end": [ 65, 54 ], "kind": "commanddeclaration" }, { "full_name": "FdRep.char_tensor'", "code": "@[simp]\ntheorem char_tensor' (V W : FdRep k G) :\n character (Action.FunctorCategoryEquivalence.inverse.obj\n (Action.FunctorCategoryEquivalence.functor.obj V βŠ—\n Action.FunctorCategoryEquivalence.functor.obj W)) = V.character * W.character", "start": [ 69, 1 ], "end": [ 74, 23 ], "kind": "commanddeclaration" }, { "full_name": "FdRep.char_iso", "code": "theorem char_iso {V W : FdRep k G} (i : V β‰… W) : V.character = W.character", "start": [ 76, 1 ], "end": [ 78, 87 ], "kind": "commanddeclaration" }, { "full_name": "FdRep.char_conj", "code": "@[simp]\ntheorem char_conj (V : FdRep k G) (g : G) (h : G) : V.character (h * g * h⁻¹) = V.character g", "start": [ 87, 1 ], "end": [ 90, 42 ], "kind": "commanddeclaration" }, { "full_name": "FdRep.char_dual", "code": "@[simp]\ntheorem char_dual (V : FdRep k G) (g : G) : (of (dual V.ρ)).character g = V.character g⁻¹", "start": [ 93, 1 ], "end": [ 95, 29 ], "kind": "commanddeclaration" }, { "full_name": "FdRep.char_linHom", "code": "@[simp]\ntheorem char_linHom (V W : FdRep k G) (g : G) :\n (of (linHom V.ρ W.ρ)).character g = V.character g⁻¹ * W.character g", "start": [ 98, 1 ], "end": [ 101, 82 ], "kind": "commanddeclaration" }, { "full_name": "FdRep.average_char_eq_finrank_invariants", "code": "theorem average_char_eq_finrank_invariants (V : FdRep k G) :\n β…Ÿ (Fintype.card G : k) β€’ βˆ‘ g : G, V.character g = finrank k (invariants V.ρ)", "start": [ 106, 1 ], "end": [ 109, 57 ], "kind": "commanddeclaration" }, { "full_name": "FdRep.char_orthonormal", "code": "theorem char_orthonormal (V W : FdRep k G) [Simple V] [Simple W] :\n β…Ÿ (Fintype.card G : k) β€’ βˆ‘ g : G, V.character g * W.character g⁻¹ =\n if Nonempty (V β‰… W) then ↑1 else ↑0", "start": [ 122, 1 ], "end": [ 142, 69 ], "kind": "commanddeclaration" } ]
Mathlib/Algebra/Homology/HomotopyCategory/SingleFunctors.lean
[ "Mathlib/CategoryTheory/Shift/SingleFunctors.lean", ".lake/packages/lean4/src/lean/Init.lean", "Mathlib/Algebra/Homology/HomotopyCategory/Shift.lean" ]
[ { "full_name": "CochainComplex.singleFunctors", "code": "noncomputable def singleFunctors : SingleFunctors C (CochainComplex C β„€) β„€ where\n functor n := single _ _ n\n shiftIso n a a' ha' := NatIso.ofComponents\n (fun X => Hom.isoOfComponents\n (fun i => eqToIso (by\n obtain rfl : a' = a + n := by omega\n dsimp [CategoryTheory.shiftFunctor, shiftMonoidalFunctor, single]\n by_cases h : i = a\n Β· subst h\n simp only [ite_true]\n Β· rw [if_neg h, if_neg (fun h' => h (by omega))])) (by simp))\n (fun {X Y} f => by\n obtain rfl : a' = a + n := by omega\n ext\n simp [single])\n shiftIso_zero a := by\n ext\n dsimp\n simp only [single, shiftFunctorZero_eq, shiftFunctorZero'_hom_app_f,\n XIsoOfEq, eqToIso.hom]\n shiftIso_add n m a a' a'' ha' ha'' := by\n ext\n dsimp\n simp only [shiftFunctorAdd_eq, shiftFunctorAdd'_hom_app_f, XIsoOfEq,\n eqToIso.hom, eqToHom_trans, id_comp]", "start": [ 31, 1 ], "end": [ 58, 43 ], "kind": "commanddeclaration" }, { "full_name": "CochainComplex.singleFunctor", "code": "noncomputable abbrev singleFunctor (n : β„€) := (singleFunctors C).functor n", "start": [ 64, 1 ], "end": [ 68, 75 ], "kind": "commanddeclaration" }, { "full_name": "HomotopyCategory.singleFunctors", "code": "noncomputable def singleFunctors : SingleFunctors C (HomotopyCategory C (ComplexShape.up β„€)) β„€ :=\n (CochainComplex.singleFunctors C).postcomp (HomotopyCategory.quotient _ _)", "start": [ 74, 1 ], "end": [ 77, 77 ], "kind": "commanddeclaration" }, { "full_name": "HomotopyCategory.singleFunctor", "code": "noncomputable abbrev singleFunctor (n : β„€) :\n C β₯€ HomotopyCategory C (ComplexShape.up β„€) :=\n (singleFunctors C).functor n", "start": [ 79, 1 ], "end": [ 83, 31 ], "kind": "commanddeclaration" }, { "full_name": "HomotopyCategory.singleFunctorsPostcompQuotientIso", "code": "noncomputable def singleFunctorsPostcompQuotientIso :\n singleFunctors C β‰…\n (CochainComplex.singleFunctors C).postcomp (HomotopyCategory.quotient _ _) :=\n Iso.refl _", "start": [ 89, 1 ], "end": [ 93, 13 ], "kind": "commanddeclaration" }, { "full_name": "HomotopyCategory.singleFunctorPostcompQuotientIso", "code": "noncomputable def singleFunctorPostcompQuotientIso (n : β„€) :\n singleFunctor C n β‰… CochainComplex.singleFunctor C n β‹™ quotient _ _ :=\n (SingleFunctors.evaluation _ _ n).mapIso (singleFunctorsPostcompQuotientIso C)", "start": [ 95, 1 ], "end": [ 98, 81 ], "kind": "commanddeclaration" } ]
Mathlib/Algebra/Lie/CartanMatrix.lean
[ "Mathlib/Data/Matrix/Notation.lean", "Mathlib/Algebra/Lie/Quotient.lean", ".lake/packages/lean4/src/lean/Init.lean", "Mathlib/Algebra/Lie/Free.lean" ]
[ { "full_name": "CartanMatrix.Generators", "code": "inductive Generators\n | H : B β†’ Generators\n | E : B β†’ Generators\n | F : B β†’ Generators", "start": [ 96, 1 ], "end": [ 101, 23 ], "kind": "commanddeclaration" }, { "full_name": "CartanMatrix.Relations.HH", "code": "def HH : B Γ— B β†’ FreeLieAlgebra R (Generators B) :=\n uncurry fun i j => ⁅H i, H j⁆", "start": [ 118, 1 ], "end": [ 120, 32 ], "kind": "commanddeclaration" }, { "full_name": "CartanMatrix.Relations.EF", "code": "def EF : B Γ— B β†’ FreeLieAlgebra R (Generators B) :=\n uncurry fun i j => if i = j then ⁅E i, F i⁆ - H i else ⁅E i, F j⁆", "start": [ 123, 1 ], "end": [ 125, 68 ], "kind": "commanddeclaration" }, { "full_name": "CartanMatrix.Relations.HE", "code": "def HE : B Γ— B β†’ FreeLieAlgebra R (Generators B) :=\n uncurry fun i j => ⁅H i, E j⁆ - A i j β€’ E j", "start": [ 128, 1 ], "end": [ 130, 46 ], "kind": "commanddeclaration" }, { "full_name": "CartanMatrix.Relations.HF", "code": "def HF : B Γ— B β†’ FreeLieAlgebra R (Generators B) :=\n uncurry fun i j => ⁅H i, F j⁆ + A i j β€’ F j", "start": [ 133, 1 ], "end": [ 135, 46 ], "kind": "commanddeclaration" }, { "full_name": "CartanMatrix.Relations.adE", "code": "def adE : B Γ— B β†’ FreeLieAlgebra R (Generators B) :=\n uncurry fun i j => ad (E i) ^ (-A i j).toNat <| ⁅E i, E j⁆", "start": [ 138, 1 ], "end": [ 144, 61 ], "kind": "commanddeclaration" }, { "full_name": "CartanMatrix.Relations.adF", "code": "def adF : B Γ— B β†’ FreeLieAlgebra R (Generators B) :=\n uncurry fun i j => ad (F i) ^ (-A i j).toNat <| ⁅F i, F j⁆", "start": [ 147, 1 ], "end": [ 151, 61 ], "kind": "commanddeclaration" }, { "full_name": "CartanMatrix.Relations.adE_of_eq_eq_zero", "code": "private theorem adE_of_eq_eq_zero (i : B) (h : A i i = 2) : adE R A ⟨i, i⟩ = 0", "start": [ 154, 1 ], "end": [ 156, 20 ], "kind": "commanddeclaration" }, { "full_name": "CartanMatrix.Relations.adF_of_eq_eq_zero", "code": "private theorem adF_of_eq_eq_zero (i : B) (h : A i i = 2) : adF R A ⟨i, i⟩ = 0", "start": [ 158, 1 ], "end": [ 160, 20 ], "kind": "commanddeclaration" }, { "full_name": "CartanMatrix.Relations.toSet", "code": "def toSet : Set (FreeLieAlgebra R (Generators B)) :=\n (Set.range <| HH R) βˆͺ (Set.range <| EF R) βˆͺ (Set.range <| HE R A) βˆͺ (Set.range <| HF R A) βˆͺ\n (Set.range <| adE R A) βˆͺ\n (Set.range <| adF R A)", "start": [ 162, 1 ], "end": [ 166, 27 ], "kind": "commanddeclaration" }, { "full_name": "CartanMatrix.Relations.toIdeal", "code": "def toIdeal : LieIdeal R (FreeLieAlgebra R (Generators B)) :=\n LieSubmodule.lieSpan R _ <| toSet R A", "start": [ 169, 1 ], "end": [ 171, 40 ], "kind": "commanddeclaration" }, { "full_name": "Matrix.ToLieAlgebra", "code": "def Matrix.ToLieAlgebra :=\n FreeLieAlgebra R _ β§Έ CartanMatrix.Relations.toIdeal R A", "start": [ 178, 1 ], "end": [ 183, 58 ], "kind": "commanddeclaration" }, { "full_name": "Matrix.ToLieAlgebra.instLieRing", "code": "instance Matrix.ToLieAlgebra.instLieRing : LieRing (Matrix.ToLieAlgebra R A) :=\n inferInstanceAs (LieRing (FreeLieAlgebra R _ β§Έ CartanMatrix.Relations.toIdeal R A))", "start": [ 187, 1 ], "end": [ 188, 86 ], "kind": "commanddeclaration" }, { "full_name": "Matrix.ToLieAlgebra.instInhabited", "code": "instance Matrix.ToLieAlgebra.instInhabited : Inhabited (Matrix.ToLieAlgebra R A) :=\n inferInstanceAs (Inhabited (FreeLieAlgebra R _ β§Έ CartanMatrix.Relations.toIdeal R A))", "start": [ 191, 1 ], "end": [ 192, 88 ], "kind": "commanddeclaration" }, { "full_name": "Matrix.ToLieAlgebra.instLieAlgebra", "code": "instance Matrix.ToLieAlgebra.instLieAlgebra : LieAlgebra R (Matrix.ToLieAlgebra R A) :=\n inferInstanceAs (LieAlgebra R (FreeLieAlgebra R _ β§Έ CartanMatrix.Relations.toIdeal R A))", "start": [ 195, 1 ], "end": [ 196, 91 ], "kind": "commanddeclaration" }, { "full_name": "CartanMatrix.E₆", "code": "def E₆ : Matrix (Fin 6) (Fin 6) β„€ :=\n !![2, 0, -1, 0, 0, 0;\n 0, 2, 0, -1, 0, 0;\n -1, 0, 2, -1, 0, 0;\n 0, -1, -1, 2, -1, 0;\n 0, 0, 0, -1, 2, -1;\n 0, 0, 0, 0, -1, 2]", "start": [ 201, 1 ], "end": [ 216, 23 ], "kind": "commanddeclaration" }, { "full_name": "CartanMatrix.E₇", "code": "def E₇ : Matrix (Fin 7) (Fin 7) β„€ :=\n !![2, 0, -1, 0, 0, 0, 0;\n 0, 2, 0, -1, 0, 0, 0;\n -1, 0, 2, -1, 0, 0, 0;\n 0, -1, -1, 2, -1, 0, 0;\n 0, 0, 0, -1, 2, -1, 0;\n 0, 0, 0, 0, -1, 2, -1;\n 0, 0, 0, 0, 0, -1, 2]", "start": [ 219, 1 ], "end": [ 235, 26 ], "kind": "commanddeclaration" }, { "full_name": "CartanMatrix.Eβ‚ˆ", "code": "def Eβ‚ˆ : Matrix (Fin 8) (Fin 8) β„€ :=\n !![2, 0, -1, 0, 0, 0, 0, 0;\n 0, 2, 0, -1, 0, 0, 0, 0;\n -1, 0, 2, -1, 0, 0, 0, 0;\n 0, -1, -1, 2, -1, 0, 0, 0;\n 0, 0, 0, -1, 2, -1, 0, 0;\n 0, 0, 0, 0, -1, 2, -1, 0;\n 0, 0, 0, 0, 0, -1, 2, -1;\n 0, 0, 0, 0, 0, 0, -1, 2]", "start": [ 238, 1 ], "end": [ 255, 29 ], "kind": "commanddeclaration" }, { "full_name": "CartanMatrix.Fβ‚„", "code": "def Fβ‚„ : Matrix (Fin 4) (Fin 4) β„€ :=\n !![2, -1, 0, 0; -1, 2, -2, 0; 0, -1, 2, -1; 0, 0, -1, 2]", "start": [ 258, 1 ], "end": [ 266, 59 ], "kind": "commanddeclaration" }, { "full_name": "CartanMatrix.Gβ‚‚", "code": "def Gβ‚‚ : Matrix (Fin 2) (Fin 2) β„€ :=\n !![2, -3; -1, 2]", "start": [ 269, 1 ], "end": [ 278, 19 ], "kind": "commanddeclaration" }, { "full_name": "LieAlgebra.e₆", "code": "abbrev e₆ :=\n CartanMatrix.E₆.ToLieAlgebra R", "start": [ 285, 1 ], "end": [ 287, 33 ], "kind": "commanddeclaration" }, { "full_name": "LieAlgebra.e₇", "code": "abbrev e₇ :=\n CartanMatrix.E₇.ToLieAlgebra R", "start": [ 290, 1 ], "end": [ 292, 33 ], "kind": "commanddeclaration" }, { "full_name": "LieAlgebra.eβ‚ˆ", "code": "abbrev eβ‚ˆ :=\n CartanMatrix.Eβ‚ˆ.ToLieAlgebra R", "start": [ 295, 1 ], "end": [ 297, 33 ], "kind": "commanddeclaration" }, { "full_name": "LieAlgebra.fβ‚„", "code": "abbrev fβ‚„ :=\n CartanMatrix.Fβ‚„.ToLieAlgebra R", "start": [ 300, 1 ], "end": [ 302, 33 ], "kind": "commanddeclaration" }, { "full_name": "LieAlgebra.gβ‚‚", "code": "abbrev gβ‚‚ :=\n CartanMatrix.Gβ‚‚.ToLieAlgebra R", "start": [ 305, 1 ], "end": [ 307, 33 ], "kind": "commanddeclaration" } ]
Mathlib/SetTheory/ZFC/Ordinal.lean
[ ".lake/packages/lean4/src/lean/Init.lean", "Mathlib/SetTheory/ZFC/Basic.lean" ]
[ { "full_name": "ZFSet.IsTransitive", "code": "def IsTransitive (x : ZFSet) : Prop :=\n βˆ€ y ∈ x, y βŠ† x", "start": [ 39, 1 ], "end": [ 41, 17 ], "kind": "commanddeclaration" }, { "full_name": "ZFSet.empty_isTransitive", "code": "@[simp]\ntheorem empty_isTransitive : IsTransitive βˆ…", "start": [ 44, 1 ], "end": [ 45, 85 ], "kind": "commanddeclaration" }, { "full_name": "ZFSet.IsTransitive.subset_of_mem", "code": "theorem IsTransitive.subset_of_mem (h : x.IsTransitive) : y ∈ x β†’ y βŠ† x", "start": [ 48, 1 ], "end": [ 49, 6 ], "kind": "commanddeclaration" }, { "full_name": "ZFSet.isTransitive_iff_mem_trans", "code": "theorem isTransitive_iff_mem_trans : z.IsTransitive ↔ βˆ€ {x y : ZFSet}, x ∈ y β†’ y ∈ z β†’ x ∈ z", "start": [ 52, 1 ], "end": [ 53, 73 ], "kind": "commanddeclaration" }, { "full_name": "ZFSet.IsTransitive.inter", "code": "protected theorem IsTransitive.inter (hx : x.IsTransitive) (hy : y.IsTransitive) :\n (x ∩ y).IsTransitive", "start": [ 59, 1 ], "end": [ 62, 53 ], "kind": "commanddeclaration" }, { "full_name": "ZFSet.IsTransitive.sUnion", "code": "protected theorem IsTransitive.sUnion (h : x.IsTransitive) :\n (⋃₀ x : ZFSet).IsTransitive", "start": [ 65, 1 ], "end": [ 68, 50 ], "kind": "commanddeclaration" }, { "full_name": "ZFSet.IsTransitive.sUnion'", "code": "theorem IsTransitive.sUnion' (H : βˆ€ y ∈ x, IsTransitive y) :\n (⋃₀ x : ZFSet).IsTransitive", "start": [ 71, 1 ], "end": [ 74, 57 ], "kind": "commanddeclaration" }, { "full_name": "ZFSet.IsTransitive.union", "code": "protected theorem IsTransitive.union (hx : x.IsTransitive) (hy : y.IsTransitive) :\n (x βˆͺ y).IsTransitive", "start": [ 77, 1 ], "end": [ 84, 14 ], "kind": "commanddeclaration" }, { "full_name": "ZFSet.IsTransitive.powerset", "code": "protected theorem IsTransitive.powerset (h : x.IsTransitive) : (powerset x).IsTransitive", "start": [ 87, 1 ], "end": [ 90, 32 ], "kind": "commanddeclaration" }, { "full_name": "ZFSet.isTransitive_iff_sUnion_subset", "code": "theorem isTransitive_iff_sUnion_subset : x.IsTransitive ↔ (⋃₀ x : ZFSet) βŠ† x", "start": [ 93, 1 ], "end": [ 96, 79 ], "kind": "commanddeclaration" }, { "full_name": "ZFSet.isTransitive_iff_subset_powerset", "code": "theorem isTransitive_iff_subset_powerset : x.IsTransitive ↔ x βŠ† powerset x", "start": [ 102, 1 ], "end": [ 103, 100 ], "kind": "commanddeclaration" } ]
Mathlib/Analysis/InnerProductSpace/LaxMilgram.lean
[ ".lake/packages/lean4/src/lean/Init.lean", "Mathlib/Analysis/InnerProductSpace/Dual.lean" ]
[ { "full_name": "IsCoercive.bounded_below", "code": "theorem bounded_below (coercive : IsCoercive B) : βˆƒ C, 0 < C ∧ βˆ€ v, C * β€–vβ€– ≀ β€–Bβ™― vβ€–", "start": [ 51, 1 ], "end": [ 62, 16 ], "kind": "commanddeclaration" }, { "full_name": "IsCoercive.antilipschitz", "code": "theorem antilipschitz (coercive : IsCoercive B) : βˆƒ C : ℝβ‰₯0, 0 < C ∧ AntilipschitzWith C Bβ™―", "start": [ 65, 1 ], "end": [ 71, 26 ], "kind": "commanddeclaration" }, { "full_name": "IsCoercive.ker_eq_bot", "code": "theorem ker_eq_bot (coercive : IsCoercive B) : ker Bβ™― = βŠ₯", "start": [ 74, 1 ], "end": [ 77, 32 ], "kind": "commanddeclaration" }, { "full_name": "IsCoercive.isClosed_range", "code": "theorem isClosed_range (coercive : IsCoercive B) : IsClosed (range Bβ™― : Set V)", "start": [ 80, 1 ], "end": [ 82, 58 ], "kind": "commanddeclaration" }, { "full_name": "IsCoercive.range_eq_top", "code": "theorem range_eq_top (coercive : IsCoercive B) : range Bβ™― = ⊀", "start": [ 87, 1 ], "end": [ 102, 26 ], "kind": "commanddeclaration" }, { "full_name": "IsCoercive.continuousLinearEquivOfBilin", "code": "def continuousLinearEquivOfBilin (coercive : IsCoercive B) : V ≃L[ℝ] V :=\n ContinuousLinearEquiv.ofBijective Bβ™― coercive.ker_eq_bot coercive.range_eq_top", "start": [ 105, 1 ], "end": [ 111, 81 ], "kind": "commanddeclaration" }, { "full_name": "IsCoercive.continuousLinearEquivOfBilin_apply", "code": "@[simp]\ntheorem continuousLinearEquivOfBilin_apply (coercive : IsCoercive B) (v w : V) :\n βŸͺcoercive.continuousLinearEquivOfBilin v, w⟫_ℝ = B v w", "start": [ 114, 1 ], "end": [ 117, 41 ], "kind": "commanddeclaration" }, { "full_name": "IsCoercive.unique_continuousLinearEquivOfBilin", "code": "theorem unique_continuousLinearEquivOfBilin (coercive : IsCoercive B) {v f : V}\n (is_lax_milgram : βˆ€ w, βŸͺf, w⟫_ℝ = B v w) : f = coercive.continuousLinearEquivOfBilin v", "start": [ 120, 1 ], "end": [ 122, 53 ], "kind": "commanddeclaration" } ]
Mathlib/Data/Buffer/Basic.lean
[ ".lake/packages/lean4/src/lean/Init.lean", "Mathlib/Init/Align.lean" ]
[]
Mathlib/NumberTheory/SiegelsLemma.lean
[ ".lake/packages/lean4/src/lean/Init.lean", "Mathlib/Tactic/Rify.lean", "Mathlib/Analysis/Matrix.lean", "Mathlib/Data/Pi/Interval.lean" ]
[ { "full_name": "Int.Matrix.image_T_subset_S", "code": "private lemma image_T_subset_S (v) (hv : v ∈ T) : A *α΅₯ v ∈ S := by\n rw [mem_Icc] at hv ⊒\n have mulVec_def : A.mulVec v =\n fun i ↦ Finset.sum univ fun j : Fin n ↦ A i j * v j := rfl\n rw [mulVec_def]\n refine ⟨fun i ↦ ?_, fun i ↦ ?_⟩\n all_goals\n simp only [mul_neg]\n gcongr βˆ‘ _ : Fin n, ?_ with j _ rw [← mul_comm (v j)] rcases le_total 0 (A i j) with hsign | hsignΒ· rw [negPart_eq_zero.2 hsign]\n exact mul_nonneg (hv.1 j) hsign\n Β· rw [negPart_eq_neg.2 hsign]\n simp only [mul_neg, neg_neg]\n exact mul_le_mul_of_nonpos_right (hv.2 j) hsign\n Β· rw [posPart_eq_self.2 hsign]\n exact mul_le_mul_of_nonneg_right (hv.2 j) hsign\n Β· rw [posPart_eq_zero.2 hsign]\n exact mul_nonpos_of_nonneg_of_nonpos (hv.1 j) hsign", "start": [ 68, 1 ], "end": [ 87, 56 ], "kind": "lemma" }, { "full_name": "Int.Matrix.card_T_eq", "code": "private lemma card_T_eq : (T).card = (B + 1) ^ n := by\n rw [Pi.card_Icc 0 B']\n simp only [Pi.zero_apply, Int.card_Icc, sub_zero, Int.toNat_ofNat_add_one, prod_const, card_fin]", "start": [ 91, 1 ], "end": [ 93, 99 ], "kind": "lemma" }, { "full_name": "Int.Matrix.N_le_P_add_one", "code": "private lemma N_le_P_add_one (i : Fin m) : N i ≀ P i + 1 := by\n calc N i\n _ ≀ 0 := by\n apply Finset.sum_nonpos\n intro j _\n simp only [mul_neg, Left.neg_nonpos_iff]\n exact mul_nonneg (Nat.cast_nonneg B) (negPart_nonneg (A i j))\n _ ≀ P i + 1 := by\n apply le_trans (Finset.sum_nonneg _) (Int.le_add_one (le_refl P i))\n intro j _\n exact mul_nonneg (Nat.cast_nonneg B) (posPart_nonneg (A i j))", "start": [ 96, 1 ], "end": [ 106, 66 ], "kind": "lemma" }, { "full_name": "Int.Matrix.card_S_eq", "code": "private lemma card_S_eq : (Finset.Icc N P).card = ∏ i : Fin m, (P i - N i + 1) := by\n rw [Pi.card_Icc N P, Nat.cast_prod]\n congr\n ext i\n rw [Int.card_Icc_of_le (N i) (P i) (N_le_P_add_one m n A i)]\n exact add_sub_right_comm (P i) 1 (N i)", "start": [ 108, 1 ], "end": [ 113, 41 ], "kind": "lemma" }, { "full_name": "Int.Matrix.one_le_norm_A_of_ne_zero", "code": "lemma one_le_norm_A_of_ne_zero : 1 ≀ β€–Aβ€– := by\n by_contra! h\n apply hA\n ext i j\n simp only [zero_apply]\n rw [norm_lt_iff Real.zero_lt_one] at h\n specialize h i j\n rw [Int.norm_eq_abs] at h\n norm_cast at h\n exact Int.abs_lt_one_iff.1 h", "start": [ 117, 1 ], "end": [ 127, 31 ], "kind": "lemma" }, { "full_name": "Int.Matrix.card_S_lt_card_T", "code": "private lemma card_S_lt_card_T : (S).card < (T).card := by\n zify rw [card_T_eq, card_S_eq]\n rify calc\n ∏ x : Fin m, (βˆ‘ x_1 : Fin n, ↑B * ↑(A x x_1)⁺ - βˆ‘ x_1 : Fin n, ↑B * -↑(A x x_1)⁻ + 1)\n ≀ (n * β€–Aβ€– * B + 1) ^ m := by\n rw [← Fin.prod_const m (n * β€–Aβ€– * B + 1)] refine Finset.prod_le_prod (fun i _ ↦ ?_) (fun i _ ↦ ?_)\n Β· have h := N_le_P_add_one m n A i\n rify at h\n linarith only [h]\n Β· simp only [mul_neg, sum_neg_distrib, sub_neg_eq_add, add_le_add_iff_right]\n have h1 : n * β€–Aβ€– * B = βˆ‘ _ : Fin n, β€–Aβ€– * B := by\n simp only [sum_const, card_univ, Fintype.card_fin, nsmul_eq_mul, mul_assoc ↑n β€–Aβ€– ↑B]\n simp_rw [h1, ← Finset.sum_add_distrib, ← mul_add, mul_comm β€–Aβ€–, ← Int.cast_add]\n gcongr with j _\n rw [posPart_add_negPart (A i j), Int.cast_abs]\n exact norm_entry_le_entrywise_sup_norm A\n _ ≀ (n * β€–Aβ€–) ^ m * (B + 1) ^ m := by\n rw [← mul_pow, mul_add, mul_one]\n gcongr\n have H : 1 ≀ (n : ℝ) := mod_cast (hm.trans hn)\n exact one_le_mul_of_one_le_of_one_le H <| one_le_norm_A_of_ne_zero m n A hA\n _ = ((n * β€–Aβ€–) ^ (m / ((n : ℝ) - m))) ^ ((n : ℝ) - m) * (B + 1) ^ m := by\n congr 1\n rw [← rpow_mul (mul_nonneg n.cast_nonneg (norm_nonneg A)), ← Real.rpow_natCast,\n div_mul_cancelβ‚€]\n exact sub_ne_zero_of_ne (mod_cast hn.ne')\n _ < (B + 1) ^ ((n : ℝ) - m) * (B + 1) ^ m := by\n gcongr\n Β· exact sub_pos.mpr (mod_cast hn)\n Β· exact Nat.lt_floor_add_one ((n * β€–Aβ€–) ^ e)\n _ = (B + 1) ^ n := by\n rw [← rpow_natCast, ← rpow_add (Nat.cast_add_one_pos B), ← rpow_natCast, sub_add_cancel]", "start": [ 133, 1 ], "end": [ 167, 97 ], "kind": "lemma" }, { "full_name": "Int.Matrix.exists_ne_zero_int_vec_norm_le", "code": "theorem exists_ne_zero_int_vec_norm_le (hA_nezero : A β‰  0) : βˆƒ t : Fin n β†’ β„€, t β‰  0 ∧\n A *α΅₯ t = 0 ∧ β€–tβ€– ≀ (n * β€–Aβ€–) ^ ((m : ℝ) / (n - m))", "start": [ 171, 1 ], "end": [ 199, 18 ], "kind": "commanddeclaration" } ]
Mathlib/Data/ZMod/Coprime.lean
[ ".lake/packages/lean4/src/lean/Init.lean", "Mathlib/RingTheory/PrincipalIdealDomain.lean", "Mathlib/Data/ZMod/Basic.lean", "Mathlib/RingTheory/Int/Basic.lean" ]
[ { "full_name": "ZMod.eq_zero_iff_gcd_ne_one", "code": "theorem eq_zero_iff_gcd_ne_one {a : β„€} {p : β„•} [pp : Fact p.Prime] :\n (a : ZMod p) = 0 ↔ a.gcd p β‰  1", "start": [ 22, 1 ], "end": [ 28, 34 ], "kind": "commanddeclaration" }, { "full_name": "ZMod.ne_zero_of_gcd_eq_one", "code": "theorem ne_zero_of_gcd_eq_one {a : β„€} {p : β„•} (pp : p.Prime) (h : a.gcd p = 1) : (a : ZMod p) β‰  0", "start": [ 31, 1 ], "end": [ 33, 69 ], "kind": "commanddeclaration" }, { "full_name": "ZMod.eq_zero_of_gcd_ne_one", "code": "theorem eq_zero_of_gcd_ne_one {a : β„€} {p : β„•} (pp : p.Prime) (h : a.gcd p β‰  1) : (a : ZMod p) = 0", "start": [ 36, 1 ], "end": [ 38, 43 ], "kind": "commanddeclaration" } ]
Mathlib/Data/Finset/Functor.lean
[ ".lake/packages/lean4/src/lean/Init.lean", "Mathlib/Data/Finset/NAry.lean", "Mathlib/Data/Finset/Lattice.lean", "Mathlib/Data/Multiset/Functor.lean" ]
[ { "full_name": "Finset.functor", "code": "protected instance functor : Functor Finset where map f s := s.image f", "start": [ 37, 1 ], "end": [ 39, 71 ], "kind": "commanddeclaration" }, { "full_name": "Finset.lawfulFunctor", "code": "instance lawfulFunctor : LawfulFunctor Finset where\n id_map s := image_id\n comp_map f g s := image_image.symm\n map_const {Ξ±} {Ξ²} := by simp only [Functor.mapConst, Functor.map]", "start": [ 41, 1 ], "end": [ 44, 68 ], "kind": "commanddeclaration" }, { "full_name": "Finset.fmap_def", "code": "@[simp]\ntheorem fmap_def {s : Finset Ξ±} (f : Ξ± β†’ Ξ²) : f <$> s = s.image f", "start": [ 46, 1 ], "end": [ 47, 73 ], "kind": "commanddeclaration" }, { "full_name": "Finset.pure", "code": "protected instance pure : Pure Finset :=\n ⟨fun x => {x}⟩", "start": [ 55, 1 ], "end": [ 56, 17 ], "kind": "commanddeclaration" }, { "full_name": "Finset.pure_def", "code": "@[simp]\ntheorem pure_def {Ξ±} : (pure : Ξ± β†’ Finset Ξ±) = singleton", "start": [ 58, 1 ], "end": [ 59, 64 ], "kind": "commanddeclaration" }, { "full_name": "Finset.applicative", "code": "protected instance applicative : Applicative Finset :=\n { Finset.functor, Finset.pure with\n seq := fun t s => t.sup fun f => (s ()).image f\n seqLeft := fun s t => if t () = βˆ… then βˆ… else s\n seqRight := fun s t => if s = βˆ… then βˆ… else t () }", "start": [ 69, 1 ], "end": [ 73, 55 ], "kind": "commanddeclaration" }, { "full_name": "Finset.seq_def", "code": "@[simp]\ntheorem seq_def (s : Finset Ξ±) (t : Finset (Ξ± β†’ Ξ²)) : t <*> s = t.sup fun f => s.image f", "start": [ 75, 1 ], "end": [ 77, 6 ], "kind": "commanddeclaration" }, { "full_name": "Finset.seqLeft_def", "code": "@[simp]\ntheorem seqLeft_def (s : Finset Ξ±) (t : Finset Ξ²) : s <* t = if t = βˆ… then βˆ… else s", "start": [ 80, 1 ], "end": [ 82, 6 ], "kind": "commanddeclaration" }, { "full_name": "Finset.seqRight_def", "code": "@[simp]\ntheorem seqRight_def (s : Finset Ξ±) (t : Finset Ξ²) : s *> t = if s = βˆ… then βˆ… else t", "start": [ 85, 1 ], "end": [ 87, 6 ], "kind": "commanddeclaration" }, { "full_name": "Finset.imageβ‚‚_def", "code": "theorem imageβ‚‚_def {Ξ± Ξ² Ξ³ : Type u} (f : Ξ± β†’ Ξ² β†’ Ξ³) (s : Finset Ξ±) (t : Finset Ξ²) :\n imageβ‚‚ f s t = f <$> s <*> t", "start": [ 90, 1 ], "end": [ 95, 17 ], "kind": "commanddeclaration" }, { "full_name": "Finset.lawfulApplicative", "code": "instance lawfulApplicative : LawfulApplicative Finset :=\n { Finset.lawfulFunctor with\n seqLeft_eq := fun s t => by\n rw [seq_def, fmap_def, seqLeft_def]\n obtain rfl | ht := t.eq_empty_or_nonempty\n Β· simp_rw [image_empty, if_true]\n exact (sup_bot _).symm\n Β· ext a\n rw [if_neg ht.ne_empty, mem_sup]\n refine ⟨fun ha => ⟨const _ a, mem_image_of_mem _ ha, mem_image_const_self.2 ht⟩, ?_⟩\n rintro ⟨f, hf, ha⟩\n rw [mem_image] at hf ha\n obtain ⟨b, hb, rfl⟩ := hf\n obtain ⟨_, _, rfl⟩ := ha\n exact hb\n seqRight_eq := fun s t => by\n rw [seq_def, fmap_def, seqRight_def]\n obtain rfl | hs := s.eq_empty_or_nonempty\n Β· rw [if_pos rfl, image_empty, sup_empty, bot_eq_empty]\n Β· ext a\n rw [if_neg hs.ne_empty, mem_sup]\n refine ⟨fun ha => ⟨id, mem_image_const_self.2 hs, by rwa [image_id]⟩, ?_⟩\n rintro ⟨f, hf, ha⟩\n rw [mem_image] at hf ha\n obtain ⟨b, hb, rfl⟩ := ha\n obtain ⟨_, _, rfl⟩ := hf\n exact hb\n pure_seq := fun f s => by simp only [pure_def, seq_def, sup_singleton, fmap_def]\n map_pure := fun f a => image_singleton _ _\n seq_pure := fun s a => sup_singleton'' _ _\n seq_assoc := fun s t u => by\n ext a\n simp_rw [seq_def, fmap_def]\n simp only [exists_prop, mem_sup, mem_image]\n constructor\n Β· rintro ⟨g, hg, b, ⟨f, hf, a, ha, rfl⟩, rfl⟩\n exact ⟨g ∘ f, ⟨comp g, ⟨g, hg, rfl⟩, f, hf, rfl⟩, a, ha, rfl⟩\n Β· rintro ⟨c, ⟨_, ⟨g, hg, rfl⟩, f, hf, rfl⟩, a, ha, rfl⟩\n exact ⟨g, hg, f a, ⟨f, hf, a, ha, rfl⟩, rfl⟩ }", "start": [ 98, 1 ], "end": [ 136, 55 ], "kind": "commanddeclaration" }, { "full_name": "Finset.commApplicative", "code": "instance commApplicative : CommApplicative Finset :=\n { Finset.lawfulApplicative with\n commutative_prod := fun s t => by\n simp_rw [seq_def, fmap_def, sup_image, sup_eq_biUnion]\n change (s.biUnion fun a => t.image fun b => (a, b))\n = t.biUnion fun b => s.image fun a => (a, b)\n trans s Γ—Λ’ t <;> [rw [product_eq_biUnion]; rw [product_eq_biUnion_right]] }", "start": [ 138, 1 ], "end": [ 144, 82 ], "kind": "commanddeclaration" }, { "full_name": "Finset.bind_def", "code": "@[simp]\ntheorem bind_def {Ξ± Ξ²} : (Β· >>= Β·) = sup (Ξ± := Finset Ξ±) (Ξ² := Ξ²)", "start": [ 158, 1 ], "end": [ 160, 6 ], "kind": "commanddeclaration" }, { "full_name": "Finset.traverse", "code": "def traverse [DecidableEq Ξ²] (f : Ξ± β†’ F Ξ²) (s : Finset Ξ±) : F (Finset Ξ²) :=\n Multiset.toFinset <$> Multiset.traverse f s.1", "start": [ 194, 1 ], "end": [ 196, 48 ], "kind": "commanddeclaration" }, { "full_name": "Finset.id_traverse", "code": "@[simp]\ntheorem id_traverse [DecidableEq Ξ±] (s : Finset Ξ±) : traverse (pure : Ξ± β†’ Id Ξ±) s = s", "start": [ 199, 1 ], "end": [ 202, 23 ], "kind": "commanddeclaration" }, { "full_name": "Finset.map_comp_coe", "code": "@[simp]\ntheorem map_comp_coe (h : Ξ± β†’ Ξ²) :\n Functor.map h ∘ Multiset.toFinset = Multiset.toFinset ∘ Functor.map h", "start": [ 207, 1 ], "end": [ 210, 33 ], "kind": "commanddeclaration" }, { "full_name": "Finset.map_traverse", "code": "theorem map_traverse (g : Ξ± β†’ G Ξ²) (h : Ξ² β†’ Ξ³) (s : Finset Ξ±) :\n Functor.map h <$> traverse g s = traverse (Functor.map h ∘ g) s", "start": [ 213, 1 ], "end": [ 217, 53 ], "kind": "commanddeclaration" } ]
Mathlib/Data/UInt.lean
[ "Mathlib/Data/ZMod/Defs.lean", ".lake/packages/lean4/src/lean/Init.lean" ]
[ { "full_name": "neZero", "code": "instance neZero : NeZero size := ⟨by decide⟩", "start": [ 31, 7 ], "end": [ 31, 51 ], "kind": "commanddeclaration" }, { "full_name": "neg_def", "code": "lemma neg_def (a : $typeName) : -a = ⟨-a.val⟩ := rfl", "start": [ 45, 7 ], "end": [ 45, 59 ], "kind": "lemma" }, { "full_name": "pow_def", "code": "lemma pow_def (a : $typeName) (n : β„•) : a ^ n = ⟨a.val ^ n⟩ := rfl", "start": [ 47, 7 ], "end": [ 47, 73 ], "kind": "lemma" }, { "full_name": "nsmul_def", "code": "lemma nsmul_def (n : β„•) (a : $typeName) : n β€’ a = ⟨n β€’ a.val⟩ := rfl", "start": [ 49, 7 ], "end": [ 49, 75 ], "kind": "lemma" }, { "full_name": "zsmul_def", "code": "lemma zsmul_def (z : β„€) (a : $typeName) : z β€’ a = ⟨z β€’ a.val⟩ := rfl", "start": [ 51, 7 ], "end": [ 51, 75 ], "kind": "lemma" }, { "full_name": "val_injective", "code": "lemma val_injective : Function.Injective val := @eq_of_val_eq", "start": [ 54, 7 ], "end": [ 54, 68 ], "kind": "lemma" }, { "full_name": "instCommMonoid", "code": "instance instCommMonoid : CommMonoid $typeName :=\n Function.Injective.commMonoid val val_injective\n rfl (fun _ _ => rfl) (fun _ _ => rfl)", "start": [ 56, 7 ], "end": [ 58, 48 ], "kind": "commanddeclaration" }, { "full_name": "instNonUnitalCommRing", "code": "instance instNonUnitalCommRing : NonUnitalCommRing $typeName :=\n Function.Injective.nonUnitalCommRing val val_injective\n rfl (fun _ _ => rfl) (fun _ _ => rfl) (fun _ => rfl) (fun _ _ => rfl)\n (fun _ _ => rfl) (fun _ _ => rfl)", "start": [ 60, 7 ], "end": [ 63, 44 ], "kind": "commanddeclaration" }, { "full_name": "instNatCast", "code": "local instance instNatCast : NatCast $typeName where\n natCast n := mk n", "start": [ 65, 7 ], "end": [ 66, 26 ], "kind": "commanddeclaration" }, { "full_name": "instIntCast", "code": "local instance instIntCast : IntCast $typeName where\n intCast z := mk z", "start": [ 68, 7 ], "end": [ 69, 26 ], "kind": "commanddeclaration" }, { "full_name": "natCast_def", "code": "lemma natCast_def (n : β„•) : (n : $typeName) = ⟨n⟩ := rfl", "start": [ 71, 7 ], "end": [ 71, 63 ], "kind": "lemma" }, { "full_name": "intCast_def", "code": "lemma intCast_def (z : β„€) : (z : $typeName) = ⟨z⟩ := rfl", "start": [ 73, 7 ], "end": [ 73, 63 ], "kind": "lemma" }, { "full_name": "instCommRing", "code": "local instance instCommRing : CommRing $typeName :=\n Function.Injective.commRing val val_injective\n rfl rfl (fun _ _ => rfl) (fun _ _ => rfl) (fun _ => rfl) (fun _ _ => rfl)\n (fun _ _ => rfl) (fun _ _ => rfl) (fun _ _ => rfl) (fun _ => rfl) (fun _ => rfl)", "start": [ 75, 7 ], "end": [ 78, 91 ], "kind": "commanddeclaration" }, { "full_name": "UInt8.isASCIIUpper", "code": "def isASCIIUpper (c : UInt8) : Bool :=\n c β‰₯ 65 && c ≀ 90", "start": [ 96, 1 ], "end": [ 98, 19 ], "kind": "commanddeclaration" }, { "full_name": "UInt8.isASCIILower", "code": "def isASCIILower (c : UInt8) : Bool :=\n c β‰₯ 97 && c ≀ 122", "start": [ 100, 1 ], "end": [ 102, 20 ], "kind": "commanddeclaration" }, { "full_name": "UInt8.isASCIIAlpha", "code": "def isASCIIAlpha (c : UInt8) : Bool :=\n c.isASCIIUpper || c.isASCIILower", "start": [ 104, 1 ], "end": [ 106, 35 ], "kind": "commanddeclaration" }, { "full_name": "UInt8.isASCIIDigit", "code": "def isASCIIDigit (c : UInt8) : Bool :=\n c β‰₯ 48 && c ≀ 57", "start": [ 108, 1 ], "end": [ 110, 19 ], "kind": "commanddeclaration" }, { "full_name": "UInt8.isASCIIAlphanum", "code": "def isASCIIAlphanum (c : UInt8) : Bool :=\n c.isASCIIAlpha || c.isASCIIDigit", "start": [ 112, 1 ], "end": [ 114, 35 ], "kind": "commanddeclaration" }, { "full_name": "UInt8.toChar", "code": "def toChar (n : UInt8) : Char := ⟨n.toUInt32, .inl (n.1.2.trans (by decide))⟩", "start": [ 122, 1 ], "end": [ 123, 78 ], "kind": "commanddeclaration" } ]
Mathlib/Order/Category/OmegaCompletePartialOrder.lean
[ "Mathlib/CategoryTheory/Limits/Shapes/Products.lean", "Mathlib/CategoryTheory/Limits/Constructions/LimitsOfProductsAndEqualizers.lean", "Mathlib/Order/OmegaCompletePartialOrder.lean", ".lake/packages/lean4/src/lean/Init.lean", "Mathlib/CategoryTheory/Limits/Shapes/Equalizers.lean", "Mathlib/CategoryTheory/ConcreteCategory/BundledHom.lean" ]
[ { "full_name": "Ο‰CPO", "code": "def Ο‰CPO : Type (u + 1) :=\n Bundled OmegaCompletePartialOrder", "start": [ 35, 1 ], "end": [ 37, 36 ], "kind": "commanddeclaration" }, { "full_name": "Ο‰CPO.of", "code": "def of (Ξ± : Type*) [OmegaCompletePartialOrder Ξ±] : Ο‰CPO :=\n Bundled.of Ξ±", "start": [ 57, 1 ], "end": [ 59, 15 ], "kind": "commanddeclaration" }, { "full_name": "Ο‰CPO.coe_of", "code": "@[simp]\ntheorem coe_of (Ξ± : Type*) [OmegaCompletePartialOrder Ξ±] : β†₯(of Ξ±) = Ξ±", "start": [ 62, 1 ], "end": [ 64, 6 ], "kind": "commanddeclaration" }, { "full_name": "Ο‰CPO.HasProducts.product", "code": "def product {J : Type v} (f : J β†’ Ο‰CPO.{v}) : Fan f :=\n Fan.mk (of (βˆ€ j, f j)) fun j => .mk (Pi.evalOrderHom j) fun _ => rfl", "start": [ 79, 1 ], "end": [ 81, 71 ], "kind": "commanddeclaration" }, { "full_name": "Ο‰CPO.HasProducts.isProduct", "code": "def isProduct (J : Type v) (f : J β†’ Ο‰CPO) : IsLimit (product f) where\n lift s :=\n ⟨⟨fun t j => (s.Ο€.app ⟨j⟩).toFun t, fun x y h j => (s.Ο€.app ⟨j⟩).monotone h⟩,\n fun x => funext fun j => (s.Ο€.app ⟨j⟩).continuous x⟩\n uniq s m w := by\n ext t; funext j change m.toFun t j = (s.Ο€.app ⟨j⟩).toFun t\n rw [← w ⟨j⟩]\n rfl\n fac s j := rfl", "start": [ 84, 1 ], "end": [ 95, 17 ], "kind": "commanddeclaration" }, { "full_name": "Ο‰CPO.omegaCompletePartialOrderEqualizer", "code": "instance omegaCompletePartialOrderEqualizer {Ξ± Ξ² : Type*} [OmegaCompletePartialOrder Ξ±]\n [OmegaCompletePartialOrder Ξ²] (f g : Ξ± →𝒄 Ξ²) :\n OmegaCompletePartialOrder { a : Ξ± // f a = g a } :=\n OmegaCompletePartialOrder.subtype _ fun c hc => by\n rw [f.continuous, g.continuous]\n congr 1\n apply OrderHom.ext; funext x apply hc _ ⟨_, rfl⟩", "start": [ 103, 1 ], "end": [ 110, 24 ], "kind": "commanddeclaration" }, { "full_name": "Ο‰CPO.HasEqualizers.equalizerΞΉ", "code": "def equalizerΞΉ {Ξ± Ξ² : Type*} [OmegaCompletePartialOrder Ξ±] [OmegaCompletePartialOrder Ξ²]\n (f g : Ξ± →𝒄 Ξ²) : { a : Ξ± // f a = g a } →𝒄 Ξ± :=\n .mk (OrderHom.Subtype.val _) fun _ => rfl", "start": [ 115, 1 ], "end": [ 118, 44 ], "kind": "commanddeclaration" }, { "full_name": "Ο‰CPO.HasEqualizers.equalizer", "code": "def equalizer {X Y : Ο‰CPO.{v}} (f g : X ⟢ Y) : Fork f g :=\n Fork.ofΞΉ (P := Ο‰CPO.of { a // f.toFun a = g.toFun a }) (equalizerΞΉ f g)\n (ContinuousHom.ext _ _ fun x => x.2)", "start": [ 121, 1 ], "end": [ 125, 41 ], "kind": "commanddeclaration" }, { "full_name": "Ο‰CPO.HasEqualizers.isEqualizer", "code": "def isEqualizer {X Y : Ο‰CPO.{v}} (f g : X ⟢ Y) : IsLimit (equalizer f g) :=\n Fork.IsLimit.mk' _ fun s =>\n ⟨{ toFun := fun x => ⟨s.ΞΉ.toFun x, by apply ContinuousHom.congr_fun s.condition⟩\n monotone' := fun x y h => s.ΞΉ.monotone h\n cont := fun x => Subtype.ext (s.ΞΉ.continuous x) }, by ext; rfl, fun hm => by\n apply ContinuousHom.ext _ _ fun x => Subtype.ext ?_ apply ContinuousHom.congr_fun hm⟩", "start": [ 128, 1 ], "end": [ 136, 40 ], "kind": "commanddeclaration" } ]
Mathlib/Analysis/Calculus/Rademacher.lean
[ "Mathlib/MeasureTheory/Measure/Lebesgue/EqHaar.lean", "Mathlib/MeasureTheory/Measure/Haar/Disintegration.lean", "Mathlib/Analysis/BoundedVariation.lean", ".lake/packages/lean4/src/lean/Init.lean", "Mathlib/Analysis/NormedSpace/FiniteDimension.lean", "Mathlib/MeasureTheory/Group/Integral.lean", "Mathlib/Analysis/Distribution/AEEqOfIntegralContDiff.lean", "Mathlib/Analysis/Calculus/LineDeriv/Measurable.lean" ]
[ { "full_name": "LipschitzWith.ae_lineDifferentiableAt", "code": "theorem ae_lineDifferentiableAt (hf : LipschitzWith C f) (v : E) :\n βˆ€α΅ p βˆ‚ΞΌ, LineDifferentiableAt ℝ f p v", "start": [ 63, 1 ], "end": [ 77, 77 ], "kind": "commanddeclaration" }, { "full_name": "LipschitzWith.memβ„’p_lineDeriv", "code": "theorem memβ„’p_lineDeriv (hf : LipschitzWith C f) (v : E) :\n Memβ„’p (fun x ↦ lineDeriv ℝ f x v) ∞ ΞΌ", "start": [ 79, 1 ], "end": [ 82, 84 ], "kind": "commanddeclaration" }, { "full_name": "LipschitzWith.locallyIntegrable_lineDeriv", "code": "theorem locallyIntegrable_lineDeriv (hf : LipschitzWith C f) (v : E) :\n LocallyIntegrable (fun x ↦ lineDeriv ℝ f x v) ΞΌ", "start": [ 84, 1 ], "end": [ 86, 50 ], "kind": "commanddeclaration" }, { "full_name": "LipschitzWith.integral_inv_smul_sub_mul_tendsto_integral_lineDeriv_mul", "code": "theorem integral_inv_smul_sub_mul_tendsto_integral_lineDeriv_mul\n (hf : LipschitzWith C f) (hg : Integrable g ΞΌ) (v : E) :\n Tendsto (fun (t : ℝ) ↦ ∫ x, (t⁻¹ β€’ (f (x + t β€’ v) - f x)) * g x βˆ‚ΞΌ) (𝓝[>] 0)\n (𝓝 (∫ x, lineDeriv ℝ f x v * g x βˆ‚ΞΌ))", "start": [ 97, 1 ], "end": [ 117, 76 ], "kind": "commanddeclaration" }, { "full_name": "LipschitzWith.integral_inv_smul_sub_mul_tendsto_integral_lineDeriv_mul'", "code": "theorem integral_inv_smul_sub_mul_tendsto_integral_lineDeriv_mul'\n (hf : LipschitzWith C f) (h'f : HasCompactSupport f) (hg : Continuous g) (v : E) :\n Tendsto (fun (t : ℝ) ↦ ∫ x, (t⁻¹ β€’ (f (x + t β€’ v) - f x)) * g x βˆ‚ΞΌ) (𝓝[>] 0)\n (𝓝 (∫ x, lineDeriv ℝ f x v * g x βˆ‚ΞΌ))", "start": [ 119, 1 ], "end": [ 160, 76 ], "kind": "commanddeclaration" }, { "full_name": "LipschitzWith.integral_lineDeriv_mul_eq", "code": "theorem integral_lineDeriv_mul_eq\n (hf : LipschitzWith C f) (hg : LipschitzWith D g) (h'g : HasCompactSupport g) (v : E) :\n ∫ x, lineDeriv ℝ f x v * g x βˆ‚ΞΌ = ∫ x, lineDeriv ℝ g x (-v) * f x βˆ‚ΞΌ", "start": [ 162, 1 ], "end": [ 195, 89 ], "kind": "commanddeclaration" }, { "full_name": "LipschitzWith.ae_lineDeriv_sum_eq", "code": "theorem ae_lineDeriv_sum_eq\n (hf : LipschitzWith C f) {ΞΉ : Type*} (s : Finset ΞΉ) (a : ΞΉ β†’ ℝ) (v : ΞΉ β†’ E) :\n βˆ€α΅ x βˆ‚ΞΌ, lineDeriv ℝ f x (βˆ‘ i ∈ s, a i β€’ v i) = βˆ‘ i ∈ s, a i β€’ lineDeriv ℝ f x (v i)", "start": [ 197, 1 ], "end": [ 233, 54 ], "kind": "commanddeclaration" }, { "full_name": "LipschitzWith.ae_exists_fderiv_of_countable", "code": "theorem ae_exists_fderiv_of_countable\n (hf : LipschitzWith C f) {s : Set E} (hs : s.Countable) :\n βˆ€α΅ x βˆ‚ΞΌ, βˆƒ (L : E β†’L[ℝ] ℝ), βˆ€ v ∈ s, HasLineDerivAt ℝ f (L v) x v", "start": [ 239, 1 ], "end": [ 253, 44 ], "kind": "commanddeclaration" }, { "full_name": "LipschitzWith.hasFderivAt_of_hasLineDerivAt_of_closure", "code": "theorem hasFderivAt_of_hasLineDerivAt_of_closure {f : E β†’ F}\n (hf : LipschitzWith C f) {s : Set E} (hs : sphere 0 1 βŠ† closure s)\n {L : E β†’L[ℝ] F} {x : E} (hL : βˆ€ v ∈ s, HasLineDerivAt ℝ f (L v) x v) :\n HasFDerivAt f L x", "start": [ 255, 1 ], "end": [ 307, 34 ], "kind": "commanddeclaration" }, { "full_name": "LipschitzWith.ae_differentiableAt_of_real", "code": "theorem ae_differentiableAt_of_real (hf : LipschitzWith C f) :\n βˆ€α΅ x βˆ‚ΞΌ, DifferentiableAt ℝ f x", "start": [ 309, 1 ], "end": [ 320, 77 ], "kind": "commanddeclaration" }, { "full_name": "LipschitzOnWith.ae_differentiableWithinAt_of_mem_of_real", "code": "theorem ae_differentiableWithinAt_of_mem_of_real (hf : LipschitzOnWith C f s) :\n βˆ€α΅ x βˆ‚ΞΌ, x ∈ s β†’ DifferentiableWithinAt ℝ f s x", "start": [ 328, 1 ], "end": [ 336, 51 ], "kind": "commanddeclaration" }, { "full_name": "LipschitzOnWith.ae_differentiableWithinAt_of_mem_pi", "code": "theorem ae_differentiableWithinAt_of_mem_pi\n {ΞΉ : Type*} [Fintype ΞΉ] {f : E β†’ ΞΉ β†’ ℝ} {s : Set E}\n (hf : LipschitzOnWith C f s) : βˆ€α΅ x βˆ‚ΞΌ, x ∈ s β†’ DifferentiableWithinAt ℝ f s x", "start": [ 338, 1 ], "end": [ 350, 54 ], "kind": "commanddeclaration" }, { "full_name": "LipschitzOnWith.ae_differentiableWithinAt_of_mem", "code": "theorem ae_differentiableWithinAt_of_mem {f : E β†’ F} (hf : LipschitzOnWith C f s) :\n βˆ€α΅ x βˆ‚ΞΌ, x ∈ s β†’ DifferentiableWithinAt ℝ f s x", "start": [ 352, 1 ], "end": [ 364, 44 ], "kind": "commanddeclaration" }, { "full_name": "LipschitzOnWith.ae_differentiableWithinAt", "code": "theorem ae_differentiableWithinAt {f : E β†’ F} (hf : LipschitzOnWith C f s)\n (hs : MeasurableSet s) :\n βˆ€α΅ x βˆ‚(ΞΌ.restrict s), DifferentiableWithinAt ℝ f s x", "start": [ 366, 1 ], "end": [ 372, 44 ], "kind": "commanddeclaration" }, { "full_name": "LipschitzWith.ae_differentiableAt", "code": "theorem LipschitzWith.ae_differentiableAt {f : E β†’ F} (h : LipschitzWith C f) :\n βˆ€α΅ x βˆ‚ΞΌ, DifferentiableAt ℝ f x", "start": [ 376, 1 ], "end": [ 381, 79 ], "kind": "commanddeclaration" } ]
Mathlib/Analysis/Complex/UnitDisc/Basic.lean
[ "Mathlib/Analysis/Complex/Circle.lean", ".lake/packages/lean4/src/lean/Init.lean", "Mathlib/Analysis/NormedSpace/BallAction.lean" ]
[ { "full_name": "Complex.UnitDisc", "code": "def UnitDisc : Type :=\n ball (0 : β„‚) 1 deriving TopologicalSpace", "start": [ 27, 1 ], "end": [ 29, 43 ], "kind": "commanddeclaration" }, { "full_name": "Complex.UnitDisc.instCommSemigroup", "code": "instance instCommSemigroup : CommSemigroup UnitDisc := by unfold UnitDisc; infer_instance", "start": [ 37, 1 ], "end": [ 37, 90 ], "kind": "commanddeclaration" }, { "full_name": "Complex.UnitDisc.instHasDistribNeg", "code": "instance instHasDistribNeg : HasDistribNeg UnitDisc := by unfold UnitDisc; infer_instance", "start": [ 38, 1 ], "end": [ 38, 90 ], "kind": "commanddeclaration" }, { "full_name": "Complex.UnitDisc.instCoe", "code": "instance instCoe : Coe UnitDisc β„‚ := ⟨Subtype.val⟩", "start": [ 39, 1 ], "end": [ 39, 51 ], "kind": "commanddeclaration" }, { "full_name": "Complex.UnitDisc.coe_injective", "code": "theorem coe_injective : Injective ((↑) : 𝔻 β†’ β„‚)", "start": [ 41, 1 ], "end": [ 42, 24 ], "kind": "commanddeclaration" }, { "full_name": "Complex.UnitDisc.abs_lt_one", "code": "theorem abs_lt_one (z : 𝔻) : abs (z : β„‚) < 1", "start": [ 45, 1 ], "end": [ 46, 26 ], "kind": "commanddeclaration" }, { "full_name": "Complex.UnitDisc.abs_ne_one", "code": "theorem abs_ne_one (z : 𝔻) : abs (z : β„‚) β‰  1", "start": [ 49, 1 ], "end": [ 50, 18 ], "kind": "commanddeclaration" }, { "full_name": "Complex.UnitDisc.normSq_lt_one", "code": "theorem normSq_lt_one (z : 𝔻) : normSq z < 1", "start": [ 53, 1 ], "end": [ 55, 25 ], "kind": "commanddeclaration" }, { "full_name": "Complex.UnitDisc.coe_ne_one", "code": "theorem coe_ne_one (z : 𝔻) : (z : β„‚) β‰  1", "start": [ 58, 1 ], "end": [ 59, 58 ], "kind": "commanddeclaration" }, { "full_name": "Complex.UnitDisc.coe_ne_neg_one", "code": "theorem coe_ne_neg_one (z : 𝔻) : (z : β„‚) β‰  -1", "start": [ 62, 1 ], "end": [ 65, 23 ], "kind": "commanddeclaration" }, { "full_name": "Complex.UnitDisc.one_add_coe_ne_zero", "code": "theorem one_add_coe_ne_zero (z : 𝔻) : (1 + z : β„‚) β‰  0", "start": [ 68, 1 ], "end": [ 69, 52 ], "kind": "commanddeclaration" }, { "full_name": "Complex.UnitDisc.coe_mul", "code": "@[simp, norm_cast]\ntheorem coe_mul (z w : 𝔻) : ↑(z * w) = (z * w : β„‚)", "start": [ 72, 1 ], "end": [ 74, 6 ], "kind": "commanddeclaration" }, { "full_name": "Complex.UnitDisc.mk", "code": "def mk (z : β„‚) (hz : abs z < 1) : 𝔻 :=\n ⟨z, mem_ball_zero_iff.2 hz⟩", "start": [ 77, 1 ], "end": [ 80, 30 ], "kind": "commanddeclaration" }, { "full_name": "Complex.UnitDisc.coe_mk", "code": "@[simp]\ntheorem coe_mk (z : β„‚) (hz : abs z < 1) : (mk z hz : β„‚) = z", "start": [ 83, 1 ], "end": [ 85, 6 ], "kind": "commanddeclaration" }, { "full_name": "Complex.UnitDisc.mk_coe", "code": "@[simp]\ntheorem mk_coe (z : 𝔻) (hz : abs (z : β„‚) < 1 := z.abs_lt_one) : mk z hz = z", "start": [ 88, 1 ], "end": [ 90, 18 ], "kind": "commanddeclaration" }, { "full_name": "Complex.UnitDisc.mk_neg", "code": "@[simp]\ntheorem mk_neg (z : β„‚) (hz : abs (-z) < 1) : mk (-z) hz = -mk z (abs.map_neg z β–Έ hz)", "start": [ 93, 1 ], "end": [ 95, 6 ], "kind": "commanddeclaration" }, { "full_name": "Complex.UnitDisc.coe_zero", "code": "@[simp]\ntheorem coe_zero : ((0 : 𝔻) : β„‚) = 0", "start": [ 104, 1 ], "end": [ 106, 6 ], "kind": "commanddeclaration" }, { "full_name": "Complex.UnitDisc.coe_eq_zero", "code": "@[simp]\ntheorem coe_eq_zero {z : 𝔻} : (z : β„‚) = 0 ↔ z = 0", "start": [ 109, 1 ], "end": [ 111, 33 ], "kind": "commanddeclaration" }, { "full_name": "Complex.UnitDisc.circleAction", "code": "instance circleAction : MulAction circle 𝔻 :=\n mulActionSphereBall", "start": [ 117, 1 ], "end": [ 118, 22 ], "kind": "commanddeclaration" }, { "full_name": "Complex.UnitDisc.isScalarTower_circle_circle", "code": "instance isScalarTower_circle_circle : IsScalarTower circle circle 𝔻 :=\n isScalarTower_sphere_sphere_ball", "start": [ 121, 1 ], "end": [ 122, 35 ], "kind": "commanddeclaration" }, { "full_name": "Complex.UnitDisc.isScalarTower_circle", "code": "instance isScalarTower_circle : IsScalarTower circle 𝔻 𝔻 :=\n isScalarTower_sphere_ball_ball", "start": [ 125, 1 ], "end": [ 126, 33 ], "kind": "commanddeclaration" }, { "full_name": "Complex.UnitDisc.instSMulCommClass_circle", "code": "instance instSMulCommClass_circle : SMulCommClass circle 𝔻 𝔻 :=\n instSMulCommClass_sphere_ball_ball", "start": [ 129, 1 ], "end": [ 130, 37 ], "kind": "commanddeclaration" }, { "full_name": "Complex.UnitDisc.instSMulCommClass_circle'", "code": "instance instSMulCommClass_circle' : SMulCommClass 𝔻 circle 𝔻 :=\n SMulCommClass.symm _ _ _", "start": [ 133, 1 ], "end": [ 134, 27 ], "kind": "commanddeclaration" }, { "full_name": "Complex.UnitDisc.coe_smul_circle", "code": "@[simp, norm_cast]\ntheorem coe_smul_circle (z : circle) (w : 𝔻) : ↑(z β€’ w) = (z * w : β„‚)", "start": [ 137, 1 ], "end": [ 139, 6 ], "kind": "commanddeclaration" }, { "full_name": "Complex.UnitDisc.closedBallAction", "code": "instance closedBallAction : MulAction (closedBall (0 : β„‚) 1) 𝔻 :=\n mulActionClosedBallBall", "start": [ 142, 1 ], "end": [ 143, 26 ], "kind": "commanddeclaration" }, { "full_name": "Complex.UnitDisc.isScalarTower_closedBall_closedBall", "code": "instance isScalarTower_closedBall_closedBall :\n IsScalarTower (closedBall (0 : β„‚) 1) (closedBall (0 : β„‚) 1) 𝔻 :=\n isScalarTower_closedBall_closedBall_ball", "start": [ 146, 1 ], "end": [ 148, 43 ], "kind": "commanddeclaration" }, { "full_name": "Complex.UnitDisc.isScalarTower_closedBall", "code": "instance isScalarTower_closedBall : IsScalarTower (closedBall (0 : β„‚) 1) 𝔻 𝔻 :=\n isScalarTower_closedBall_ball_ball", "start": [ 151, 1 ], "end": [ 152, 37 ], "kind": "commanddeclaration" }, { "full_name": "Complex.UnitDisc.instSMulCommClass_closedBall", "code": "instance instSMulCommClass_closedBall : SMulCommClass (closedBall (0 : β„‚) 1) 𝔻 𝔻 :=\n ⟨fun _ _ _ => Subtype.ext <| mul_left_comm _ _ _⟩", "start": [ 155, 1 ], "end": [ 156, 52 ], "kind": "commanddeclaration" }, { "full_name": "Complex.UnitDisc.instSMulCommClass_closedBall'", "code": "instance instSMulCommClass_closedBall' : SMulCommClass 𝔻 (closedBall (0 : β„‚) 1) 𝔻 :=\n SMulCommClass.symm _ _ _", "start": [ 159, 1 ], "end": [ 160, 27 ], "kind": "commanddeclaration" }, { "full_name": "Complex.UnitDisc.instSMulCommClass_circle_closedBall", "code": "instance instSMulCommClass_circle_closedBall : SMulCommClass circle (closedBall (0 : β„‚) 1) 𝔻 :=\n instSMulCommClass_sphere_closedBall_ball", "start": [ 163, 1 ], "end": [ 164, 43 ], "kind": "commanddeclaration" }, { "full_name": "Complex.UnitDisc.instSMulCommClass_closedBall_circle", "code": "instance instSMulCommClass_closedBall_circle : SMulCommClass (closedBall (0 : β„‚) 1) circle 𝔻 :=\n SMulCommClass.symm _ _ _", "start": [ 167, 1 ], "end": [ 168, 27 ], "kind": "commanddeclaration" }, { "full_name": "Complex.UnitDisc.coe_smul_closedBall", "code": "@[simp, norm_cast]\ntheorem coe_smul_closedBall (z : closedBall (0 : β„‚) 1) (w : 𝔻) : ↑(z β€’ w) = (z * w : β„‚)", "start": [ 171, 1 ], "end": [ 173, 6 ], "kind": "commanddeclaration" }, { "full_name": "Complex.UnitDisc.re", "code": "def re (z : 𝔻) : ℝ :=\n Complex.re z", "start": [ 176, 1 ], "end": [ 178, 15 ], "kind": "commanddeclaration" }, { "full_name": "Complex.UnitDisc.im", "code": "def im (z : 𝔻) : ℝ :=\n Complex.im z", "start": [ 181, 1 ], "end": [ 183, 15 ], "kind": "commanddeclaration" }, { "full_name": "Complex.UnitDisc.re_coe", "code": "@[simp, norm_cast]\ntheorem re_coe (z : 𝔻) : (z : β„‚).re = z.re", "start": [ 186, 1 ], "end": [ 188, 6 ], "kind": "commanddeclaration" }, { "full_name": "Complex.UnitDisc.im_coe", "code": "@[simp, norm_cast]\ntheorem im_coe (z : 𝔻) : (z : β„‚).im = z.im", "start": [ 191, 1 ], "end": [ 193, 6 ], "kind": "commanddeclaration" }, { "full_name": "Complex.UnitDisc.re_neg", "code": "@[simp]\ntheorem re_neg (z : 𝔻) : (-z).re = -z.re", "start": [ 196, 1 ], "end": [ 198, 6 ], "kind": "commanddeclaration" }, { "full_name": "Complex.UnitDisc.im_neg", "code": "@[simp]\ntheorem im_neg (z : 𝔻) : (-z).im = -z.im", "start": [ 201, 1 ], "end": [ 203, 6 ], "kind": "commanddeclaration" }, { "full_name": "Complex.UnitDisc.conj", "code": "def conj (z : 𝔻) : 𝔻 :=\n mk (conj' ↑z) <| (abs_conj z).symm β–Έ z.abs_lt_one", "start": [ 206, 1 ], "end": [ 208, 52 ], "kind": "commanddeclaration" }, { "full_name": "Complex.UnitDisc.coe_conj", "code": "@[simp]\ntheorem coe_conj (z : 𝔻) : (z.conj : β„‚) = conj' ↑z", "start": [ 213, 1 ], "end": [ 215, 6 ], "kind": "commanddeclaration" }, { "full_name": "Complex.UnitDisc.conj_zero", "code": "@[simp]\ntheorem conj_zero : conj 0 = 0", "start": [ 218, 1 ], "end": [ 220, 33 ], "kind": "commanddeclaration" }, { "full_name": "Complex.UnitDisc.conj_conj", "code": "@[simp]\ntheorem conj_conj (z : 𝔻) : conj (conj z) = z", "start": [ 223, 1 ], "end": [ 225, 45 ], "kind": "commanddeclaration" }, { "full_name": "Complex.UnitDisc.conj_neg", "code": "@[simp]\ntheorem conj_neg (z : 𝔻) : (-z).conj = -z.conj", "start": [ 228, 1 ], "end": [ 230, 6 ], "kind": "commanddeclaration" }, { "full_name": "Complex.UnitDisc.re_conj", "code": "@[simp]\ntheorem re_conj (z : 𝔻) : z.conj.re = z.re", "start": [ 233, 1 ], "end": [ 235, 6 ], "kind": "commanddeclaration" }, { "full_name": "Complex.UnitDisc.im_conj", "code": "@[simp]\ntheorem im_conj (z : 𝔻) : z.conj.im = -z.im", "start": [ 238, 1 ], "end": [ 240, 6 ], "kind": "commanddeclaration" }, { "full_name": "Complex.UnitDisc.conj_mul", "code": "@[simp]\ntheorem conj_mul (z w : 𝔻) : (z * w).conj = z.conj * w.conj", "start": [ 243, 1 ], "end": [ 245, 31 ], "kind": "commanddeclaration" } ]
Mathlib/Algebra/Order/Group/Bounds.lean
[ "Mathlib/Algebra/Order/Group/Defs.lean", ".lake/packages/lean4/src/lean/Init.lean", "Mathlib/Order/Bounds/Basic.lean" ]
[ { "full_name": "IsGLB.exists_between_self_add", "code": "theorem IsGLB.exists_between_self_add (h : IsGLB s a) (hΞ΅ : 0 < Ξ΅) : βˆƒ b ∈ s, a ≀ b ∧ b < a + Ξ΅", "start": [ 19, 1 ], "end": [ 20, 47 ], "kind": "commanddeclaration" }, { "full_name": "IsGLB.exists_between_self_add'", "code": "theorem IsGLB.exists_between_self_add' (h : IsGLB s a) (hβ‚‚ : a βˆ‰ s) (hΞ΅ : 0 < Ξ΅) :\n βˆƒ b ∈ s, a < b ∧ b < a + Ξ΅", "start": [ 23, 1 ], "end": [ 25, 51 ], "kind": "commanddeclaration" }, { "full_name": "IsLUB.exists_between_sub_self", "code": "theorem IsLUB.exists_between_sub_self (h : IsLUB s a) (hΞ΅ : 0 < Ξ΅) : βˆƒ b ∈ s, a - Ξ΅ < b ∧ b ≀ a", "start": [ 28, 1 ], "end": [ 29, 39 ], "kind": "commanddeclaration" }, { "full_name": "IsLUB.exists_between_sub_self'", "code": "theorem IsLUB.exists_between_sub_self' (h : IsLUB s a) (hβ‚‚ : a βˆ‰ s) (hΞ΅ : 0 < Ξ΅) :\n βˆƒ b ∈ s, a - Ξ΅ < b ∧ b < a", "start": [ 32, 1 ], "end": [ 34, 43 ], "kind": "commanddeclaration" } ]
Mathlib/Lean/Expr.lean
[ "Mathlib/Lean/Expr/Basic.lean", ".lake/packages/lean4/src/lean/Init.lean", "Mathlib/Lean/Expr/ReplaceRec.lean" ]
[]
Mathlib/CategoryTheory/Limits/EpiMono.lean
[ ".lake/packages/lean4/src/lean/Init.lean", "Mathlib/CategoryTheory/Limits/Shapes/CommSq.lean" ]
[ { "full_name": "CategoryTheory.mono_iff_fst_eq_snd", "code": "lemma mono_iff_fst_eq_snd : Mono f ↔ c.fst = c.snd := by\n constructor\n Β· intro hf\n simpa only [← cancel_mono f] using c.condition\n Β· intro hf\n constructor\n intro Z g g' h\n obtain βŸ¨Ο†, rfl, rfl⟩ := PullbackCone.IsLimit.lift' hc g g' h\n rw [hf]", "start": [ 38, 1 ], "end": [ 46, 12 ], "kind": "lemma" }, { "full_name": "CategoryTheory.mono_iff_isIso_fst", "code": "lemma mono_iff_isIso_fst : Mono f ↔ IsIso c.fst := by\n rw [mono_iff_fst_eq_snd hc]\n constructor\n Β· intro h\n obtain βŸ¨Ο†, hφ₁, hΟ†β‚‚βŸ© := PullbackCone.IsLimit.lift' hc (πŸ™ X) (πŸ™ X) (by simp)\n refine βŸ¨Ο†, PullbackCone.IsLimit.hom_ext hc ?_ ?_, hΟ†β‚βŸ©\n Β· dsimp\n simp only [assoc, hφ₁, id_comp, comp_id]\n Β· dsimp\n simp only [assoc, hΟ†β‚‚, id_comp, comp_id, h]\n Β· intro\n obtain βŸ¨Ο†, hφ₁, hΟ†β‚‚βŸ© := PullbackCone.IsLimit.lift' hc (πŸ™ X) (πŸ™ X) (by simp)\n have : IsSplitEpi Ο† := IsSplitEpi.mk ⟨SplitEpi.mk c.fst (by\n rw [← cancel_mono c.fst, assoc, id_comp, hφ₁, comp_id])⟩\n rw [← cancel_epi Ο†, hφ₁, hΟ†β‚‚]", "start": [ 48, 1 ], "end": [ 62, 34 ], "kind": "lemma" }, { "full_name": "CategoryTheory.mono_iff_isIso_snd", "code": "lemma mono_iff_isIso_snd : Mono f ↔ IsIso c.snd :=\n mono_iff_isIso_fst (PullbackCone.flipIsLimit hc)", "start": [ 64, 1 ], "end": [ 65, 51 ], "kind": "lemma" }, { "full_name": "CategoryTheory.mono_iff_isPullback", "code": "lemma mono_iff_isPullback : Mono f ↔ IsPullback (πŸ™ X) (πŸ™ X) f f := by\n constructor\n Β· intro\n exact IsPullback.of_isLimit (PullbackCone.isLimitMkIdId f)\n Β· intro hf\n exact (mono_iff_fst_eq_snd hf.isLimit).2 rfl", "start": [ 69, 1 ], "end": [ 74, 49 ], "kind": "lemma" }, { "full_name": "CategoryTheory.epi_iff_inl_eq_inr", "code": "lemma epi_iff_inl_eq_inr : Epi f ↔ c.inl = c.inr := by\n constructor\n Β· intro hf\n simpa only [← cancel_epi f] using c.condition\n Β· intro hf\n constructor\n intro Z g g' h\n obtain βŸ¨Ο†, rfl, rfl⟩ := PushoutCocone.IsColimit.desc' hc g g' h\n rw [hf]", "start": [ 82, 1 ], "end": [ 90, 12 ], "kind": "lemma" }, { "full_name": "CategoryTheory.epi_iff_isIso_inl", "code": "lemma epi_iff_isIso_inl : Epi f ↔ IsIso c.inl := by\n rw [epi_iff_inl_eq_inr hc]\n constructor\n Β· intro h\n obtain βŸ¨Ο†, hφ₁, hΟ†β‚‚βŸ© := PushoutCocone.IsColimit.desc' hc (πŸ™ Y) (πŸ™ Y) (by simp)\n refine βŸ¨Ο†, hφ₁, PushoutCocone.IsColimit.hom_ext hc ?_ ?_⟩\n Β· dsimp\n simp only [comp_id, reassoc_of% hφ₁]\n Β· dsimp\n simp only [comp_id, h, reassoc_of% hΟ†β‚‚]\n Β· intro\n obtain βŸ¨Ο†, hφ₁, hΟ†β‚‚βŸ© := PushoutCocone.IsColimit.desc' hc (πŸ™ Y) (πŸ™ Y) (by simp)\n have : IsSplitMono Ο† := IsSplitMono.mk ⟨SplitMono.mk c.inl (by\n rw [← cancel_epi c.inl, reassoc_of% hφ₁, comp_id])⟩\n rw [← cancel_mono Ο†, hφ₁, hΟ†β‚‚]", "start": [ 92, 1 ], "end": [ 106, 35 ], "kind": "lemma" }, { "full_name": "CategoryTheory.epi_iff_isIso_inr", "code": "lemma epi_iff_isIso_inr : Epi f ↔ IsIso c.inr :=\n epi_iff_isIso_inl (PushoutCocone.flipIsColimit hc)", "start": [ 108, 1 ], "end": [ 109, 53 ], "kind": "lemma" }, { "full_name": "CategoryTheory.epi_iff_isPushout", "code": "lemma epi_iff_isPushout : Epi f ↔ IsPushout f f (πŸ™ Y) (πŸ™ Y) := by\n constructor\n Β· intro\n exact IsPushout.of_isColimit (PushoutCocone.isColimitMkIdId f)\n Β· intro hf\n exact (epi_iff_inl_eq_inr hf.isColimit).2 rfl", "start": [ 113, 1 ], "end": [ 118, 50 ], "kind": "lemma" } ]
Mathlib/Data/Vector/Mem.lean
[ ".lake/packages/lean4/src/lean/Init.lean", "Mathlib/Data/Vector/Basic.lean" ]
[ { "full_name": "Vector.get_mem", "code": "@[simp]\ntheorem get_mem (i : Fin n) (v : Vector Ξ± n) : v.get i ∈ v.toList", "start": [ 25, 1 ], "end": [ 28, 27 ], "kind": "commanddeclaration" }, { "full_name": "Vector.mem_iff_get", "code": "theorem mem_iff_get (v : Vector Ξ± n) : a ∈ v.toList ↔ βˆƒ i, v.get i = a", "start": [ 31, 1 ], "end": [ 35, 38 ], "kind": "commanddeclaration" }, { "full_name": "Vector.not_mem_nil", "code": "theorem not_mem_nil : a βˆ‰ (Vector.nil : Vector Ξ± 0).toList", "start": [ 38, 1 ], "end": [ 41, 7 ], "kind": "commanddeclaration" }, { "full_name": "Vector.not_mem_zero", "code": "theorem not_mem_zero (v : Vector Ξ± 0) : a βˆ‰ v.toList", "start": [ 44, 1 ], "end": [ 45, 41 ], "kind": "commanddeclaration" }, { "full_name": "Vector.mem_cons_iff", "code": "theorem mem_cons_iff (v : Vector Ξ± n) : a' ∈ (a ::α΅₯ v).toList ↔ a' = a ∨ a' ∈ v.toList", "start": [ 48, 1 ], "end": [ 49, 41 ], "kind": "commanddeclaration" }, { "full_name": "Vector.mem_succ_iff", "code": "theorem mem_succ_iff (v : Vector Ξ± (n + 1)) : a ∈ v.toList ↔ a = v.head ∨ a ∈ v.tail.toList", "start": [ 52, 1 ], "end": [ 54, 71 ], "kind": "commanddeclaration" }, { "full_name": "Vector.mem_cons_self", "code": "theorem mem_cons_self (v : Vector Ξ± n) : a ∈ (a ::α΅₯ v).toList", "start": [ 57, 1 ], "end": [ 58, 67 ], "kind": "commanddeclaration" }, { "full_name": "Vector.head_mem", "code": "@[simp]\ntheorem head_mem (v : Vector Ξ± (n + 1)) : v.head ∈ v.toList", "start": [ 61, 1 ], "end": [ 63, 57 ], "kind": "commanddeclaration" }, { "full_name": "Vector.mem_cons_of_mem", "code": "theorem mem_cons_of_mem (v : Vector Ξ± n) (ha' : a' ∈ v.toList) : a' ∈ (a ::α΅₯ v).toList", "start": [ 66, 1 ], "end": [ 67, 46 ], "kind": "commanddeclaration" }, { "full_name": "Vector.mem_of_mem_tail", "code": "theorem mem_of_mem_tail (v : Vector Ξ± n) (ha : a ∈ v.tail.toList) : a ∈ v.toList", "start": [ 70, 1 ], "end": [ 73, 43 ], "kind": "commanddeclaration" }, { "full_name": "Vector.mem_map_iff", "code": "theorem mem_map_iff (b : Ξ²) (v : Vector Ξ± n) (f : Ξ± β†’ Ξ²) :\n b ∈ (v.map f).toList ↔ βˆƒ a : Ξ±, a ∈ v.toList ∧ f a = b", "start": [ 76, 1 ], "end": [ 78, 39 ], "kind": "commanddeclaration" }, { "full_name": "Vector.not_mem_map_zero", "code": "theorem not_mem_map_zero (b : Ξ²) (v : Vector Ξ± 0) (f : Ξ± β†’ Ξ²) : b βˆ‰ (v.map f).toList", "start": [ 81, 1 ], "end": [ 82, 91 ], "kind": "commanddeclaration" }, { "full_name": "Vector.mem_map_succ_iff", "code": "theorem mem_map_succ_iff (b : Ξ²) (v : Vector Ξ± (n + 1)) (f : Ξ± β†’ Ξ²) :\n b ∈ (v.map f).toList ↔ f v.head = b ∨ βˆƒ a : Ξ±, a ∈ v.tail.toList ∧ f a = b", "start": [ 85, 1 ], "end": [ 87, 67 ], "kind": "commanddeclaration" } ]
Mathlib/CategoryTheory/Functor/Derived/RightDerived.lean
[ ".lake/packages/lean4/src/lean/Init.lean", "Mathlib/CategoryTheory/Localization/Predicate.lean", "Mathlib/CategoryTheory/Functor/KanExtension/Basic.lean" ]
[ { "full_name": "CategoryTheory.Functor.IsRightDerivedFunctor", "code": "class IsRightDerivedFunctor [L.IsLocalization W] : Prop where\n isLeftKanExtension' : RF.IsLeftKanExtension Ξ±", "start": [ 47, 1 ], "end": [ 52, 48 ], "kind": "commanddeclaration" }, { "full_name": "CategoryTheory.Functor.IsRightDerivedFunctor.isLeftKanExtension", "code": "lemma IsRightDerivedFunctor.isLeftKanExtension\n [L.IsLocalization W] [RF.IsRightDerivedFunctor Ξ± W] :\n RF.IsLeftKanExtension Ξ± :=\n IsRightDerivedFunctor.isLeftKanExtension' W", "start": [ 54, 1 ], "end": [ 57, 46 ], "kind": "lemma" }, { "full_name": "CategoryTheory.Functor.isRightDerivedFunctor_iff_isLeftKanExtension", "code": "lemma isRightDerivedFunctor_iff_isLeftKanExtension [L.IsLocalization W] :\n RF.IsRightDerivedFunctor Ξ± W ↔ RF.IsLeftKanExtension Ξ± := by\n constructor\n Β· exact fun _ => IsRightDerivedFunctor.isLeftKanExtension RF Ξ± W\n Β· exact fun h => ⟨h⟩", "start": [ 59, 1 ], "end": [ 63, 23 ], "kind": "lemma" }, { "full_name": "CategoryTheory.Functor.isRightDerivedFunctor_iff_of_iso", "code": "lemma isRightDerivedFunctor_iff_of_iso (Ξ±' : F ⟢ L β‹™ RF') (W : MorphismProperty C)\n [L.IsLocalization W] (e : RF β‰… RF') (comm : Ξ± ≫ whiskerLeft L e.hom = Ξ±') :\n RF.IsRightDerivedFunctor Ξ± W ↔ RF'.IsRightDerivedFunctor Ξ±' W := by\n simp only [isRightDerivedFunctor_iff_isLeftKanExtension]\n exact isLeftKanExtension_iff_of_iso e _ _ comm", "start": [ 66, 1 ], "end": [ 70, 49 ], "kind": "lemma" }, { "full_name": "CategoryTheory.Functor.rightDerivedDesc", "code": "noncomputable def rightDerivedDesc (G : D β₯€ H) (Ξ² : F ⟢ L β‹™ G) : RF ⟢ G :=\n have := IsRightDerivedFunctor.isLeftKanExtension RF Ξ± W\n RF.descOfIsLeftKanExtension Ξ± G Ξ²", "start": [ 77, 1 ], "end": [ 80, 36 ], "kind": "commanddeclaration" }, { "full_name": "CategoryTheory.Functor.rightDerived_fac", "code": "@[reassoc (attr := simp)]\nlemma rightDerived_fac (G : D β₯€ H) (Ξ² : F ⟢ L β‹™ G) :\n Ξ± ≫ whiskerLeft L (RF.rightDerivedDesc Ξ± W G Ξ²) = Ξ² :=\n have := IsRightDerivedFunctor.isLeftKanExtension RF Ξ± W\n RF.descOfIsLeftKanExtension_fac Ξ± G Ξ²", "start": [ 82, 1 ], "end": [ 86, 40 ], "kind": "lemma" }, { "full_name": "CategoryTheory.Functor.rightDerived_fac_app", "code": "@[reassoc (attr := simp)]\nlemma rightDerived_fac_app (G : D β₯€ H) (Ξ² : F ⟢ L β‹™ G) (X : C):\n Ξ±.app X ≫ (RF.rightDerivedDesc Ξ± W G Ξ²).app (L.obj X) = Ξ².app X :=\n have := IsRightDerivedFunctor.isLeftKanExtension RF Ξ± W\n RF.descOfIsLeftKanExtension_fac_app Ξ± G Ξ² X", "start": [ 88, 1 ], "end": [ 92, 46 ], "kind": "lemma" }, { "full_name": "CategoryTheory.Functor.rightDerived_ext", "code": "lemma rightDerived_ext (G : D β₯€ H) (γ₁ Ξ³β‚‚ : RF ⟢ G)\n (hΞ³ : Ξ± ≫ whiskerLeft L γ₁ = Ξ± ≫ whiskerLeft L Ξ³β‚‚) : γ₁ = Ξ³β‚‚ :=\n have := IsRightDerivedFunctor.isLeftKanExtension RF Ξ± W\n RF.hom_ext_of_isLeftKanExtension Ξ± γ₁ Ξ³β‚‚ hΞ³", "start": [ 94, 1 ], "end": [ 97, 46 ], "kind": "lemma" }, { "full_name": "CategoryTheory.Functor.rightDerivedNatTrans", "code": "noncomputable def rightDerivedNatTrans (Ο„ : F ⟢ F') : RF ⟢ RF' :=\n RF.rightDerivedDesc Ξ± W RF' (Ο„ ≫ Ξ±')", "start": [ 99, 1 ], "end": [ 102, 39 ], "kind": "commanddeclaration" }, { "full_name": "CategoryTheory.Functor.rightDerivedNatTrans_fac", "code": "@[reassoc (attr := simp)]\nlemma rightDerivedNatTrans_fac (Ο„ : F ⟢ F') :\n Ξ± ≫ whiskerLeft L (rightDerivedNatTrans RF RF' Ξ± Ξ±' W Ο„) = Ο„ ≫ Ξ±' := by\n dsimp only [rightDerivedNatTrans]\n simp", "start": [ 104, 1 ], "end": [ 108, 7 ], "kind": "lemma" }, { "full_name": "CategoryTheory.Functor.rightDerivedNatTrans_app", "code": "@[reassoc (attr := simp)]\nlemma rightDerivedNatTrans_app (Ο„ : F ⟢ F') (X : C) :\n Ξ±.app X ≫ (rightDerivedNatTrans RF RF' Ξ± Ξ±' W Ο„).app (L.obj X) =\n Ο„.app X ≫ Ξ±'.app X := by\n dsimp only [rightDerivedNatTrans]\n simp", "start": [ 110, 1 ], "end": [ 115, 7 ], "kind": "lemma" }, { "full_name": "CategoryTheory.Functor.rightDerivedNatTrans_id", "code": "@[simp]\nlemma rightDerivedNatTrans_id :\n rightDerivedNatTrans RF RF Ξ± Ξ± W (πŸ™ F) = πŸ™ RF :=\n rightDerived_ext RF Ξ± W _ _ _ (by aesop_cat)", "start": [ 117, 1 ], "end": [ 120, 47 ], "kind": "lemma" }, { "full_name": "CategoryTheory.Functor.rightDerivedNatTrans_comp", "code": "@[reassoc (attr:= simp)]\nlemma rightDerivedNatTrans_comp (Ο„ : F ⟢ F') (Ο„' : F' ⟢ F'') :\n rightDerivedNatTrans RF RF' Ξ± Ξ±' W Ο„ ≫ rightDerivedNatTrans RF' RF'' Ξ±' Ξ±'' W Ο„' =\n rightDerivedNatTrans RF RF'' Ξ± Ξ±'' W (Ο„ ≫ Ο„') :=\n rightDerived_ext RF Ξ± W _ _ _ (by aesop_cat)", "start": [ 122, 1 ], "end": [ 126, 47 ], "kind": "lemma" }, { "full_name": "CategoryTheory.Functor.rightDerivedNatIso", "code": "@[simps]\nnoncomputable def rightDerivedNatIso (Ο„ : F β‰… F') :\n RF β‰… RF' where\n hom := rightDerivedNatTrans RF RF' Ξ± Ξ±' W Ο„.hom\n inv := rightDerivedNatTrans RF' RF Ξ±' Ξ± W Ο„.inv", "start": [ 128, 1 ], "end": [ 134, 50 ], "kind": "commanddeclaration" }, { "full_name": "CategoryTheory.Functor.rightDerivedUnique", "code": "noncomputable abbrev rightDerivedUnique [RF'.IsRightDerivedFunctor Ξ±'β‚‚ W] : RF β‰… RF' :=\n rightDerivedNatIso RF RF' Ξ± Ξ±'β‚‚ W (Iso.refl F)", "start": [ 136, 1 ], "end": [ 138, 49 ], "kind": "commanddeclaration" }, { "full_name": "CategoryTheory.Functor.isRightDerivedFunctor_iff_isIso_rightDerivedDesc", "code": "lemma isRightDerivedFunctor_iff_isIso_rightDerivedDesc (G : D β₯€ H) (Ξ² : F ⟢ L β‹™ G) :\n G.IsRightDerivedFunctor Ξ² W ↔ IsIso (RF.rightDerivedDesc Ξ± W G Ξ²) := by\n rw [isRightDerivedFunctor_iff_isLeftKanExtension]\n have := IsRightDerivedFunctor.isLeftKanExtension _ Ξ± W\n exact isLeftKanExtension_iff_isIso _ Ξ± _ (by simp)", "start": [ 140, 1 ], "end": [ 144, 53 ], "kind": "lemma" }, { "full_name": "CategoryTheory.Functor.HasRightDerivedFunctor", "code": "class HasRightDerivedFunctor : Prop where\n hasLeftKanExtension' : HasLeftKanExtension W.Q F", "start": [ 150, 1 ], "end": [ 155, 51 ], "kind": "commanddeclaration" }, { "full_name": "CategoryTheory.Functor.hasRightDerivedFunctor_iff", "code": "lemma hasRightDerivedFunctor_iff :\n F.HasRightDerivedFunctor W ↔ HasLeftKanExtension L F := by\n have : HasRightDerivedFunctor F W ↔ HasLeftKanExtension W.Q F :=\n ⟨fun h => h.hasLeftKanExtension', fun h => ⟨h⟩⟩\n rw [this, hasLeftExtension_iff_postcomp₁ (Localization.compUniqFunctor W.Q L W) F]", "start": [ 160, 1 ], "end": [ 164, 85 ], "kind": "lemma" }, { "full_name": "CategoryTheory.Functor.hasRightDerivedFunctor_iff_of_iso", "code": "lemma hasRightDerivedFunctor_iff_of_iso :\n HasRightDerivedFunctor F W ↔ HasRightDerivedFunctor F' W := by\n rw [hasRightDerivedFunctor_iff F W.Q W, hasRightDerivedFunctor_iff F' W.Q W,\n hasLeftExtension_iff_of_isoβ‚‚ W.Q e]", "start": [ 168, 1 ], "end": [ 171, 40 ], "kind": "lemma" }, { "full_name": "CategoryTheory.Functor.HasRightDerivedFunctor.hasLeftKanExtension", "code": "lemma HasRightDerivedFunctor.hasLeftKanExtension [HasRightDerivedFunctor F W] :\n HasLeftKanExtension L F := by\n simpa only [← hasRightDerivedFunctor_iff F L W]", "start": [ 175, 1 ], "end": [ 177, 50 ], "kind": "lemma" }, { "full_name": "CategoryTheory.Functor.HasRightDerivedFunctor.mk'", "code": "lemma HasRightDerivedFunctor.mk' [RF.IsRightDerivedFunctor Ξ± W] :\n HasRightDerivedFunctor F W := by\n have := IsRightDerivedFunctor.isLeftKanExtension RF Ξ± W\n simpa only [hasRightDerivedFunctor_iff F L W] using HasLeftKanExtension.mk RF Ξ±", "start": [ 181, 1 ], "end": [ 184, 82 ], "kind": "lemma" }, { "full_name": "CategoryTheory.Functor.totalRightDerived", "code": "noncomputable def totalRightDerived : D β₯€ H :=\n have := HasRightDerivedFunctor.hasLeftKanExtension F L W\n leftKanExtension L F", "start": [ 190, 1 ], "end": [ 195, 23 ], "kind": "commanddeclaration" }, { "full_name": "CategoryTheory.Functor.totalRightDerivedUnit", "code": "noncomputable def totalRightDerivedUnit : F ⟢ L β‹™ F.totalRightDerived L W :=\n have := HasRightDerivedFunctor.hasLeftKanExtension F L W\n leftKanExtensionUnit L F", "start": [ 197, 1 ], "end": [ 200, 27 ], "kind": "commanddeclaration" } ]
Mathlib/NumberTheory/Modular.lean
[ "Mathlib/LinearAlgebra/Matrix/GeneralLinearGroup.lean", "Mathlib/Analysis/Complex/UpperHalfPlane/Basic.lean", "Mathlib/Topology/Algebra/Module/FiniteDimension.lean", "Mathlib/LinearAlgebra/GeneralLinearGroup.lean", ".lake/packages/lean4/src/lean/Init.lean", "Mathlib/Topology/Instances/Matrix.lean" ]
[ { "full_name": "ModularGroup.bottom_row_coprime", "code": "theorem bottom_row_coprime {R : Type*} [CommRing R] (g : SL(2, R)) :\n IsCoprime ((↑g : Matrix (Fin 2) (Fin 2) R) 1 0) ((↑g : Matrix (Fin 2) (Fin 2) R) 1 1)", "start": [ 84, 1 ], "end": [ 89, 18 ], "kind": "commanddeclaration" }, { "full_name": "ModularGroup.bottom_row_surj", "code": "theorem bottom_row_surj {R : Type*} [CommRing R] :\n Set.SurjOn (fun g : SL(2, R) => (↑g : Matrix (Fin 2) (Fin 2) R) 1) Set.univ\n {cd | IsCoprime (cd 0) (cd 1)}", "start": [ 92, 1 ], "end": [ 104, 16 ], "kind": "commanddeclaration" }, { "full_name": "ModularGroup.tendsto_normSq_coprime_pair", "code": "theorem tendsto_normSq_coprime_pair :\n Filter.Tendsto (fun p : Fin 2 β†’ β„€ => normSq ((p 0 : β„‚) * z + p 1)) cofinite atTop", "start": [ 115, 1 ], "end": [ 161, 76 ], "kind": "commanddeclaration" }, { "full_name": "ModularGroup.lcRow0", "code": "def lcRow0 (p : Fin 2 β†’ β„€) : Matrix (Fin 2) (Fin 2) ℝ β†’β‚—[ℝ] ℝ :=\n ((p 0 : ℝ) β€’ LinearMap.proj (0 : Fin 2) +\n (p 1 : ℝ) β€’ LinearMap.proj (1 : Fin 2) : (Fin 2 β†’ ℝ) β†’β‚—[ℝ] ℝ).comp\n (LinearMap.proj 0)", "start": [ 164, 1 ], "end": [ 170, 23 ], "kind": "commanddeclaration" }, { "full_name": "ModularGroup.lcRow0_apply", "code": "@[simp]\ntheorem lcRow0_apply (p : Fin 2 β†’ β„€) (g : Matrix (Fin 2) (Fin 2) ℝ) :\n lcRow0 p g = p 0 * g 0 0 + p 1 * g 0 1", "start": [ 173, 1 ], "end": [ 176, 6 ], "kind": "commanddeclaration" }, { "full_name": "ModularGroup.lcRow0Extend", "code": "@[simps!]\ndef lcRow0Extend {cd : Fin 2 β†’ β„€} (hcd : IsCoprime (cd 0) (cd 1)) :\n Matrix (Fin 2) (Fin 2) ℝ ≃ₗ[ℝ] Matrix (Fin 2) (Fin 2) ℝ :=\n LinearEquiv.piCongrRight\n ![by\n refine\n LinearMap.GeneralLinearGroup.generalLinearEquiv ℝ (Fin 2 β†’ ℝ)\n (GeneralLinearGroup.toLinear (planeConformalMatrix (cd 0 : ℝ) (-(cd 1 : ℝ)) ?_))\n norm_cast\n rw [neg_sq]\n exact hcd.sq_add_sq_ne_zero, LinearEquiv.refl ℝ (Fin 2 β†’ ℝ)]", "start": [ 179, 1 ], "end": [ 191, 67 ], "kind": "commanddeclaration" }, { "full_name": "ModularGroup.tendsto_lcRow0", "code": "theorem tendsto_lcRow0 {cd : Fin 2 β†’ β„€} (hcd : IsCoprime (cd 0) (cd 1)) :\n Tendsto (fun g : { g : SL(2, β„€) // (β†‘β‚˜g) 1 = cd } => lcRow0 cd ↑(↑g : SL(2, ℝ))) cofinite\n (cocompact ℝ)", "start": [ 197, 1 ], "end": [ 236, 8 ], "kind": "commanddeclaration" }, { "full_name": "ModularGroup.smul_eq_lcRow0_add", "code": "theorem smul_eq_lcRow0_add {p : Fin 2 β†’ β„€} (hp : IsCoprime (p 0) (p 1)) (hg : (β†‘β‚˜g) 1 = p) :\n ↑(g β€’ z) =\n (lcRow0 p ↑(g : SL(2, ℝ)) : β„‚) / ((p 0 : β„‚) ^ 2 + (p 1 : β„‚) ^ 2) +\n ((p 1 : β„‚) * z - p 0) / (((p 0 : β„‚) ^ 2 + (p 1 : β„‚) ^ 2) * (p 0 * z + p 1))", "start": [ 239, 1 ], "end": [ 255, 7 ], "kind": "commanddeclaration" }, { "full_name": "ModularGroup.tendsto_abs_re_smul", "code": "theorem tendsto_abs_re_smul {p : Fin 2 β†’ β„€} (hp : IsCoprime (p 0) (p 1)) :\n Tendsto\n (fun g : { g : SL(2, β„€) // (β†‘β‚˜g) 1 = p } => |((g : SL(2, β„€)) β€’ z).re|) cofinite atTop", "start": [ 258, 1 ], "end": [ 276, 68 ], "kind": "commanddeclaration" }, { "full_name": "ModularGroup.exists_max_im", "code": "theorem exists_max_im : βˆƒ g : SL(2, β„€), βˆ€ g' : SL(2, β„€), (g' β€’ z).im ≀ (g β€’ z).im", "start": [ 287, 1 ], "end": [ 301, 31 ], "kind": "commanddeclaration" }, { "full_name": "ModularGroup.exists_row_one_eq_and_min_re", "code": "theorem exists_row_one_eq_and_min_re {cd : Fin 2 β†’ β„€} (hcd : IsCoprime (cd 0) (cd 1)) :\n βˆƒ g : SL(2, β„€), (β†‘β‚˜g) 1 = cd ∧ βˆ€ g' : SL(2, β„€), (β†‘β‚˜g) 1 = (β†‘β‚˜g') 1 β†’\n |(g β€’ z).re| ≀ |(g' β€’ z).re|", "start": [ 304, 1 ], "end": [ 318, 22 ], "kind": "commanddeclaration" }, { "full_name": "ModularGroup.coe_T_zpow_smul_eq", "code": "theorem coe_T_zpow_smul_eq {n : β„€} : (↑(T ^ n β€’ z) : β„‚) = z + n", "start": [ 321, 1 ], "end": [ 323, 43 ], "kind": "commanddeclaration" }, { "full_name": "ModularGroup.re_T_zpow_smul", "code": "theorem re_T_zpow_smul (n : β„€) : (T ^ n β€’ z).re = z.re + n", "start": [ 326, 1 ], "end": [ 327, 64 ], "kind": "commanddeclaration" }, { "full_name": "ModularGroup.im_T_zpow_smul", "code": "theorem im_T_zpow_smul (n : β„€) : (T ^ n β€’ z).im = z.im", "start": [ 330, 1 ], "end": [ 331, 74 ], "kind": "commanddeclaration" }, { "full_name": "ModularGroup.re_T_smul", "code": "theorem re_T_smul : (T β€’ z).re = z.re + 1", "start": [ 334, 1 ], "end": [ 334, 79 ], "kind": "commanddeclaration" }, { "full_name": "ModularGroup.im_T_smul", "code": "theorem im_T_smul : (T β€’ z).im = z.im", "start": [ 337, 1 ], "end": [ 337, 75 ], "kind": "commanddeclaration" }, { "full_name": "ModularGroup.re_T_inv_smul", "code": "theorem re_T_inv_smul : (T⁻¹ β€’ z).re = z.re - 1", "start": [ 340, 1 ], "end": [ 340, 88 ], "kind": "commanddeclaration" }, { "full_name": "ModularGroup.im_T_inv_smul", "code": "theorem im_T_inv_smul : (T⁻¹ β€’ z).im = z.im", "start": [ 343, 1 ], "end": [ 343, 84 ], "kind": "commanddeclaration" }, { "full_name": "ModularGroup.exists_eq_T_zpow_of_c_eq_zero", "code": "theorem exists_eq_T_zpow_of_c_eq_zero (hc : (β†‘β‚˜g) 1 0 = 0) :\n βˆƒ n : β„€, βˆ€ z : ℍ, g β€’ z = T ^ n β€’ z", "start": [ 349, 1 ], "end": [ 361, 83 ], "kind": "commanddeclaration" }, { "full_name": "ModularGroup.g_eq_of_c_eq_one", "code": "theorem g_eq_of_c_eq_one (hc : (β†‘β‚˜g) 1 0 = 1) : g = T ^ (β†‘β‚˜g) 0 0 * S * T ^ (β†‘β‚˜g) 1 1", "start": [ 365, 1 ], "end": [ 372, 37 ], "kind": "commanddeclaration" }, { "full_name": "ModularGroup.normSq_S_smul_lt_one", "code": "theorem normSq_S_smul_lt_one (h : 1 < normSq z) : normSq ↑(S β€’ z) < 1", "start": [ 375, 1 ], "end": [ 377, 78 ], "kind": "commanddeclaration" }, { "full_name": "ModularGroup.im_lt_im_S_smul", "code": "theorem im_lt_im_S_smul (h : normSq z < 1) : z.im < (S β€’ z).im", "start": [ 380, 1 ], "end": [ 388, 22 ], "kind": "commanddeclaration" }, { "full_name": "ModularGroup.fd", "code": "def fd : Set ℍ :=\n {z | 1 ≀ normSq (z : β„‚) ∧ |z.re| ≀ (1 : ℝ) / 2}", "start": [ 391, 1 ], "end": [ 393, 50 ], "kind": "commanddeclaration" }, { "full_name": "ModularGroup.fdo", "code": "def fdo : Set ℍ :=\n {z | 1 < normSq (z : β„‚) ∧ |z.re| < (1 : ℝ) / 2}", "start": [ 396, 1 ], "end": [ 398, 50 ], "kind": "commanddeclaration" }, { "full_name": "ModularGroup.abs_two_mul_re_lt_one_of_mem_fdo", "code": "theorem abs_two_mul_re_lt_one_of_mem_fdo (h : z ∈ π’Ÿα΅’) : |2 * z.re| < 1", "start": [ 409, 1 ], "end": [ 411, 12 ], "kind": "commanddeclaration" }, { "full_name": "ModularGroup.three_lt_four_mul_im_sq_of_mem_fdo", "code": "theorem three_lt_four_mul_im_sq_of_mem_fdo (h : z ∈ π’Ÿα΅’) : 3 < 4 * z.im ^ 2", "start": [ 414, 1 ], "end": [ 417, 37 ], "kind": "commanddeclaration" }, { "full_name": "ModularGroup.one_lt_normSq_T_zpow_smul", "code": "theorem one_lt_normSq_T_zpow_smul (hz : z ∈ π’Ÿα΅’) (n : β„€) : 1 < normSq (T ^ n β€’ z : ℍ)", "start": [ 420, 1 ], "end": [ 425, 52 ], "kind": "commanddeclaration" }, { "full_name": "ModularGroup.eq_zero_of_mem_fdo_of_T_zpow_mem_fdo", "code": "theorem eq_zero_of_mem_fdo_of_T_zpow_mem_fdo {n : β„€} (hz : z ∈ π’Ÿα΅’) (hg : T ^ n β€’ z ∈ π’Ÿα΅’) :\n n = 0", "start": [ 428, 1 ], "end": [ 438, 26 ], "kind": "commanddeclaration" }, { "full_name": "ModularGroup.exists_smul_mem_fd", "code": "theorem exists_smul_mem_fd (z : ℍ) : βˆƒ g : SL(2, β„€), g β€’ z ∈ π’Ÿ", "start": [ 441, 1 ], "end": [ 472, 83 ], "kind": "commanddeclaration" }, { "full_name": "ModularGroup.abs_c_le_one", "code": "theorem abs_c_le_one (hz : z ∈ π’Ÿα΅’) (hg : g β€’ z ∈ π’Ÿα΅’) : |(β†‘β‚˜g) 1 0| ≀ 1", "start": [ 477, 1 ], "end": [ 509, 42 ], "kind": "commanddeclaration" }, { "full_name": "ModularGroup.c_eq_zero", "code": "theorem c_eq_zero (hz : z ∈ π’Ÿα΅’) (hg : g β€’ z ∈ π’Ÿα΅’) : (β†‘β‚˜g) 1 0 = 0", "start": [ 512, 1 ], "end": [ 531, 71 ], "kind": "commanddeclaration" }, { "full_name": "ModularGroup.eq_smul_self_of_mem_fdo_mem_fdo", "code": "theorem eq_smul_self_of_mem_fdo_mem_fdo (hz : z ∈ π’Ÿα΅’) (hg : g β€’ z ∈ π’Ÿα΅’) : z = g β€’ z", "start": [ 534, 1 ], "end": [ 539, 62 ], "kind": "commanddeclaration" } ]
Mathlib/Topology/ContinuousFunction/Sigma.lean
[ ".lake/packages/lean4/src/lean/Init.lean", "Mathlib/Topology/CompactOpen.lean" ]
[ { "full_name": "ContinuousMap.embedding_sigmaMk_comp", "code": "theorem embedding_sigmaMk_comp [Nonempty X] :\n Embedding (fun g : Ξ£ i, C(X, Y i) ↦ (sigmaMk g.1).comp g.2) where", "start": [ 44, 1 ], "end": [ 54, 21 ], "kind": "commanddeclaration" }, { "full_name": "ContinuousMap.exists_lift_sigma", "code": "theorem exists_lift_sigma (f : C(X, Ξ£ i, Y i)) : βˆƒ i g, f = (sigmaMk i).comp g", "start": [ 60, 1 ], "end": [ 67, 34 ], "kind": "commanddeclaration" }, { "full_name": "ContinuousMap.sigmaCodHomeomorph", "code": "@[simps! symm_apply]\ndef sigmaCodHomeomorph : C(X, Ξ£ i, Y i) β‰ƒβ‚œ Ξ£ i, C(X, Y i) :=\n .symm <| Equiv.toHomeomorphOfInducing\n (.ofBijective _ ⟨embedding_sigmaMk_comp.inj, fun f ↦\n let ⟨i, g, hg⟩ := f.exists_lift_sigma; ⟨⟨i, g⟩, hg.symm⟩⟩)\n embedding_sigmaMk_comp.toInducing", "start": [ 71, 1 ], "end": [ 81, 38 ], "kind": "commanddeclaration" } ]
Mathlib/Data/Finset/NatDivisors.lean
[ "Mathlib/Data/Nat/Order/Lemmas.lean", "Mathlib/Data/Finset/Pointwise.lean", ".lake/packages/lean4/src/lean/Init.lean", "Mathlib/NumberTheory/Divisors.lean" ]
[ { "full_name": "Nat.divisors_mul", "code": "lemma Nat.divisors_mul (m n : β„•) : divisors (m * n) = divisors m * divisors n := by\n ext k\n simp_rw [mem_mul, mem_divisors, dvd_mul, mul_ne_zero_iff, ← exists_and_left, ← exists_and_right]\n simp only [and_assoc, and_comm, and_left_comm]", "start": [ 20, 1 ], "end": [ 25, 49 ], "kind": "lemma" }, { "full_name": "Nat.divisorsHom", "code": "@[simps]\ndef Nat.divisorsHom : β„• β†’* Finset β„• where\n toFun := Nat.divisors\n map_mul' := divisors_mul\n map_one' := divisors_one", "start": [ 27, 1 ], "end": [ 32, 27 ], "kind": "commanddeclaration" }, { "full_name": "Nat.Prime.divisors_sq", "code": "lemma Nat.Prime.divisors_sq {p : β„•} (hp : p.Prime) : (p ^ 2).divisors = {p ^ 2, p, 1} := by\n simp [divisors_prime_pow hp, range_succ]", "start": [ 34, 1 ], "end": [ 35, 43 ], "kind": "lemma" }, { "full_name": "List.nat_divisors_prod", "code": "lemma List.nat_divisors_prod (l : List β„•) : divisors l.prod = (l.map divisors).prod :=\n map_list_prod Nat.divisorsHom l", "start": [ 37, 1 ], "end": [ 38, 34 ], "kind": "lemma" }, { "full_name": "Multiset.nat_divisors_prod", "code": "lemma Multiset.nat_divisors_prod (s : Multiset β„•) : divisors s.prod = (s.map divisors).prod :=\n map_multiset_prod Nat.divisorsHom s", "start": [ 40, 1 ], "end": [ 41, 38 ], "kind": "lemma" }, { "full_name": "Finset.nat_divisors_prod", "code": "lemma Finset.nat_divisors_prod {ΞΉ : Type*} (s : Finset ΞΉ) (f : ΞΉ β†’ β„•) :\n divisors (∏ i ∈ s, f i) = ∏ i ∈ s, divisors (f i) :=\n map_prod Nat.divisorsHom f s", "start": [ 43, 1 ], "end": [ 45, 31 ], "kind": "lemma" } ]
Mathlib/GroupTheory/GroupAction/Sum.lean
[ ".lake/packages/lean4/src/lean/Init.lean", "Mathlib/Algebra/Group/Action/Defs.lean" ]
[ { "full_name": "Sum.smul_def", "code": "@[to_additive]\ntheorem smul_def : a β€’ x = x.map (a β€’ Β·) (a β€’ Β·)", "start": [ 37, 1 ], "end": [ 39, 6 ], "kind": "commanddeclaration" }, { "full_name": "Sum.smul_inl", "code": "@[to_additive (attr := simp)]\ntheorem smul_inl : a β€’ (inl b : Sum Ξ± Ξ²) = inl (a β€’ b)", "start": [ 43, 1 ], "end": [ 45, 6 ], "kind": "commanddeclaration" }, { "full_name": "Sum.smul_inr", "code": "@[to_additive (attr := simp)]\ntheorem smul_inr : a β€’ (inr c : Sum Ξ± Ξ²) = inr (a β€’ c)", "start": [ 49, 1 ], "end": [ 51, 6 ], "kind": "commanddeclaration" }, { "full_name": "Sum.smul_swap", "code": "@[to_additive (attr := simp)]\ntheorem smul_swap : (a β€’ x).swap = a β€’ x.swap", "start": [ 55, 1 ], "end": [ 56, 68 ], "kind": "commanddeclaration" }, { "full_name": "Sum.FaithfulSMulLeft", "code": "@[to_additive]\ninstance FaithfulSMulLeft [FaithfulSMul M Ξ±] : FaithfulSMul M (Sum Ξ± Ξ²) :=\n ⟨fun h => eq_of_smul_eq_smul fun a : Ξ± => by injection h (inl a)⟩", "start": [ 78, 1 ], "end": [ 80, 68 ], "kind": "commanddeclaration" }, { "full_name": "Sum.FaithfulSMulRight", "code": "@[to_additive]\ninstance FaithfulSMulRight [FaithfulSMul M Ξ²] : FaithfulSMul M (Sum Ξ± Ξ²) :=\n ⟨fun h => eq_of_smul_eq_smul fun b : Ξ² => by injection h (inr b)⟩", "start": [ 84, 1 ], "end": [ 86, 68 ], "kind": "commanddeclaration" } ]
Mathlib/Init/Data/Int/Lemmas.lean
[ "Mathlib/Mathport/Rename.lean", ".lake/packages/lean4/src/lean/Init.lean" ]
[]
Mathlib/NumberTheory/PrimesCongruentOne.lean
[ ".lake/packages/lean4/src/lean/Init.lean", "Mathlib/RingTheory/Polynomial/Cyclotomic/Eval.lean" ]
[ { "full_name": "Nat.exists_prime_gt_modEq_one", "code": "theorem exists_prime_gt_modEq_one {k : β„•} (n : β„•) (hk0 : k β‰  0) :\n βˆƒ p : β„•, Nat.Prime p ∧ n < p ∧ p ≑ 1 [MOD k]", "start": [ 24, 1 ], "end": [ 57, 54 ], "kind": "commanddeclaration" }, { "full_name": "Nat.frequently_atTop_modEq_one", "code": "theorem frequently_atTop_modEq_one {k : β„•} (hk0 : k β‰  0) :\n βˆƒαΆ  p in atTop, Nat.Prime p ∧ p ≑ 1 [MOD k]", "start": [ 60, 1 ], "end": [ 64, 39 ], "kind": "commanddeclaration" }, { "full_name": "Nat.infinite_setOf_prime_modEq_one", "code": "theorem infinite_setOf_prime_modEq_one {k : β„•} (hk0 : k β‰  0) :\n Set.Infinite {p : β„• | Nat.Prime p ∧ p ≑ 1 [MOD k]}", "start": [ 67, 1 ], "end": [ 70, 67 ], "kind": "commanddeclaration" } ]
Mathlib/LinearAlgebra/TensorProduct/Matrix.lean
[ "Mathlib/LinearAlgebra/TensorProduct/Basis.lean", ".lake/packages/lean4/src/lean/Init.lean", "Mathlib/LinearAlgebra/Matrix/ToLin.lean", "Mathlib/Data/Matrix/Kronecker.lean" ]
[ { "full_name": "TensorProduct.toMatrix_map", "code": "theorem TensorProduct.toMatrix_map (f : M β†’β‚—[R] M') (g : N β†’β‚—[R] N') :\n toMatrix (bM.tensorProduct bN) (bM'.tensorProduct bN') (TensorProduct.map f g) =\n toMatrix bM bM' f βŠ—β‚– toMatrix bN bN' g", "start": [ 37, 1 ], "end": [ 44, 65 ], "kind": "commanddeclaration" }, { "full_name": "Matrix.toLin_kronecker", "code": "theorem Matrix.toLin_kronecker (A : Matrix ΞΉ' ΞΉ R) (B : Matrix ΞΊ' ΞΊ R) :\n toLin (bM.tensorProduct bN) (bM'.tensorProduct bN') (A βŠ—β‚– B) =\n TensorProduct.map (toLin bM bM' A) (toLin bN bN' B)", "start": [ 47, 1 ], "end": [ 53, 20 ], "kind": "commanddeclaration" }, { "full_name": "TensorProduct.toMatrix_comm", "code": "theorem TensorProduct.toMatrix_comm :\n toMatrix (bM.tensorProduct bN) (bN.tensorProduct bM) (TensorProduct.comm R M N) =\n (1 : Matrix (ΞΉ Γ— ΞΊ) (ΞΉ Γ— ΞΊ) R).submatrix Prod.swap _root_.id", "start": [ 56, 1 ], "end": [ 64, 75 ], "kind": "commanddeclaration" }, { "full_name": "TensorProduct.toMatrix_assoc", "code": "theorem TensorProduct.toMatrix_assoc :\n toMatrix ((bM.tensorProduct bN).tensorProduct bP) (bM.tensorProduct (bN.tensorProduct bP))\n (TensorProduct.assoc R M N P) =\n (1 : Matrix (ΞΉ Γ— ΞΊ Γ— Ο„) (ΞΉ Γ— ΞΊ Γ— Ο„) R).submatrix _root_.id (Equiv.prodAssoc _ _ _)", "start": [ 67, 1 ], "end": [ 78, 21 ], "kind": "commanddeclaration" } ]
.lake/packages/lean4/src/lean/Lean/Compiler/IR/LLVMBindings.lean
[ ".lake/packages/lean4/src/lean/Init/System/IO.lean" ]
[ { "full_name": "LLVM.CodegenFileType", "code": "structure CodegenFileType where\n private mk :: val : UInt64", "start": [ 20, 1 ], "end": [ 21, 29 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.CodegenFileType.AssemblyFile", "code": "def CodegenFileType.AssemblyFile : CodegenFileType := { val := 0 }", "start": [ 23, 1 ], "end": [ 23, 67 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.CodegenFileType.ObjectFile", "code": "def CodegenFileType.ObjectFile : CodegenFileType := { val := 1 }", "start": [ 24, 1 ], "end": [ 24, 65 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.IntPredicate", "code": "structure IntPredicate where\n private mk :: val : UInt64", "start": [ 27, 1 ], "end": [ 28, 29 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.IntPredicate.EQ", "code": "def IntPredicate.EQ : IntPredicate := { val := 32 }", "start": [ 30, 1 ], "end": [ 30, 52 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.IntPredicate.NE", "code": "def IntPredicate.NE : IntPredicate := { val := IntPredicate.EQ.val + 1 }", "start": [ 31, 1 ], "end": [ 31, 73 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.IntPredicate.UGT", "code": "def IntPredicate.UGT : IntPredicate := { val := IntPredicate.NE.val + 1 }", "start": [ 32, 1 ], "end": [ 32, 74 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.AttributeIndex", "code": "structure AttributeIndex where\n private mk :: val : UInt64", "start": [ 35, 1 ], "end": [ 36, 29 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.AttributeIndex.AttributeReturnIndex", "code": "def AttributeIndex.AttributeReturnIndex : AttributeIndex := { val := 0 }", "start": [ 38, 1 ], "end": [ 38, 73 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.AttributeIndex.AttributeFunctionIndex", "code": "def AttributeIndex.AttributeFunctionIndex : AttributeIndex := { val := 18446744073709551615 }", "start": [ 40, 1 ], "end": [ 40, 94 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.BasicBlock", "code": "structure BasicBlock (ctx : Context) where\n private mk :: ptr : USize", "start": [ 42, 1 ], "end": [ 43, 28 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.Builder", "code": "structure Builder (ctx : Context) where\n private mk :: ptr : USize", "start": [ 46, 1 ], "end": [ 47, 28 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.Context", "code": "structure Context where\n private mk :: ptr : USize", "start": [ 50, 1 ], "end": [ 51, 28 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.LLVMType", "code": "structure LLVMType (ctx : Context) where\n private mk :: ptr : USize", "start": [ 54, 1 ], "end": [ 55, 28 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.MemoryBuffer", "code": "structure MemoryBuffer (ctx : Context) where\n private mk :: ptr : USize", "start": [ 58, 1 ], "end": [ 59, 28 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.Module", "code": "structure Module (ctx : Context) where\n private mk :: ptr : USize", "start": [ 62, 1 ], "end": [ 63, 28 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.PassManager", "code": "structure PassManager (ctx : Context) where\n private mk :: ptr : USize", "start": [ 66, 1 ], "end": [ 67, 28 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.PassManagerBuilder", "code": "structure PassManagerBuilder (ctx : Context) where\n private mk :: ptr : USize", "start": [ 70, 1 ], "end": [ 71, 28 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.Target", "code": "structure Target (ctx : Context) where\n private mk :: ptr : USize", "start": [ 74, 1 ], "end": [ 75, 28 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.TargetMachine", "code": "structure TargetMachine (ctx : Context) where\n private mk :: ptr : USize", "start": [ 78, 1 ], "end": [ 79, 28 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.Value", "code": "structure Value (ctx : Context) where\n private mk :: ptr : USize", "start": [ 82, 1 ], "end": [ 83, 28 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.Value.isNull", "code": "def Value.isNull (v : Value ctx) : Bool := v.ptr == 0", "start": [ 86, 1 ], "end": [ 87, 54 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.Value.getName", "code": "@[extern \"lean_llvm_get_value_name2\"]\nopaque Value.getName {ctx : Context} (value : Value ctx) : BaseIO String", "start": [ 89, 1 ], "end": [ 90, 73 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.Attribute", "code": "structure Attribute (ctx : Context) where\n private mk :: ptr : USize", "start": [ 92, 1 ], "end": [ 93, 28 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.llvmInitializeTargetInfo", "code": "@[extern \"lean_llvm_initialize_target_info\"]\nopaque llvmInitializeTargetInfo : BaseIO (Unit)", "start": [ 96, 1 ], "end": [ 97, 48 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.createContext", "code": "@[extern \"lean_llvm_create_context\"]\nopaque createContext : BaseIO (Context)", "start": [ 99, 1 ], "end": [ 100, 40 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.createModule", "code": "@[extern \"lean_llvm_create_module\"]\nopaque createModule (ctx : Context) (name : @&String) : BaseIO (Module ctx)", "start": [ 102, 1 ], "end": [ 103, 76 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.moduleToString", "code": "@[extern \"lean_llvm_module_to_string\"]\nopaque moduleToString (m : Module ctx) : BaseIO String", "start": [ 105, 1 ], "end": [ 106, 55 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.writeBitcodeToFile", "code": "@[extern \"lean_llvm_write_bitcode_to_file\"]\nopaque writeBitcodeToFile (m : Module ctx) (path : @&String) : BaseIO Unit", "start": [ 108, 1 ], "end": [ 109, 75 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.addFunction", "code": "@[extern \"lean_llvm_add_function\"]\nopaque addFunction (m : Module ctx) (name : @&String) (type : LLVMType ctx) : BaseIO (Value ctx)", "start": [ 111, 1 ], "end": [ 112, 97 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.getFirstFunction", "code": "@[extern \"lean_llvm_get_first_function\"]\nopaque getFirstFunction (m : Module ctx) : BaseIO (Value ctx)", "start": [ 114, 1 ], "end": [ 115, 62 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.getNextFunction", "code": "@[extern \"lean_llvm_get_next_function\"]\nopaque getNextFunction (glbl : Value ctx) : BaseIO (Value ctx)", "start": [ 117, 1 ], "end": [ 118, 63 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.getNamedFunction", "code": "@[extern \"lean_llvm_get_named_function\"]\nopaque getNamedFunction (m : Module ctx) (name : @&String) : BaseIO (Option (Value ctx))", "start": [ 120, 1 ], "end": [ 121, 89 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.addGlobal", "code": "@[extern \"lean_llvm_add_global\"]\nopaque addGlobal (m : Module ctx) (name : @&String) (type : LLVMType ctx) : BaseIO (Value ctx)", "start": [ 123, 1 ], "end": [ 124, 95 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.getNamedGlobal", "code": "@[extern \"lean_llvm_get_named_global\"]\nopaque getNamedGlobal (m : Module ctx) (name : @&String) : BaseIO (Option (Value ctx))", "start": [ 126, 1 ], "end": [ 127, 87 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.getFirstGlobal", "code": "@[extern \"lean_llvm_get_first_global\"]\nopaque getFirstGlobal (m : Module ctx) : BaseIO (Value ctx)", "start": [ 129, 1 ], "end": [ 130, 60 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.getNextGlobal", "code": "@[extern \"lean_llvm_get_next_global\"]\nopaque getNextGlobal (glbl : Value ctx) : BaseIO (Value ctx)", "start": [ 132, 1 ], "end": [ 133, 61 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.buildGlobalString", "code": "@[extern \"lean_llvm_build_global_string\"]\nopaque buildGlobalString (builder : Builder ctx) (value : @&String) (name : @&String := \"\") : BaseIO (Value ctx)", "start": [ 135, 1 ], "end": [ 136, 113 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.isDeclaration", "code": "@[extern \"llvm_is_declaration\"]\nopaque isDeclaration (global : Value ctx) : BaseIO Bool", "start": [ 138, 1 ], "end": [ 139, 56 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.setInitializer", "code": "@[extern \"lean_llvm_set_initializer\"]\nopaque setInitializer (glbl : Value ctx) (val : Value ctx) : BaseIO Unit", "start": [ 141, 1 ], "end": [ 142, 73 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.functionType", "code": "@[extern \"lean_llvm_function_type\"]\nopaque functionType (retty : LLVMType ctx) (args : @&Array (LLVMType ctx)) (isVarArg : Bool := false) : BaseIO (LLVMType ctx)", "start": [ 144, 1 ], "end": [ 145, 126 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.voidType", "code": "@[extern \"lean_llvm_void_type_in_context\"]\nopaque voidType (ctx : Context) : BaseIO (LLVMType ctx)", "start": [ 147, 1 ], "end": [ 148, 56 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.intTypeInContext", "code": "@[extern \"lean_llvm_int_type_in_context\"]\nopaque intTypeInContext (ctx : Context) (width : UInt64) : BaseIO (LLVMType ctx)", "start": [ 150, 1 ], "end": [ 151, 81 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.opaquePointerTypeInContext", "code": "@[extern \"lean_llvm_opaque_pointer_type_in_context\"]\nopaque opaquePointerTypeInContext (ctx : Context) (addrspace: UInt64 := 0) : BaseIO (LLVMType ctx)", "start": [ 153, 1 ], "end": [ 154, 99 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.floatTypeInContext", "code": "@[extern \"lean_llvm_float_type_in_context\"]\nopaque floatTypeInContext (ctx : Context) : BaseIO (LLVMType ctx)", "start": [ 156, 1 ], "end": [ 157, 66 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.doubleTypeInContext", "code": "@[extern \"lean_llvm_double_type_in_context\"]\nopaque doubleTypeInContext (ctx : Context) : BaseIO (LLVMType ctx)", "start": [ 159, 1 ], "end": [ 160, 67 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.pointerType", "code": "@[extern \"lean_llvm_pointer_type\"]\nopaque pointerType (elemty : LLVMType ctx) : BaseIO (LLVMType ctx)", "start": [ 162, 1 ], "end": [ 163, 67 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.arrayType", "code": "@[extern \"lean_llvm_array_type\"]\nopaque arrayType (elemty : LLVMType ctx) (nelem : UInt64) : BaseIO (LLVMType ctx)", "start": [ 165, 1 ], "end": [ 166, 82 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.constArray", "code": "@[extern \"lean_llvm_const_array\"]\nopaque constArray (elemty : LLVMType ctx) (vals : @&Array (Value ctx)) : BaseIO (LLVMType ctx)", "start": [ 168, 1 ], "end": [ 169, 95 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.constString", "code": "@[extern \"lean_llvm_const_string\"]\nopaque constString (ctx : Context) (str : @&String) : BaseIO (Value ctx)", "start": [ 172, 1 ], "end": [ 173, 73 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.constPointerNull", "code": "@[extern \"lean_llvm_const_pointer_null\"]\nopaque constPointerNull (elemty : LLVMType ctx) : BaseIO (Value ctx)", "start": [ 175, 1 ], "end": [ 176, 69 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.getUndef", "code": "@[extern \"lean_llvm_get_undef\"]\nopaque getUndef (elemty : LLVMType ctx) : BaseIO (Value ctx)", "start": [ 178, 1 ], "end": [ 179, 61 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.createBuilderInContext", "code": "@[extern \"lean_llvm_create_builder_in_context\"]\nopaque createBuilderInContext (ctx : Context) : BaseIO (Builder ctx)", "start": [ 181, 1 ], "end": [ 182, 69 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.appendBasicBlockInContext", "code": "@[extern \"lean_llvm_append_basic_block_in_context\"]\nopaque appendBasicBlockInContext (ctx : Context) (fn : Value ctx) (name : @&String) : BaseIO (BasicBlock ctx)", "start": [ 184, 1 ], "end": [ 185, 112 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.countBasicBlocks", "code": "@[extern \"lean_llvm_count_basic_blocks\"]\nopaque countBasicBlocks (fn : Value ctx) : BaseIO UInt64", "start": [ 187, 1 ], "end": [ 188, 57 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.getEntryBasicBlock", "code": "@[extern \"lean_llvm_get_entry_basic_block\"]\nopaque getEntryBasicBlock (fn : Value ctx) : BaseIO (BasicBlock ctx)", "start": [ 190, 1 ], "end": [ 191, 69 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.getFirstInstruction", "code": "@[extern \"lean_llvm_get_first_instruction\"]\nopaque getFirstInstruction (bb : BasicBlock ctx) : BaseIO (Option (Value ctx))", "start": [ 193, 1 ], "end": [ 194, 79 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.positionBuilderBefore", "code": "@[extern \"lean_llvm_position_builder_before\"]\nopaque positionBuilderBefore (builder : Builder ctx) (instr : Value ctx) : BaseIO Unit", "start": [ 196, 1 ], "end": [ 197, 87 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.positionBuilderAtEnd", "code": "@[extern \"lean_llvm_position_builder_at_end\"]\nopaque positionBuilderAtEnd (builder : Builder ctx) (bb : BasicBlock ctx) : BaseIO Unit", "start": [ 199, 1 ], "end": [ 200, 89 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.buildCall2", "code": "@[extern \"lean_llvm_build_call2\"]\nopaque buildCall2 (builder : Builder ctx) (ty: LLVMType ctx) (fn : Value ctx) (args : @&Array (Value ctx)) (name : @&String := \"\") : BaseIO (Value ctx)", "start": [ 202, 1 ], "end": [ 203, 153 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.setTailCall", "code": "@[extern \"lean_llvm_set_tail_call\"]\nopaque setTailCall (fn : Value ctx) (istail : Bool) : BaseIO Unit", "start": [ 205, 1 ], "end": [ 206, 66 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.buildCondBr", "code": "@[extern \"lean_llvm_build_cond_br\"]\nopaque buildCondBr (builder : Builder ctx) (if_ : Value ctx) (thenbb : BasicBlock ctx) (elsebb : BasicBlock ctx) : BaseIO (Value ctx)", "start": [ 208, 1 ], "end": [ 209, 134 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.buildBr", "code": "@[extern \"lean_llvm_build_br\"]\nopaque buildBr (builder : Builder ctx) (bb : BasicBlock ctx) : BaseIO (Value ctx)", "start": [ 211, 1 ], "end": [ 212, 82 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.buildAlloca", "code": "@[extern \"lean_llvm_build_alloca\"]\nopaque buildAlloca (builder : Builder ctx) (ty : LLVMType ctx) (name : @&String := \"\") : BaseIO (Value ctx)", "start": [ 214, 1 ], "end": [ 215, 108 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.buildLoad2", "code": "@[extern \"lean_llvm_build_load2\"]\nopaque buildLoad2 (builder : Builder ctx) (ty: LLVMType ctx) (val : Value ctx) (name : @&String := \"\") : BaseIO (Value ctx)", "start": [ 217, 1 ], "end": [ 218, 124 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.buildStore", "code": "@[extern \"lean_llvm_build_store\"]\nopaque buildStore (builder : Builder ctx) (val : Value ctx) (store_loc_ptr : Value ctx) : BaseIO Unit", "start": [ 220, 1 ], "end": [ 221, 102 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.buildRet", "code": "@[extern \"lean_llvm_build_ret\"]\nopaque buildRet (builder : Builder ctx) (val : Value ctx) : BaseIO (Value ctx)", "start": [ 223, 1 ], "end": [ 224, 79 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.buildUnreachable", "code": "@[extern \"lean_llvm_build_unreachable\"]\nopaque buildUnreachable (builder : Builder ctx) : BaseIO (Value ctx)", "start": [ 226, 1 ], "end": [ 227, 69 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.buildGEP2", "code": "@[extern \"lean_llvm_build_gep2\"]\nopaque buildGEP2 (builder : Builder ctx) (ty: LLVMType ctx) (base : Value ctx) (ixs : @&Array (Value ctx)) (name : @&String := \"\") : BaseIO (Value ctx)", "start": [ 229, 1 ], "end": [ 230, 152 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.buildInBoundsGEP2", "code": "@[extern \"lean_llvm_build_inbounds_gep2\"]\nopaque buildInBoundsGEP2 (builder : Builder ctx) (ty: LLVMType ctx) (base : Value ctx) (ixs : @&Array (Value ctx)) (name : @&String := \"\") : BaseIO (Value ctx)", "start": [ 232, 1 ], "end": [ 233, 160 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.buildSext", "code": "@[extern \"lean_llvm_build_sext\"]\nopaque buildSext (builder : Builder ctx) (val : Value ctx) (destTy : LLVMType ctx) (name : @&String := \"\") : BaseIO (Value ctx)", "start": [ 235, 1 ], "end": [ 236, 128 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.buildZext", "code": "@[extern \"lean_llvm_build_zext\"]\nopaque buildZext (builder : Builder ctx) (val : Value ctx) (destTy : LLVMType ctx) (name : @&String := \"\") : BaseIO (Value ctx)", "start": [ 238, 1 ], "end": [ 239, 128 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.buildSextOrTrunc", "code": "@[extern \"lean_llvm_build_sext_or_trunc\"]\nopaque buildSextOrTrunc (builder : Builder ctx) (val : Value ctx) (destTy : LLVMType ctx) (name : @&String := \"\") : BaseIO (Value ctx)", "start": [ 241, 1 ], "end": [ 242, 135 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.buildSwitch", "code": "@[extern \"lean_llvm_build_switch\"]\nopaque buildSwitch (builder : Builder ctx) (val : Value ctx) (elseBB : BasicBlock ctx) (numCasesHint : UInt64) : BaseIO (Value ctx)", "start": [ 244, 1 ], "end": [ 245, 132 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.buildPtrToInt", "code": "@[extern \"lean_llvm_build_ptr_to_int\"]\nopaque buildPtrToInt (builder : Builder ctx) (ptr : Value ctx) (destTy : LLVMType ctx) (name : @&String := \"\") : BaseIO (Value ctx)", "start": [ 247, 1 ], "end": [ 248, 132 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.buildMul", "code": "@[extern \"lean_llvm_build_mul\"]\nopaque buildMul (builder : Builder ctx) (x y : Value ctx) (name : @&String := \"\") : BaseIO (Value ctx)", "start": [ 250, 1 ], "end": [ 251, 103 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.buildAdd", "code": "@[extern \"lean_llvm_build_add\"]\nopaque buildAdd (builder : Builder ctx) (x y : Value ctx) (name : @&String := \"\") : BaseIO (Value ctx)", "start": [ 253, 1 ], "end": [ 254, 103 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.buildSub", "code": "@[extern \"lean_llvm_build_sub\"]\nopaque buildSub (builder : Builder ctx) (x y : Value ctx) (name : @&String := \"\") : BaseIO (Value ctx)", "start": [ 256, 1 ], "end": [ 257, 103 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.buildNot", "code": "@[extern \"lean_llvm_build_not\"]\nopaque buildNot (builder : Builder ctx) (x : Value ctx) (name : @&String := \"\") : BaseIO (Value ctx)", "start": [ 259, 1 ], "end": [ 260, 101 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.buildICmp", "code": "@[extern \"lean_llvm_build_icmp\"]\nopaque buildICmp (builder : Builder ctx) (predicate : IntPredicate) (x y : Value ctx) (name : @&String := \"\") : BaseIO (Value ctx)", "start": [ 262, 1 ], "end": [ 263, 131 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.addCase", "code": "@[extern \"lean_llvm_add_case\"]\nopaque addCase (switch onVal : Value ctx) (destBB : BasicBlock ctx) : BaseIO Unit", "start": [ 265, 1 ], "end": [ 266, 82 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.getInsertBlock", "code": "@[extern \"lean_llvm_get_insert_block\"]\nopaque getInsertBlock (builder : Builder ctx) : BaseIO (BasicBlock ctx)", "start": [ 268, 1 ], "end": [ 269, 72 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.clearInsertionPosition", "code": "@[extern \"lean_llvm_clear_insertion_position\"]\nopaque clearInsertionPosition (builder : Builder ctx) : BaseIO Unit", "start": [ 271, 1 ], "end": [ 272, 68 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.getBasicBlockParent", "code": "@[extern \"lean_llvm_get_basic_block_parent\"]\nopaque getBasicBlockParent (bb : BasicBlock ctx) : BaseIO (Value ctx)", "start": [ 274, 1 ], "end": [ 275, 70 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.typeOf", "code": "@[extern \"lean_llvm_type_of\"]\nopaque typeOf (val : Value ctx) : BaseIO (LLVMType ctx)", "start": [ 277, 1 ], "end": [ 278, 56 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.constInt", "code": "@[extern \"lean_llvm_const_int\"]\nopaque constInt (intty : LLVMType ctx) (value : UInt64) (signExtend : @Bool := false) : BaseIO (Value ctx)", "start": [ 280, 1 ], "end": [ 281, 107 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.printModuletoString", "code": "@[extern \"lean_llvm_print_module_to_string\"]\nopaque printModuletoString (mod : Module ctx) : BaseIO (String)", "start": [ 283, 1 ], "end": [ 284, 64 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.printModuletoFile", "code": "@[extern \"lean_llvm_print_module_to_file\"]\nopaque printModuletoFile (mod : Module ctx) (file : @&String) : BaseIO Unit", "start": [ 286, 1 ], "end": [ 287, 76 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.countParams", "code": "@[extern \"llvm_count_params\"]\nopaque countParams (fn : Value ctx) : BaseIO UInt64", "start": [ 289, 1 ], "end": [ 290, 52 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.getParam", "code": "@[extern \"llvm_get_param\"]\nopaque getParam (fn : Value ctx) (ix : UInt64) : BaseIO (Value ctx)", "start": [ 292, 1 ], "end": [ 293, 68 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.createMemoryBufferWithContentsOfFile", "code": "@[extern \"lean_llvm_create_memory_buffer_with_contents_of_file\"]\nopaque createMemoryBufferWithContentsOfFile (path : @&String) : BaseIO (MemoryBuffer ctx)", "start": [ 295, 1 ], "end": [ 296, 90 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.parseBitcode", "code": "@[extern \"lean_llvm_parse_bitcode\"]\nopaque parseBitcode (ctx : Context) (membuf : MemoryBuffer ctx) : BaseIO (Module ctx)", "start": [ 298, 1 ], "end": [ 299, 86 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.linkModules", "code": "@[extern \"lean_llvm_link_modules\"]\nopaque linkModules (dest : Module ctx) (src : Module ctx) : BaseIO Unit", "start": [ 301, 1 ], "end": [ 302, 72 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.getDefaultTargetTriple", "code": "@[extern \"lean_llvm_get_default_target_triple\"]\nopaque getDefaultTargetTriple : BaseIO String", "start": [ 304, 1 ], "end": [ 305, 46 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.getTargetFromTriple", "code": "@[extern \"lean_llvm_get_target_from_triple\"]\nopaque getTargetFromTriple (triple : @&String) : BaseIO (Target ctx)", "start": [ 307, 1 ], "end": [ 308, 69 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.createTargetMachine", "code": "@[extern \"lean_llvm_create_target_machine\"]\nopaque createTargetMachine (target : Target ctx) (tripleStr : @&String) (cpu : @&String) (features : @&String) : BaseIO (TargetMachine ctx)", "start": [ 310, 1 ], "end": [ 311, 140 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.targetMachineEmitToFile", "code": "@[extern \"lean_llvm_target_machine_emit_to_file\"]\nopaque targetMachineEmitToFile (targetMachine : TargetMachine ctx) (module : Module ctx) (filepath : @&String) (codegenType : LLVM.CodegenFileType) : BaseIO Unit", "start": [ 313, 1 ], "end": [ 314, 162 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.createPassManager", "code": "@[extern \"lean_llvm_create_pass_manager\"]\nopaque createPassManager : BaseIO (PassManager ctx)", "start": [ 316, 1 ], "end": [ 317, 52 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.disposePassManager", "code": "@[extern \"lean_llvm_dispose_pass_manager\"]\nopaque disposePassManager (pm : PassManager ctx) : BaseIO Unit", "start": [ 319, 1 ], "end": [ 320, 63 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.runPassManager", "code": "@[extern \"lean_llvm_run_pass_manager\"]\nopaque runPassManager (pm : PassManager ctx) (mod : Module ctx): BaseIO Unit", "start": [ 322, 1 ], "end": [ 323, 77 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.createPassManagerBuilder", "code": "@[extern \"lean_llvm_create_pass_manager_builder\"]\nopaque createPassManagerBuilder : BaseIO (PassManagerBuilder ctx)", "start": [ 325, 1 ], "end": [ 326, 66 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.disposePassManagerBuilder", "code": "@[extern \"lean_llvm_dispose_pass_manager_builder\"]\nopaque disposePassManagerBuilder (pmb : PassManagerBuilder ctx) : BaseIO Unit", "start": [ 328, 1 ], "end": [ 329, 78 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.PassManagerBuilder.setOptLevel", "code": "@[extern \"lean_llvm_pass_manager_builder_set_opt_level\"]\nopaque PassManagerBuilder.setOptLevel (pmb : PassManagerBuilder ctx) (optLevel : unsigned) : BaseIO Unit", "start": [ 331, 1 ], "end": [ 332, 105 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.PassManagerBuilder.populateModulePassManager", "code": "@[extern \"lean_llvm_pass_manager_builder_populate_module_pass_manager\"]\nopaque PassManagerBuilder.populateModulePassManager (pmb : PassManagerBuilder ctx) (pm : PassManager ctx): BaseIO Unit", "start": [ 334, 1 ], "end": [ 335, 119 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.disposeTargetMachine", "code": "@[extern \"lean_llvm_dispose_target_machine\"]\nopaque disposeTargetMachine (tm : TargetMachine ctx) : BaseIO Unit", "start": [ 337, 1 ], "end": [ 338, 67 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.disposeModule", "code": "@[extern \"lean_llvm_dispose_module\"]\nopaque disposeModule (m : Module ctx) : BaseIO Unit", "start": [ 340, 1 ], "end": [ 341, 52 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.verifyModule", "code": "@[extern \"lean_llvm_verify_module\"]\nopaque verifyModule (m : Module ctx) : BaseIO (Option String)", "start": [ 343, 1 ], "end": [ 344, 62 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.createStringAttribute", "code": "@[extern \"lean_llvm_create_string_attribute\"]\nopaque createStringAttribute (key : String) (value : String) : BaseIO (Attribute ctx)", "start": [ 346, 1 ], "end": [ 347, 86 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.addAttributeAtIndex", "code": "@[extern \"lean_llvm_add_attribute_at_index\"]\nopaque addAttributeAtIndex (fn : Value ctx) (idx: AttributeIndex) (attr: Attribute ctx) : BaseIO Unit", "start": [ 349, 1 ], "end": [ 350, 102 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.Visibility", "code": "structure Visibility where\n private mk :: val : UInt64", "start": [ 354, 1 ], "end": [ 355, 29 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.Visibility.default", "code": "def Visibility.default : Visibility := { val := 0 }", "start": [ 357, 1 ], "end": [ 357, 54 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.Visibility.hidden", "code": "def Visibility.hidden : Visibility := { val := 1 }", "start": [ 358, 1 ], "end": [ 358, 54 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.Visibility.protected", "code": "def Visibility.protected : Visibility := { val := 2 }", "start": [ 359, 1 ], "end": [ 359, 54 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.setVisibility", "code": "@[extern \"lean_llvm_set_visibility\"]\nopaque setVisibility {ctx : Context} (value : Value ctx) (visibility : Visibility) : BaseIO Unit", "start": [ 361, 1 ], "end": [ 362, 97 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.DLLStorageClass", "code": "structure DLLStorageClass where\n private mk :: val : UInt64", "start": [ 365, 1 ], "end": [ 366, 29 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.DLLStorageClass.default", "code": "def DLLStorageClass.default : DLLStorageClass := { val := 0 }", "start": [ 368, 1 ], "end": [ 368, 62 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.DLLStorageClass.import", "code": "def DLLStorageClass.import : DLLStorageClass := { val := 1 }", "start": [ 369, 1 ], "end": [ 369, 62 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.DLLStorageClass.export", "code": "def DLLStorageClass.export : DLLStorageClass := { val := 2 }", "start": [ 370, 1 ], "end": [ 370, 62 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.setDLLStorageClass", "code": "@[extern \"lean_llvm_set_dll_storage_class\"]\nopaque setDLLStorageClass {ctx : Context} (value : Value ctx) (dllStorageClass : DLLStorageClass) : BaseIO Unit", "start": [ 372, 1 ], "end": [ 373, 112 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.Linkage", "code": "structure Linkage where\n private mk :: val : UInt64", "start": [ 376, 1 ], "end": [ 377, 29 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.Linkage.external", "code": "def Linkage.external : Linkage := { val := 0 }", "start": [ 379, 1 ], "end": [ 380, 47 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.Linkage.availableExternally", "code": "def Linkage.availableExternally : Linkage := { val := 1 }", "start": [ 381, 1 ], "end": [ 381, 58 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.Linkage.linkOnceAny", "code": "def Linkage.linkOnceAny : Linkage := { val := 2 }", "start": [ 382, 1 ], "end": [ 383, 50 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.Linkage.linkOnceODR", "code": "def Linkage.linkOnceODR : Linkage := { val := 3 }", "start": [ 384, 1 ], "end": [ 385, 50 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.Linkage.linkOnceODRAutoHide", "code": "def Linkage.linkOnceODRAutoHide : Linkage := { val := 4 }", "start": [ 386, 1 ], "end": [ 387, 58 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.Linkage.weakAny", "code": "def Linkage.weakAny : Linkage := { val := 5 }", "start": [ 388, 1 ], "end": [ 389, 46 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.Linkage.weakODR", "code": "def Linkage.weakODR : Linkage := { val := 6 }", "start": [ 390, 1 ], "end": [ 391, 46 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.Linkage.appending", "code": "def Linkage.appending : Linkage := { val := 7 }", "start": [ 392, 1 ], "end": [ 393, 48 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.Linkage.internal", "code": "def Linkage.internal : Linkage := { val := 8 }", "start": [ 394, 1 ], "end": [ 395, 47 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.Linkage.private", "code": "def Linkage.private : Linkage := { val := 9 }", "start": [ 396, 1 ], "end": [ 397, 46 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.Linkage.dllImport", "code": "def Linkage.dllImport : Linkage := { val := 10 }", "start": [ 398, 1 ], "end": [ 399, 49 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.Linkage.dllExport", "code": "def Linkage.dllExport : Linkage := { val := 11 }", "start": [ 400, 1 ], "end": [ 401, 49 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.Linkage.externalWeak", "code": "def Linkage.externalWeak : Linkage := { val := 12 }", "start": [ 402, 1 ], "end": [ 403, 52 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.Linkage.ghost", "code": "def Linkage.ghost : Linkage := { val := 13 }", "start": [ 404, 1 ], "end": [ 405, 45 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.Linkage.common", "code": "def Linkage.common : Linkage := { val := 14 }", "start": [ 406, 1 ], "end": [ 407, 46 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.Linkage.linkerPrivate", "code": "def Linkage.linkerPrivate : Linkage := { val := 15 }", "start": [ 408, 1 ], "end": [ 409, 53 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.Linkage.linkerPrivateWeak", "code": "def Linkage.linkerPrivateWeak : Linkage := { val := 16 }", "start": [ 410, 1 ], "end": [ 411, 57 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.setLinkage", "code": "@[extern \"lean_llvm_set_linkage\"]\nopaque setLinkage {ctx : Context} (value : Value ctx) (linkage : Linkage) : BaseIO Unit", "start": [ 413, 1 ], "end": [ 414, 88 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.i1Type", "code": "def i1Type (ctx : LLVM.Context) : BaseIO (LLVM.LLVMType ctx) :=\n LLVM.intTypeInContext ctx 1", "start": [ 417, 1 ], "end": [ 418, 30 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.i8Type", "code": "def i8Type (ctx : LLVM.Context) : BaseIO (LLVM.LLVMType ctx) :=\n LLVM.intTypeInContext ctx 8", "start": [ 420, 1 ], "end": [ 421, 30 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.i16Type", "code": "def i16Type (ctx : LLVM.Context) : BaseIO (LLVM.LLVMType ctx) :=\n LLVM.intTypeInContext ctx 16", "start": [ 423, 1 ], "end": [ 424, 31 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.i32Type", "code": "def i32Type (ctx : LLVM.Context) : BaseIO (LLVM.LLVMType ctx) :=\n LLVM.intTypeInContext ctx 32", "start": [ 426, 1 ], "end": [ 427, 31 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.i64Type", "code": "def i64Type (ctx : LLVM.Context) : BaseIO (LLVM.LLVMType ctx) :=\n LLVM.intTypeInContext ctx 64", "start": [ 429, 1 ], "end": [ 430, 31 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.voidPtrType", "code": "def voidPtrType (ctx : LLVM.Context) : BaseIO (LLVM.LLVMType ctx) :=\n do LLVM.pointerType (← LLVM.intTypeInContext ctx 8)", "start": [ 432, 1 ], "end": [ 433, 54 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.i8PtrType", "code": "def i8PtrType (ctx : LLVM.Context) : BaseIO (LLVM.LLVMType ctx) :=\n voidPtrType ctx", "start": [ 435, 1 ], "end": [ 436, 18 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.constTrue", "code": "def constTrue (ctx : Context) : BaseIO (Value ctx) :=\n do constInt (← i1Type ctx) 1 (signExtend := false)", "start": [ 438, 1 ], "end": [ 439, 53 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.constFalse", "code": "def constFalse (ctx : Context) : BaseIO (Value ctx) :=\n do constInt (← i1Type ctx) 0 (signExtend := false)", "start": [ 441, 1 ], "end": [ 442, 53 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.constInt'", "code": "def constInt' (ctx : Context) (width : UInt64) (value : UInt64) (signExtend : Bool := false) : BaseIO (Value ctx) :=\n do constInt (← LLVM.intTypeInContext ctx width) value signExtend", "start": [ 444, 1 ], "end": [ 445, 66 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.constInt1", "code": "def constInt1 (ctx : Context) (value : UInt64) (signExtend : Bool := false) : BaseIO (Value ctx) :=\n constInt' ctx 1 value signExtend", "start": [ 447, 1 ], "end": [ 448, 35 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.constInt8", "code": "def constInt8 (ctx : Context) (value : UInt64) (signExtend : Bool := false) : BaseIO (Value ctx) :=\n constInt' ctx 8 value signExtend", "start": [ 450, 1 ], "end": [ 451, 35 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.constInt32", "code": "def constInt32 (ctx : Context) (value : UInt64) (signExtend : Bool := false) : BaseIO (Value ctx) :=\n constInt' ctx 32 value signExtend", "start": [ 453, 1 ], "end": [ 454, 36 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.constInt64", "code": "def constInt64 (ctx : Context) (value : UInt64) (signExtend : Bool := false) : BaseIO (Value ctx) :=\n constInt' ctx 64 value signExtend", "start": [ 456, 1 ], "end": [ 457, 36 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.constIntSizeT", "code": "def constIntSizeT (ctx : Context) (value : UInt64) (signExtend : Bool := false) : BaseIO (Value ctx) :=\n constInt' ctx 64 value signExtend", "start": [ 459, 1 ], "end": [ 461, 36 ], "kind": "commanddeclaration" }, { "full_name": "LLVM.constIntUnsigned", "code": "def constIntUnsigned (ctx : Context) (value : UInt64) (signExtend : Bool := false) : BaseIO (Value ctx) :=\n constInt' ctx 32 value signExtend", "start": [ 463, 1 ], "end": [ 465, 36 ], "kind": "commanddeclaration" } ]
.lake/packages/lean4/src/lean/lake/Lake.lean
[ ".lake/packages/lean4/src/lean/lake/Lake/Config.lean", ".lake/packages/lean4/src/lean/Init.lean", ".lake/packages/lean4/src/lean/lake/Lake/Toml.lean", ".lake/packages/lean4/src/lean/lake/Lake/DSL.lean", ".lake/packages/lean4/src/lean/lake/Lake/Version.lean", ".lake/packages/lean4/src/lean/lake/Lake/Build.lean", ".lake/packages/lean4/src/lean/lake/Lake/CLI/Actions.lean" ]
[]
.lake/packages/lean4/src/lean/lake/Lake/CLI.lean
[ ".lake/packages/lean4/src/lean/Init.lean", ".lake/packages/lean4/src/lean/lake/Lake/CLI/Main.lean" ]
[]
Mathlib.lean
[ "Mathlib/Data/Finset/Union.lean", "Mathlib/LinearAlgebra/TensorProduct/Matrix.lean", "Mathlib/NumberTheory/PrimesCongruentOne.lean", "Mathlib/Init/Data/Int/Lemmas.lean", "Mathlib/Topology/Homotopy/Equiv.lean", "Mathlib/CategoryTheory/Functor/Functorial.lean", "Mathlib/GroupTheory/GroupAction/Sum.lean", "Mathlib/Analysis/InnerProductSpace/Calculus.lean", "Mathlib/Data/Rat/Cast/Lemmas.lean", "Mathlib/Algebra/Category/ModuleCat/Presheaf/Sheafification.lean", "Mathlib/Topology/Connected/LocallyConnected.lean", "Mathlib/ModelTheory/Encoding.lean", "Mathlib/Tactic/Linarith/Oracle/SimplexAlgorithm/SimplexAlgorithm.lean", "Mathlib/LinearAlgebra/FreeModule/StrongRankCondition.lean", "Mathlib/RingTheory/Ideal/Basic.lean", "Mathlib/Data/Finset/NatDivisors.lean", "Mathlib/NumberTheory/LegendreSymbol/QuadraticReciprocity.lean", "Mathlib/Tactic/CC/Datatypes.lean", "Mathlib/Topology/ContinuousFunction/Sigma.lean", "Mathlib/Tactic/PPWithUniv.lean", "Mathlib/RingTheory/Polynomial/Eisenstein/Basic.lean", "Mathlib/MeasureTheory/Integral/ExpDecay.lean", "Mathlib/Analysis/InnerProductSpace/NormPow.lean", "Mathlib/ModelTheory/Skolem.lean", "Mathlib/Analysis/LocallyConvex/Basic.lean", "Mathlib/NumberTheory/Modular.lean", "Mathlib/Algebra/GroupWithZero/Hom.lean", "Mathlib/Topology/Algebra/Module/Multilinear/Basic.lean", "Mathlib/Order/CompactlyGenerated/Basic.lean", "Mathlib/AlgebraicTopology/DoldKan/Homotopies.lean", "Mathlib/Data/Multiset/NatAntidiagonal.lean", "Mathlib/Analysis/Distribution/AEEqOfIntegralContDiff.lean", "Mathlib/Algebra/Order/BigOperators/Group/Multiset.lean", "Mathlib/RingTheory/FiniteStability.lean", "Mathlib/Control/Fix.lean", "Mathlib/Topology/ContinuousFunction/Algebra.lean", "Mathlib/CategoryTheory/Sites/Coherent/ExtensiveSheaves.lean", "Mathlib/CategoryTheory/Functor/Derived/RightDerived.lean", "Mathlib/Deprecated/Group.lean", "Mathlib/LinearAlgebra/TensorAlgebra/Basic.lean", "Mathlib/Topology/Order/Hom/Basic.lean", "Mathlib/Data/Sign.lean", "Mathlib/ModelTheory/Satisfiability.lean", "Mathlib/Data/Vector/Mem.lean", "Mathlib/Topology/MetricSpace/Dilation.lean", "Mathlib/Topology/Order/IntermediateValue.lean", "Mathlib/Analysis/Convex/Between.lean", "Mathlib/Topology/Algebra/Group/Basic.lean", "Mathlib/Topology/Sheaves/Limits.lean", "Mathlib/Logic/IsEmpty.lean", "Mathlib/Algebra/GroupWithZero/Divisibility.lean", "Mathlib/CategoryTheory/Limits/EpiMono.lean", "Mathlib/CategoryTheory/Limits/Shapes/Biproducts.lean", "Mathlib/CategoryTheory/Shift/CommShift.lean", "Mathlib/Tactic/Choose.lean", "Mathlib/Control/Basic.lean", "Mathlib/Tactic/Sat/FromLRAT.lean", "Mathlib/GroupTheory/Transfer.lean", "Mathlib/LinearAlgebra/DirectSum/Finsupp.lean", "Mathlib/Algebra/Category/Grp/Basic.lean", "Mathlib/RingTheory/Polynomial/Cyclotomic/Eval.lean", "Mathlib/Topology/Order/T5.lean", "Mathlib/Algebra/MvPolynomial/Cardinal.lean", "Mathlib/Lean/Expr.lean", "Mathlib/Algebra/Group/Semiconj/Units.lean", "Mathlib/Data/List/TFAE.lean", "Mathlib/Order/Filter/ENNReal.lean", "Mathlib/Order/Filter/CountableSeparatingOn.lean", "Mathlib/Algebra/Category/FGModuleCat/Basic.lean", "Mathlib/Data/Matroid/Basic.lean", "Mathlib/LinearAlgebra/Dimension/Finrank.lean", "Mathlib/Algebra/Order/Group/Bounds.lean", "Mathlib/Data/Fin/Tuple/Sort.lean", "Mathlib/Tactic/Positivity.lean", "Mathlib/Topology/MetricSpace/Thickening.lean", "Mathlib/Analysis/Complex/UnitDisc/Basic.lean", "Mathlib/Analysis/Calculus/Rademacher.lean", "Mathlib/Order/Category/OmegaCompletePartialOrder.lean", "Mathlib/Logic/Pairwise.lean", "Mathlib/Analysis/PSeriesComplex.lean", "Mathlib/CategoryTheory/LiftingProperties/Adjunction.lean", "Mathlib/CategoryTheory/Sites/Coherent/Basic.lean", "Mathlib/Combinatorics/SimpleGraph/Hasse.lean", "Mathlib/Computability/PartrecCode.lean", "Mathlib/Control/Monad/Basic.lean", "Mathlib/Algebra/Category/Ring/Constructions.lean", "Mathlib/Data/Complex/BigOperators.lean", "Mathlib/Data/UInt.lean", "Mathlib/MeasureTheory/OuterMeasure/AE.lean", "Mathlib/ModelTheory/Syntax.lean", "Mathlib/Order/Filter/AtTopBot.lean", "Mathlib/NumberTheory/Zsqrtd/Basic.lean", "Mathlib/Tactic/Conv.lean", "Mathlib/Combinatorics/Derangements/Basic.lean", "Mathlib/Topology/UrysohnsBounded.lean", "Mathlib/Data/Finset/Functor.lean", "Mathlib/LinearAlgebra/DirectSum/TensorProduct.lean", "Mathlib/Topology/Order/Bornology.lean", "Mathlib/Topology/ContinuousFunction/FunctionalCalculus.lean", "Mathlib/CategoryTheory/Filtered/Final.lean", "Mathlib/RingTheory/Coprime/Lemmas.lean", "Mathlib/Data/ZMod/Coprime.lean", "Mathlib/MeasureTheory/Integral/Bochner.lean", "Mathlib/MeasureTheory/Function/ConditionalExpectation/CondexpL1.lean", "Mathlib/NumberTheory/SiegelsLemma.lean", "Mathlib/CategoryTheory/Sites/ConcreteSheafification.lean", "Mathlib/Data/Buffer/Basic.lean", "Mathlib/Analysis/InnerProductSpace/LaxMilgram.lean", "Mathlib/SetTheory/ZFC/Ordinal.lean", "Mathlib/Data/Nat/ModEq.lean", "Mathlib/GroupTheory/CoprodI.lean", "Mathlib/Data/Nat/Log.lean", "Mathlib/Algebra/Homology/ComplexShape.lean", "Mathlib/FieldTheory/IsAlgClosed/AlgebraicClosure.lean", "Mathlib/NumberTheory/NumberField/Embeddings.lean", "Mathlib/Algebra/Lie/CartanMatrix.lean", "Mathlib/LinearAlgebra/Span.lean", "Mathlib/Algebra/Homology/HomotopyCategory/SingleFunctors.lean", "Mathlib/Algebra/Star/Unitary.lean", "Mathlib/CategoryTheory/Limits/Shapes/ZeroObjects.lean", "Mathlib/RingTheory/TensorProduct/MvPolynomial.lean", "Mathlib/RepresentationTheory/Character.lean", "Mathlib/Algebra/Order/Positive/Ring.lean", "Mathlib/Lean/EnvExtension.lean", "Mathlib/Algebra/Group/Pi/Basic.lean", "Mathlib/Algebra/ContinuedFractions/Computation/CorrectnessTerminating.lean", "Mathlib/CategoryTheory/Limits/Shapes/BinaryProducts.lean", "Mathlib/Data/Subtype.lean", "Mathlib/Tactic/Ring/PNat.lean", "Mathlib/Topology/Category/Locale.lean", "Mathlib/Algebra/Ring/Subsemiring/Pointwise.lean", "Mathlib/Util/CountHeartbeats.lean", "Mathlib/CategoryTheory/IsomorphismClasses.lean", "Mathlib/LinearAlgebra/LinearPMap.lean", "Mathlib/Algebra/EuclideanDomain/Basic.lean", "Mathlib/Analysis/Convex/StrictConvexBetween.lean", "Mathlib/RingTheory/WittVector/DiscreteValuationRing.lean", "Mathlib/Algebra/Squarefree/Basic.lean", "Mathlib/Algebra/Order/CauSeq/Basic.lean", "Mathlib/Analysis/Convex/Radon.lean", "Mathlib/Data/Nat/Factors.lean", "Mathlib/Data/Set/Function.lean", "Mathlib/Order/BoundedOrder.lean", "Mathlib/Order/Closure.lean", "Mathlib/RingTheory/IntegralClosure.lean", "Mathlib/CategoryTheory/Limits/Preserves/FunctorCategory.lean", "Mathlib/Analysis/Analytic/Composition.lean", "Mathlib/Analysis/Calculus/InverseFunctionTheorem/FiniteDimensional.lean", "Mathlib/CategoryTheory/Adjunction/Unique.lean", "Mathlib/Algebra/Order/Ring/Abs.lean", "Mathlib/Condensed/Light/Module.lean", "Mathlib/Algebra/Order/GroupWithZero/Unbundled.lean", "Mathlib/Analysis/Fourier/RiemannLebesgueLemma.lean", "Mathlib/RingTheory/MvPowerSeries/Inverse.lean", "Mathlib/Topology/Semicontinuous.lean", "Mathlib/Data/Complex/Cardinality.lean", "Mathlib/LinearAlgebra/Matrix/Trace.lean", "Mathlib/Algebra/Algebra/Subalgebra/Basic.lean", "Mathlib/Data/Multiset/Antidiagonal.lean", "Mathlib/Algebra/Lie/EngelSubalgebra.lean", "Mathlib/CategoryTheory/MorphismProperty/Concrete.lean", "Mathlib/Analysis/NormedSpace/Star/ContinuousFunctionalCalculus/Instances.lean", "Mathlib/Algebra/Category/ModuleCat/Adjunctions.lean", "Mathlib/Algebra/Module/Injective.lean", "Mathlib/Data/Finset/Card.lean", "Mathlib/CategoryTheory/Localization/FiniteProducts.lean", "Mathlib/CategoryTheory/Limits/HasLimits.lean", "Mathlib/AlgebraicGeometry/OpenImmersion.lean", "Mathlib/Algebra/Star/Prod.lean", "Mathlib/CategoryTheory/Limits/Shapes/FiniteProducts.lean", "Mathlib/CategoryTheory/Limits/FinallySmall.lean", "Mathlib/Tactic/ComputeDegree.lean", "Mathlib/Topology/Order/Lattice.lean", "Mathlib/Combinatorics/SimpleGraph/Regularity/Equitabilise.lean", "Mathlib/AlgebraicTopology/DoldKan/FunctorN.lean", "Mathlib/Tactic/Linarith/Datatypes.lean", "Mathlib/Algebra/Homology/HomologySequenceLemmas.lean", "Mathlib/Geometry/RingedSpace/Stalks.lean", "Mathlib/Tactic/NormNum/GCD.lean", "Mathlib/Analysis/Complex/PhragmenLindelof.lean", "Mathlib/AlgebraicGeometry/Cover/Open.lean", "Mathlib/Topology/Sheaves/SheafCondition/OpensLeCover.lean", "Mathlib/Topology/PartialHomeomorph.lean", "Mathlib/Analysis/Convex/EGauge.lean", "Mathlib/Tactic/ScopedNS.lean", "Mathlib/Analysis/Calculus/LineDeriv/Basic.lean", "Mathlib/CategoryTheory/Sites/DenseSubsite.lean", "Mathlib/CategoryTheory/Sites/LocallyInjective.lean", "Mathlib/GroupTheory/Subgroup/Center.lean", "Mathlib/Logic/Equiv/List.lean", "Mathlib/Topology/Order/Hom/Esakia.lean", "Mathlib/Order/RelIso/Set.lean", "Mathlib/NumberTheory/NumberField/ClassNumber.lean", "Mathlib/LinearAlgebra/FinsuppVectorSpace.lean", "Mathlib/Geometry/Manifold/DerivationBundle.lean", "Mathlib/Geometry/Euclidean/Sphere/Ptolemy.lean", "Mathlib/Data/Finset/Fin.lean", "Mathlib/Data/Real/Star.lean", "Mathlib/LinearAlgebra/BilinearForm/TensorProduct.lean", "Mathlib/Analysis/Calculus/LocalExtr/Rolle.lean", "Mathlib/Topology/Sheaves/Forget.lean", "Mathlib/Tactic/Widget/Calc.lean", "Mathlib/Tactic/IntervalCases.lean", "Mathlib/CategoryTheory/Abelian/Exact.lean", "Mathlib/Topology/CompactOpen.lean", "Mathlib/LinearAlgebra/Matrix/Dual.lean", "Mathlib/Order/Filter/Interval.lean", "Mathlib/MeasureTheory/Measure/Haar/OfBasis.lean", "Mathlib/Algebra/ContinuedFractions/TerminatedStable.lean", "Mathlib/Order/OrderIsoNat.lean", "Mathlib/CategoryTheory/Limits/Shapes/Diagonal.lean", "Mathlib/FieldTheory/Laurent.lean", "Mathlib/Algebra/Polynomial/Monic.lean", "Mathlib/LinearAlgebra/CliffordAlgebra/Basic.lean", "Mathlib/RepresentationTheory/FdRep.lean", "Mathlib/Tactic/FunProp/Core.lean", "Mathlib/Algebra/CharP/Subring.lean", "Mathlib/Tactic/Relation/Symm.lean", "Mathlib/Algebra/Group/Invertible/Basic.lean", "Mathlib/LinearAlgebra/Dimension/DivisionRing.lean", "Mathlib/ModelTheory/Basic.lean", "Mathlib/CategoryTheory/Preadditive/InjectiveResolution.lean", "Mathlib/Combinatorics/Configuration.lean", "Mathlib/Data/QPF/Multivariate/Constructions/Const.lean", "Mathlib/Algebra/MonoidAlgebra/Ideal.lean", "Mathlib/CategoryTheory/Monoidal/Functorial.lean", "Mathlib/LinearAlgebra/TensorAlgebra/Grading.lean", "Mathlib/Analysis/Calculus/Gradient/Basic.lean", "Mathlib/Analysis/Convex/SimplicialComplex/Basic.lean", "Mathlib/Algebra/Algebra/Subalgebra/Rank.lean", "Mathlib/CategoryTheory/Triangulated/Basic.lean", "Mathlib/GroupTheory/GroupAction/DomAct/Basic.lean", "Mathlib/Data/Rat/Denumerable.lean", "Mathlib/Algebra/Category/Grp/EpiMono.lean", "Mathlib/Data/Finsupp/Interval.lean", "Mathlib/Lean/CoreM.lean", "Mathlib/LinearAlgebra/QuadraticForm/Prod.lean", "Mathlib/LinearAlgebra/AffineSpace/Pointwise.lean", "Mathlib/Algebra/Order/Monoid/Unbundled/Defs.lean", "Mathlib/Algebra/Module/Algebra.lean", "Mathlib/Analysis/SpecialFunctions/Gaussian/FourierTransform.lean", "Mathlib/Topology/DiscreteSubset.lean", "Mathlib/Combinatorics/SetFamily/Compression/UV.lean", "Mathlib/Algebra/Category/ModuleCat/Sheaf/Colimits.lean", "Mathlib/Order/Category/BddOrd.lean", "Mathlib/Probability/BorelCantelli.lean", "Mathlib/Algebra/Order/BigOperators/Ring/Multiset.lean", "Mathlib/GroupTheory/Abelianization.lean", "Mathlib/SetTheory/Cardinal/Subfield.lean", "Mathlib/SetTheory/Game/Birthday.lean", "Mathlib/Algebra/AddConstMap/Basic.lean", "Mathlib/CategoryTheory/Idempotents/KaroubiKaroubi.lean", "Mathlib/Logic/Equiv/TransferInstance.lean", "Mathlib/Control/Random.lean", "Mathlib/RingTheory/AdicCompletion/Basic.lean", "Mathlib/Tactic/NthRewrite.lean", "Mathlib/Tactic/Have.lean", "Mathlib/Topology/MetricSpace/Pseudo/Defs.lean", "Mathlib/Tactic/ExtendDoc.lean", "Mathlib/RingTheory/Flat/Basic.lean", "Mathlib/Topology/MetricSpace/DilationEquiv.lean", "Mathlib/RingTheory/FinitePresentation.lean", "Mathlib/Algebra/Ring/Nat.lean", "Mathlib/Algebra/Order/Antidiag/Pi.lean", "Mathlib/Algebra/BigOperators/Intervals.lean", "Mathlib/CategoryTheory/Abelian/Subobject.lean", "Mathlib/Algebra/Homology/SingleHomology.lean", "Mathlib/Algebra/Polynomial/Bivariate.lean", "Mathlib/CategoryTheory/Triangulated/Rotate.lean", "Mathlib/Data/Int/LeastGreatest.lean", "Mathlib/Algebra/CharP/Pi.lean", "Mathlib/Logic/Encodable/Lattice.lean", "Mathlib/Analysis/Convex/Quasiconvex.lean", "Mathlib/Tactic/NormNum.lean", "Mathlib/CategoryTheory/Limits/Yoneda.lean", "Mathlib/Analysis/Calculus/ContDiff/RCLike.lean", "Mathlib/Data/Nat/Set.lean", "Mathlib/Geometry/Euclidean/Angle/Oriented/RightAngle.lean", "Mathlib/LinearAlgebra/TensorProduct/DirectLimit.lean", "Mathlib/Algebra/Homology/TotalComplexShift.lean", "Mathlib/Combinatorics/SimpleGraph/StronglyRegular.lean", "Mathlib/LinearAlgebra/CliffordAlgebra/Grading.lean", "Mathlib/Data/Rbtree/Find.lean", "Mathlib/LinearAlgebra/Multilinear/Basis.lean", "Mathlib/Tactic/Simps/NotationClass.lean", "Mathlib/Analysis/Normed/Group/Pointwise.lean", "Mathlib/Topology/NoetherianSpace.lean", "Mathlib/Data/Finsupp/Fin.lean", "Mathlib/GroupTheory/QuotientGroup.lean", "Mathlib/CategoryTheory/Bicategory/Extension.lean", "Mathlib/NumberTheory/Harmonic/Int.lean", "Mathlib/Geometry/RingedSpace/PresheafedSpace.lean", "Mathlib/AlgebraicTopology/DoldKan/Equivalence.lean", "Mathlib/MeasureTheory/Function/LocallyIntegrable.lean", "Mathlib/Topology/EMetricSpace/Basic.lean", "Mathlib/Analysis/Calculus/InverseFunctionTheorem/ApproximatesLinearOn.lean", "Mathlib/MeasureTheory/Measure/Content.lean", "Mathlib/CategoryTheory/Adjunction/Opposites.lean", "Mathlib/Data/Matrix/Hadamard.lean", "Mathlib/Algebra/Group/Invertible/Defs.lean", "Mathlib/Data/Nat/EvenOddRec.lean", "Mathlib/CategoryTheory/Preadditive/Generator.lean", "Mathlib/MeasureTheory/Integral/Periodic.lean", "Mathlib/Analysis/InnerProductSpace/PiL2.lean", "Mathlib/Algebra/Order/Group/Basic.lean", "Mathlib/Data/Nat/Factorial/Basic.lean", "Mathlib/Tactic/Lemma.lean", "Mathlib/Analysis/Complex/Conformal.lean", "Mathlib/Order/Minimal.lean", "Mathlib/RingTheory/Polynomial/RationalRoot.lean", "Mathlib/Topology/UniformSpace/CompactConvergence.lean", "Mathlib/Analysis/Normed/Group/AddCircle.lean", "Mathlib/MeasureTheory/Measure/HasOuterApproxClosed.lean", "Mathlib/Order/SuccPred/IntervalSucc.lean", "Mathlib/Algebra/Module/Bimodule.lean", "Mathlib/Algebra/Homology/Single.lean", "Mathlib/Analysis/Calculus/FDeriv/RestrictScalars.lean", "Mathlib/CategoryTheory/Subobject/WellPowered.lean", "Mathlib/Combinatorics/SimpleGraph/Matching.lean", "Mathlib/CategoryTheory/ConcreteCategory/Elementwise.lean", "Mathlib/Data/Ordmap/Ordnode.lean", "Mathlib/Analysis/Convex/Cone/Extension.lean", "Mathlib/Order/Bounds/OrderIso.lean", "Mathlib/Testing/SlimCheck/Testable.lean", "Mathlib/RingTheory/Ideal/Maps.lean", "Mathlib/Analysis/Normed/Group/Basic.lean", "Mathlib/Analysis/Convex/StoneSeparation.lean", "Mathlib/LinearAlgebra/BilinearForm/Properties.lean", "Mathlib/Init/Data/List/Lemmas.lean", "Mathlib/Analysis/NormedSpace/Star/Multiplier.lean", "Mathlib/Geometry/Euclidean/Inversion/Basic.lean", "Mathlib/Algebra/Category/Grp/EnoughInjectives.lean", "Mathlib/Analysis/Calculus/ParametricIntegral.lean", "Mathlib/CategoryTheory/Sites/CoverLifting.lean", "Mathlib/Util/AddRelatedDecl.lean", "Mathlib/Algebra/Homology/HomologicalComplexLimits.lean", "Mathlib/Analysis/Calculus/FDeriv/Analytic.lean", "Mathlib/Algebra/Order/Monoid/Defs.lean", "Mathlib/Algebra/Polynomial/Reverse.lean", "Mathlib/MeasureTheory/Function/LpSeminorm/ChebyshevMarkov.lean", "Mathlib/CategoryTheory/Limits/Preserves/Finite.lean", "Mathlib/Algebra/IsPrimePow.lean", "Mathlib/Algebra/Category/Semigrp/Basic.lean", "Mathlib/Data/Nat/Fib/Zeckendorf.lean", "Mathlib/Topology/SeparatedMap.lean", "Mathlib/Algebra/Homology/Opposite.lean", "Mathlib/RingTheory/WittVector/Defs.lean", "Mathlib/Data/Finset/PImage.lean", "Mathlib/Init/Align.lean", "Mathlib/ModelTheory/Algebra/Ring/Basic.lean", "Mathlib/Topology/ContinuousFunction/Bounded.lean", "Mathlib/RingTheory/Derivation/Lie.lean", "Mathlib/Algebra/Lie/Submodule.lean", "Mathlib/GroupTheory/Commutator.lean", "Mathlib/Dynamics/Circle/RotationNumber/TranslationNumber.lean", "Mathlib/Algebra/Category/ModuleCat/Basic.lean", "Mathlib/Analysis/MeanInequalitiesPow.lean", "Mathlib/Data/Multiset/Lattice.lean", "Mathlib/Order/Sublattice.lean", "Mathlib/LinearAlgebra/QuadraticForm/TensorProduct.lean", "Mathlib/Order/Interval/Set/UnorderedInterval.lean", "Mathlib/Geometry/Euclidean/Angle/Unoriented/Basic.lean", "Mathlib/Geometry/Manifold/Algebra/SmoothFunctions.lean", "Mathlib/Combinatorics/SimpleGraph/Prod.lean", "Mathlib/MeasureTheory/Function/L2Space.lean", "Mathlib/Algebra/BigOperators/WithTop.lean", "Mathlib/Combinatorics/SetFamily/AhlswedeZhang.lean", "Mathlib/Combinatorics/SimpleGraph/Connectivity/Subgraph.lean", "Mathlib/RingTheory/Localization/Integer.lean", "Mathlib/CategoryTheory/Limits/Constructions/Equalizers.lean", "Mathlib/Algebra/Order/Module/Synonym.lean", "Mathlib/RingTheory/Polynomial/IrreducibleRing.lean", "Mathlib/RingTheory/PowerSeries/Order.lean", "Mathlib/Analysis/BoxIntegral/Partition/Split.lean", "Mathlib/RingTheory/Generators.lean", "Mathlib/MeasureTheory/Integral/Marginal.lean", "Mathlib/Logic/Function/OfArity.lean", "Mathlib/RingTheory/Polynomial/Opposites.lean", "Mathlib/CategoryTheory/Preadditive/EilenbergMoore.lean", "Mathlib/Combinatorics/SimpleGraph/Acyclic.lean", "Mathlib/Data/Finset/Image.lean", "Mathlib/Analysis/NormedSpace/PiTensorProduct/InjectiveSeminorm.lean", "Mathlib/CategoryTheory/MorphismProperty/Composition.lean", "Mathlib/CategoryTheory/ConcreteCategory/UnbundledHom.lean", "Mathlib/Data/Num/Bitwise.lean", "Mathlib/LinearAlgebra/Basis/Flag.lean", "Mathlib/MeasureTheory/Integral/Indicator.lean", "Mathlib/Data/Matroid/Restrict.lean", "Mathlib/RingTheory/WittVector/Teichmuller.lean", "Mathlib/Order/Category/FinBddDistLat.lean", "Mathlib/Data/Int/Cast/Field.lean", "Mathlib/Algebra/Ring/Action/Group.lean", "Mathlib/Order/Monotone/Monovary.lean", "Mathlib/Tactic/LinearCombination.lean", "Mathlib/CategoryTheory/Sites/LeftExact.lean", "Mathlib/Tactic/Linter/HashCommandLinter.lean", "Mathlib/Algebra/Order/Archimedean.lean", "Mathlib/Computability/RegularExpressions.lean", "Mathlib/Tactic/RenameBVar.lean", "Mathlib/Logic/Function/Conjugate.lean", "Mathlib/LinearAlgebra/Matrix/Polynomial.lean", "Mathlib/MeasureTheory/Measure/GiryMonad.lean", "Mathlib/Tactic/Contrapose.lean", "Mathlib/Data/Semiquot.lean", "Mathlib/GroupTheory/Index.lean", "Mathlib/Geometry/Manifold/VectorBundle/Tangent.lean", "Mathlib/AlgebraicGeometry/FunctionField.lean", "Mathlib/Combinatorics/SimpleGraph/Connectivity.lean", "Mathlib/Logic/Small/Ring.lean", "Mathlib/LinearAlgebra/Matrix/AbsoluteValue.lean", "Mathlib/LinearAlgebra/AffineSpace/AffineEquiv.lean", "Mathlib/Data/Multiset/Pi.lean", "Mathlib/Analysis/Analytic/Polynomial.lean", "Mathlib/Data/ENNReal/Operations.lean", "Mathlib/Analysis/SpecialFunctions/Exp.lean", "Mathlib/Data/Matrix/ColumnRowPartitioned.lean", "Mathlib/Analysis/Calculus/Dslope.lean", "Mathlib/Algebra/Category/ModuleCat/Sheaf/Generators.lean", "Mathlib/LinearAlgebra/Matrix/Nondegenerate.lean", "Mathlib/NumberTheory/ArithmeticFunction.lean", "Mathlib/RingTheory/NormTrace.lean", "Mathlib/MeasureTheory/Constructions/EventuallyMeasurable.lean", "Mathlib/NumberTheory/Primorial.lean", "Mathlib/Order/Synonym.lean", "Mathlib/Algebra/Homology/HomologicalComplexBiprod.lean", "Mathlib/Combinatorics/Additive/RuzsaCovering.lean", "Mathlib/Analysis/RCLike/Basic.lean", "Mathlib/CategoryTheory/Limits/Shapes/DisjointCoproduct.lean", "Mathlib/Data/Erased.lean", "Mathlib/RingTheory/Polynomial/Vieta.lean", "Mathlib/Algebra/Polynomial/Degree/Lemmas.lean", "Mathlib/Analysis/Calculus/Deriv/Pow.lean", "Mathlib/CategoryTheory/Localization/Bousfield.lean", "Mathlib/Algebra/BigOperators/Ring/Multiset.lean", "Mathlib/Topology/CompletelyRegular.lean", "Mathlib/CategoryTheory/Sites/Abelian.lean", "Mathlib/Analysis/Calculus/Deriv/Support.lean", "Mathlib/Combinatorics/SimpleGraph/Triangle/Removal.lean", "Mathlib/Topology/Category/TopCat/Opens.lean", "Mathlib/Topology/Algebra/ConstMulAction.lean", "Mathlib/Analysis/Convex/Independent.lean", "Mathlib/Topology/Sheaves/Functors.lean", "Mathlib/Algebra/Polynomial/Degree/CardPowDegree.lean", "Mathlib/RingTheory/Polynomial/Cyclotomic/Roots.lean", "Mathlib/CategoryTheory/ChosenFiniteProducts.lean", "Mathlib/NumberTheory/Liouville/LiouvilleNumber.lean", "Mathlib/RingTheory/Regular/RegularSequence.lean", "Mathlib/Algebra/Lie/Weights/RootSystem.lean", "Mathlib/GroupTheory/Submonoid/Centralizer.lean", "Mathlib/RingTheory/UniqueFactorizationDomain.lean", "Mathlib/MeasureTheory/Measure/Lebesgue/Complex.lean", "Mathlib/CategoryTheory/Sites/EffectiveEpimorphic.lean", "Mathlib/Analysis/Calculus/Deriv/Comp.lean", "Mathlib/Algebra/LinearRecurrence.lean", "Mathlib/AlgebraicGeometry/Morphisms/QuasiCompact.lean", "Mathlib/Order/GameAdd.lean", "Mathlib/Algebra/Category/ModuleCat/EpiMono.lean", "Mathlib/Data/List/Chain.lean", "Mathlib/Algebra/Group/NatPowAssoc.lean", "Mathlib/Analysis/ODE/PicardLindelof.lean", "Mathlib/Order/JordanHolder.lean", "Mathlib/Analysis/InnerProductSpace/Symmetric.lean", "Mathlib/AlgebraicTopology/KanComplex.lean", "Mathlib/Analysis/Normed/Order/Basic.lean", "Mathlib/Algebra/BigOperators/Ring.lean", "Mathlib/RingTheory/Localization/Finiteness.lean", "Mathlib/Analysis/SpecialFunctions/Log/ENNReal.lean", "Mathlib/Algebra/Homology/ShortComplex/HomologicalComplex.lean", "Mathlib/Analysis/Convex/Cone/Proper.lean", "Mathlib/CategoryTheory/GradedObject.lean", "Mathlib/GroupTheory/Congruence/Basic.lean", "Mathlib/CategoryTheory/Filtered/Connected.lean", "Mathlib/Algebra/Category/ModuleCat/Subobject.lean", "Mathlib/CategoryTheory/Limits/Shapes/StrictInitial.lean", "Mathlib/CategoryTheory/Conj.lean", "Mathlib/Topology/Order/ExtrClosure.lean", "Mathlib/Order/CompleteSublattice.lean", "Mathlib/RingTheory/RingHom/Surjective.lean", "Mathlib/Combinatorics/SetFamily/LYM.lean", "Mathlib/Analysis/Calculus/Monotone.lean", "Mathlib/Analysis/Asymptotics/AsymptoticEquivalent.lean", "Mathlib/Order/Interval/Set/OrderIso.lean", "Mathlib/NumberTheory/Liouville/Basic.lean", "Mathlib/Algebra/Algebra/Quasispectrum.lean", "Mathlib/CategoryTheory/Monoidal/NaturalTransformation.lean", "Mathlib/RingTheory/WittVector/Compare.lean", "Mathlib/Algebra/Homology/HomologicalComplexAbelian.lean", "Mathlib/SetTheory/Surreal/Multiplication.lean", "Mathlib/Analysis/Calculus/InverseFunctionTheorem/ContDiff.lean", "Mathlib/Control/Traversable/Lemmas.lean", "Mathlib/Data/MLList/Dedup.lean", "Mathlib/Geometry/Manifold/IntegralCurve.lean", "Mathlib/NumberTheory/Cyclotomic/Basic.lean", "Mathlib/Probability/Martingale/Centering.lean", "Mathlib/RingTheory/DedekindDomain/IntegralClosure.lean", "Mathlib/Algebra/Polynomial/Coeff.lean", "Mathlib/LinearAlgebra/Determinant.lean", "Mathlib/Lean/Json.lean", "Mathlib/RingTheory/RingHom/Finite.lean", "Mathlib/Init/Data/Sigma/Lex.lean", "Mathlib/Algebra/Category/Grp/ZModuleEquivalence.lean", "Mathlib/MeasureTheory/Integral/Gamma.lean", "Mathlib/Analysis/Calculus/BumpFunction/FiniteDimension.lean", "Mathlib/Data/Int/GCD.lean", "Mathlib/CategoryTheory/Closed/Monoidal.lean", "Mathlib/CategoryTheory/Functor/ReflectsIso.lean", "Mathlib/SetTheory/Game/Domineering.lean", "Mathlib/RingTheory/Localization/AtPrime.lean", "Mathlib/Analysis/Complex/Schwarz.lean", "Mathlib/RingTheory/Bezout.lean", "Mathlib/Algebra/Order/Group/Nat.lean", "Mathlib/RingTheory/Ideal/Basis.lean", "Mathlib/Analysis/BoundedVariation.lean", "Mathlib/Data/String/Lemmas.lean", "Mathlib/Algebra/Category/Ring/FilteredColimits.lean", "Mathlib/Probability/Kernel/IntegralCompProd.lean", "Mathlib/Algebra/Ring/Opposite.lean", "Mathlib/Analysis/Normed/Group/Seminorm.lean", "Mathlib/CategoryTheory/Functor/Currying.lean", "Mathlib/MeasureTheory/Function/AEEqOfIntegral.lean", "Mathlib/Analysis/NormedSpace/OperatorNorm/Prod.lean", "Mathlib/LinearAlgebra/Dimension/FreeAndStrongRankCondition.lean", "Mathlib/Tactic/Rename.lean", "Mathlib/Combinatorics/SetFamily/Intersecting.lean", "Mathlib/Tactic/MkIffOfInductiveProp.lean", "Mathlib/MeasureTheory/Integral/PeakFunction.lean", "Mathlib/Algebra/Polynomial/FieldDivision.lean", "Mathlib/Topology/Homotopy/Contractible.lean", "Mathlib/Condensed/Explicit.lean", "Mathlib/AlgebraicTopology/FundamentalGroupoid/Product.lean", "Mathlib/CategoryTheory/Limits/Shapes/Countable.lean", "Mathlib/Data/Int/ModEq.lean", "Mathlib/Analysis/BoxIntegral/DivergenceTheorem.lean", "Mathlib/NumberTheory/Multiplicity.lean", "Mathlib/MeasureTheory/Function/StronglyMeasurable/Inner.lean", "Mathlib/RingTheory/Polynomial/Basic.lean", "Mathlib/Analysis/InnerProductSpace/LinearPMap.lean", "Mathlib/FieldTheory/IsPerfectClosure.lean", "Mathlib/LinearAlgebra/CliffordAlgebra/Fold.lean", "Mathlib/Algebra/Ring/Int.lean", "Mathlib/Data/List/GetD.lean", "Mathlib/Tactic/DeriveFintype.lean", "Mathlib/Tactic/FunProp/ContDiff.lean", "Mathlib/Topology/Algebra/InfiniteSum/Real.lean", "Mathlib/Topology/Connected/PathConnected.lean", "Mathlib/CategoryTheory/Sites/Limits.lean", "Mathlib/CategoryTheory/Sites/InducedTopology.lean", "Mathlib/Data/Stream/Init.lean", "Mathlib/Algebra/Field/Opposite.lean", "Mathlib/CategoryTheory/Limits/Preserves/Shapes/Pullbacks.lean", "Mathlib/CategoryTheory/Limits/Constructions/Over/Products.lean", "Mathlib/CategoryTheory/NatIso.lean", "Mathlib/Data/ULift.lean", "Mathlib/CategoryTheory/Limits/Cones.lean", "Mathlib/RingTheory/FiniteType.lean", "Mathlib/Probability/Kernel/Condexp.lean", "Mathlib/Topology/UniformSpace/AbsoluteValue.lean", "Mathlib/Analysis/NormedSpace/Banach.lean", "Mathlib/MeasureTheory/Measure/EverywherePos.lean", "Mathlib/Tactic/Variable.lean", "Mathlib/Algebra/Category/Grp/Kernels.lean", "Mathlib/Logic/Small/Set.lean", "Mathlib/Topology/Baire/LocallyCompactRegular.lean", "Mathlib/MeasureTheory/Integral/IntegralEqImproper.lean", "Mathlib/Algebra/CharP/Defs.lean", "Mathlib/LinearAlgebra/Coevaluation.lean", "Mathlib/Combinatorics/SimpleGraph/Triangle/Counting.lean", "Mathlib/Init/Data/Bool/Basic.lean", "Mathlib/Topology/Algebra/InfiniteSum/Basic.lean", "Mathlib/CategoryTheory/Abelian/DiagramLemmas/Four.lean", "Mathlib/Analysis/SpecialFunctions/Pow/NNReal.lean", "Mathlib/Topology/UniformSpace/Pi.lean", "Mathlib/Algebra/Homology/ShortComplex/Ab.lean", "Mathlib/Analysis/Convex/Hull.lean", "Mathlib/CategoryTheory/Monad/Basic.lean", "Mathlib/CategoryTheory/Monoidal/Functor.lean", "Mathlib/Order/Interval/Finset/Basic.lean", "Mathlib/Data/Nat/Factorization/Root.lean", "Mathlib/Order/Zorn.lean", "Mathlib/Data/NNRat/Lemmas.lean", "Mathlib/Topology/UniformSpace/AbstractCompletion.lean", "Mathlib/MeasureTheory/OuterMeasure/Operations.lean", "Mathlib/Data/Bool/Set.lean", "Mathlib/MeasureTheory/Covering/LiminfLimsup.lean", "Mathlib/Topology/Order/LocalExtr.lean", "Mathlib/MeasureTheory/Function/StronglyMeasurable/Lemmas.lean", "Mathlib/Algebra/Polynomial/Expand.lean", "Mathlib/LinearAlgebra/Multilinear/TensorProduct.lean", "Mathlib/Data/Multiset/Bind.lean", "Mathlib/AlgebraicTopology/DoldKan/EquivalencePseudoabelian.lean", "Mathlib/AlgebraicTopology/DoldKan/NReflectsIso.lean", "Mathlib/Topology/Algebra/ProperConstSMul.lean", "Mathlib/Algebra/Field/Rat.lean", "Mathlib/Algebra/Category/MonCat/Adjunctions.lean", "Mathlib/Data/List/MinMax.lean", "Mathlib/Probability/Distributions/Uniform.lean", "Mathlib/Algebra/MvPolynomial/Basic.lean", "Mathlib/Data/Nat/Count.lean", "Mathlib/Analysis/NormedSpace/Complemented.lean", "Mathlib/Data/Complex/Module.lean", "Mathlib/Algebra/Module/Submodule/Map.lean", "Mathlib/CategoryTheory/Sites/IsSheafOneHypercover.lean", "Mathlib/Data/Rbtree/Insert.lean", "Mathlib/Algebra/Tropical/Lattice.lean", "Mathlib/CategoryTheory/FinCategory/Basic.lean", "Mathlib/Computability/TMToPartrec.lean", "Mathlib/LinearAlgebra/AffineSpace/Basis.lean", "Mathlib/Logic/Equiv/Fintype.lean", "Mathlib/Algebra/Order/Ring/Star.lean", "Mathlib/MeasureTheory/Constructions/BorelSpace/Complex.lean", "Mathlib/RingTheory/GradedAlgebra/Basic.lean", "Mathlib/Data/FunLike/Fintype.lean", "Mathlib/SetTheory/Cardinal/UnivLE.lean", "Mathlib/Algebra/Star/Basic.lean", "Mathlib/Algebra/GradedMonoid.lean", "Mathlib/Tactic/Eval.lean", "Mathlib/CategoryTheory/Category/Quiv.lean", "Mathlib/Analysis/Calculus/FDeriv/Extend.lean", "Mathlib/Analysis/Convex/Jensen.lean", "Mathlib/Order/Directed.lean", "Mathlib/Data/Int/ConditionallyCompleteOrder.lean", "Mathlib/Data/Multiset/Range.lean", "Mathlib/Algebra/BigOperators/GroupWithZero/Finset.lean", "Mathlib/CategoryTheory/Sites/LocallySurjective.lean", "Mathlib/RingTheory/Polynomial/Hermite/Basic.lean", "Mathlib/Algebra/Homology/ShortComplex/PreservesHomology.lean", "Mathlib/Data/Set/Card.lean", "Mathlib/RingTheory/Etale/Basic.lean", "Mathlib/Analysis/SpecialFunctions/Arsinh.lean", "Mathlib/CategoryTheory/Limits/Shapes/KernelPair.lean", "Mathlib/CategoryTheory/Monoidal/Internal/Module.lean", "Mathlib/Topology/IndicatorConstPointwise.lean", "Mathlib/MeasureTheory/Covering/DensityTheorem.lean", "Mathlib/Tactic/FunProp/RefinedDiscrTree.lean", "Mathlib/Algebra/Category/Grp/Injective.lean", "Mathlib/CategoryTheory/Functor/Basic.lean", "Mathlib/Data/Matroid/Dual.lean", "Mathlib/CategoryTheory/Sites/Coherent/CoherentSheaves.lean", "Mathlib/Order/BooleanAlgebra.lean", "Mathlib/LinearAlgebra/Basis/VectorSpace.lean", "Mathlib/Order/Filter/EventuallyConst.lean", "Mathlib/Analysis/Complex/AbelLimit.lean", "Mathlib/Analysis/Calculus/AffineMap.lean", "Mathlib/CategoryTheory/Preadditive/HomOrthogonal.lean", "Mathlib/Combinatorics/Hindman.lean", "Mathlib/Algebra/Lie/Weights/Killing.lean", "Mathlib/Topology/Algebra/Module/StrongTopology.lean", "Mathlib/Data/Nat/Choose/Multinomial.lean", "Mathlib/Topology/Bornology/Constructions.lean", "Mathlib/Order/Notation.lean", "Mathlib/Topology/MetricSpace/CantorScheme.lean", "Mathlib/RingTheory/LaurentSeries.lean", "Mathlib/CategoryTheory/Limits/Shapes/FunctorCategory.lean", "Mathlib/Algebra/Category/ModuleCat/Sheaf/Free.lean", "Mathlib/Algebra/Lie/DirectSum.lean", "Mathlib/RingTheory/Discriminant.lean", "Mathlib/Logic/Small/Group.lean", "Mathlib/CategoryTheory/DiscreteCategory.lean", "Mathlib/NumberTheory/ZetaValues.lean", "Mathlib/Data/List/ToFinsupp.lean", "Mathlib/GroupTheory/Subgroup/Simple.lean", "Mathlib/Analysis/InnerProductSpace/Orthogonal.lean", "Mathlib/NumberTheory/ModularForms/CongruenceSubgroups.lean", "Mathlib/RingTheory/Noetherian.lean", "Mathlib/Logic/Nontrivial/Basic.lean", "Mathlib/Data/Nat/Choose/Vandermonde.lean", "Mathlib/Tactic/CancelDenoms/Core.lean", "Mathlib/CategoryTheory/Monad/Limits.lean", "Mathlib/Analysis/NormedSpace/HahnBanach/Separation.lean", "Mathlib/Algebra/Order/Monoid/ToMulBot.lean", "Mathlib/RingTheory/Presentation.lean", "Mathlib/Order/Filter/Prod.lean", "Mathlib/Analysis/Calculus/UniformLimitsDeriv.lean", "Mathlib/CategoryTheory/Sites/Subsheaf.lean", "Mathlib/Tactic/Ring.lean", "Mathlib/Data/List/Range.lean", "Mathlib/MeasureTheory/Function/AEMeasurableOrder.lean", "Mathlib/Topology/Algebra/OpenSubgroup.lean", "Mathlib/Tactic/CC.lean", "Mathlib/Algebra/Homology/HomotopyCategory/HomComplex.lean", "Mathlib/Analysis/Complex/Angle.lean", "Mathlib/Geometry/Manifold/ContMDiff/Atlas.lean", "Mathlib/Topology/Algebra/Ring/Basic.lean", "Mathlib/Data/Matrix/Rank.lean", "Mathlib/NumberTheory/ModularForms/Basic.lean", "Mathlib/Topology/Connected/Separation.lean", "Mathlib/Topology/CountableSeparatingOn.lean", "Mathlib/Topology/LocallyFinite.lean", "Mathlib/Order/LiminfLimsup.lean", "Mathlib/Algebra/Ring/Subsemiring/Basic.lean", "Mathlib/Tactic/HigherOrder.lean", "Mathlib/Topology/Support.lean", "Mathlib/Algebra/Algebra/Equiv.lean", "Mathlib/Algebra/Star/StarAlgHom.lean", "Mathlib/AlgebraicGeometry/Pullbacks.lean", "Mathlib/Analysis/Convex/Deriv.lean", "Mathlib/Analysis/NormedSpace/Completion.lean", "Mathlib/CategoryTheory/MorphismProperty/IsInvertedBy.lean", "Mathlib/CategoryTheory/Preadditive/Yoneda/Limits.lean", "Mathlib/Order/Interval/Finset/Defs.lean", "Mathlib/Analysis/SpecialFunctions/PolynomialExp.lean", "Mathlib/Init/Data/Quot.lean", "Mathlib/MeasureTheory/Function/AEMeasurableSequence.lean", "Mathlib/GroupTheory/GroupAction/Hom.lean", "Mathlib/Tactic/CategoryTheory/Coherence.lean", "Mathlib/Algebra/ModEq.lean", "Mathlib/Algebra/Polynomial/EraseLead.lean", "Mathlib/Analysis/Convex/Function.lean", "Mathlib/Algebra/Ring/CentroidHom.lean", "Mathlib/CategoryTheory/Idempotents/SimplicialObject.lean", "Mathlib/CategoryTheory/Limits/Preserves/Opposites.lean", "Mathlib/LinearAlgebra/AffineSpace/Basic.lean", "Mathlib/LinearAlgebra/AffineSpace/Independent.lean", "Mathlib/Order/WellFoundedSet.lean", "Mathlib/SetTheory/Cardinal/Finite.lean", "Mathlib/Topology/Baire/Lemmas.lean", "Mathlib/Data/Seq/Parallel.lean", "Mathlib/Probability/Notation.lean", "Mathlib/CategoryTheory/Adjunction/Whiskering.lean", "Mathlib/Algebra/Module/FinitePresentation.lean", "Mathlib/CategoryTheory/PEmpty.lean", "Mathlib/RingTheory/Nilpotent/Basic.lean", "Mathlib/Util/SynthesizeUsing.lean", "Mathlib/LinearAlgebra/Matrix/SpecialLinearGroup.lean", "Mathlib/AlgebraicGeometry/Morphisms/UniversallyClosed.lean", "Mathlib/Algebra/Algebra/Spectrum.lean", "Mathlib/Data/Prod/PProd.lean", "Mathlib/Probability/Martingale/BorelCantelli.lean", "Mathlib/Data/List/Pairwise.lean", "Mathlib/Topology/Basic.lean", "Mathlib/Order/RelIso/Group.lean", "Mathlib/RingTheory/DiscreteValuationRing/Basic.lean", "Mathlib/CategoryTheory/Grothendieck.lean", "Mathlib/Geometry/Manifold/VectorBundle/SmoothSection.lean", "Mathlib/MeasureTheory/Measure/Haar/Quotient.lean", "Mathlib/MeasureTheory/Measure/Tilted.lean", "Mathlib/Algebra/Star/Pi.lean", "Mathlib/Analysis/LocallyConvex/AbsConvex.lean", "Mathlib/GroupTheory/FreeAbelianGroup.lean", "Mathlib/Probability/IdentDistrib.lean", "Mathlib/RingTheory/DedekindDomain/Basic.lean", "Mathlib/CategoryTheory/GradedObject/Associator.lean", "Mathlib/CategoryTheory/Products/Associator.lean", "Mathlib/SetTheory/Cardinal/ToNat.lean", "Mathlib/Init/Quot.lean", "Mathlib/Analysis/Complex/CauchyIntegral.lean", "Mathlib/Algebra/Lie/NonUnitalNonAssocAlgebra.lean", "Mathlib/CategoryTheory/Preadditive/Yoneda/Basic.lean", "Mathlib/CategoryTheory/Sites/SheafOfTypes.lean", "Mathlib/FieldTheory/Finiteness.lean", "Mathlib/Geometry/Manifold/VectorBundle/Pullback.lean", "Mathlib/Order/Filter/IndicatorFunction.lean", "Mathlib/Topology/Category/LightProfinite/Basic.lean", "Mathlib/Algebra/Group/WithOne/Defs.lean", "Mathlib/Algebra/Module/CharacterModule.lean", "Mathlib/Algebra/Lie/Semisimple/Basic.lean", "Mathlib/Probability/Distributions/Gaussian.lean", "Mathlib/Probability/ProbabilityMassFunction/Binomial.lean", "Mathlib/Topology/ContinuousFunction/Ideals.lean", "Mathlib/AlgebraicGeometry/EllipticCurve/Group.lean", "Mathlib/Probability/Kernel/Disintegration/Integral.lean", "Mathlib/CategoryTheory/Limits/Shapes/Products.lean", "Mathlib/NumberTheory/Divisors.lean", "Mathlib/Algebra/Module/Equiv.lean", "Mathlib/Topology/ProperMap.lean", "Mathlib/AlgebraicTopology/DoldKan/Normalized.lean", "Mathlib/Algebra/Lie/Derivation/Basic.lean", "Mathlib/CategoryTheory/FiberedCategory/Cartesian.lean", "Mathlib/LinearAlgebra/Orientation.lean", "Mathlib/Topology/Defs/Sequences.lean", "Mathlib/GroupTheory/GroupAction/Embedding.lean", "Mathlib/AlgebraicTopology/SimplicialCategory/Basic.lean", "Mathlib/LinearAlgebra/Dimension/RankNullity.lean", "Mathlib/Order/WithBot.lean", "Mathlib/NumberTheory/LegendreSymbol/GaussEisensteinLemmas.lean", "Mathlib/CategoryTheory/Sites/Closed.lean", "Mathlib/Control/Applicative.lean", "Mathlib/Topology/UniformSpace/UniformConvergence.lean", "Mathlib/Data/Nat/Cast/Prod.lean", "Mathlib/RingTheory/Norm.lean", "Mathlib/Topology/VectorBundle/Hom.lean", "Mathlib/Order/Atoms/Finite.lean", "Mathlib/Init/Classical.lean", "Mathlib/Algebra/Group/Submonoid/Units.lean", "Mathlib/Analysis/Complex/UpperHalfPlane/Topology.lean", "Mathlib/SetTheory/Game/Impartial.lean", "Mathlib/Algebra/CharP/Algebra.lean", "Mathlib/Data/List/Lattice.lean", "Mathlib/Combinatorics/SimpleGraph/Init.lean", "Mathlib/Data/Fin/SuccPred.lean", "Mathlib/GroupTheory/NoncommPiCoprod.lean", "Mathlib/Data/SProd.lean", "Mathlib/Analysis/InnerProductSpace/Projection.lean", "Mathlib/Analysis/Calculus/MeanValue.lean", "Mathlib/GroupTheory/Coxeter/Matrix.lean", "Mathlib/Analysis/Calculus/Implicit.lean", "Mathlib/Topology/Instances/RealVectorSpace.lean", "Mathlib/CategoryTheory/Monoidal/Braided/Opposite.lean", "Mathlib/Algebra/Group/Commute/Units.lean", "Mathlib/Order/Filter/Basic.lean", "Mathlib/Topology/Algebra/InfiniteSum/Group.lean", "Mathlib/Data/List/Sections.lean", "Mathlib/Algebra/Order/Module/Defs.lean", "Mathlib/MeasureTheory/Integral/IntegrableOn.lean", "Mathlib/Algebra/Ring/Aut.lean", "Mathlib/CategoryTheory/Sites/PreservesSheafification.lean", "Mathlib/NumberTheory/EulerProduct/Basic.lean", "Mathlib/CategoryTheory/Localization/CalculusOfFractions/ComposableArrows.lean", "Mathlib/Testing/SlimCheck/Functions.lean", "Mathlib/CategoryTheory/Category/Cat/Limit.lean", "Mathlib/Order/Disjointed.lean", "Mathlib/Algebra/Category/Ring/Adjunctions.lean", "Mathlib/Analysis/Asymptotics/Asymptotics.lean", "Mathlib/CategoryTheory/Monoidal/Opposite.lean", "Mathlib/Logic/Godel/GodelBetaFunction.lean", "Mathlib/Data/Nat/Bitwise.lean", "Mathlib/RingTheory/Bialgebra/Equiv.lean", "Mathlib/Tactic/Linarith/Lemmas.lean", "Mathlib/CategoryTheory/Limits/FullSubcategory.lean", "Mathlib/Algebra/BigOperators/RingEquiv.lean", "Mathlib/Analysis/SpecialFunctions/ImproperIntegrals.lean", "Mathlib/Data/Array/ExtractLemmas.lean", "Mathlib/Tactic/Spread.lean", "Mathlib/Topology/Category/Stonean/Limits.lean", "Mathlib/Order/Interval/Finset/Nat.lean", "Mathlib/Algebra/Module/Submodule/Pointwise.lean", "Mathlib/NumberTheory/FunctionField.lean", "Mathlib/Algebra/Lie/Weights/Chain.lean", "Mathlib/Algebra/CharP/Reduced.lean", "Mathlib/Algebra/Order/Monoid/Unbundled/Basic.lean", "Mathlib/Algebra/CharP/Two.lean", "Mathlib/Analysis/BoxIntegral/Box/Basic.lean", "Mathlib/Order/Hom/Set.lean", "Mathlib/RingTheory/Polynomial/Bernstein.lean", "Mathlib/Geometry/Euclidean/Inversion/Calculus.lean", "Mathlib/AlgebraicTopology/DoldKan/FunctorGamma.lean", "Mathlib/Topology/QuasiSeparated.lean", "Mathlib/Tactic/HaveI.lean", "Mathlib/Data/Prod/Lex.lean", "Mathlib/Analysis/ConstantSpeed.lean", "Mathlib/Order/Filter/NAry.lean", "Mathlib/Algebra/Homology/Embedding/Basic.lean", "Mathlib/Geometry/RingedSpace/SheafedSpace.lean", "Mathlib/Algebra/Star/RingQuot.lean", "Mathlib/Algebra/Module/LinearMap/End.lean", "Mathlib/CategoryTheory/Idempotents/Karoubi.lean", "Mathlib/Topology/Algebra/UniformConvergence.lean", "Mathlib/Computability/Encoding.lean", "Mathlib/CategoryTheory/Localization/Adjunction.lean", "Mathlib/CategoryTheory/Galois/Prorepresentability.lean", "Mathlib/CategoryTheory/Adjunction/AdjointFunctorTheorems.lean", "Mathlib/FieldTheory/ChevalleyWarning.lean", "Mathlib/Algebra/Module/Submodule/Order.lean", "Mathlib/Topology/Category/Stonean/EffectiveEpi.lean", "Mathlib/RingTheory/HahnSeries/Summable.lean", "Mathlib/Analysis/Convex/Integral.lean", "Mathlib/Analysis/Calculus/Deriv/Polynomial.lean", "Mathlib/Algebra/BigOperators/Finsupp.lean", "Mathlib/Algebra/MonoidAlgebra/ToDirectSum.lean", "Mathlib/Analysis/Calculus/FDeriv/Pi.lean", "Mathlib/Order/Hom/Lattice.lean", "Mathlib/Probability/Integration.lean", "Mathlib/NumberTheory/Rayleigh.lean", "Mathlib/Algebra/GCDMonoid/IntegrallyClosed.lean", "Mathlib/Order/Monotone/Basic.lean", "Mathlib/LinearAlgebra/QuadraticForm/Dual.lean", "Mathlib/FieldTheory/SeparableDegree.lean", "Mathlib/Order/ZornAtoms.lean", "Mathlib/MeasureTheory/OuterMeasure/Basic.lean", "Mathlib/Order/Heyting/Boundary.lean", "Mathlib/MeasureTheory/Measure/ProbabilityMeasure.lean", "Mathlib/Algebra/Group/ConjFinite.lean", "Mathlib/Probability/Martingale/Basic.lean", "Mathlib/Tactic/CasesM.lean", "Mathlib/Data/Finset/NoncommProd.lean", "Mathlib/MeasureTheory/Constructions/Cylinders.lean", "Mathlib/LinearAlgebra/Finsupp.lean", "Mathlib/CategoryTheory/Sites/Plus.lean", "Mathlib/Data/List/Perm.lean", "Mathlib/CategoryTheory/Preadditive/EndoFunctor.lean", "Mathlib/CategoryTheory/Limits/Shapes/Multiequalizer.lean", "Mathlib/GroupTheory/SpecificGroups/Dihedral.lean", "Mathlib/NumberTheory/LSeries/HurwitzZetaValues.lean", "Mathlib/Util/AtomM.lean", "Mathlib/Analysis/Complex/Liouville.lean", "Mathlib/Algebra/Category/Grp/Subobject.lean", "Mathlib/Combinatorics/Derangements/Exponential.lean", "Mathlib/Data/Finset/Lattice.lean", "Mathlib/SetTheory/Ordinal/Arithmetic.lean", "Mathlib/Algebra/Category/ModuleCat/Tannaka.lean", "Mathlib/CategoryTheory/Monoidal/Transport.lean", "Mathlib/Data/Nat/Hyperoperation.lean", "Mathlib/RingTheory/Localization/Away/AdjoinRoot.lean", "Mathlib/LinearAlgebra/Matrix/SesquilinearForm.lean", "Mathlib/Tactic/ProjectionNotation.lean", "Mathlib/GroupTheory/Perm/Cycle/Concrete.lean", "Mathlib/LinearAlgebra/Eigenspace/Zero.lean", "Mathlib/Dynamics/Ergodic/Ergodic.lean", "Mathlib/Algebra/Order/Nonneg/Ring.lean", "Mathlib/RingTheory/Polynomial/Cyclotomic/Expand.lean", "Mathlib/CategoryTheory/Limits/IsLimit.lean", "Mathlib/Topology/Algebra/Star.lean", "Mathlib/Geometry/Manifold/MFDeriv/FDeriv.lean", "Mathlib/Topology/ContinuousFunction/LocallyConstant.lean", "Mathlib/Util/WithWeakNamespace.lean", "Mathlib/Algebra/CharZero/Defs.lean", "Mathlib/LinearAlgebra/FreeAlgebra.lean", "Mathlib/CategoryTheory/Sigma/Basic.lean", "Mathlib/MeasureTheory/Integral/Lebesgue.lean", "Mathlib/Algebra/Module/Submodule/EqLocus.lean", "Mathlib/CategoryTheory/Limits/Preserves/Shapes/Terminal.lean", "Mathlib/SetTheory/Game/Short.lean", "Mathlib/Algebra/Module/Hom.lean", "Mathlib/Data/PFunctor/Multivariate/Basic.lean", "Mathlib/Analysis/InnerProductSpace/OfNorm.lean", "Mathlib/Algebra/Homology/ShortComplex/Limits.lean", "Mathlib/RingTheory/Perfection.lean", "Mathlib/CategoryTheory/Yoneda.lean", "Mathlib/Data/ZMod/IntUnitsPower.lean", "Mathlib/GroupTheory/Coxeter/Length.lean", "Mathlib/CategoryTheory/Limits/Connected.lean", "Mathlib/MeasureTheory/Function/LpSpace/DomAct/Basic.lean", "Mathlib/CategoryTheory/GradedObject/Unitor.lean", "Mathlib/Algebra/GroupWithZero/Semiconj.lean", "Mathlib/Algebra/Order/Floor/Div.lean", "Mathlib/NumberTheory/Padics/RingHoms.lean", "Mathlib/Data/HashMap.lean", "Mathlib/Dynamics/Newton.lean", ".lake/packages/lean4/src/lean/Init.lean", "Mathlib/Algebra/MonoidAlgebra/Basic.lean", "Mathlib/Data/ZMod/Algebra.lean", "Mathlib/Algebra/Module/Opposites.lean", "Mathlib/Topology/Instances/PNat.lean", "Mathlib/FieldTheory/Tower.lean", "Mathlib/Analysis/Calculus/Taylor.lean", "Mathlib/LinearAlgebra/CrossProduct.lean", "Mathlib/Topology/ShrinkingLemma.lean", "Mathlib/Probability/Independence/Basic.lean", "Mathlib/Data/Setoid/Partition.lean", "Mathlib/CategoryTheory/ConcreteCategory/ReflectsIso.lean", "Mathlib/Topology/Order/LeftRight.lean", "Mathlib/Tactic/NormNum/DivMod.lean", "Mathlib/Algebra/Group/ULift.lean", "Mathlib/MeasureTheory/Constructions/Polish.lean", "Mathlib/Topology/MetricSpace/Basic.lean", "Mathlib/Data/List/Prime.lean", "Mathlib/RingTheory/Valuation/ValuationRing.lean", "Mathlib/Algebra/Polynomial/Derivation.lean", "Mathlib/Tactic/Generalize.lean", "Mathlib/Algebra/Order/Floor/Prime.lean", "Mathlib/NumberTheory/ModularForms/Identities.lean", "Mathlib/CategoryTheory/Sums/Basic.lean", "Mathlib/Deprecated/Submonoid.lean", "Mathlib/NumberTheory/SmoothNumbers.lean", "Mathlib/RingTheory/FreeCommRing.lean", "Mathlib/Algebra/Order/GroupWithZero/Canonical.lean", "Mathlib/Algebra/Polynomial/Induction.lean", "Mathlib/Combinatorics/SimpleGraph/LapMatrix.lean", "Mathlib/CategoryTheory/Functor/Category.lean", "Mathlib/Data/DList/Defs.lean", "Mathlib/Tactic/Attr/Core.lean", "Mathlib/Topology/Metrizable/ContinuousMap.lean", "Mathlib/Algebra/Opposites.lean", "Mathlib/CategoryTheory/Products/Basic.lean", "Mathlib/Topology/MetricSpace/PiNat.lean", "Mathlib/CategoryTheory/Monoidal/FunctorCategory.lean", "Mathlib/Analysis/Normed/Group/Completeness.lean", "Mathlib/Algebra/Ring/WithZero.lean", "Mathlib/Data/Rat/Cast/CharZero.lean", "Mathlib/Order/Category/BddDistLat.lean", "Mathlib/Algebra/BigOperators/Group/List.lean", "Mathlib/Algebra/MvPolynomial/Expand.lean", "Mathlib/Algebra/Star/StarRingHom.lean", "Mathlib/Order/SuccPred/Limit.lean", "Mathlib/Data/Fin/Tuple/Reflection.lean", "Mathlib/Geometry/Manifold/ContMDiff/Product.lean", "Mathlib/Data/Finset/Pointwise.lean", "Mathlib/Algebra/Star/Rat.lean", "Mathlib/Data/NNReal/Basic.lean", "Mathlib/Init/ZeroOne.lean", "Mathlib/MeasureTheory/Measure/WithDensityVectorMeasure.lean", "Mathlib/Order/Antichain.lean", "Mathlib/Topology/Algebra/Module/Multilinear/Topology.lean", "Mathlib/CategoryTheory/Abelian/Images.lean", "Mathlib/CategoryTheory/Limits/Preserves/Basic.lean", "Mathlib/Logic/UnivLE.lean", "Mathlib/MeasureTheory/Integral/CircleIntegral.lean", "Mathlib/Algebra/Ring/Parity.lean", "Mathlib/CategoryTheory/Category/Init.lean", "Mathlib/FieldTheory/Fixed.lean", "Mathlib/Order/Filter/Pointwise.lean", "Mathlib/Algebra/Algebra/Subalgebra/Order.lean", "Mathlib/Algebra/ContinuedFractions/Computation/ApproximationCorollaries.lean", "Mathlib/CategoryTheory/Limits/EssentiallySmall.lean", "Mathlib/Data/List/Rotate.lean", "Mathlib/NumberTheory/KummerDedekind.lean", "Mathlib/Algebra/Order/Group/MinMax.lean", "Mathlib/Algebra/Order/Chebyshev.lean", "Mathlib/SetTheory/Ordinal/NaturalOps.lean", "Mathlib/CategoryTheory/Monoidal/Internal/Types.lean", "Mathlib/MeasureTheory/Measure/FiniteMeasureProd.lean", "Mathlib/Geometry/Euclidean/Triangle.lean", "Mathlib/LinearAlgebra/Matrix/ZPow.lean", "Mathlib/GroupTheory/Coxeter/Inversion.lean", "Mathlib/Data/QPF/Multivariate/Constructions/Fix.lean", "Mathlib/Tactic/Linarith.lean", "Mathlib/Order/Fin.lean", "Mathlib/Combinatorics/Quiver/Subquiver.lean", "Mathlib/Analysis/Fourier/FourierTransform.lean", "Mathlib/Data/Rat/Star.lean", "Mathlib/Topology/MetricSpace/Sequences.lean", "Mathlib/Algebra/Order/Group/DenselyOrdered.lean", "Mathlib/GroupTheory/Order/Min.lean", "Mathlib/NumberTheory/Cyclotomic/Three.lean", "Mathlib/Data/List/Palindrome.lean", "Mathlib/RingTheory/RingInvo.lean", "Mathlib/CategoryTheory/Limits/SmallComplete.lean", "Mathlib/Topology/Instances/Rat.lean", "Mathlib/CategoryTheory/Abelian/InjectiveResolution.lean", "Mathlib/Analysis/Calculus/BumpFunction/Basic.lean", "Mathlib/Data/FunLike/Basic.lean", "Mathlib/Init/Function.lean", "Mathlib/NumberTheory/Harmonic/Bounds.lean", "Mathlib/Topology/Algebra/Order/LiminfLimsup.lean", "Mathlib/Order/Filter/SmallSets.lean", "Mathlib/GroupTheory/GroupAction/Prod.lean", "Mathlib/CategoryTheory/Category/Bipointed.lean", "Mathlib/Data/Set/Countable.lean", "Mathlib/NumberTheory/LegendreSymbol/QuadraticChar/Basic.lean", "Mathlib/Analysis/InnerProductSpace/Dual.lean", "Mathlib/CategoryTheory/Galois/Examples.lean", "Mathlib/Topology/Algebra/Monoid.lean", "Mathlib/ModelTheory/ElementaryMaps.lean", "Mathlib/Topology/Algebra/GroupWithZero.lean", "Mathlib/Algebra/Homology/HomologySequence.lean", "Mathlib/Topology/MetricSpace/Pseudo/Lemmas.lean", "Mathlib/Probability/ProbabilityMassFunction/Integrals.lean", "Mathlib/Algebra/Polynomial/Eval.lean", "Mathlib/CategoryTheory/Localization/Resolution.lean", "Mathlib/Analysis/Analytic/Inverse.lean", "Mathlib/CategoryTheory/Types.lean", "Mathlib/Topology/Algebra/Order/Rolle.lean", "Mathlib/Data/Rbtree/DefaultLt.lean", "Mathlib/Combinatorics/Schnirelmann.lean", "Mathlib/RingTheory/MvPolynomial/Localization.lean", "Mathlib/Probability/ProbabilityMassFunction/Constructions.lean", "Mathlib/SetTheory/Ordinal/FixedPoint.lean", "Mathlib/Algebra/Polynomial/DenomsClearable.lean", "Mathlib/CategoryTheory/CatCommSq.lean", "Mathlib/Analysis/NormedSpace/OperatorNorm/Basic.lean", "Mathlib/CategoryTheory/Bicategory/Kan/Adjunction.lean", "Mathlib/Combinatorics/SetFamily/FourFunctions.lean", "Mathlib/RingTheory/PowerSeries/Trunc.lean", "Mathlib/Analysis/SpecialFunctions/Gamma/Deligne.lean", "Mathlib/Topology/GDelta.lean", "Mathlib/Tactic/FBinop.lean", "Mathlib/Topology/Category/TopCat/Limits/Products.lean", "Mathlib/Logic/Equiv/Fin.lean", "Mathlib/Data/Fintype/Quotient.lean", "Mathlib/AlgebraicTopology/DoldKan/Degeneracies.lean", "Mathlib/Analysis/BoxIntegral/Box/SubboxInduction.lean", "Mathlib/Algebra/Group/Defs.lean", "Mathlib/Data/Nat/Cast/Order.lean", "Mathlib/Algebra/Ring/Equiv.lean", "Mathlib/Dynamics/Minimal.lean", "Mathlib/Data/Set/MulAntidiagonal.lean", "Mathlib/GroupTheory/Congruence/BigOperators.lean", "Mathlib/CategoryTheory/Limits/Shapes/WidePullbacks.lean", "Mathlib/LinearAlgebra/BilinearMap.lean", "Mathlib/Algebra/Tropical/Basic.lean", "Mathlib/NumberTheory/LSeries/Convolution.lean", "Mathlib/NumberTheory/ModularForms/SlashActions.lean", "Mathlib/Analysis/Normed/Group/Int.lean", "Mathlib/Data/Set/Finite.lean", "Mathlib/Order/Cover.lean", "Mathlib/Analysis/SpecialFunctions/Trigonometric/Complex.lean", "Mathlib/Order/Category/NonemptyFinLinOrd.lean", "Mathlib/Analysis/Convex/Extreme.lean", "Mathlib/Algebra/Order/Group/Indicator.lean", "Mathlib/Algebra/CharP/CharAndCard.lean", "Mathlib/Analysis/Convex/Star.lean", "Mathlib/Algebra/GroupPower/IterateHom.lean", "Mathlib/CategoryTheory/FiberedCategory/BasedCategory.lean", "Mathlib/Data/W/Cardinal.lean", "Mathlib/Data/W/Basic.lean", "Mathlib/Algebra/Star/SelfAdjoint.lean", "Mathlib/Data/BitVec.lean", "Mathlib/Topology/UniformSpace/CompleteSeparated.lean", "Mathlib/GroupTheory/GroupAction/Group.lean", "Mathlib/MeasureTheory/Function/LpSeminorm/CompareExp.lean", "Mathlib/FieldTheory/Perfect.lean", "Mathlib/Analysis/MellinInversion.lean", "Mathlib/Algebra/Lie/Normalizer.lean", "Mathlib/Analysis/Convex/AmpleSet.lean", "Mathlib/FieldTheory/IsAlgClosed/Classification.lean", "Mathlib/Topology/Sheaves/Sheafify.lean", "Mathlib/Order/Copy.lean", "Mathlib/LinearAlgebra/Matrix/IsDiag.lean", "Mathlib/Algebra/Module/LinearMap/Defs.lean", "Mathlib/RingTheory/Ideal/AssociatedPrime.lean", "Mathlib/Analysis/SpecialFunctions/Complex/Circle.lean", "Mathlib/Data/Real/Irrational.lean", "Mathlib/Topology/Algebra/Module/Simple.lean", "Mathlib/Algebra/Group/Embedding.lean", "Mathlib/Data/Nat/MaxPowDiv.lean", "Mathlib/Tactic/Monotonicity/Basic.lean", "Mathlib/LinearAlgebra/Alternating/Basic.lean", "Mathlib/Topology/Category/LightProfinite/EffectiveEpi.lean", "Mathlib/CategoryTheory/NatTrans.lean", "Mathlib/Data/Set/Functor.lean", "Mathlib/MeasureTheory/Function/StronglyMeasurable/Basic.lean", "Mathlib/Topology/Algebra/GroupCompletion.lean", "Mathlib/Data/Finset/Sort.lean", "Mathlib/Data/Prod/TProd.lean", "Mathlib/LinearAlgebra/Lagrange.lean", "Mathlib/LinearAlgebra/Alternating/DomCoprod.lean", "Mathlib/Order/Category/Preord.lean", "Mathlib/Data/PSigma/Order.lean", "Mathlib/RingTheory/Valuation/PrimeMultiplicity.lean", "Mathlib/Probability/Moments.lean", "Mathlib/Topology/NhdsSet.lean", "Mathlib/Topology/UniformSpace/UniformEmbedding.lean", "Mathlib/Data/SetLike/Fintype.lean", "Mathlib/RingTheory/Jacobson.lean", "Mathlib/Tactic/FunProp/Attr.lean", "Mathlib/Algebra/DirectSum/Basic.lean", "Mathlib/Util/WhatsNew.lean", "Mathlib/RepresentationTheory/Invariants.lean", "Mathlib/Data/Set/Equitable.lean", "Mathlib/Topology/MetricSpace/Bounded.lean", "Mathlib/NumberTheory/FLT/Four.lean", "Mathlib/CategoryTheory/Subobject/Limits.lean", "Mathlib/Data/Rbtree/Main.lean", "Mathlib/LinearAlgebra/QuadraticForm/TensorProduct/Isometries.lean", "Mathlib/RingTheory/HahnSeries/Multiplication.lean", "Mathlib/NumberTheory/ModularForms/JacobiTheta/OneVariable.lean", "Mathlib/Algebra/Category/Grp/Adjunctions.lean", "Mathlib/Data/Matroid/IndepAxioms.lean", "Mathlib/Combinatorics/Additive/PluenneckeRuzsa.lean", "Mathlib/Data/List/Nodup.lean", "Mathlib/Data/ENat/Lattice.lean", "Mathlib/GroupTheory/GroupAction/DomAct/ActionHom.lean", "Mathlib/GroupTheory/PresentedGroup.lean", "Mathlib/NumberTheory/NumberField/Discriminant.lean", "Mathlib/Tactic/Recall.lean", "Mathlib/Data/Nat/Nth.lean", "Mathlib/Topology/Defs/Induced.lean", "Mathlib/Algebra/Group/Submonoid/Pointwise.lean", "Mathlib/Tactic/DeprecateMe.lean", "Mathlib/Analysis/Complex/Isometry.lean", "Mathlib/NumberTheory/NumberField/Units/Regulator.lean", "Mathlib/Data/Fin/Tuple/BubbleSortInduction.lean", "Mathlib/Topology/Algebra/WithZeroTopology.lean", "Mathlib/CategoryTheory/Limits/ConcreteCategory.lean", "Mathlib/Data/Real/Sign.lean", "Mathlib/Algebra/Ring/Semiconj.lean", "Mathlib/Algebra/Ring/Action/Invariant.lean", "Mathlib/Init/Data/Option/Init/Lemmas.lean", "Mathlib/Algebra/Lie/Abelian.lean", "Mathlib/CategoryTheory/Localization/HasLocalization.lean", "Mathlib/Algebra/Group/UniqueProds.lean", "Mathlib/Analysis/LocallyConvex/ContinuousOfBounded.lean", "Mathlib/Order/SupClosed.lean", "Mathlib/Logic/Function/Iterate.lean", "Mathlib/Tactic/SplitIfs.lean", "Mathlib/Topology/Algebra/Polynomial.lean", "Mathlib/Topology/Order/Category/FrameAdjunction.lean", "Mathlib/Topology/Separation.lean", "Mathlib/Topology/MetricSpace/Perfect.lean", "Mathlib/Topology/Sheaves/PresheafOfFunctions.lean", "Mathlib/Topology/Algebra/MulAction.lean", "Mathlib/CategoryTheory/Monoidal/Cartesian/Comon_.lean", "Mathlib/Order/Estimator.lean", "Mathlib/Geometry/Manifold/MFDeriv/Atlas.lean", "Mathlib/RingTheory/Polynomial/Nilpotent.lean", "Mathlib/AlgebraicTopology/DoldKan/EquivalenceAdditive.lean", "Mathlib/Topology/UniformSpace/Basic.lean", "Mathlib/Analysis/Calculus/FDeriv/Equiv.lean", "Mathlib/Probability/Process/Stopping.lean", "Mathlib/LinearAlgebra/Matrix/GeneralLinearGroup.lean", "Mathlib/Analysis/SpecialFunctions/Trigonometric/EulerSineProd.lean", "Mathlib/Tactic/FunProp/AEMeasurable.lean", "Mathlib/RingTheory/QuotSMulTop.lean", "Mathlib/Topology/Algebra/Algebra.lean", "Mathlib/Data/Sigma/Order.lean", "Mathlib/Algebra/Homology/ShortComplex/ShortExact.lean", "Mathlib/Analysis/NormedSpace/Int.lean", "Mathlib/Control/Bitraversable/Instances.lean", "Mathlib/Data/Finite/Defs.lean", "Mathlib/Analysis/Convex/Cone/Pointed.lean", "Mathlib/Condensed/Light/Functors.lean", "Mathlib/Condensed/Functors.lean", "Mathlib/Data/Finmap.lean", "Mathlib/LinearAlgebra/CliffordAlgebra/Contraction.lean", "Mathlib/Data/Complex/Exponential.lean", "Mathlib/Algebra/Polynomial/Cardinal.lean", "Mathlib/LinearAlgebra/Matrix/Determinant/Misc.lean", "Mathlib/CategoryTheory/Limits/Preserves/Shapes/Biproducts.lean", "Mathlib/CategoryTheory/Limits/Elements.lean", "Mathlib/CategoryTheory/Opposites.lean", "Mathlib/RepresentationTheory/GroupCohomology/LowDegree.lean", "Mathlib/Analysis/FunctionalSpaces/SobolevInequality.lean", "Mathlib/Lean/Elab/Tactic/Basic.lean", "Mathlib/GroupTheory/DoubleCoset.lean", "Mathlib/Order/ConditionallyCompleteLattice/Finset.lean", "Mathlib/CategoryTheory/Limits/Shapes/Equalizers.lean", "Mathlib/LinearAlgebra/Matrix/ProjectiveSpecialLinearGroup.lean", "Mathlib/SetTheory/Ordinal/Topology.lean", "Mathlib/Algebra/Ring/Subsemiring/Order.lean", "Mathlib/Data/Nat/Cast/NeZero.lean", "Mathlib/Algebra/Order/Group/OrderIso.lean", "Mathlib/CategoryTheory/Idempotents/HomologicalComplex.lean", "Mathlib/CategoryTheory/Category/Factorisation.lean", "Mathlib/Condensed/Solid.lean", "Mathlib/Topology/Sheaves/SheafCondition/UniqueGluing.lean", "Mathlib/NumberTheory/Zsqrtd/ToReal.lean", "Mathlib/Analysis/Calculus/LagrangeMultipliers.lean", "Mathlib/CategoryTheory/Limits/Preserves/Shapes/Products.lean", "Mathlib/Data/List/FinRange.lean", "Mathlib/RingTheory/Coalgebra/Equiv.lean", "Mathlib/Algebra/Homology/ShortComplex/Linear.lean", "Mathlib/LinearAlgebra/TensorProduct/RightExactness.lean", "Mathlib/RingTheory/Localization/Submodule.lean", "Mathlib/Algebra/Category/ModuleCat/Products.lean", "Mathlib/Topology/Algebra/StarSubalgebra.lean", "Mathlib/Algebra/MvPolynomial/Degrees.lean", "Mathlib/Topology/Connected/TotallyDisconnected.lean", "Mathlib/Data/Vector/Zip.lean", "Mathlib/GroupTheory/GroupAction/Pointwise.lean", "Mathlib/Data/Nat/Bits.lean", "Mathlib/CategoryTheory/Localization/DerivabilityStructure/Basic.lean", "Mathlib/Combinatorics/Additive/FreimanHom.lean", "Mathlib/NumberTheory/Dioph.lean", "Mathlib/LinearAlgebra/Matrix/Gershgorin.lean", "Mathlib/Topology/MetricSpace/ThickenedIndicator.lean", "Mathlib/Topology/Category/Profinite/AsLimit.lean", "Mathlib/Order/Circular.lean", "Mathlib/RingTheory/MvPowerSeries/Basic.lean", "Mathlib/Analysis/Convex/Join.lean", "Mathlib/Data/List/NodupEquivFin.lean", "Mathlib/GroupTheory/Perm/ClosureSwap.lean", "Mathlib/Data/PFunctor/Univariate/M.lean", "Mathlib/Analysis/Asymptotics/Theta.lean", "Mathlib/Algebra/Category/Grp/Biproducts.lean", "Mathlib/MeasureTheory/Constructions/BorelSpace/Real.lean", "Mathlib/Algebra/Category/Grp/FilteredColimits.lean", "Mathlib/NumberTheory/ModularForms/EisensteinSeries/MDifferentiable.lean", "Mathlib/CategoryTheory/Monoidal/Free/Basic.lean", "Mathlib/Data/Rbtree/Init.lean", "Mathlib/Data/Fin/Fin2.lean", "Mathlib/Data/NNRat/BigOperators.lean", "Mathlib/CategoryTheory/Limits/Shapes/ConcreteCategory.lean", "Mathlib/LinearAlgebra/FreeModule/IdealQuotient.lean", "Mathlib/Analysis/SumIntegralComparisons.lean", "Mathlib/GroupTheory/GroupAction/Quotient.lean", "Mathlib/Order/Filter/Germ.lean", "Mathlib/Order/SuccPred/CompleteLinearOrder.lean", "Mathlib/Tactic/GuardHypNums.lean", "Mathlib/LinearAlgebra/Projectivization/Basic.lean", "Mathlib/Tactic/InferParam.lean", "Mathlib/Data/Countable/Defs.lean", "Mathlib/SetTheory/Cardinal/SchroederBernstein.lean", "Mathlib/CategoryTheory/Monoidal/Bimon_.lean", "Mathlib/MeasureTheory/Function/ConditionalExpectation/AEMeasurable.lean", "Mathlib/Algebra/Category/GrpWithZero.lean", "Mathlib/Analysis/InnerProductSpace/ConformalLinearMap.lean", "Mathlib/Topology/Algebra/Module/LinearPMap.lean", "Mathlib/Analysis/Normed/Group/Uniform.lean", "Mathlib/Tactic/Rify.lean", "Mathlib/MeasureTheory/Measure/Sub.lean", "Mathlib/Data/Fintype/Shrink.lean", "Mathlib/RepresentationTheory/GroupCohomology/Hilbert90.lean", "Mathlib/LinearAlgebra/PerfectPairing.lean", "Mathlib/Order/Interval/Set/ProjIcc.lean", "Mathlib/CategoryTheory/Adjunction/Mates.lean", "Mathlib/LinearAlgebra/AffineSpace/FiniteDimensional.lean", "Mathlib/CategoryTheory/Sites/OneHypercover.lean", "Mathlib/Analysis/Convex/PartitionOfUnity.lean", "Mathlib/RingTheory/Valuation/ExtendToLocalization.lean", "Mathlib/Combinatorics/SimpleGraph/Regularity/Lemma.lean", "Mathlib/Algebra/Order/Group/Abs.lean", "Mathlib/Algebra/BigOperators/Associated.lean", "Mathlib/CategoryTheory/Category/GaloisConnection.lean", "Mathlib/CategoryTheory/Monoidal/Types/Symmetric.lean", "Mathlib/Analysis/Calculus/Deriv/ZPow.lean", "Mathlib/Algebra/Category/Grp/Limits.lean", "Mathlib/Data/Int/SuccPred.lean", "Mathlib/Data/List/Zip.lean", "Mathlib/NumberTheory/LucasLehmer.lean", "Mathlib/MeasureTheory/Group/FundamentalDomain.lean", "Mathlib/RingTheory/MatrixAlgebra.lean", "Mathlib/Lean/PrettyPrinter/Delaborator.lean", "Mathlib/LinearAlgebra/Projectivization/Subspace.lean", "Mathlib/Algebra/Homology/Exact.lean", "Mathlib/Data/Ordmap/Ordset.lean", "Mathlib/Algebra/CharZero/Infinite.lean", "Mathlib/Data/Set/Pairwise/Lattice.lean", "Mathlib/LinearAlgebra/Pi.lean", "Mathlib/Data/Complex/Basic.lean", "Mathlib/NumberTheory/Cyclotomic/Rat.lean", "Mathlib/Combinatorics/Additive/AP/Three/Behrend.lean", "Mathlib/NumberTheory/LegendreSymbol/QuadraticChar/GaussSum.lean", "Mathlib/Data/Matrix/DMatrix.lean", "Mathlib/LinearAlgebra/Projectivization/Independence.lean", "Mathlib/GroupTheory/Solvable.lean", "Mathlib/Logic/Nonempty.lean", "Mathlib/LinearAlgebra/AffineSpace/ContinuousAffineEquiv.lean", "Mathlib/Analysis/SpecificLimits/FloorPow.lean", "Mathlib/Data/Char.lean", "Mathlib/MeasureTheory/Function/SimpleFuncDenseLp.lean", "Mathlib/Data/Finsupp/Notation.lean", "Mathlib/Analysis/Complex/UpperHalfPlane/FunctionsBoundedAtInfty.lean", "Mathlib/CategoryTheory/Subobject/Comma.lean", "Mathlib/Topology/StoneCech.lean", "Mathlib/Combinatorics/SimpleGraph/Regularity/Chunk.lean", "Mathlib/Analysis/LocallyConvex/Bounded.lean", "Mathlib/Order/Filter/Curry.lean", "Mathlib/Algebra/Category/ModuleCat/Sheaf/ChangeOfRings.lean", "Mathlib/Analysis/SpecialFunctions/Pow/Real.lean", "Mathlib/Algebra/Lie/BaseChange.lean", "Mathlib/CategoryTheory/Shift/Basic.lean", "Mathlib/SetTheory/ZFC/Basic.lean", "Mathlib/Algebra/Polynomial/Mirror.lean", "Mathlib/Tactic/Nontriviality.lean", "Mathlib/Topology/Algebra/Order/Archimedean.lean", "Mathlib/CategoryTheory/EffectiveEpi/Enough.lean", "Mathlib/LinearAlgebra/Eigenspace/Semisimple.lean", "Mathlib/FieldTheory/NormalClosure.lean", "Mathlib/Algebra/Module/ULift.lean", "Mathlib/Analysis/Calculus/DiffContOnCl.lean", "Mathlib/NumberTheory/ClassNumber/FunctionField.lean", "Mathlib/Tactic/Common.lean", "Mathlib/LinearAlgebra/SymplecticGroup.lean", "Mathlib/Topology/DenseEmbedding.lean", "Mathlib/Data/ENat/Basic.lean", "Mathlib/Data/Set/Lattice.lean", "Mathlib/NumberTheory/FLT/Three.lean", "Mathlib/Analysis/Complex/Hadamard.lean", "Mathlib/Analysis/Complex/OperatorNorm.lean", "Mathlib/Data/Bool/Basic.lean", "Mathlib/RingTheory/Polynomial/Tower.lean", "Mathlib/Data/QPF/Multivariate/Constructions/Sigma.lean", "Mathlib/MeasureTheory/Measure/Haar/InnerProductSpace.lean", "Mathlib/Probability/CondCount.lean", "Mathlib/Topology/Category/Stonean/Adjunctions.lean", "Mathlib/MeasureTheory/Constructions/Pi.lean", "Mathlib/Topology/MetricSpace/Holder.lean", "Mathlib/Algebra/DualQuaternion.lean", "Mathlib/CategoryTheory/Limits/ExactFunctor.lean", "Mathlib/Topology/Algebra/Semigroup.lean", "Mathlib/RingTheory/Localization/LocalizationLocalization.lean", "Mathlib/Tactic/ApplyFun.lean", "Mathlib/Order/Partition/Finpartition.lean", "Mathlib/Order/Partition/Equipartition.lean", "Mathlib/LinearAlgebra/CliffordAlgebra/Conjugation.lean", "Mathlib/Order/Interval/Set/SurjOn.lean", "Mathlib/RingTheory/MvPolynomial/WeightedHomogeneous.lean", "Mathlib/Topology/Order/UpperLowerSetTopology.lean", "Mathlib/Data/List/AList.lean", "Mathlib/Algebra/Algebra/Subalgebra/MulOpposite.lean", "Mathlib/Analysis/NormedSpace/HahnBanach/Extension.lean", "Mathlib/CategoryTheory/Abelian/RightDerived.lean", "Mathlib/Data/Fin/VecNotation.lean", "Mathlib/Data/Vector/Snoc.lean", "Mathlib/Deprecated/Subring.lean", "Mathlib/Lean/LocalContext.lean", "Mathlib/Algebra/Order/Module/Pointwise.lean", "Mathlib/CategoryTheory/Groupoid/FreeGroupoid.lean", "Mathlib/Control/Traversable/Equiv.lean", "Mathlib/RingTheory/RootsOfUnity/Minpoly.lean", "Mathlib/CategoryTheory/Limits/Presheaf.lean", "Mathlib/SetTheory/Cardinal/CountableCover.lean", "Mathlib/CategoryTheory/Abelian/EpiWithInjectiveKernel.lean", "Mathlib/CategoryTheory/Balanced.lean", "Mathlib/Geometry/Euclidean/Angle/Sphere.lean", "Mathlib/Algebra/BigOperators/Ring/List.lean", "Mathlib/MeasureTheory/Measure/AEDisjoint.lean", "Mathlib/MeasureTheory/OuterMeasure/Defs.lean", "Mathlib/Probability/Cdf.lean", "Mathlib/Combinatorics/SimpleGraph/Finite.lean", "Mathlib/MeasureTheory/Measure/Lebesgue/EqHaar.lean", "Mathlib/Topology/Covering.lean", "Mathlib/Algebra/Order/UpperLower.lean", "Mathlib/Algebra/Order/Hom/Basic.lean", "Mathlib/Topology/Metrizable/Uniformity.lean", "Mathlib/Dynamics/BirkhoffSum/Basic.lean", "Mathlib/MeasureTheory/Integral/Pi.lean", "Mathlib/SetTheory/Cardinal/Cofinality.lean", "Mathlib/Algebra/Ring/Subring/MulOpposite.lean", "Mathlib/CategoryTheory/Limits/Shapes/NormalMono/Basic.lean", "Mathlib/Combinatorics/SimpleGraph/Operations.lean", "Mathlib/Algebra/Order/Module/OrderedSMul.lean", "Mathlib/FieldTheory/IsSepClosed.lean", "Mathlib/CategoryTheory/Limits/Shapes/Types.lean", "Mathlib/MeasureTheory/MeasurableSpace/CountablyGenerated.lean", "Mathlib/Algebra/Polynomial/Identities.lean", "Mathlib/LinearAlgebra/Matrix/Charpoly/Minpoly.lean", "Mathlib/RingTheory/AdicCompletion/Exactness.lean", "Mathlib/Algebra/Module/Submodule/IterateMapComap.lean", "Mathlib/Probability/Kernel/MeasurableIntegral.lean", "Mathlib/RingTheory/Valuation/Quotient.lean", "Mathlib/Tactic/Monotonicity/Attr.lean", "Mathlib/Topology/UnitInterval.lean", "Mathlib/Algebra/Homology/HomotopyCategory.lean", "Mathlib/CategoryTheory/Linear/Yoneda.lean", "Mathlib/AlgebraicTopology/MooreComplex.lean", "Mathlib/Data/MLList/BestFirst.lean", "Mathlib/CategoryTheory/Limits/Preserves/Shapes/Kernels.lean", "Mathlib/Algebra/Group/Subgroup/MulOpposite.lean", "Mathlib/Data/Setoid/Basic.lean", "Mathlib/Topology/Algebra/ContinuousMonoidHom.lean", "Mathlib/Algebra/Order/Field/InjSurj.lean", "Mathlib/NumberTheory/LSeries/Convergence.lean", "Mathlib/MeasureTheory/Decomposition/RadonNikodym.lean", "Mathlib/CategoryTheory/Idempotents/Biproducts.lean", "Mathlib/Algebra/Star/BigOperators.lean", "Mathlib/LinearAlgebra/Projection.lean", "Mathlib/MeasureTheory/Covering/VitaliFamily.lean", "Mathlib/LinearAlgebra/Eigenspace/Triangularizable.lean", "Mathlib/Data/DFinsupp/Lex.lean", "Mathlib/CategoryTheory/UnivLE.lean", "Mathlib/Data/Nat/SuccPred.lean", "Mathlib/Tactic/NormNum/Inv.lean", "Mathlib/Data/Real/EReal.lean", "Mathlib/FieldTheory/Finite/GaloisField.lean", "Mathlib/Tactic/CongrM.lean", "Mathlib/Logic/Function/FromTypes.lean", "Mathlib/Algebra/Homology/ShortComplex/Exact.lean", "Mathlib/Control/LawfulFix.lean", "Mathlib/Algebra/Algebra/Subalgebra/Unitization.lean", "Mathlib/CategoryTheory/GlueData.lean", "Mathlib/Algebra/Order/Group/Int.lean", "Mathlib/CategoryTheory/ConcreteCategory/Bundled.lean", "Mathlib/Data/Finset/Basic.lean", "Mathlib/Logic/Embedding/Basic.lean", "Mathlib/Algebra/Ring/Pi.lean", "Mathlib/RingTheory/Coalgebra/Hom.lean", "Mathlib/Analysis/NormedSpace/ProdLp.lean", "Mathlib/Analysis/Convex/Slope.lean", "Mathlib/RingTheory/Regular/IsSMulRegular.lean", "Mathlib/RingTheory/Valuation/ValuationSubring.lean", "Mathlib/MeasureTheory/Integral/FundThmCalculus.lean", "Mathlib/MeasureTheory/Constructions/BorelSpace/Order.lean", "Mathlib/MeasureTheory/Function/EssSup.lean", "Mathlib/Control/EquivFunctor/Instances.lean", "Mathlib/Probability/Kernel/Composition.lean", "Mathlib/Data/List/Dedup.lean", "Mathlib/Probability/Kernel/Basic.lean", "Mathlib/Algebra/Group/Subgroup/Basic.lean", "Mathlib/MeasureTheory/Measure/Haar/Unique.lean", "Mathlib/Data/Rat/Encodable.lean", "Mathlib/RingTheory/LocalProperties.lean", "Mathlib/MeasureTheory/Constructions/Projective.lean", "Mathlib/Util/Qq.lean", "Mathlib/Data/Seq/WSeq.lean", "Mathlib/Order/KrullDimension.lean", "Mathlib/Tactic/Measurability/Init.lean", "Mathlib/RingTheory/PowerSeries/Inverse.lean", "Mathlib/Tactic/GCongr/ForwardAttr.lean", "Mathlib/SetTheory/Ordinal/Principal.lean", "Mathlib/CategoryTheory/Monoidal/CoherenceLemmas.lean", "Mathlib/Data/Fin/FlagRange.lean", "Mathlib/LinearAlgebra/GeneralLinearGroup.lean", "Mathlib/Data/Real/Pointwise.lean", "Mathlib/Order/PropInstances.lean", "Mathlib/Analysis/SpecialFunctions/Complex/Arg.lean", "Mathlib/RingTheory/FractionalIdeal/Basic.lean", "Mathlib/CategoryTheory/Monoidal/End.lean", "Mathlib/Algebra/ContinuedFractions/Computation/Basic.lean", "Mathlib/CategoryTheory/Limits/Shapes/FunctorToTypes.lean", "Mathlib/Probability/Kernel/Disintegration/Basic.lean", "Mathlib/Algebra/CharP/IntermediateField.lean", "Mathlib/Analysis/Complex/TaylorSeries.lean", "Mathlib/CategoryTheory/Limits/FintypeCat.lean", "Mathlib/MeasureTheory/Decomposition/UnsignedHahn.lean", "Mathlib/Init/Data/Ordering/Lemmas.lean", "Mathlib/RingTheory/Algebraic.lean", "Mathlib/Algebra/GroupWithZero/Defs.lean", "Mathlib/CategoryTheory/Core.lean", "Mathlib/Algebra/Polynomial/Degree/Definitions.lean", "Mathlib/CategoryTheory/GuitartExact/VerticalComposition.lean", "Mathlib/RingTheory/MvPolynomial/Homogeneous.lean", "Mathlib/Analysis/Complex/Basic.lean", "Mathlib/Tactic/Substs.lean", "Mathlib/Algebra/Group/Nat.lean", "Mathlib/CategoryTheory/Sites/Sheaf.lean", "Mathlib/Tactic/Replace.lean", "Mathlib/Algebra/Category/ModuleCat/Injective.lean", "Mathlib/Data/Finset/MulAntidiagonal.lean", "Mathlib/Algebra/MvPolynomial/Monad.lean", "Mathlib/LinearAlgebra/Trace.lean", "Mathlib/Data/Matrix/Basis.lean", "Mathlib/Probability/Martingale/Upcrossing.lean", "Mathlib/Combinatorics/SimpleGraph/Regularity/Energy.lean", "Mathlib/FieldTheory/AbelRuffini.lean", "Mathlib/CategoryTheory/Monoidal/Category.lean", "Mathlib/Data/Finite/Card.lean", "Mathlib/Order/ConditionallyCompleteLattice/Group.lean", "Mathlib/SetTheory/Game/Basic.lean", "Mathlib/Algebra/Group/Hom/CompTypeclasses.lean", "Mathlib/CategoryTheory/Sites/EpiMono.lean", "Mathlib/GroupTheory/FreeGroup/IsFreeGroup.lean", "Mathlib/Algebra/Category/ModuleCat/Sheaf/Abelian.lean", "Mathlib/Algebra/Divisibility/Prod.lean", "Mathlib/Algebra/Order/Monoid/Unbundled/Pow.lean", "Mathlib/NumberTheory/FLT/Basic.lean", "Mathlib/Probability/Process/HittingTime.lean", "Mathlib/Tactic/Coe.lean", "Mathlib/Data/PNat/Interval.lean", "Mathlib/GroupTheory/GroupAction/Option.lean", "Mathlib/Algebra/BigOperators/Finprod.lean", "Mathlib/LinearAlgebra/BilinearForm/Basic.lean", "Mathlib/Algebra/Ring/Regular.lean", "Mathlib/Algebra/Homology/ShortComplex/SnakeLemma.lean", "Mathlib/Combinatorics/Additive/Corner/Roth.lean", "Mathlib/NumberTheory/Padics/PadicNorm.lean", "Mathlib/Analysis/SpecialFunctions/NonIntegrable.lean", "Mathlib/NumberTheory/Harmonic/EulerMascheroni.lean", "Mathlib/RingTheory/HahnSeries/Basic.lean", "Mathlib/SetTheory/Ordinal/Notation.lean", "Mathlib/Analysis/Seminorm.lean", "Mathlib/Order/SuccPred/Relation.lean", "Mathlib/Data/Matrix/Kronecker.lean", "Mathlib/Init/Algebra/Classes.lean", "Mathlib/Analysis/Normed/Group/AddTorsor.lean", "Mathlib/CategoryTheory/Limits/Preserves/Shapes/Images.lean", "Mathlib/Probability/Distributions/Geometric.lean", "Mathlib/Order/OmegaCompletePartialOrder.lean", "Mathlib/Tactic/Polyrith.lean", "Mathlib/LinearAlgebra/FiniteDimensional.lean", "Mathlib/NumberTheory/LegendreSymbol/AddCharacter.lean", "Mathlib/Data/Nat/Choose/Bounds.lean", "Mathlib/CategoryTheory/Abelian/ProjectiveResolution.lean", "Mathlib/MeasureTheory/Function/AEEqFun/DomAct.lean", "Mathlib/Tactic/NormNum/Core.lean", "Mathlib/Data/NNReal/Star.lean", "Mathlib/RingTheory/WittVector/Basic.lean", "Mathlib/Analysis/Complex/RemovableSingularity.lean", "Mathlib/Data/Finset/Finsupp.lean", "Mathlib/Data/Multiset/Dedup.lean", "Mathlib/Data/Int/CharZero.lean", "Mathlib/Algebra/MonoidAlgebra/Support.lean", "Mathlib/Data/List/Join.lean", "Mathlib/NumberTheory/LSeries/MellinEqDirichlet.lean", "Mathlib/MeasureTheory/SetSemiring.lean", "Mathlib/GroupTheory/SchurZassenhaus.lean", "Mathlib/FieldTheory/RatFunc/AsPolynomial.lean", "Mathlib/Analysis/NormedSpace/ENorm.lean", "Mathlib/Topology/Order/Priestley.lean", "Mathlib/Order/Iterate.lean", "Mathlib/CategoryTheory/Shift/Predicate.lean", "Mathlib/RingTheory/IntegrallyClosed.lean", "Mathlib/Algebra/Group/Submonoid/Operations.lean", "Mathlib/Topology/Algebra/FilterBasis.lean", "Mathlib/Order/Interval/Set/OrdConnectedComponent.lean", "Mathlib/Topology/MetricSpace/Cauchy.lean", "Mathlib/CategoryTheory/Bicategory/Strict.lean", "Mathlib/Data/PNat/Xgcd.lean", "Mathlib/Algebra/DirectSum/Internal.lean", "Mathlib/Data/Nat/Squarefree.lean", "Mathlib/Dynamics/Ergodic/Conservative.lean", "Mathlib/Geometry/RingedSpace/OpenImmersion.lean", "Mathlib/RingTheory/Adjoin/Field.lean", "Mathlib/Algebra/Lie/TraceForm.lean", "Mathlib/Data/PNat/Defs.lean", "Mathlib/Init/Data/Nat/Notation.lean", "Mathlib/MeasureTheory/Covering/Besicovitch.lean", "Mathlib/RingTheory/Unramified/Derivations.lean", "Mathlib/MeasureTheory/Function/LpSpace.lean", "Mathlib/Tactic/FunProp/Theorems.lean", "Mathlib/Algebra/Order/Field/Power.lean", "Mathlib/Data/Multiset/Functor.lean", "Mathlib/Topology/Category/Compactum.lean", "Mathlib/Topology/List.lean", "Mathlib/Topology/Algebra/Module/WeakDual.lean", "Mathlib/Algebra/Group/Equiv/TypeTags.lean", "Mathlib/Algebra/Homology/ExactSequence.lean", "Mathlib/Algebra/Polynomial/Module/AEval.lean", "Mathlib/MeasureTheory/Integral/DominatedConvergence.lean", "Mathlib/Data/List/Lemmas.lean", "Mathlib/Data/Finsupp/AList.lean", "Mathlib/Analysis/Calculus/BumpFunction/Convolution.lean", "Mathlib/Algebra/Order/Pi.lean", "Mathlib/CategoryTheory/Abelian/Generator.lean", "Mathlib/Data/PNat/Prime.lean", "Mathlib/Algebra/Category/Grp/Preadditive.lean", "Mathlib/Logic/Unique.lean", "Mathlib/Data/Set/Notation.lean", "Mathlib/Tactic/Positivity/Core.lean", "Mathlib/Analysis/Fourier/AddCircle.lean", "Mathlib/Data/Multiset/Sum.lean", "Mathlib/Algebra/Group/Hom/Defs.lean", "Mathlib/Analysis/SpecialFunctions/Stirling.lean", "Mathlib/Topology/UniformSpace/Completion.lean", "Mathlib/Geometry/Manifold/Algebra/LeftInvariantDerivation.lean", "Mathlib/GroupTheory/GroupAction/Sigma.lean", "Mathlib/Analysis/Normed/Group/ZeroAtInfty.lean", "Mathlib/Analysis/NormedSpace/Star/Basic.lean", "Mathlib/Data/ZMod/Quotient.lean", "Mathlib/Order/Monotone/Odd.lean", "Mathlib/CategoryTheory/Monoidal/OfChosenFiniteProducts/Symmetric.lean", "Mathlib/Lean/Thunk.lean", "Mathlib/Data/Finset/Grade.lean", "Mathlib/RingTheory/PowerSeries/Derivative.lean", "Mathlib/Geometry/Manifold/BumpFunction.lean", "Mathlib/Algebra/Category/ModuleCat/Differentials/Presheaf.lean", "Mathlib/Lean/Meta/Basic.lean", "Mathlib/Order/Radical.lean", "Mathlib/Tactic/GuardGoalNums.lean", "Mathlib/Analysis/SpecialFunctions/Complex/LogDeriv.lean", "Mathlib/NumberTheory/LSeries/Dirichlet.lean", "Mathlib/Data/Sum/Lattice.lean", "Mathlib/Data/Matroid/Map.lean", "Mathlib/CategoryTheory/Limits/Constructions/Filtered.lean", "Mathlib/Order/Category/BoolAlg.lean", "Mathlib/Algebra/Order/Group/Units.lean", "Mathlib/Data/Finset/Powerset.lean", "Mathlib/Analysis/NormedSpace/Star/GelfandDuality.lean", "Mathlib/Computability/DFA.lean", "Mathlib/AlgebraicTopology/FundamentalGroupoid/InducedMaps.lean", "Mathlib/CategoryTheory/Limits/Over.lean", "Mathlib/AlgebraicTopology/SimplicialObject.lean", "Mathlib/Analysis/NormedSpace/OperatorNorm/Asymptotics.lean", "Mathlib/Analysis/Convex/Uniform.lean", "Mathlib/CategoryTheory/Sites/Coherent/LocallySurjective.lean", "Mathlib/FieldTheory/AbsoluteGaloisGroup.lean", "Mathlib/Algebra/Order/CauSeq/BigOperators.lean", "Mathlib/LinearAlgebra/TensorProduct/Submodule.lean", "Mathlib/Algebra/Category/ModuleCat/Monoidal/Closed.lean", "Mathlib/Order/Extension/Linear.lean", "Mathlib/Analysis/Calculus/IteratedDeriv/Defs.lean", "Mathlib/Geometry/Manifold/SmoothManifoldWithCorners.lean", "Mathlib/Topology/Metrizable/Basic.lean", "Mathlib/NumberTheory/SumPrimeReciprocals.lean", "Mathlib/Data/Nat/PartENat.lean", "Mathlib/Analysis/NormedSpace/SphereNormEquiv.lean", "Mathlib/NumberTheory/NumberField/Units/DirichletTheorem.lean", "Mathlib/Tactic/ClearExclamation.lean", "Mathlib/Order/ConditionallyCompleteLattice/Basic.lean", "Mathlib/LinearAlgebra/StdBasis.lean", "Mathlib/CategoryTheory/Abelian/Pseudoelements.lean", "Mathlib/Algebra/Group/TypeTags.lean", "Mathlib/FieldTheory/MvPolynomial.lean", "Mathlib/Algebra/Star/Order.lean", "Mathlib/Algebra/GroupWithZero/NonZeroDivisors.lean", "Mathlib/RepresentationTheory/Action/Continuous.lean", "Mathlib/Data/Multiset/Fintype.lean", "Mathlib/RingTheory/EuclideanDomain.lean", "Mathlib/Geometry/Manifold/Algebra/Structures.lean", "Mathlib/Order/RelIso/Basic.lean", "Mathlib/Algebra/Order/Monoid/TypeTags.lean", "Mathlib/Analysis/SpecialFunctions/Log/Basic.lean", "Mathlib/Data/DList/Instances.lean", "Mathlib/Data/Finset/NAry.lean", "Mathlib/Topology/Bornology/Hom.lean", "Mathlib/Data/Finset/Update.lean", "Mathlib/Data/Countable/Small.lean", "Mathlib/CategoryTheory/Shift/ShiftSequence.lean", "Mathlib/Tactic/Linter/OldObtain.lean", "Mathlib/CategoryTheory/Sites/Preserves.lean", "Mathlib/Algebra/Lie/SkewAdjoint.lean", "Mathlib/AlgebraicGeometry/EllipticCurve/DivisionPolynomial/Basic.lean", "Mathlib/RingTheory/Derivation/Basic.lean", "Mathlib/CategoryTheory/Limits/Types.lean", "Mathlib/Analysis/SpecialFunctions/Gamma/BohrMollerup.lean", "Mathlib/ModelTheory/Order.lean", "Mathlib/Tactic/Clean.lean", "Mathlib/Algebra/Group/Submonoid/Membership.lean", "Mathlib/Topology/Sheaves/Operations.lean", "Mathlib/Analysis/NormedSpace/TrivSqZeroExt.lean", "Mathlib/Topology/Category/TopCat/EffectiveEpi.lean", "Mathlib/Analysis/Convex/GaugeRescale.lean", "Mathlib/Order/Ideal.lean", "Mathlib/RepresentationTheory/Maschke.lean", "Mathlib/RingTheory/Congruence/BigOperators.lean", "Mathlib/Algebra/Category/BialgebraCat/Basic.lean", "Mathlib/Data/Multiset/Fold.lean", "Mathlib/Data/Prod/Basic.lean", "Mathlib/Data/FunLike/Embedding.lean", "Mathlib/SetTheory/Cardinal/Continuum.lean", "Mathlib/Tactic/TermCongr.lean", "Mathlib/Topology/Algebra/Order/Compact.lean", "Mathlib/Algebra/PUnitInstances.lean", "Mathlib/Combinatorics/SimpleGraph/Density.lean", "Mathlib/Analysis/NormedSpace/Algebra.lean", "Mathlib/Analysis/NormedSpace/WeakDual.lean", "Mathlib/Analysis/Complex/UpperHalfPlane/Metric.lean", "Mathlib/MeasureTheory/Integral/LebesgueNormedSpace.lean", "Mathlib/Geometry/Manifold/LocalDiffeomorph.lean", "Mathlib/Deprecated/Subgroup.lean", "Mathlib/Algebra/Ring/Units.lean", "Mathlib/CategoryTheory/Monoidal/Types/Basic.lean", "Mathlib/Topology/Instances/Sign.lean", "Mathlib/CategoryTheory/Localization/Predicate.lean", "Mathlib/Algebra/Quaternion.lean", "Mathlib/AlgebraicTopology/DoldKan/PInfty.lean", "Mathlib/Geometry/Manifold/Instances/Real.lean", "Mathlib/Topology/Instances/Real.lean", "Mathlib/Combinatorics/SimpleGraph/Regularity/Uniform.lean", "Mathlib/Topology/Instances/Nat.lean", "Mathlib/Analysis/Normed/Field/Basic.lean", "Mathlib/CategoryTheory/Sites/Spaces.lean", "Mathlib/Topology/Algebra/Nonarchimedean/Bases.lean", "Mathlib/Combinatorics/SimpleGraph/Ends/Defs.lean", "Mathlib/Data/Real/Basic.lean", "Mathlib/Data/Nat/Order/Lemmas.lean", "Mathlib/Topology/VectorBundle/Basic.lean", "Mathlib/AlgebraicTopology/FundamentalGroupoid/SimplyConnected.lean", "Mathlib/AlgebraicTopology/DoldKan/Notations.lean", "Mathlib/Algebra/BigOperators/Group/Multiset.lean", "Mathlib/CategoryTheory/Filtered/Small.lean", "Mathlib/Algebra/Group/Commutator.lean", "Mathlib/Data/QPF/Multivariate/Basic.lean", "Mathlib/Dynamics/Ergodic/Function.lean", "Mathlib/ModelTheory/Ultraproducts.lean", "Mathlib/FieldTheory/IntermediateField.lean", "Mathlib/CategoryTheory/Limits/MonoCoprod.lean", "Mathlib/Combinatorics/SetFamily/Compression/Down.lean", "Mathlib/LinearAlgebra/CliffordAlgebra/Equivs.lean", "Mathlib/MeasureTheory/Measure/Haar/Basic.lean", "Mathlib/Tactic/ClearExcept.lean", "Mathlib/CategoryTheory/Bicategory/Functor/Oplax.lean", "Mathlib/Topology/MetricSpace/Antilipschitz.lean", "Mathlib/Condensed/Light/Discrete.lean", "Mathlib/Probability/Density.lean", "Mathlib/Algebra/Homology/DerivedCategory/ExactFunctor.lean", "Mathlib/Algebra/Module/Zlattice/Basic.lean", "Mathlib/Geometry/Euclidean/Sphere/Power.lean", "Mathlib/MeasureTheory/Order/UpperLower.lean", "Mathlib/Algebra/HierarchyDesign.lean", "Mathlib/Algebra/MvPolynomial/CommRing.lean", "Mathlib/NumberTheory/WellApproximable.lean", "Mathlib/RepresentationTheory/Action/Concrete.lean", "Mathlib/LinearAlgebra/QuotientPi.lean", "Mathlib/Order/PFilter.lean", "Mathlib/Tactic/DeriveTraversable.lean", "Mathlib/Tactic/Linter/Style.lean", "Mathlib/Order/Category/FinPartOrd.lean", "Mathlib/Computability/Primrec.lean", "Mathlib/Data/Finset/Pi.lean", "Mathlib/Topology/MetricSpace/ShrinkingLemma.lean", "Mathlib/CategoryTheory/Linear/FunctorCategory.lean", "Mathlib/Combinatorics/Quiver/Arborescence.lean", "Mathlib/Topology/ContinuousFunction/ContinuousMapZero.lean", "Mathlib/CategoryTheory/Sites/Sieves.lean", "Mathlib/MeasureTheory/Measure/Regular.lean", "Mathlib/Topology/Category/Profinite/Limits.lean", "Mathlib/Init/Data/Int/Basic.lean", "Mathlib/Algebra/Group/Action/Defs.lean", "Mathlib/Data/Seq/Computation.lean", "Mathlib/Order/Filter/Cocardinal.lean", "Mathlib/Data/Stream/Defs.lean", "Mathlib/Analysis/InnerProductSpace/l2Space.lean", "Mathlib/NumberTheory/GaussSum.lean", "Mathlib/Data/Fintype/Parity.lean", "Mathlib/AlgebraicTopology/SingularSet.lean", "Mathlib/Algebra/Divisibility/Basic.lean", "Mathlib/Algebra/Homology/Bifunctor.lean", "Mathlib/RingTheory/PowerSeries/Basic.lean", "Mathlib/Analysis/NormedSpace/ConformalLinearMap.lean", "Mathlib/NumberTheory/FrobeniusNumber.lean", "Mathlib/Combinatorics/SetFamily/CauchyDavenport.lean", "Mathlib/AlgebraicTopology/SimplicialSet/Monoidal.lean", "Mathlib/AlgebraicGeometry/Spec.lean", "Mathlib/MeasureTheory/Function/LpSeminorm/Basic.lean", "Mathlib/Logic/Embedding/Set.lean", "Mathlib/Combinatorics/Additive/AP/Three/Defs.lean", "Mathlib/Algebra/Algebra/Basic.lean", "Mathlib/LinearAlgebra/Dual.lean", "Mathlib/Order/Interval/Set/WithBotTop.lean", "Mathlib/CategoryTheory/Adjunction/Over.lean", "Mathlib/Topology/Algebra/InfiniteSum/NatInt.lean", "Mathlib/Algebra/CubicDiscriminant.lean", "Mathlib/NumberTheory/LSeries/HurwitzZetaOdd.lean", "Mathlib/Topology/ContinuousFunction/StoneWeierstrass.lean", "Mathlib/CategoryTheory/Functor/FullyFaithful.lean", "Mathlib/Order/RelSeries.lean", "Mathlib/Algebra/Group/Commute/Basic.lean", "Mathlib/Data/Matrix/RowCol.lean", "Mathlib/Geometry/Manifold/Algebra/LieGroup.lean", "Mathlib/CategoryTheory/Limits/Constructions/ZeroObjects.lean", "Mathlib/Logic/Function/Basic.lean", "Mathlib/NumberTheory/NumberField/CanonicalEmbedding/Basic.lean", "Mathlib/Analysis/NormedSpace/Star/Matrix.lean", "Mathlib/Logic/Equiv/Embedding.lean", "Mathlib/Tactic/Linter.lean", "Mathlib/Lean/Meta.lean", "Mathlib/Topology/Sheaves/Sheaf.lean", "Mathlib/Analysis/Calculus/FormalMultilinearSeries.lean", "Mathlib/Analysis/Calculus/Deriv/Pi.lean", "Mathlib/CategoryTheory/Sites/Coherent/Equivalence.lean", "Mathlib/MeasureTheory/Group/Prod.lean", "Mathlib/Order/CompletePartialOrder.lean", "Mathlib/Data/Vector/Defs.lean", "Mathlib/Order/Monotone/Extension.lean", "Mathlib/RingTheory/RingHomProperties.lean", "Mathlib/Topology/AlexandrovDiscrete.lean", "Mathlib/Algebra/Bounds.lean", "Mathlib/Algebra/Module/GradedModule.lean", "Mathlib/Analysis/Complex/OpenMapping.lean", "Mathlib/Analysis/Calculus/LHopital.lean", "Mathlib/Analysis/LocallyConvex/WithSeminorms.lean", "Mathlib/CategoryTheory/Bicategory/NaturalTransformation.lean", "Mathlib/Data/Fin/Tuple/Monotone.lean", "Mathlib/Data/Real/Pi/Wallis.lean", "Mathlib/Geometry/Manifold/AnalyticManifold.lean", "Mathlib/Geometry/Manifold/MFDeriv/UniqueDifferential.lean", "Mathlib/LinearAlgebra/Charpoly/Basic.lean", "Mathlib/ModelTheory/Algebra/Field/CharP.lean", "Mathlib/Topology/MetricSpace/Gluing.lean", "Mathlib/Tactic/DeriveToExpr.lean", "Mathlib/Algebra/Ring/Idempotents.lean", "Mathlib/Util/AssertNoSorry.lean", "Mathlib/Data/ENNReal/Inv.lean", "Mathlib/Geometry/Manifold/ContMDiff/Defs.lean", "Mathlib/LinearAlgebra/Semisimple.lean", "Mathlib/Analysis/SpecialFunctions/Pow/Integral.lean", "Mathlib/Dynamics/BirkhoffSum/Average.lean", "Mathlib/LinearAlgebra/Matrix/ToLin.lean", "Mathlib/NumberTheory/LSeries/Linearity.lean", "Mathlib/Analysis/NormedSpace/RCLike.lean", "Mathlib/Topology/Irreducible.lean", "Mathlib/NumberTheory/ModularForms/SlashInvariantForms.lean", "Mathlib/Analysis/Calculus/Conformal/InnerProduct.lean", "Mathlib/NumberTheory/Padics/PadicNumbers.lean", "Mathlib/Algebra/Module/PID.lean", "Mathlib/RingTheory/MvPolynomial/Tower.lean", "Mathlib/Topology/Algebra/MvPolynomial.lean", "Mathlib/GroupTheory/Perm/Cycle/Type.lean", "Mathlib/CategoryTheory/Limits/IndYoneda.lean", "Mathlib/Topology/UniformSpace/Matrix.lean", "Mathlib/Analysis/Convex/Side.lean", "Mathlib/LinearAlgebra/QuadraticForm/Basic.lean", "Mathlib/Lean/Meta/DiscrTree.lean", "Mathlib/RingTheory/Localization/InvSubmonoid.lean", "Mathlib/Data/Sym/Basic.lean", "Mathlib/Algebra/Polynomial/BigOperators.lean", "Mathlib/Analysis/Normed/Field/UnitBall.lean", "Mathlib/Analysis/LocallyConvex/WeakDual.lean", "Mathlib/CategoryTheory/Monoidal/Mon_.lean", "Mathlib/CategoryTheory/EssentiallySmall.lean", "Mathlib/Combinatorics/SetFamily/Shadow.lean", "Mathlib/NumberTheory/DiophantineApproximation.lean", "Mathlib/NumberTheory/ModularForms/JacobiTheta/Manifold.lean", "Mathlib/Algebra/Category/AlgebraCat/Limits.lean", "Mathlib/Data/Real/Hyperreal.lean", "Mathlib/Order/Filter/CountableInter.lean", "Mathlib/CategoryTheory/Limits/Shapes/Reflexive.lean", "Mathlib/RingTheory/RootsOfUnity/Lemmas.lean", "Mathlib/RingTheory/Valuation/Integral.lean", "Mathlib/CategoryTheory/Monad/EquivMon.lean", "Mathlib/Data/Nat/Cast/Field.lean", "Mathlib/CategoryTheory/Localization/Pi.lean", "Mathlib/MeasureTheory/Decomposition/SignedHahn.lean", "Mathlib/Topology/FiberBundle/IsHomeomorphicTrivialBundle.lean", "Mathlib/CategoryTheory/Limits/Shapes/CombinedProducts.lean", "Mathlib/CategoryTheory/Category/PartialFun.lean", "Mathlib/RepresentationTheory/GroupCohomology/Resolution.lean", "Mathlib/Analysis/Normed/Group/SemiNormedGrp/Kernels.lean", "Mathlib/AlgebraicTopology/DoldKan/Projections.lean", "Mathlib/Algebra/Polynomial/Laurent.lean", "Mathlib/CategoryTheory/Quotient/Linear.lean", "Mathlib/Data/Complex/Abs.lean", "Mathlib/Analysis/SpecialFunctions/Trigonometric/Inverse.lean", "Mathlib/Tactic/SlimCheck.lean", "Mathlib/RingTheory/Adjoin/Tower.lean", "Mathlib/AlgebraicGeometry/PrimeSpectrum/Basic.lean", "Mathlib/CategoryTheory/Abelian/LeftDerived.lean", "Mathlib/Data/Equiv/Functor.lean", "Mathlib/RingTheory/PiTensorProduct.lean", "Mathlib/RingTheory/Adjoin/FG.lean", "Mathlib/RingTheory/Polynomial/Pochhammer.lean", "Mathlib/Data/PFunctor/Univariate/Basic.lean", "Mathlib/Data/PNat/Factors.lean", "Mathlib/CategoryTheory/Preadditive/SingleObj.lean", "Mathlib/Topology/Compactness/Lindelof.lean", "Mathlib/Analysis/InnerProductSpace/Orientation.lean", "Mathlib/Analysis/Calculus/Deriv/Linear.lean", "Mathlib/Topology/Algebra/Module/Star.lean", "Mathlib/Algebra/Category/Ring/Basic.lean", "Mathlib/Algebra/Lie/OfAssociative.lean", "Mathlib/Analysis/InnerProductSpace/Rayleigh.lean", "Mathlib/Order/IsWellOrderLimitElement.lean", "Mathlib/CategoryTheory/GuitartExact/Basic.lean", "Mathlib/Analysis/SpecialFunctions/CompareExp.lean", "Mathlib/CategoryTheory/Sites/ConstantSheaf.lean", "Mathlib/Combinatorics/SetFamily/HarrisKleitman.lean", "Mathlib/Tactic/Clear_.lean", "Mathlib/Topology/Category/FinTopCat.lean", "Mathlib/Data/Vector3.lean", "Mathlib/Order/Lattice.lean", "Mathlib/Data/Fintype/Sum.lean", "Mathlib/Tactic/Explode/Pretty.lean", "Mathlib/Data/List/ReduceOption.lean", "Mathlib/Combinatorics/SimpleGraph/Partition.lean", "Mathlib/MeasureTheory/MeasurableSpace/Invariants.lean", "Mathlib/RingTheory/Polynomial/Quotient.lean", "Mathlib/LinearAlgebra/TensorPower.lean", "Mathlib/RingTheory/Fintype.lean", "Mathlib/GroupTheory/FixedPointFree.lean", "Mathlib/Topology/Algebra/Order/Floor.lean", "Mathlib/Algebra/Homology/HomotopyCategory/ShiftSequence.lean", "Mathlib/AlgebraicTopology/SimplicialSet.lean", "Mathlib/CategoryTheory/Bicategory/FunctorBicategory.lean", "Mathlib/CategoryTheory/Bicategory/Adjunction.lean", "Mathlib/Init/Data/Option/Lemmas.lean", "Mathlib/Data/Int/NatPrime.lean", "Mathlib/Lean/Meta/Simp.lean", "Mathlib/Algebra/Algebra/RestrictScalars.lean", "Mathlib/Data/Multiset/FinsetOps.lean", "Mathlib/Algebra/Order/Ring/Pow.lean", "Mathlib/LinearAlgebra/Eigenspace/Matrix.lean", "Mathlib/LinearAlgebra/Matrix/Charpoly/Coeff.lean", "Mathlib/ModelTheory/Definability.lean", "Mathlib/Analysis/MellinTransform.lean", "Mathlib/Data/Real/Pi/Leibniz.lean", "Mathlib/Algebra/Order/Pointwise.lean", "Mathlib/RingTheory/WittVector/InitTail.lean", "Mathlib/Algebra/Group/Semiconj/Defs.lean", "Mathlib/CategoryTheory/Sites/Coherent/ReflectsPrecoherent.lean", "Mathlib/Data/W/Constructions.lean", "Mathlib/RepresentationTheory/Action/Limits.lean", "Mathlib/Algebra/Group/Hom/End.lean", "Mathlib/Combinatorics/Quiver/Basic.lean", "Mathlib/MeasureTheory/Measure/Haar/Disintegration.lean", "Mathlib/Topology/Constructions.lean", "Mathlib/Algebra/CharZero/Quotient.lean", "Mathlib/Probability/Independence/ZeroOne.lean", "Mathlib/CategoryTheory/Sites/Coherent/Comparison.lean", "Mathlib/Combinatorics/Quiver/Push.lean", "Mathlib/Algebra/Ring/Defs.lean", "Mathlib/RingTheory/IsTensorProduct.lean", "Mathlib/CategoryTheory/Sites/Coherent/SheafComparison.lean", "Mathlib/Lean/Message.lean", "Mathlib/SetTheory/Ordinal/Exponential.lean", "Mathlib/CategoryTheory/GradedObject/Single.lean", "Mathlib/Algebra/Order/Antidiag/Prod.lean", "Mathlib/Analysis/Calculus/Darboux.lean", "Mathlib/RingTheory/AlgebraicIndependent.lean", "Mathlib/Algebra/Order/Nonneg/Module.lean", "Mathlib/Control/Traversable/Instances.lean", "Mathlib/Data/Array/Defs.lean", "Mathlib/Topology/Algebra/Module/Determinant.lean", "Mathlib/Data/Fintype/Units.lean", "Mathlib/CategoryTheory/Functor/EpiMono.lean", "Mathlib/Analysis/NormedSpace/Dual.lean", "Mathlib/Logic/Encodable/Basic.lean", "Mathlib/Combinatorics/Hall/Finite.lean", "Mathlib/LinearAlgebra/Matrix/BilinearForm.lean", "Mathlib/Topology/Instances/ENNReal.lean", "Mathlib/Computability/EpsilonNFA.lean", "Mathlib/CategoryTheory/Monoidal/Linear.lean", "Mathlib/GroupTheory/Perm/List.lean", "Mathlib/Data/Finset/Sym.lean", "Mathlib/Topology/Order/LeftRightLim.lean", "Mathlib/Data/Fintype/List.lean", "Mathlib/RingTheory/Localization/Cardinality.lean", "Mathlib/Analysis/Analytic/IsolatedZeros.lean", "Mathlib/Algebra/Order/Nonneg/Floor.lean", "Mathlib/Algebra/Order/Floor.lean", "Mathlib/CategoryTheory/Limits/FunctorToTypes.lean", "Mathlib/LinearAlgebra/Matrix/Transvection.lean", "Mathlib/RingTheory/Kaehler/Basic.lean", "Mathlib/CategoryTheory/ConcreteCategory/BundledHom.lean", "Mathlib/LinearAlgebra/RootSystem/Basic.lean", "Mathlib/CategoryTheory/Shift/Pullback.lean", "Mathlib/Tactic/SudoSetOption.lean", "Mathlib/CategoryTheory/Sites/Over.lean", "Mathlib/CategoryTheory/Pi/Basic.lean", "Mathlib/Data/List/Destutter.lean", "Mathlib/NumberTheory/ModularForms/JacobiTheta/TwoVariable.lean", "Mathlib/Algebra/Lie/TensorProduct.lean", "Mathlib/Init/Data/List/Basic.lean", "Mathlib/RingTheory/Ideal/Colon.lean", "Mathlib/Algebra/GroupWithZero/Indicator.lean", "Mathlib/Tactic/FunProp/Types.lean", "Mathlib/Tactic/Zify.lean", "Mathlib/CategoryTheory/Triangulated/TriangleShift.lean", "Mathlib/Algebra/Polynomial/Monomial.lean", "Mathlib/Data/Fintype/Perm.lean", "Mathlib/LinearAlgebra/FreeModule/Finite/Matrix.lean", "Mathlib/Topology/ContinuousFunction/Compact.lean", "Mathlib/Algebra/Category/MonCat/Limits.lean", "Mathlib/Algebra/Ring/Action/Basic.lean", "Mathlib/Algebra/Expr.lean", "Mathlib/LinearAlgebra/CliffordAlgebra/EvenEquiv.lean", "Mathlib/Data/Fintype/Sort.lean", "Mathlib/LinearAlgebra/Eigenspace/Minpoly.lean", "Mathlib/Data/Finset/Fold.lean", "Mathlib/Topology/ContinuousFunction/Ordered.lean", "Mathlib/Analysis/NormedSpace/MStructure.lean", "Mathlib/Analysis/SpecialFunctions/Gaussian/PoissonSummation.lean", "Mathlib/Control/Traversable/Basic.lean", "Mathlib/Data/Finset/Interval.lean", "Mathlib/AlgebraicTopology/ExtraDegeneracy.lean", "Mathlib/NumberTheory/LSeries/HurwitzZeta.lean", "Mathlib/Topology/Sober.lean", "Mathlib/Algebra/GroupWithZero/Conj.lean", "Mathlib/Data/Finset/Sigma.lean", "Mathlib/CategoryTheory/Adjunction/Restrict.lean", "Mathlib/Data/List/EditDistance/Defs.lean", "Mathlib/CategoryTheory/Category/Pointed.lean", "Mathlib/Algebra/Order/Monoid/Unbundled/MinMax.lean", "Mathlib/GroupTheory/EckmannHilton.lean", "Mathlib/Tactic/NormNum/Eq.lean", "Mathlib/RingTheory/Coalgebra/Basic.lean", "Mathlib/CategoryTheory/Simple.lean", "Mathlib/Tactic/ApplyCongr.lean", "Mathlib/Analysis/Calculus/FDeriv/Mul.lean", "Mathlib/CategoryTheory/Galois/Decomposition.lean", "Mathlib/Algebra/Homology/TotalComplex.lean", "Mathlib/Algebra/Order/Ring/Defs.lean", "Mathlib/LinearAlgebra/AffineSpace/Ordered.lean", "Mathlib/Algebra/Order/Ring/Rat.lean", "Mathlib/Algebra/Star/NonUnitalSubalgebra.lean", "Mathlib/CategoryTheory/Sites/LocallyBijective.lean", "Mathlib/Order/SuccPred/LinearLocallyFinite.lean", "Mathlib/Data/Int/Cast/Defs.lean", "Mathlib/Data/Fintype/Powerset.lean", "Mathlib/GroupTheory/Subsemigroup/Center.lean", "Mathlib/RingTheory/DiscreteValuationRing/TFAE.lean", "Mathlib/LinearAlgebra/QuadraticForm/Real.lean", "Mathlib/Topology/UniformSpace/Cauchy.lean", "Mathlib/Order/Grade.lean", "Mathlib/AlgebraicGeometry/ProjectiveSpectrum/Scheme.lean", "Mathlib/MeasureTheory/Measure/WithDensity.lean", "Mathlib/Algebra/Order/Antidiag/Finsupp.lean", "Mathlib/Util/FormatTable.lean", "Mathlib/ModelTheory/Bundled.lean", "Mathlib/Data/Nat/Periodic.lean", "Mathlib/Algebra/Order/Group/Lattice.lean", "Mathlib/Analysis/BoxIntegral/Partition/Measure.lean", "Mathlib/Topology/Sheaves/Skyscraper.lean", "Mathlib/Analysis/SpecialFunctions/ExpDeriv.lean", "Mathlib/Topology/MetricSpace/Lipschitz.lean", "Mathlib/CategoryTheory/Functor/OfSequence.lean", "Mathlib/Algebra/FreeMonoid/Count.lean", "Mathlib/Analysis/SpecificLimits/RCLike.lean", "Mathlib/Analysis/Subadditive.lean", "Mathlib/Algebra/MvPolynomial/Division.lean", "Mathlib/Topology/Algebra/InfiniteSum/Constructions.lean", "Mathlib/Algebra/Field/Subfield.lean", "Mathlib/CategoryTheory/ChosenFiniteProducts/FunctorCategory.lean", "Mathlib/Combinatorics/Optimization/ValuedCSP.lean", "Mathlib/Data/Finset/Pointwise/Interval.lean", "Mathlib/Analysis/Calculus/InverseFunctionTheorem/Deriv.lean", "Mathlib/Tactic/ApplyWith.lean", "Mathlib/CategoryTheory/Functor/Const.lean", "Mathlib/GroupTheory/NoncommCoprod.lean", "Mathlib/Algebra/Lie/Matrix.lean", "Mathlib/Data/DFinsupp/Multiset.lean", "Mathlib/RingTheory/DedekindDomain/PID.lean", "Mathlib/Topology/Order/OrderClosed.lean", "Mathlib/Combinatorics/SimpleGraph/Dart.lean", "Mathlib/Algebra/Group/FiniteSupport.lean", "Mathlib/CategoryTheory/Triangulated/HomologicalFunctor.lean", "Mathlib/NumberTheory/Harmonic/GammaDeriv.lean", "Mathlib/Analysis/LocallyConvex/Polar.lean", "Mathlib/CategoryTheory/Subterminal.lean", "Mathlib/CategoryTheory/Category/Pairwise.lean", "Mathlib/Analysis/NormedSpace/AffineIsometry.lean", "Mathlib/Algebra/Category/ModuleCat/Colimits.lean", "Mathlib/Combinatorics/SimpleGraph/Hamiltonian.lean", "Mathlib/GroupTheory/ClassEquation.lean", "Mathlib/Topology/Category/Profinite/CofilteredLimit.lean", "Mathlib/Algebra/Category/Grp/Colimits.lean", "Mathlib/Algebra/Module/Pi.lean", "Mathlib/CategoryTheory/IsConnected.lean", "Mathlib/Algebra/GeomSum.lean", "Mathlib/Topology/Category/CompHausLike/Basic.lean", "Mathlib/Data/UnionFind.lean", "Mathlib/Order/CompleteLatticeIntervals.lean", "Mathlib/RingTheory/DedekindDomain/Ideal.lean", "Mathlib/Algebra/Order/Field/Rat.lean", "Mathlib/RingTheory/Polynomial/Selmer.lean", "Mathlib/Order/Interval/Basic.lean", "Mathlib/LinearAlgebra/Matrix/NonsingularInverse.lean", "Mathlib/NumberTheory/Liouville/LiouvilleWith.lean", "Mathlib/RingTheory/PrincipalIdealDomain.lean", "Mathlib/Analysis/Normed/Group/HomCompletion.lean", "Mathlib/Algebra/CharZero/Lemmas.lean", "Mathlib/Data/Int/Cast/Prod.lean", "Mathlib/Geometry/Manifold/ContMDiffMap.lean", "Mathlib/Analysis/VonNeumannAlgebra/Basic.lean", "Mathlib/CategoryTheory/Sites/Equivalence.lean", "Mathlib/Order/WellFounded.lean", "Mathlib/CategoryTheory/Whiskering.lean", "Mathlib/RingTheory/HopfAlgebra.lean", "Mathlib/Data/List/Infix.lean", "Mathlib/CategoryTheory/Endomorphism.lean", "Mathlib/Tactic/Group.lean", "Mathlib/Probability/Independence/Conditional.lean", "Mathlib/RingTheory/GradedAlgebra/Radical.lean", "Mathlib/Combinatorics/Quiver/Symmetric.lean", "Mathlib/CategoryTheory/FintypeCat.lean", "Mathlib/Data/Int/Order/Units.lean", "Mathlib/Topology/ExtendFrom.lean", "Mathlib/CategoryTheory/Products/Unitor.lean", "Mathlib/Data/Set/Subsingleton.lean", "Mathlib/Analysis/BoxIntegral/Partition/Filter.lean", "Mathlib/Analysis/PSeries.lean", "Mathlib/Data/Set/Sups.lean", "Mathlib/Order/Concept.lean", "Mathlib/LinearAlgebra/Matrix/Charpoly/LinearMap.lean", "Mathlib/AlgebraicGeometry/ProjectiveSpectrum/Topology.lean", "Mathlib/RingTheory/ClassGroup.lean", "Mathlib/Data/Finset/Preimage.lean", "Mathlib/Topology/Order.lean", "Mathlib/Analysis/LocallyConvex/Barrelled.lean", "Mathlib/LinearAlgebra/AffineSpace/Midpoint.lean", "Mathlib/Topology/Bornology/BoundedOperation.lean", "Mathlib/RingTheory/RingHom/Integral.lean", "Mathlib/MeasureTheory/Function/ConditionalExpectation/Basic.lean", "Mathlib/RingTheory/Ideal/LocalRing.lean", "Mathlib/RingTheory/Localization/NormTrace.lean", "Mathlib/Algebra/MvPolynomial/Polynomial.lean", "Mathlib/Tactic/NormNum/BigOperators.lean", "Mathlib/GroupTheory/MonoidLocalization.lean", "Mathlib/ModelTheory/Semantics.lean", "Mathlib/RingTheory/Valuation/RankOne.lean", "Mathlib/Data/Fin/Tuple/NatAntidiagonal.lean", "Mathlib/Tactic/Find.lean", "Mathlib/CategoryTheory/Limits/Fubini.lean", "Mathlib/Combinatorics/Derangements/Finite.lean", "Mathlib/Topology/Instances/Irrational.lean", "Mathlib/Algebra/Category/AlgebraCat/Symmetric.lean", "Mathlib/RingTheory/Localization/FractionRing.lean", "Mathlib/Algebra/Homology/ShortComplex/RightHomology.lean", "Mathlib/Algebra/Ring/Subring/Units.lean", "Mathlib/Algebra/Order/Group/PosPart.lean", "Mathlib/RingTheory/Ideal/IsPrimary.lean", "Mathlib/CategoryTheory/Monad/Products.lean", "Mathlib/Data/Set/Constructions.lean", "Mathlib/Data/Real/ENatENNReal.lean", "Mathlib/Topology/Category/TopCat/OpenNhds.lean", "Mathlib/Algebra/Group/Opposite.lean", "Mathlib/Analysis/NormedSpace/lpSpace.lean", "Mathlib/GroupTheory/GroupAction/ConjAct.lean", "Mathlib/Topology/MetricSpace/HausdorffDistance.lean", "Mathlib/Analysis/Normed/Group/Bounded.lean", "Mathlib/CategoryTheory/Sites/Types.lean", "Mathlib/Order/PrimeSeparator.lean", "Mathlib/Algebra/Order/EuclideanAbsoluteValue.lean", "Mathlib/Combinatorics/SetFamily/Kleitman.lean", "Mathlib/Analysis/Analytic/Meromorphic.lean", "Mathlib/MeasureTheory/Covering/Differentiation.lean", "Mathlib/MeasureTheory/Group/Integral.lean", "Mathlib/CategoryTheory/Monoidal/Internal/FunctorCategory.lean", "Mathlib/CategoryTheory/SmallObject/Iteration.lean", "Mathlib/Topology/Algebra/ContinuousAffineMap.lean", "Mathlib/Algebra/Homology/HomotopyCategory/ShortExact.lean", "Mathlib/Analysis/Convex/Segment.lean", "Mathlib/CategoryTheory/Comma/Arrow.lean", "Mathlib/Combinatorics/Hall/Basic.lean", "Mathlib/RingTheory/HahnSeries/Addition.lean", "Mathlib/Algebra/Order/Invertible.lean", "Mathlib/Analysis/Calculus/Deriv/Star.lean", "Mathlib/GroupTheory/OrderOfElement.lean", "Mathlib/MeasureTheory/Measure/AEMeasurable.lean", "Mathlib/RingTheory/Adjoin/PowerBasis.lean", "Mathlib/Analysis/NormedSpace/Exponential.lean", "Mathlib/Data/Nat/Choose/Sum.lean", "Mathlib/LinearAlgebra/InvariantBasisNumber.lean", "Mathlib/Algebra/Order/Group/Cone.lean", "Mathlib/Algebra/Order/Monovary.lean", "Mathlib/Analysis/NormedSpace/LpEquiv.lean", "Mathlib/CategoryTheory/Linear/LinearFunctor.lean", "Mathlib/MeasureTheory/Measure/LogLikelihoodRatio.lean", "Mathlib/Probability/Independence/Kernel.lean", "Mathlib/MeasureTheory/Constructions/Prod/Basic.lean", "Mathlib/Algebra/Group/Subgroup/Pointwise.lean", "Mathlib/MeasureTheory/Measure/FiniteMeasure.lean", "Mathlib/Topology/UniformSpace/Equiv.lean", "Mathlib/Algebra/Order/Group/Prod.lean", "Mathlib/Topology/ContinuousFunction/T0Sierpinski.lean", "Mathlib/CategoryTheory/Comma/Basic.lean", "Mathlib/CategoryTheory/Sites/Adjunction.lean", "Mathlib/CategoryTheory/Bicategory/Functor/Pseudofunctor.lean", "Mathlib/Data/List/Enum.lean", "Mathlib/Order/BooleanGenerators.lean", "Mathlib/FieldTheory/SeparableClosure.lean", "Mathlib/LinearAlgebra/AffineSpace/Slope.lean", "Mathlib/LinearAlgebra/TensorProduct/Basic.lean", "Mathlib/AlgebraicGeometry/EllipticCurve/Jacobian.lean", "Mathlib/Tactic/FinCases.lean", "Mathlib/Algebra/Group/Subsemigroup/Membership.lean", "Mathlib/LinearAlgebra/Matrix/SchurComplement.lean", "Mathlib/Algebra/Category/Grp/EquivalenceGroupAddGroup.lean", "Mathlib/Data/Finsupp/BigOperators.lean", "Mathlib/Data/Nat/Defs.lean", "Mathlib/Tactic/Relation/Rfl.lean", "Mathlib/RingTheory/Bialgebra/Hom.lean", "Mathlib/Tactic/Use.lean", "Mathlib/LinearAlgebra/PID.lean", "Mathlib/NumberTheory/ClassNumber/Finite.lean", "Mathlib/Analysis/NormedSpace/Star/ContinuousFunctionalCalculus/Restrict.lean", "Mathlib/Algebra/ContinuedFractions/Computation/Translations.lean", "Mathlib/Algebra/Lie/Semisimple/Defs.lean", "Mathlib/LinearAlgebra/FreeModule/PID.lean", "Mathlib/Data/Finsupp/Order.lean", "Mathlib/NumberTheory/FermatPsp.lean", "Mathlib/Algebra/Order/Algebra.lean", "Mathlib/Analysis/ODE/Gronwall.lean", "Mathlib/Tactic/GCongr.lean", "Mathlib/Algebra/Group/Units/Hom.lean", "Mathlib/Topology/Category/TopCommRingCat.lean", "Mathlib/LinearAlgebra/AnnihilatingPolynomial.lean", "Mathlib/NumberTheory/LSeries/HurwitzZetaEven.lean", "Mathlib/Tactic/SwapVar.lean", "Mathlib/CategoryTheory/EpiMono.lean", "Mathlib/Util/DischargerAsTactic.lean", "Mathlib/Analysis/InnerProductSpace/TwoDim.lean", "Mathlib/Control/Bifunctor.lean", "Mathlib/CategoryTheory/Limits/Preserves/Ulift.lean", "Mathlib/Algebra/ContinuedFractions/Computation/TerminatesIffRat.lean", "Mathlib/Data/Finset/Sum.lean", "Mathlib/Analysis/Calculus/FDeriv/Bilinear.lean", "Mathlib/Util/Superscript.lean", "Mathlib/Algebra/Category/ModuleCat/Sheaf/PushforwardContinuous.lean", "Mathlib/Analysis/Calculus/Deriv/AffineMap.lean", "Mathlib/Init/Set.lean", "Mathlib/RingTheory/Complex.lean", "Mathlib/Tactic/CancelDenoms.lean", "Mathlib/Topology/VectorBundle/Constructions.lean", "Mathlib/Algebra/Category/MonCat/Basic.lean", "Mathlib/MeasureTheory/Measure/Doubling.lean", "Mathlib/Topology/Category/TopCat/Basic.lean", "Mathlib/CategoryTheory/Idempotents/Basic.lean", "Mathlib/Algebra/GCDMonoid/Finset.lean", "Mathlib/LinearAlgebra/TensorAlgebra/ToTensorPower.lean", "Mathlib/Order/UpperLower/LocallyFinite.lean", "Mathlib/RingTheory/DedekindDomain/FiniteAdeleRing.lean", "Mathlib/Geometry/Euclidean/Sphere/SecondInter.lean", "Mathlib/Algebra/Vertex/HVertexOperator.lean", "Mathlib/RingTheory/QuotientNilpotent.lean", "Mathlib/Tactic/SimpIntro.lean", "Mathlib/Data/Int/Interval.lean", "Mathlib/Topology/MetricSpace/Closeds.lean", "Mathlib/NumberTheory/EulerProduct/DirichletLSeries.lean", "Mathlib/Data/Nat/Choose/Central.lean", "Mathlib/Topology/ContinuousFunction/Basic.lean", "Mathlib/CategoryTheory/Functor/KanExtension/Adjunction.lean", "Mathlib/CategoryTheory/Iso.lean", "Mathlib/Algebra/BigOperators/Fin.lean", "Mathlib/CategoryTheory/Subobject/Basic.lean", "Mathlib/Control/EquivFunctor.lean", "Mathlib/Data/Sigma/Basic.lean", "Mathlib/Algebra/Lie/IdealOperations.lean", "Mathlib/MeasureTheory/Covering/Vitali.lean", "Mathlib/Algebra/Category/ModuleCat/Monoidal/Symmetric.lean", "Mathlib/GroupTheory/GroupAction/SubMulAction.lean", "Mathlib/RingTheory/Flat/Algebra.lean", "Mathlib/Algebra/Order/Field/Canonical/Defs.lean", "Mathlib/CategoryTheory/ClosedUnderIsomorphisms.lean", "Mathlib/Tactic/Attr/Register.lean", "Mathlib/Analysis/SpecialFunctions/Complex/Arctan.lean", "Mathlib/Data/DFinsupp/NeLocus.lean", "Mathlib/MeasureTheory/Tactic.lean", "Mathlib/Algebra/ContinuedFractions/ConvergentsEquiv.lean", "Mathlib/Combinatorics/Additive/ETransform.lean", "Mathlib/CategoryTheory/Shift/ShiftedHom.lean", "Mathlib/Data/Finsupp/Defs.lean", "Mathlib/Geometry/Manifold/Diffeomorph.lean", "Mathlib/LinearAlgebra/Matrix/InvariantBasisNumber.lean", "Mathlib/Tactic/NormNum/Pow.lean", "Mathlib/Topology/Instances/EReal.lean", "Mathlib/Algebra/MonoidAlgebra/Division.lean", "Mathlib/Analysis/Complex/Arg.lean", "Mathlib/CategoryTheory/Elementwise.lean", "Mathlib/Data/Multiset/Basic.lean", "Mathlib/Data/Int/CardIntervalMod.lean", "Mathlib/RingTheory/JacobsonIdeal.lean", "Mathlib/Analysis/Normed/Group/Hom.lean", "Mathlib/Topology/Sheaves/Init.lean", "Mathlib/Algebra/Order/Interval/Finset.lean", "Mathlib/Probability/Kernel/Disintegration/CdfToKernel.lean", "Mathlib/Algebra/Polynomial/PartialFractions.lean", "Mathlib/Topology/Bases.lean", "Mathlib/AlgebraicGeometry/Limits.lean", "Mathlib/Tactic/HelpCmd.lean", "Mathlib/CategoryTheory/Adjunction/FullyFaithful.lean", "Mathlib/Analysis/Complex/Polynomial.lean", "Mathlib/MeasureTheory/Order/Lattice.lean", "Mathlib/Algebra/Category/ModuleCat/Simple.lean", "Mathlib/Condensed/Discrete.lean", "Mathlib/Data/Num/Lemmas.lean", "Mathlib/Analysis/SpecialFunctions/Sqrt.lean", "Mathlib/Analysis/SpecialFunctions/Log/Deriv.lean", "Mathlib/Analysis/Normed/Group/Completion.lean", "Mathlib/Algebra/Module/LinearMap/Star.lean", "Mathlib/Data/Fintype/Card.lean", "Mathlib/Data/TypeMax.lean", "Mathlib/LinearAlgebra/AffineSpace/Restrict.lean", "Mathlib/Algebra/Order/Group/PiLex.lean", "Mathlib/Computability/NFA.lean", "Mathlib/Analysis/Calculus/Deriv/Inv.lean", "Mathlib/Data/Matrix/Notation.lean", "Mathlib/CategoryTheory/Monoidal/Braided/Basic.lean", "Mathlib/Probability/Kernel/MeasureCompProd.lean", "Mathlib/Algebra/CharP/Invertible.lean", "Mathlib/Analysis/Calculus/ContDiff/FiniteDimension.lean", "Mathlib/Tactic/ToExpr.lean", "Mathlib/Data/List/Intervals.lean", "Mathlib/CategoryTheory/CofilteredSystem.lean", "Mathlib/Algebra/Category/ModuleCat/Algebra.lean", "Mathlib/MeasureTheory/Group/AddCircle.lean", "Mathlib/Analysis/SpecialFunctions/Pow/Asymptotics.lean", "Mathlib/Algebra/Category/ModuleCat/Limits.lean", "Mathlib/Analysis/BoxIntegral/Basic.lean", "Mathlib/Data/List/ProdSigma.lean", "Mathlib/Data/Fin/Tuple/Curry.lean", "Mathlib/MeasureTheory/Integral/BoundedContinuousFunction.lean", "Mathlib/Algebra/ContinuedFractions/Basic.lean", "Mathlib/CategoryTheory/Monoidal/CommMon_.lean", "Mathlib/ModelTheory/Graph.lean", "Mathlib/MeasureTheory/Function/LpSeminorm/TriangleInequality.lean", "Mathlib/Tactic/Ring/RingNF.lean", "Mathlib/NumberTheory/ModularForms/EisensteinSeries/UniformConvergence.lean", "Mathlib/Topology/MetricSpace/Contracting.lean", "Mathlib/RingTheory/FractionalIdeal/Norm.lean", "Mathlib/AlgebraicGeometry/Morphisms/RingHomProperties.lean", "Mathlib/Logic/Small/Basic.lean", "Mathlib/Computability/Reduce.lean", "Mathlib/GroupTheory/Perm/Basic.lean", "Mathlib/MeasureTheory/OuterMeasure/Caratheodory.lean", "Mathlib/Data/Matrix/DualNumber.lean", "Mathlib/Data/Finite/Set.lean", "Mathlib/Data/Finset/Order.lean", "Mathlib/Analysis/Convex/Caratheodory.lean", "Mathlib/CategoryTheory/Limits/KanExtension.lean", "Mathlib/Order/Interval/Finset/Fin.lean", "Mathlib/Algebra/Field/MinimalAxioms.lean", "Mathlib/Data/DFinsupp/Basic.lean", "Mathlib/Algebra/Algebra/Subalgebra/Pointwise.lean", "Mathlib/LinearAlgebra/Contraction.lean", "Mathlib/Algebra/Group/WithOne/Basic.lean", "Mathlib/Analysis/Analytic/Basic.lean", "Mathlib/Tactic/CategoryTheory/MonoidalComp.lean", "Mathlib/Topology/Algebra/InfiniteSum/Defs.lean", "Mathlib/Topology/Algebra/Order/Group.lean", "Mathlib/Algebra/Order/Ring/Int.lean", "Mathlib/Combinatorics/SimpleGraph/Finsubgraph.lean", "Mathlib/Algebra/Module/MinimalAxioms.lean", "Mathlib/LinearAlgebra/BilinearForm/DualLattice.lean", "Mathlib/Algebra/Ring/AddAut.lean", "Mathlib/Analysis/Calculus/FDeriv/Add.lean", "Mathlib/Topology/Algebra/Localization.lean", "Mathlib/Algebra/Pointwise/Stabilizer.lean", "Mathlib/CategoryTheory/Subobject/FactorThru.lean", "Mathlib/Geometry/Manifold/ContMDiffMFDeriv.lean", "Mathlib/Combinatorics/SimpleGraph/Metric.lean", "Mathlib/Topology/Algebra/Order/UpperLower.lean", "Mathlib/Condensed/TopComparison.lean", "Mathlib/Order/RelClasses.lean", "Mathlib/Algebra/Order/BigOperators/Ring/Finset.lean", "Mathlib/RingTheory/Int/Basic.lean", "Mathlib/LinearAlgebra/QuadraticForm/QuadraticModuleCat/Monoidal.lean", "Mathlib/RingTheory/Coprime/Ideal.lean", "Mathlib/Topology/Category/CompHaus/Projective.lean", "Mathlib/Util/SleepHeartbeats.lean", "Mathlib/Data/Num/Prime.lean", "Mathlib/Tactic/Continuity/Init.lean", "Mathlib/Algebra/CharP/MixedCharZero.lean", "Mathlib/SetTheory/Cardinal/Ordinal.lean", "Mathlib/Analysis/Complex/UpperHalfPlane/Manifold.lean", "Mathlib/Order/Extension/Well.lean", "Mathlib/Analysis/Normed/Group/Submodule.lean", "Mathlib/RingTheory/Unramified/Basic.lean", "Mathlib/LinearAlgebra/Matrix/Adjugate.lean", "Mathlib/Algebra/Order/Ring/Cast.lean", "Mathlib/Data/TwoPointing.lean", "Mathlib/RingTheory/Polynomial/Content.lean", "Mathlib/LinearAlgebra/Basis.lean", "Mathlib/AlgebraicGeometry/Sites/BigZariski.lean", "Mathlib/RingTheory/Smooth/Basic.lean", "Mathlib/AlgebraicGeometry/PrimeSpectrum/Maximal.lean", "Mathlib/CategoryTheory/Localization/Equivalence.lean", "Mathlib/AlgebraicGeometry/Scheme.lean", "Mathlib/LinearAlgebra/CliffordAlgebra/Inversion.lean", "Mathlib/LinearAlgebra/Matrix/Charpoly/Eigs.lean", "Mathlib/Logic/Basic.lean", "Mathlib/Topology/Category/TopCat/Limits/Konig.lean", "Mathlib/Analysis/NormedSpace/PiTensorProduct/ProjectiveSeminorm.lean", "Mathlib/Data/Set/UnionLift.lean", "Mathlib/Topology/ContinuousFunction/Weierstrass.lean", "Mathlib/RingTheory/MvPolynomial/Symmetric.lean", "Mathlib/Algebra/Ring/CompTypeclasses.lean", "Mathlib/LinearAlgebra/ExteriorAlgebra/Grading.lean", "Mathlib/Tactic/Monotonicity/Lemmas.lean", "Mathlib/CategoryTheory/Limits/Shapes/NormalMono/Equalizers.lean", "Mathlib/Data/Set/Opposite.lean", "Mathlib/Analysis/Normed/Group/BallSphere.lean", "Mathlib/Order/Filter/Ring.lean", "Mathlib/Data/Finsupp/WellFounded.lean", "Mathlib/Combinatorics/SimpleGraph/Regularity/Bound.lean", "Mathlib/Analysis/Convex/SpecificFunctions/Pow.lean", "Mathlib/GroupTheory/Perm/Closure.lean", "Mathlib/NumberTheory/Harmonic/ZetaAsymp.lean", "Mathlib/CategoryTheory/Limits/Shapes/StrongEpi.lean", "Mathlib/Topology/Compactness/SigmaCompact.lean", "Mathlib/Topology/ContinuousFunction/StarOrdered.lean", "Mathlib/Analysis/SpecialFunctions/Log/NegMulLog.lean", "Mathlib/MeasureTheory/Measure/Trim.lean", "Mathlib/Algebra/Module/Prod.lean", "Mathlib/Algebra/Group/Commute/Hom.lean", "Mathlib/GroupTheory/GroupAction/Period.lean", "Mathlib/Algebra/Ring/NegOnePow.lean", "Mathlib/Algebra/Lie/Engel.lean", "Mathlib/LinearAlgebra/DFinsupp.lean", "Mathlib/Order/Filter/Partial.lean", "Mathlib/NumberTheory/LSeries/AbstractFuncEq.lean", "Mathlib/Data/Nat/PrimeFin.lean", "Mathlib/CategoryTheory/Limits/VanKampen.lean", "Mathlib/LinearAlgebra/FreeModule/Finite/Basic.lean", "Mathlib/Init/Control/Lawful.lean", "Mathlib/Tactic/ExistsI.lean", "Mathlib/Order/Irreducible.lean", "Mathlib/LinearAlgebra/Matrix/Hermitian.lean", "Mathlib/CategoryTheory/Elements.lean", "Mathlib/RingTheory/Localization/Ideal.lean", "Mathlib/Geometry/Euclidean/Angle/Unoriented/Affine.lean", "Mathlib/NumberTheory/ModularForms/JacobiTheta/Bounds.lean", "Mathlib/Tactic/Trace.lean", "Mathlib/GroupTheory/GroupAction/FixedPoints.lean", "Mathlib/Algebra/Category/ModuleCat/Free.lean", "Mathlib/Data/Set/Basic.lean", "Mathlib/Analysis/SpecialFunctions/Log/Base.lean", "Mathlib/CategoryTheory/Preadditive/ProjectiveResolution.lean", "Mathlib/Data/Nat/Size.lean", "Mathlib/Data/Sum/Basic.lean", "Mathlib/Topology/Category/CompHaus/Basic.lean", "Mathlib/CategoryTheory/Limits/Lattice.lean", "Mathlib/Algebra/Category/Grp/Abelian.lean", "Mathlib/Topology/ClopenBox.lean", "Mathlib/GroupTheory/Torsion.lean", "Mathlib/Analysis/NormedSpace/BanachSteinhaus.lean", "Mathlib/Tactic/ModCases.lean", "Mathlib/CategoryTheory/Bicategory/Basic.lean", "Mathlib/Analysis/Complex/Circle.lean", "Mathlib/Data/Finset/Piecewise.lean", "Mathlib/Analysis/Calculus/FDeriv/Measurable.lean", "Mathlib/Data/List/Sublists.lean", "Mathlib/Order/Hom/Order.lean", "Mathlib/Order/PrimeIdeal.lean", "Mathlib/Topology/LocalAtTarget.lean", "Mathlib/Tactic/Positivity/Finset.lean", "Mathlib/Topology/LocallyConstant/Algebra.lean", "Mathlib/Data/Sum/Order.lean", "Mathlib/Logic/Equiv/Functor.lean", "Mathlib/Data/Finset/Attr.lean", "Mathlib/FieldTheory/PolynomialGaloisGroup.lean", "Mathlib/RingTheory/Localization/Away/Basic.lean", "Mathlib/Topology/UniformSpace/Equicontinuity.lean", "Mathlib/Algebra/Homology/HomotopyCategory/Shift.lean", "Mathlib/CategoryTheory/Sites/Canonical.lean", "Mathlib/Algebra/Module/Submodule/Ker.lean", "Mathlib/Algebra/DirectSum/Module.lean", "Mathlib/FieldTheory/Finite/Basic.lean", "Mathlib/GroupTheory/Sylow.lean", "Mathlib/Topology/Bornology/Absorbs.lean", "Mathlib/Geometry/Euclidean/Angle/Oriented/Basic.lean", "Mathlib/Logic/Equiv/Array.lean", "Mathlib/CategoryTheory/Functor/KanExtension/Pointwise.lean", "Mathlib/CategoryTheory/Filtered/Basic.lean", "Mathlib/Data/List/Sigma.lean", "Mathlib/Logic/Lemmas.lean", "Mathlib/Algebra/Polynomial/Module/FiniteDimensional.lean", "Mathlib/Algebra/Lie/CartanExists.lean", "Mathlib/NumberTheory/Pell.lean", "Mathlib/Tactic/RSuffices.lean", "Mathlib/Data/Option/NAry.lean", "Mathlib/Topology/Instances/Matrix.lean", "Mathlib/Util/Delaborators.lean", "Mathlib/Order/CompleteBooleanAlgebra.lean", "Mathlib/CategoryTheory/Quotient/Preadditive.lean", "Mathlib/Order/Disjoint.lean", "Mathlib/Algebra/Order/Sub/Prod.lean", "Mathlib/Geometry/Manifold/ConformalGroupoid.lean", "Mathlib/RingTheory/FreeRing.lean", "Mathlib/Algebra/MvPolynomial/PDeriv.lean", "Mathlib/CategoryTheory/Localization/CalculusOfFractions.lean", "Mathlib/Tactic/Explode/Datatypes.lean", "Mathlib/Algebra/Order/Monoid/Units.lean", "Mathlib/GroupTheory/Perm/Finite.lean", "Mathlib/Algebra/Order/Group/Synonym.lean", "Mathlib/Logic/Small/List.lean", "Mathlib/CategoryTheory/Abelian/Injective.lean", "Mathlib/MeasureTheory/Measure/MutuallySingular.lean", "Mathlib/Analysis/SpecialFunctions/Trigonometric/Series.lean", "Mathlib/Data/Real/Archimedean.lean", "Mathlib/Algebra/Order/Module/Algebra.lean", "Mathlib/AlgebraicGeometry/PrimeSpectrum/IsOpenComapC.lean", "Mathlib/Control/Bitraversable/Lemmas.lean", "Mathlib/FieldTheory/IsAlgClosed/Basic.lean", "Mathlib/AlgebraicGeometry/EllipticCurve/DivisionPolynomial/Degree.lean", "Mathlib/CategoryTheory/FiberedCategory/HomLift.lean", "Mathlib/Geometry/RingedSpace/PresheafedSpace/HasColimits.lean", "Mathlib/MeasureTheory/MeasurableSpace/Embedding.lean", "Mathlib/Algebra/Lie/Subalgebra.lean", "Mathlib/RingTheory/EisensteinCriterion.lean", "Mathlib/CategoryTheory/Triangulated/Functor.lean", "Mathlib/Topology/Specialization.lean", "Mathlib/FieldTheory/RatFunc/Basic.lean", "Mathlib/Tactic/Linarith/Verification.lean", "Mathlib/Algebra/Module/Submodule/Range.lean", "Mathlib/CategoryTheory/SingleObj.lean", "Mathlib/Analysis/SpecialFunctions/PolarCoord.lean", "Mathlib/RingTheory/Polynomial/Dickson.lean", "Mathlib/Topology/Order/IsLUB.lean", "Mathlib/Algebra/PEmptyInstances.lean", "Mathlib/NumberTheory/SumFourSquares.lean", "Mathlib/FieldTheory/IsAlgClosed/Spectrum.lean", "Mathlib/Algebra/Group/MinimalAxioms.lean", "Mathlib/Topology/Algebra/UniformField.lean", "Mathlib/GroupTheory/GroupAction/Ring.lean", "Mathlib/Algebra/Algebra/Pi.lean", "Mathlib/Algebra/Order/Kleene.lean", "Mathlib/Topology/Sets/Closeds.lean", "Mathlib/Order/FixedPoints.lean", "Mathlib/RingTheory/Congruence/Basic.lean", "Mathlib/MeasureTheory/Function/AEEqFun.lean", "Mathlib/Algebra/Field/IsField.lean", "Mathlib/Data/Rat/Floor.lean", "Mathlib/CategoryTheory/Triangulated/Pretriangulated.lean", "Mathlib/RingTheory/Polynomial/Eisenstein/IsIntegral.lean", "Mathlib/Topology/Category/CompHaus/Limits.lean", "Mathlib/Topology/TietzeExtension.lean", "Mathlib/Data/Fintype/Order.lean", "Mathlib/Algebra/Ring/Identities.lean", "Mathlib/Algebra/Category/ModuleCat/Biproducts.lean", "Mathlib/CategoryTheory/Monoidal/Limits.lean", "Mathlib/Data/Analysis/Topology.lean", "Mathlib/MeasureTheory/Function/ConditionalExpectation/Unique.lean", "Mathlib/AlgebraicTopology/SimplexCategory.lean", "Mathlib/Algebra/NeZero.lean", "Mathlib/Init/Data/Rat/Basic.lean", "Mathlib/RingTheory/Localization/Module.lean", "Mathlib/Algebra/Category/ModuleCat/Presheaf.lean", "Mathlib/GroupTheory/Subgroup/Saturated.lean", "Mathlib/RingTheory/PowerBasis.lean", "Mathlib/Control/Monad/Writer.lean", "Mathlib/Order/Interval/Set/Image.lean", "Mathlib/AlgebraicGeometry/Restrict.lean", "Mathlib/Data/PFun.lean", "Mathlib/Tactic/Linter/GlobalAttributeIn.lean", "Mathlib/Init/Data/Int/DivMod.lean", "Mathlib/FieldTheory/SplittingField/Construction.lean", "Mathlib/Combinatorics/SetFamily/Shatter.lean", "Mathlib/GroupTheory/Subgroup/Centralizer.lean", "Mathlib/Data/Set/Pointwise/ListOfFn.lean", "Mathlib/Algebra/Order/Nonneg/Field.lean", "Mathlib/Control/Bitraversable/Basic.lean", "Mathlib/CategoryTheory/Sums/Associator.lean", "Mathlib/Computability/Language.lean", "Mathlib/Dynamics/PeriodicPts.lean", "Mathlib/CategoryTheory/Sites/Coherent/ReflectsPreregular.lean", "Mathlib/Analysis/NormedSpace/Units.lean", "Mathlib/Data/Nat/Upto.lean", "Mathlib/CategoryTheory/Limits/FilteredColimitCommutesFiniteLimit.lean", "Mathlib/Geometry/Manifold/MFDeriv/SpecificFunctions.lean", "Mathlib/Topology/MetricSpace/MetricSeparated.lean", "Mathlib/Data/MLList/IO.lean", "Mathlib/Topology/Algebra/Module/Basic.lean", "Mathlib/Algebra/GroupWithZero/Units/Lemmas.lean", "Mathlib/Algebra/Group/Fin.lean", "Mathlib/Analysis/Convex/Cone/InnerDual.lean", "Mathlib/Tactic/WLOG.lean", "Mathlib/NumberTheory/NumberField/Norm.lean", "Mathlib/RingTheory/NonUnitalSubring/Basic.lean", "Mathlib/GroupTheory/SpecificGroups/KleinFour.lean", "Mathlib/Analysis/SpecialFunctions/Complex/Analytic.lean", "Mathlib/MeasureTheory/Group/GeometryOfNumbers.lean", "Mathlib/Order/Hom/Bounded.lean", "Mathlib/Data/Bundle.lean", "Mathlib/Algebra/Homology/DifferentialObject.lean", "Mathlib/MeasureTheory/Covering/BesicovitchVectorSpace.lean", "Mathlib/LinearAlgebra/Matrix/Reindex.lean", "Mathlib/RingTheory/Polynomial/Hermite/Gaussian.lean", "Mathlib/CategoryTheory/Limits/Constructions/Over/Basic.lean", "Mathlib/CategoryTheory/CommSq.lean", "Mathlib/CategoryTheory/Groupoid/Basic.lean", "Mathlib/CategoryTheory/Preadditive/Biproducts.lean", "Mathlib/Algebra/Polynomial/Lifts.lean", "Mathlib/Analysis/Calculus/FDeriv/Symmetric.lean", "Mathlib/CategoryTheory/Monoidal/Types/Coyoneda.lean", "Mathlib/LinearAlgebra/FiniteSpan.lean", "Mathlib/Tactic/Linter/UnusedTactic.lean", "Mathlib/CategoryTheory/Enriched/Basic.lean", "Mathlib/MeasureTheory/Constructions/HaarToSphere.lean", "Mathlib/CategoryTheory/Closed/Cartesian.lean", "Mathlib/CategoryTheory/Monad/Types.lean", "Mathlib/NumberTheory/ClassNumber/AdmissibleAbs.lean", "Mathlib/GroupTheory/Finiteness.lean", "Mathlib/Init/Data/Option/Basic.lean", "Mathlib/NumberTheory/Ostrowski.lean", "Mathlib/MeasureTheory/Measure/Dirac.lean", "Mathlib/RingTheory/Nilpotent/Lemmas.lean", "Mathlib/Init/Data/Prod.lean", "Mathlib/Algebra/Ring/Subsemiring/MulOpposite.lean", "Mathlib/MeasureTheory/Integral/IntervalAverage.lean", "Mathlib/Algebra/Category/CoalgebraCat/Basic.lean", "Mathlib/Algebra/GroupWithZero/WithZero.lean", "Mathlib/AlgebraicGeometry/Morphisms/Basic.lean", "Mathlib/Data/Nat/Digits.lean", "Mathlib/NumberTheory/DirichletCharacter/Basic.lean", "Mathlib/FieldTheory/Minpoly/Field.lean", "Mathlib/Topology/Algebra/Module/Multilinear/Bounded.lean", "Mathlib/AlgebraicTopology/DoldKan/Faces.lean", "Mathlib/Data/Int/Order/Lemmas.lean", "Mathlib/Algebra/Order/Group/TypeTags.lean", "Mathlib/Order/Filter/Pi.lean", "Mathlib/RingTheory/DedekindDomain/SelmerGroup.lean", "Mathlib/NumberTheory/NumberField/Units/Basic.lean", "Mathlib/Geometry/Euclidean/Circumcenter.lean", "Mathlib/RingTheory/MvPolynomial/Ideal.lean", "Mathlib/RingTheory/Polynomial/IntegralNormalization.lean", "Mathlib/Algebra/Order/Monoid/NatCast.lean", "Mathlib/Analysis/Complex/ReImTopology.lean", "Mathlib/RingTheory/Artinian.lean", "Mathlib/Algebra/CharP/Basic.lean", "Mathlib/Lean/Exception.lean", "Mathlib/MeasureTheory/Function/ConditionalExpectation/Real.lean", "Mathlib/Tactic/Cases.lean", "Mathlib/Util/Tactic.lean", "Mathlib/Topology/Sheaves/Stalks.lean", "Mathlib/SetTheory/Ordinal/Basic.lean", "Mathlib/SetTheory/Surreal/Basic.lean", "Mathlib/Topology/Partial.lean", "Mathlib/RingTheory/WittVector/FrobeniusFractionField.lean", "Mathlib/AlgebraicTopology/DoldKan/NCompGamma.lean", "Mathlib/LinearAlgebra/ExteriorAlgebra/Basic.lean", "Mathlib/RingTheory/WittVector/WittPolynomial.lean", "Mathlib/MeasureTheory/Measure/Typeclasses.lean", "Mathlib/Topology/Order/Filter.lean", "Mathlib/Algebra/Order/Group/Instances.lean", "Mathlib/Analysis/Asymptotics/SuperpolynomialDecay.lean", "Mathlib/Analysis/Normed/Group/Tannery.lean", "Mathlib/CategoryTheory/Closed/Functor.lean", "Mathlib/Condensed/Limits.lean", "Mathlib/MeasureTheory/OuterMeasure/Induced.lean", "Mathlib/Algebra/Category/ModuleCat/Sheaf/Quasicoherent.lean", "Mathlib/Algebra/DirectSum/Finsupp.lean", "Mathlib/FieldTheory/Separable.lean", "Mathlib/Topology/ContinuousFunction/ZeroAtInfty.lean", "Mathlib/Probability/ConditionalExpectation.lean", "Mathlib/Init/Data/Int/Order.lean", "Mathlib/Algebra/GCDMonoid/Multiset.lean", "Mathlib/MeasureTheory/Measure/VectorMeasure.lean", "Mathlib/SetTheory/Cardinal/Divisibility.lean", "Mathlib/Combinatorics/SimpleGraph/Coloring.lean", "Mathlib/LinearAlgebra/TensorProduct/Graded/External.lean", "Mathlib/CategoryTheory/EffectiveEpi/Extensive.lean", "Mathlib/Algebra/Order/Monoid/Submonoid.lean", "Mathlib/CategoryTheory/Endofunctor/Algebra.lean", "Mathlib/Algebra/Category/FGModuleCat/Limits.lean", "Mathlib/Algebra/Category/ModuleCat/Presheaf/Pushforward.lean", "Mathlib/Data/Pi/Interval.lean", "Mathlib/Topology/MetricSpace/Equicontinuity.lean", "Mathlib/Algebra/Group/Ext.lean", "Mathlib/Algebra/Group/Subgroup/Finite.lean", "Mathlib/Topology/Sheaves/SheafCondition/PairwiseIntersections.lean", "Mathlib/Data/Fintype/CardEmbedding.lean", "Mathlib/Probability/Kernel/RadonNikodym.lean", "Mathlib/CategoryTheory/EffectiveEpi/RegularEpi.lean", "Mathlib/Algebra/CharP/ExpChar.lean", "Mathlib/CategoryTheory/Category/RelCat.lean", "Mathlib/Data/Finsupp/Lex.lean", "Mathlib/LinearAlgebra/CliffordAlgebra/Prod.lean", "Mathlib/Analysis/NormedSpace/OperatorNorm/NNNorm.lean", "Mathlib/Topology/Algebra/Field.lean", "Mathlib/FieldTheory/RatFunc/Defs.lean", "Mathlib/Combinatorics/SimpleGraph/Basic.lean", "Mathlib/RingTheory/Localization/Integral.lean", "Mathlib/Data/Nat/Totient.lean", "Mathlib/GroupTheory/SpecificGroups/Quaternion.lean", "Mathlib/Algebra/Polynomial/AlgebraMap.lean", "Mathlib/Lean/Meta/CongrTheorems.lean", "Mathlib/Analysis/Analytic/Constructions.lean", "Mathlib/Analysis/Normed/Group/CocompactMap.lean", "Mathlib/Analysis/NormedSpace/Pointwise.lean", "Mathlib/Data/Nat/Choose/Basic.lean", "Mathlib/Topology/Algebra/Module/Alternating/Basic.lean", "Mathlib/RingTheory/RootsOfUnity/Complex.lean", "Mathlib/Analysis/Calculus/ContDiff/Defs.lean", "Mathlib/CategoryTheory/Sites/Grothendieck.lean", "Mathlib/Analysis/Calculus/FDeriv/Comp.lean", "Mathlib/CategoryTheory/Limits/ColimitLimit.lean", "Mathlib/Analysis/SpecialFunctions/Integrals.lean", "Mathlib/ModelTheory/Algebra/Field/Basic.lean", "Mathlib/Tactic/ExtractGoal.lean", "Mathlib/AlgebraicTopology/SplitSimplicialObject.lean", "Mathlib/CategoryTheory/Adjunction/Lifting.lean", "Mathlib/RingTheory/Congruence/Opposite.lean", "Mathlib/CategoryTheory/Category/ULift.lean", "Mathlib/Analysis/Normed/Group/SemiNormedGrp/Completion.lean", "Mathlib/GroupTheory/Archimedean.lean", "Mathlib/Init/Order/LinearOrder.lean", "Mathlib/Algebra/SMulWithZero.lean", "Mathlib/Analysis/LocallyConvex/BalancedCoreHull.lean", "Mathlib/Analysis/MeanInequalities.lean", "Mathlib/Topology/ContinuousFunction/CompactlySupported.lean", "Mathlib/Algebra/GroupWithZero/Prod.lean", "Mathlib/Algebra/Polynomial/Module/Basic.lean", "Mathlib/Analysis/Convolution.lean", "Mathlib/Algebra/Homology/HomotopyCategory/DegreewiseSplit.lean", "Mathlib/Tactic/Says.lean", "Mathlib/MeasureTheory/Measure/Lebesgue/Basic.lean", "Mathlib/Algebra/Order/Ring/Synonym.lean", "Mathlib/Analysis/Distribution/SchwartzSpace.lean", "Mathlib/LinearAlgebra/Matrix/Determinant/Basic.lean", "Mathlib/MeasureTheory/Order/Group/Lattice.lean", "Mathlib/Algebra/Homology/HomologicalComplex.lean", "Mathlib/CategoryTheory/MorphismProperty/Basic.lean", "Mathlib/NumberTheory/Cyclotomic/Gal.lean", "Mathlib/Probability/Process/Adapted.lean", "Mathlib/LinearAlgebra/TensorProduct/Opposite.lean", "Mathlib/Order/Interval/Set/Basic.lean", "Mathlib/Topology/MetricSpace/CauSeqFilter.lean", "Mathlib/Algebra/Group/Center.lean", "Mathlib/Data/Nat/WithBot.lean", "Mathlib/NumberTheory/Bernoulli.lean", "Mathlib/Util/CompileInductive.lean", "Mathlib/MeasureTheory/Constructions/UnitInterval.lean", "Mathlib/Analysis/Calculus/Deriv/Basic.lean", "Mathlib/AlgebraicGeometry/Gluing.lean", "Mathlib/CategoryTheory/EffectiveEpi/Basic.lean", "Mathlib/CategoryTheory/Triangulated/Opposite.lean", "Mathlib/Topology/Homotopy/HSpaces.lean", "Mathlib/CategoryTheory/Abelian/Ext.lean", "Mathlib/CategoryTheory/Sites/Localization.lean", "Mathlib/RingTheory/Flat/Stability.lean", "Mathlib/Algebra/Star/Center.lean", "Mathlib/CategoryTheory/Sites/Coherent/ExtensiveTopology.lean", "Mathlib/LinearAlgebra/Matrix/Orthogonal.lean", "Mathlib/RingTheory/WittVector/MulP.lean", "Mathlib/Data/Rat/BigOperators.lean", "Mathlib/RingTheory/Ideal/IdempotentFG.lean", "Mathlib/AlgebraicGeometry/EllipticCurve/Projective.lean", "Mathlib/Data/Finsupp/Multiset.lean", "Mathlib/Algebra/Order/Ring/WithTop.lean", "Mathlib/CategoryTheory/Comma/Presheaf.lean", "Mathlib/Data/FinEnum.lean", "Mathlib/CategoryTheory/Linear/Basic.lean", "Mathlib/MeasureTheory/Function/SimpleFunc.lean", "Mathlib/LinearAlgebra/Reflection.lean", "Mathlib/Algebra/MvPolynomial/Comap.lean", "Mathlib/Algebra/GroupWithZero/Pi.lean", "Mathlib/Order/Nat.lean", "Mathlib/RingTheory/Ideal/Prod.lean", "Mathlib/Tactic/CC/Addition.lean", "Mathlib/Topology/ContinuousFunction/NonUnitalFunctionalCalculus.lean", "Mathlib/Topology/Filter.lean", "Mathlib/Algebra/Category/ModuleCat/Presheaf/Sheafify.lean", "Mathlib/Data/Part.lean", "Mathlib/Tactic/UnsetOption.lean", "Mathlib/RingTheory/DedekindDomain/Different.lean", "Mathlib/Algebra/Tropical/BigOperators.lean", "Mathlib/Analysis/Calculus/Conformal/NormedSpace.lean", "Mathlib/Algebra/Category/ModuleCat/Sheaf/Limits.lean", "Mathlib/RingTheory/SimpleModule.lean", "Mathlib/RingTheory/Valuation/RamificationGroup.lean", "Mathlib/AlgebraicTopology/TopologicalSimplex.lean", "Mathlib/Algebra/Star/Subalgebra.lean", "Mathlib/Order/Filter/ModEq.lean", "Mathlib/Probability/ConditionalProbability.lean", "Mathlib/RingTheory/WittVector/Verschiebung.lean", "Mathlib/Algebra/GroupWithZero/Units/Basic.lean", "Mathlib/Algebra/Field/Equiv.lean", "Mathlib/Analysis/Calculus/Deriv/Inverse.lean", "Mathlib/Data/FP/Basic.lean", "Mathlib/Topology/Instances/Complex.lean", "Mathlib/Topology/Category/TopCat/Limits/Basic.lean", "Mathlib/Geometry/Euclidean/Inversion/ImageHyperplane.lean", "Mathlib/CategoryTheory/Limits/Pi.lean", "Mathlib/Tactic/ByContra.lean", "Mathlib/Algebra/Homology/Additive.lean", "Mathlib/Analysis/Calculus/ContDiff/Basic.lean", "Mathlib/LinearAlgebra/PiTensorProduct.lean", "Mathlib/RingTheory/Ideal/Over.lean", "Mathlib/Combinatorics/Enumerative/Partition.lean", "Mathlib/Analysis/Calculus/LineDeriv/Measurable.lean", "Mathlib/Combinatorics/SimpleGraph/Triangle/Tripartite.lean", "Mathlib/Order/Category/Semilat.lean", "Mathlib/Topology/Algebra/NormedValued.lean", "Mathlib/Data/Nat/GCD/BigOperators.lean", "Mathlib/Data/List/Duplicate.lean", "Mathlib/Analysis/Calculus/FDeriv/Linear.lean", "Mathlib/Order/SuccPred/Basic.lean", "Mathlib/CategoryTheory/Generator.lean", "Mathlib/FieldTheory/Cardinality.lean", "Mathlib/CategoryTheory/EffectiveEpi/Coproduct.lean", "Mathlib/Geometry/Euclidean/Angle/Unoriented/RightAngle.lean", "Mathlib/Algebra/Module/LinearMap/Polynomial.lean", "Mathlib/Analysis/Analytic/Linear.lean", "Mathlib/Data/Set/Subset.lean", "Mathlib/Tactic/Simps/Basic.lean", "Mathlib/CategoryTheory/Limits/Preserves/Filtered.lean", "Mathlib/CategoryTheory/Localization/Opposite.lean", "Mathlib/Analysis/Calculus/InverseFunctionTheorem/FDeriv.lean", "Mathlib/Topology/PartitionOfUnity.lean", "Mathlib/LinearAlgebra/QuadraticForm/Complex.lean", "Mathlib/Algebra/Order/Monoid/Canonical/Defs.lean", "Mathlib/CategoryTheory/Limits/Indization/IndObject.lean", "Mathlib/ModelTheory/Algebra/Ring/FreeCommRing.lean", "Mathlib/Probability/Process/Filtration.lean", "Mathlib/NumberTheory/LucasPrimality.lean", "Mathlib/MeasureTheory/Group/LIntegral.lean", "Mathlib/LinearAlgebra/Matrix/Charpoly/FiniteField.lean", "Mathlib/Topology/UrysohnsLemma.lean", "Mathlib/Algebra/Order/Field/Basic.lean", "Mathlib/Topology/Homotopy/Product.lean", "Mathlib/NumberTheory/Padics/PadicVal.lean", "Mathlib/Tactic/NormNum/Result.lean", "Mathlib/Algebra/Homology/DerivedCategory/ShortExact.lean", "Mathlib/Order/Interval/Set/OrderEmbedding.lean", "Mathlib/Tactic/ArithMult.lean", "Mathlib/Algebra/Homology/ComplexShapeSigns.lean", "Mathlib/LinearAlgebra/Dimension/Constructions.lean", "Mathlib/Data/List/Sym.lean", "Mathlib/MeasureTheory/OuterMeasure/OfFunction.lean", "Mathlib/Tactic/NormNum/LegendreSymbol.lean", "Mathlib/Topology/Order/PartialSups.lean", "Mathlib/CategoryTheory/Comma/Over.lean", "Mathlib/Data/Finsupp/PWO.lean", "Mathlib/CategoryTheory/FullSubcategory.lean", "Mathlib/Data/Finset/Prod.lean", "Mathlib/Tactic/TypeCheck.lean", "Mathlib/CategoryTheory/Localization/HomEquiv.lean", "Mathlib/Algebra/Polynomial/SpecificDegree.lean", "Mathlib/Data/Finsupp/Antidiagonal.lean", "Mathlib/Mathport/Syntax.lean", "Mathlib/Algebra/Category/AlgebraCat/Basic.lean", "Mathlib/Tactic/Eqns.lean", "Mathlib/Algebra/Associated.lean", "Mathlib/Algebra/Category/ModuleCat/Sheaf.lean", "Mathlib/CategoryTheory/Preadditive/Yoneda/Injective.lean", "Mathlib/MeasureTheory/Constructions/BorelSpace/Metric.lean", "Mathlib/Topology/Homeomorph.lean", "Mathlib/CategoryTheory/Category/Grpd.lean", "Mathlib/Tactic/SuppressCompilation.lean", "Mathlib/Algebra/Polynomial/Roots.lean", "Mathlib/Algebra/Homology/Functor.lean", "Mathlib/Algebra/Ring/BooleanRing.lean", "Mathlib/Combinatorics/SimpleGraph/Regularity/Increment.lean", "Mathlib/CategoryTheory/Adjunction/Comma.lean", "Mathlib/RingTheory/Polynomial/Chebyshev.lean", "Mathlib/Algebra/DualNumber.lean", "Mathlib/CategoryTheory/Abelian/Homology.lean", "Mathlib/RingTheory/AdjoinRoot.lean", "Mathlib/Analysis/NormedSpace/RieszLemma.lean", "Mathlib/Data/Sym/Sym2/Init.lean", "Mathlib/Data/Nat/PSub.lean", "Mathlib/Algebra/Module/Card.lean", "Mathlib/CategoryTheory/Limits/FunctorCategory.lean", "Mathlib/Algebra/Lie/Free.lean", "Mathlib/CategoryTheory/Monoidal/Comon_.lean", "Mathlib/FieldTheory/KrullTopology.lean", "Mathlib/Analysis/SumOverResidueClass.lean", "Mathlib/RingTheory/Finiteness.lean", "Mathlib/Data/List/Forall2.lean", "Mathlib/AlgebraicGeometry/Morphisms/QuasiSeparated.lean", "Mathlib/CategoryTheory/Bicategory/Coherence.lean", "Mathlib/Combinatorics/Colex.lean", "Mathlib/Topology/Homotopy/Path.lean", "Mathlib/LinearAlgebra/Isomorphisms.lean", "Mathlib/Algebra/Order/Field/Defs.lean", "Mathlib/Order/Filter/Bases.lean", "Mathlib/Probability/StrongLaw.lean", "Mathlib/Tactic/CategoryTheory/BicategoryCoherence.lean", "Mathlib/Topology/IsLocalHomeomorph.lean", "Mathlib/MeasureTheory/Integral/IntervalIntegral.lean", "Mathlib/Algebra/BigOperators/Option.lean", "Mathlib/Algebra/DirectSum/Decomposition.lean", "Mathlib/NumberTheory/ADEInequality.lean", "Mathlib/Tactic/NormNum/OfScientific.lean", "Mathlib/Data/Sum/Interval.lean", "Mathlib/RingTheory/PowerSeries/WellKnown.lean", "Mathlib/RingTheory/Ideal/IsPrincipal.lean", "Mathlib/Topology/Category/TopCat/Yoneda.lean", "Mathlib/Topology/FiberBundle/Constructions.lean", "Mathlib/Data/Finset/Slice.lean", "Mathlib/LinearAlgebra/Matrix/PosDef.lean", "Mathlib/MeasureTheory/PiSystem.lean", "Mathlib/Algebra/Homology/HomotopyCategory/MappingCone.lean", "Mathlib/Topology/Algebra/Constructions.lean", "Mathlib/Order/Chain.lean", "Mathlib/Algebra/Group/Subgroup/Order.lean", "Mathlib/Topology/UniformSpace/CompareReals.lean", "Mathlib/Tactic/Widget/SelectInsertParamsClass.lean", "Mathlib/Logic/Equiv/Set.lean", "Mathlib/Algebra/Order/Rearrangement.lean", "Mathlib/Analysis/NormedSpace/Real.lean", "Mathlib/CategoryTheory/Monad/Kleisli.lean", "Mathlib/Geometry/Manifold/PartitionOfUnity.lean", "Mathlib/RingTheory/RingHom/FiniteType.lean", "Mathlib/Algebra/Homology/ShortComplex/ConcreteCategory.lean", "Mathlib/Topology/Category/TopCat/Adjunctions.lean", "Mathlib/Algebra/Module/BigOperators.lean", "Mathlib/LinearAlgebra/AffineSpace/MidpointZero.lean", "Mathlib/CategoryTheory/ComposableArrows.lean", "Mathlib/MeasureTheory/MeasurableSpace/Card.lean", "Mathlib/CategoryTheory/Monoidal/Mod_.lean", "Mathlib/Algebra/Group/Semiconj/Basic.lean", "Mathlib/MeasureTheory/Measure/Stieltjes.lean", "Mathlib/Algebra/Category/Ring/Colimits.lean", "Mathlib/Algebra/Lie/Weights/Cartan.lean", "Mathlib/GroupTheory/FreeAbelianGroupFinsupp.lean", "Mathlib/RingTheory/Flat/EquationalCriterion.lean", "Mathlib/Algebra/Group/InjSurj.lean", "Mathlib/Data/DFinsupp/Notation.lean", "Mathlib/Algebra/GroupWithZero/Basic.lean", "Mathlib/CategoryTheory/Localization/DerivabilityStructure/Constructor.lean", "Mathlib/Geometry/Manifold/MFDeriv/Defs.lean", "Mathlib/MeasureTheory/Function/Egorov.lean", "Mathlib/RingTheory/DedekindDomain/SInteger.lean", "Mathlib/Tactic/TypeStar.lean", "Mathlib/Order/Category/CompleteLat.lean", "Mathlib/NumberTheory/NumberField/FractionalIdeal.lean", "Mathlib/Util/MemoFix.lean", "Mathlib/AlgebraicGeometry/EllipticCurve/Weierstrass.lean", "Mathlib/Data/QPF/Multivariate/Constructions/Quot.lean", "Mathlib/Topology/MetricSpace/HausdorffDimension.lean", "Mathlib/Algebra/Field/Defs.lean", "Mathlib/Topology/Perfect.lean", "Mathlib/Algebra/Module/Submodule/LinearMap.lean", "Mathlib/Geometry/Manifold/Instances/Sphere.lean", "Mathlib/Tactic/Ring/Basic.lean", "Mathlib/Condensed/Module.lean", "Mathlib/Algebra/Star/Free.lean", "Mathlib/Analysis/Convex/Gauge.lean", "Mathlib/Algebra/DirectSum/LinearMap.lean", "Mathlib/Data/Fintype/Prod.lean", "Mathlib/MeasureTheory/Measure/Count.lean", "Mathlib/Tactic/SimpRw.lean", "Mathlib/Logic/Nontrivial/Defs.lean", "Mathlib/Tactic/Widget/Conv.lean", "Mathlib/CategoryTheory/Sites/Coherent/RegularSheaves.lean", "Mathlib/NumberTheory/VonMangoldt.lean", "Mathlib/CategoryTheory/Preadditive/FunctorCategory.lean", "Mathlib/AlgebraicTopology/DoldKan/SplitSimplicialObject.lean", "Mathlib/Tactic/TryThis.lean", "Mathlib/Tactic/CategoryTheory/Elementwise.lean", "Mathlib/Topology/Algebra/InfiniteSum/Order.lean", "Mathlib/Algebra/Group/Prod.lean", "Mathlib/AlgebraicTopology/FundamentalGroupoid/PUnit.lean", "Mathlib/RingTheory/Bialgebra/Basic.lean", "Mathlib/GroupTheory/Perm/Cycle/Factors.lean", "Mathlib/Geometry/Manifold/LocalInvariantProperties.lean", "Mathlib/Tactic/Linter/Lint.lean", "Mathlib/Topology/Category/Profinite/Basic.lean", "Mathlib/Probability/ProbabilityMassFunction/Monad.lean", "Mathlib/Topology/OmegaCompletePartialOrder.lean", "Mathlib/Analysis/NormedSpace/ContinuousAffineMap.lean", "Mathlib/Data/Finsupp/NeLocus.lean", "Mathlib/Data/Complex/ExponentialBounds.lean", "Mathlib/Algebra/Group/Even.lean", "Mathlib/Algebra/Ring/Prod.lean", "Mathlib/Analysis/Calculus/Deriv/Slope.lean", "Mathlib/Init/Data/Fin/Basic.lean", "Mathlib/NumberTheory/MulChar/Basic.lean", "Mathlib/Data/Fin/Basic.lean", "Mathlib/Data/Multiset/Sym.lean", "Mathlib/Data/Set/Defs.lean", "Mathlib/Probability/Kernel/Disintegration/MeasurableStieltjes.lean", "Mathlib/Analysis/Convex/Measure.lean", "Mathlib/Order/Category/BddLat.lean", "Mathlib/Data/PNat/Equiv.lean", "Mathlib/Tactic/NormNum/Prime.lean", "Mathlib/Logic/Hydra.lean", "Mathlib/Algebra/Ring/Ext.lean", "Mathlib/Order/Interval/Set/OrdConnected.lean", "Mathlib/Topology/ContinuousFunction/CocompactMap.lean", "Mathlib/Topology/Category/Profinite/Projective.lean", "Mathlib/Algebra/Order/Interval/Set/Group.lean", "Mathlib/CategoryTheory/Limits/Creates.lean", "Mathlib/Analysis/NormedSpace/Extend.lean", "Mathlib/Algebra/Order/Ring/InjSurj.lean", "Mathlib/LinearAlgebra/Vandermonde.lean", "Mathlib/Tactic/ToAdditive.lean", "Mathlib/SetTheory/Game/Ordinal.lean", "Mathlib/NumberTheory/Wilson.lean", "Mathlib/CategoryTheory/Category/KleisliCat.lean", "Mathlib/Tactic/Measurability.lean", "Mathlib/Data/Finsupp/Basic.lean", "Mathlib/Topology/Separation/NotNormal.lean", "Mathlib/LinearAlgebra/Quotient.lean", "Mathlib/Algebra/Module/Submodule/Bilinear.lean", "Mathlib/CategoryTheory/Adjunction/Limits.lean", "Mathlib/Data/QPF/Multivariate/Constructions/Comp.lean", "Mathlib/CategoryTheory/Limits/Bicones.lean", "Mathlib/Data/Real/GoldenRatio.lean", "Mathlib/Algebra/EuclideanDomain/Instances.lean", "Mathlib/SetTheory/Ordinal/FixedPointApproximants.lean", "Mathlib/RepresentationTheory/Rep.lean", "Mathlib/Combinatorics/Additive/Dissociation.lean", "Mathlib/CategoryTheory/Bicategory/LocallyDiscrete.lean", "Mathlib/Logic/Function/CompTypeclasses.lean", "Mathlib/Tactic/Inhabit.lean", "Mathlib/Algebra/Homology/Embedding/Restriction.lean", "Mathlib/Analysis/NormedSpace/Multilinear/Curry.lean", "Mathlib/Algebra/Order/Sub/Defs.lean", "Mathlib/Algebra/Category/ModuleCat/Differentials/Basic.lean", "Mathlib/Analysis/SpecialFunctions/Trigonometric/InverseDeriv.lean", "Mathlib/CategoryTheory/Groupoid.lean", "Mathlib/GroupTheory/Perm/Option.lean", "Mathlib/Tactic/FunProp/StateList.lean", "Mathlib/Tactic/FunProp.lean", "Mathlib/Data/Fintype/Lattice.lean", "Mathlib/Analysis/SpecialFunctions/Trigonometric/ComplexDeriv.lean", "Mathlib/CategoryTheory/Limits/Comma.lean", "Mathlib/Algebra/Algebra/Defs.lean", "Mathlib/Algebra/Order/AbsoluteValue.lean", "Mathlib/RingTheory/WittVector/MulCoeff.lean", "Mathlib/Tactic/RewriteSearch.lean", "Mathlib/GroupTheory/Submonoid/Inverses.lean", "Mathlib/CategoryTheory/Limits/Shapes/Equivalence.lean", "Mathlib/NumberTheory/DirichletCharacter/Bounds.lean", "Mathlib/GroupTheory/Congruence/Opposite.lean", "Mathlib/CategoryTheory/Limits/Shapes/SplitCoequalizer.lean", "Mathlib/Tactic/CategoryTheory/Slice.lean", "Mathlib/MeasureTheory/Covering/OneDim.lean", "Mathlib/RingTheory/QuotientNoetherian.lean", "Mathlib/CategoryTheory/Sites/NonabelianCohomology/H1.lean", "Mathlib/CategoryTheory/Bicategory/Free.lean", "Mathlib/RingTheory/WittVector/Identities.lean", "Mathlib/CategoryTheory/Closed/Zero.lean", "Mathlib/Data/Set/NAry.lean", "Mathlib/CategoryTheory/Limits/Preserves/Shapes/Equalizers.lean", "Mathlib/LinearAlgebra/SModEq.lean", "Mathlib/Order/Height.lean", "Mathlib/Probability/Distributions/Poisson.lean", "Mathlib/Lean/Name.lean", "Mathlib/Tactic/Recover.lean", "Mathlib/Topology/Algebra/Module/FiniteDimension.lean", "Mathlib/CategoryTheory/MorphismProperty/Factorization.lean", "Mathlib/Data/List/InsertNth.lean", "Mathlib/Topology/Order/Monotone.lean", "Mathlib/Algebra/Module/Projective.lean", "Mathlib/NumberTheory/Cyclotomic/PID.lean", "Mathlib/Analysis/Hofer.lean", "Mathlib/AlgebraicGeometry/Morphisms/ClosedImmersion.lean", "Mathlib/Analysis/NormedSpace/WithLp.lean", "Mathlib/AlgebraicTopology/Nerve.lean", "Mathlib/Data/Finsupp/Fintype.lean", "Mathlib/Geometry/Manifold/ContMDiff/NormedSpace.lean", "Mathlib/LinearAlgebra/BilinearForm/Hom.lean", "Mathlib/Logic/Equiv/Basic.lean", "Mathlib/FieldTheory/Finite/Polynomial.lean", "Mathlib/CategoryTheory/Preadditive/OfBiproducts.lean", "Mathlib/MeasureTheory/Function/SpecialFunctions/Basic.lean", "Mathlib/Tactic/NormNum/Ineq.lean", "Mathlib/Data/Int/AbsoluteValue.lean", "Mathlib/NumberTheory/BernoulliPolynomials.lean", "Mathlib/Analysis/Fourier/PoissonSummation.lean", "Mathlib/CategoryTheory/Idempotents/FunctorExtension.lean", "Mathlib/Algebra/Algebra/NonUnitalHom.lean", "Mathlib/Topology/Category/TopCat/EpiMono.lean", "Mathlib/Tactic/ProxyType.lean", "Mathlib/RingTheory/Ideal/Cotangent.lean", "Mathlib/GroupTheory/Schreier.lean", "Mathlib/Data/DFinsupp/WellFounded.lean", "Mathlib/Tactic/Linter/TextBased.lean", "Mathlib/Order/CompleteLattice.lean", "Mathlib/Analysis/Normed/Group/Constructions.lean", "Mathlib/Analysis/NormedSpace/HomeomorphBall.lean", "Mathlib/Order/Atoms.lean", "Mathlib/Algebra/Category/ModuleCat/ChangeOfRings.lean", "Mathlib/Analysis/NormedSpace/Ray.lean", "Mathlib/Geometry/Euclidean/Angle/Oriented/Affine.lean", "Mathlib/Algebra/Order/GroupWithZero/Synonym.lean", "Mathlib/Algebra/Polynomial/Degree/TrailingDegree.lean", "Mathlib/GroupTheory/FreeGroup/NielsenSchreier.lean", "Mathlib/ModelTheory/DirectLimit.lean", "Mathlib/MeasureTheory/MeasurableSpace/Defs.lean", "Mathlib/Algebra/ContinuedFractions/Computation/Approximations.lean", "Mathlib/Analysis/Asymptotics/SpecificAsymptotics.lean", "Mathlib/Data/Int/Associated.lean", "Mathlib/Data/Rat/Lemmas.lean", "Mathlib/Algebra/Order/ZeroLEOne.lean", "Mathlib/Order/Heyting/Regular.lean", "Mathlib/Data/List/Lex.lean", "Mathlib/GroupTheory/SpecificGroups/Alternating.lean", "Mathlib/Analysis/Calculus/ContDiff/Bounds.lean", "Mathlib/Order/InitialSeg.lean", "Mathlib/Geometry/Euclidean/Basic.lean", "Mathlib/Algebra/Algebra/Hom.lean", "Mathlib/Geometry/RingedSpace/LocallyRingedSpace.lean", "Mathlib/Logic/Equiv/Defs.lean", "Mathlib/LinearAlgebra/Dimension/StrongRankCondition.lean", "Mathlib/Analysis/Convex/Mul.lean", "Mathlib/Data/Nat/Cast/Synonym.lean", "Mathlib/LinearAlgebra/FreeModule/Norm.lean", "Mathlib/AlgebraicGeometry/Modules/Presheaf.lean", "Mathlib/Data/Int/Cast/Lemmas.lean", "Mathlib/Algebra/Order/Interval/Basic.lean", "Mathlib/Algebra/Module/Submodule/Basic.lean", "Mathlib/Analysis/NormedSpace/Basic.lean", "Mathlib/Algebra/Homology/ShortComplex/FunctorEquivalence.lean", "Mathlib/Analysis/NormedSpace/LinearIsometry.lean", "Mathlib/Analysis/SpecialFunctions/Gaussian/GaussianIntegral.lean", "Mathlib/Geometry/Manifold/WhitneyEmbedding.lean", "Mathlib/Algebra/MvPolynomial/Rename.lean", "Mathlib/Order/Filter/Lift.lean", "Mathlib/Probability/Process/PartitionFiltration.lean", "Mathlib/Data/Fintype/BigOperators.lean", "Mathlib/Algebra/Group/Commute/Defs.lean", "Mathlib/Analysis/NormedSpace/Star/Exponential.lean", "Mathlib/Topology/Maps.lean", "Mathlib/Init/Control/Combinators.lean", "Mathlib/Algebra/Module/Submodule/Lattice.lean", "Mathlib/Algebra/Category/Grp/Images.lean", "Mathlib/CategoryTheory/Abelian/Opposite.lean", "Mathlib/Data/Opposite.lean", "Mathlib/MeasureTheory/Function/Floor.lean", "Mathlib/Tactic/SetLike.lean", "Mathlib/Order/Max.lean", "Mathlib/Data/Option/Basic.lean", "Mathlib/Analysis/NormedSpace/FiniteDimension.lean", "Mathlib/Algebra/CharP/LocalRing.lean", "Mathlib/Algebra/Polynomial/CancelLeads.lean", "Mathlib/Analysis/NormedSpace/PiLp.lean", "Mathlib/Algebra/Order/ToIntervalMod.lean", "Mathlib/Data/Fintype/Pi.lean", "Mathlib/Data/Fintype/Option.lean", "Mathlib/MeasureTheory/Decomposition/SignedLebesgue.lean", "Mathlib/Topology/Algebra/Module/LocallyConvex.lean", "Mathlib/Topology/Algebra/UniformGroup.lean", "Mathlib/Analysis/Calculus/FDeriv/Star.lean", "Mathlib/Data/Complex/FiniteDimensional.lean", "Mathlib/Data/Real/ConjExponents.lean", "Mathlib/Topology/ContinuousOn.lean", "Mathlib/Data/Matrix/Reflection.lean", "Mathlib/Topology/MetricSpace/Algebra.lean", "Mathlib/Geometry/Manifold/Sheaf/LocallyRingedSpace.lean", "Mathlib/Algebra/MonoidAlgebra/NoZeroDivisors.lean", "Mathlib/Analysis/NormedSpace/HahnBanach/SeparatingDual.lean", "Mathlib/Analysis/NormedSpace/Star/ContinuousFunctionalCalculus/Order.lean", "Mathlib/CategoryTheory/Category/TwoP.lean", "Mathlib/LinearAlgebra/Matrix/ToLinearEquiv.lean", "Mathlib/Lean/Expr/ReplaceRec.lean", "Mathlib/CategoryTheory/FinCategory/AsType.lean", "Mathlib/Topology/Category/Stonean/Basic.lean", "Mathlib/Topology/Baire/CompleteMetrizable.lean", "Mathlib/Init/Data/Nat/Basic.lean", "Mathlib/Tactic/ApplyAt.lean", "Mathlib/Algebra/DirectSum/Algebra.lean", "Mathlib/GroupTheory/GroupAction/Units.lean", "Mathlib/RingTheory/WittVector/IsPoly.lean", "Mathlib/Geometry/Manifold/ContMDiff/Basic.lean", "Mathlib/Tactic/NormNum/NatSqrt.lean", "Mathlib/Algebra/Module/LinearMap/Basic.lean", "Mathlib/Data/Nat/Fib/Basic.lean", "Mathlib/Algebra/Order/Ring/Nat.lean", "Mathlib/AlgebraicGeometry/StructureSheaf.lean", "Mathlib/Data/Fintype/Sigma.lean", "Mathlib/Topology/Compactness/LocallyCompact.lean", "Mathlib/Analysis/Calculus/ParametricIntervalIntegral.lean", "Mathlib/Algebra/Quandle.lean", "Mathlib/Analysis/Convex/Contractible.lean", "Mathlib/Logic/Equiv/Option.lean", "Mathlib/RepresentationTheory/Action/Basic.lean", "Mathlib/Algebra/Module/Basic.lean", "Mathlib/MeasureTheory/Function/SimpleFuncDense.lean", "Mathlib/Algebra/Field/Basic.lean", "Mathlib/Algebra/Group/Conj.lean", "Mathlib/Algebra/Order/BigOperators/Ring/List.lean", "Mathlib/CategoryTheory/Closed/Types.lean", "Mathlib/MeasureTheory/Function/LpOrder.lean", "Mathlib/Data/Set/Pointwise/BigOperators.lean", "Mathlib/SetTheory/Lists.lean", "Mathlib/Analysis/Convex/Normed.lean", "Mathlib/Algebra/Ring/Divisibility/Lemmas.lean", "Mathlib/Algebra/QuaternionBasis.lean", "Mathlib/Data/Matrix/Block.lean", "Mathlib/Data/Int/Range.lean", "Mathlib/Data/ZMod/Defs.lean", "Mathlib/Combinatorics/SimpleGraph/AdjMatrix.lean", "Mathlib/Algebra/Module/PointwisePi.lean", "Mathlib/Topology/Category/Born.lean", "Mathlib/MeasureTheory/Measure/LevyProkhorovMetric.lean", "Mathlib/Order/Filter/Ker.lean", "Mathlib/Tactic/Abel.lean", "Mathlib/Data/List/Sort.lean", "Mathlib/Algebra/Lie/Nilpotent.lean", "Mathlib/Algebra/DirectSum/Ring.lean", "Mathlib/Analysis/NormedSpace/Extr.lean", "Mathlib/Algebra/Category/ModuleCat/Presheaf/Limits.lean", "Mathlib/FieldTheory/Adjoin.lean", "Mathlib/Probability/Distributions/Gamma.lean", "Mathlib/Algebra/Field/Power.lean", "Mathlib/CategoryTheory/Localization/Composition.lean", "Mathlib/Tactic/Constructor.lean", "Mathlib/RingTheory/OrzechProperty.lean", "Mathlib/Data/Set/Pointwise/Finite.lean", "Mathlib/FieldTheory/PrimitiveElement.lean", "Mathlib/Topology/Clopen.lean", "Mathlib/Algebra/Category/AlgebraCat/Monoidal.lean", "Mathlib/Data/Nat/Cast/WithTop.lean", "Mathlib/Lean/Expr/ExtraRecognizers.lean", "Mathlib/Topology/Category/Profinite/Product.lean", "Mathlib/Tactic/ToLevel.lean", "Mathlib/Algebra/Polynomial/RingDivision.lean", "Mathlib/MeasureTheory/Group/Pointwise.lean", "Mathlib/Data/NNRat/Defs.lean", "Mathlib/Algebra/Order/Field/Pi.lean", "Mathlib/Data/ZMod/Parity.lean", "Mathlib/Tactic/ITauto.lean", "Mathlib/Algebra/GroupWithZero/NeZero.lean", "Mathlib/Geometry/Manifold/Complex.lean", "Mathlib/Data/Set/Prod.lean", "Mathlib/Util/AssertExists.lean", "Mathlib/Order/Bounds/Basic.lean", "Mathlib/AlgebraicGeometry/Morphisms/OpenImmersion.lean", "Mathlib/Algebra/Order/Monoid/Prod.lean", "Mathlib/Algebra/Algebra/Subalgebra/Prod.lean", "Mathlib/Probability/Kernel/Disintegration/Unique.lean", "Mathlib/Tactic/FunProp/Mor.lean", "Mathlib/Tactic/Linarith/Oracle/SimplexAlgorithm.lean", "Mathlib/Algebra/AlgebraicCard.lean", "Mathlib/MeasureTheory/Integral/TorusIntegral.lean", "Mathlib/Data/Nat/Cast/SetInterval.lean", "Mathlib/Logic/Small/Defs.lean", "Mathlib/GroupTheory/GroupAction/Pi.lean", "Mathlib/RingTheory/ReesAlgebra.lean", "Mathlib/Algebra/Order/Interval/Set/Monoid.lean", "Mathlib/Algebra/Lie/Basic.lean", "Mathlib/AlgebraicGeometry/Morphisms/Separated.lean", "Mathlib/Algebra/Order/Field/Subfield.lean", "Mathlib/Analysis/Complex/AbsMax.lean", "Mathlib/RingTheory/MvPolynomial/NewtonIdentities.lean", "Mathlib/Topology/MetricSpace/Completion.lean", "Mathlib/NumberTheory/LSeries/RiemannZeta.lean", "Mathlib/Order/Filter/Ultrafilter.lean", "Mathlib/Algebra/GroupWithZero/Invertible.lean", "Mathlib/Data/Nat/Factorial/DoubleFactorial.lean", "Mathlib/Algebra/Order/Sub/Basic.lean", "Mathlib/Analysis/Fourier/FourierTransformDeriv.lean", "Mathlib/Data/Fin/Tuple/Basic.lean", "Mathlib/Geometry/RingedSpace/LocallyRingedSpace/HasColimits.lean", "Mathlib/Algebra/Category/ModuleCat/FilteredColimits.lean", "Mathlib/SetTheory/Surreal/Dyadic.lean", "Mathlib/Topology/Hom/Open.lean", "Mathlib/Algebra/Group/Subsemigroup/Operations.lean", "Mathlib/Analysis/NormedSpace/UnitizationL1.lean", "Mathlib/Topology/Order/Category/AlexDisc.lean", "Mathlib/Algebra/MvPolynomial/Funext.lean", "Mathlib/CategoryTheory/Localization/CalculusOfFractions/Preadditive.lean", "Mathlib/Algebra/Homology/LocalCohomology.lean", "Mathlib/RingTheory/DedekindDomain/AdicValuation.lean", "Mathlib/Tactic/Positivity/Basic.lean", "Mathlib/Algebra/Regular/SMul.lean", "Mathlib/GroupTheory/GroupAction/Opposite.lean", "Mathlib/Analysis/NormedSpace/OperatorNorm/Mul.lean", "Mathlib/Order/Filter/ListTraverse.lean", "Mathlib/Algebra/Homology/ShortComplex/LeftHomology.lean", "Mathlib/CategoryTheory/Limits/Constructions/WeaklyInitial.lean", "Mathlib/MeasureTheory/Constructions/BorelSpace/Basic.lean", "Mathlib/Analysis/SpecialFunctions/SmoothTransition.lean", "Mathlib/Topology/Order/ScottTopology.lean", "Mathlib/CategoryTheory/Subobject/Lattice.lean", "Mathlib/Analysis/NormedSpace/BallAction.lean", "Mathlib/Analysis/NormedSpace/FunctionSeries.lean", "Mathlib/Data/List/Count.lean", "Mathlib/Topology/ExtremallyDisconnected.lean", "Mathlib/Analysis/Convex/Extrema.lean", "Mathlib/Algebra/CharP/Quotient.lean", "Mathlib/GroupTheory/PushoutI.lean", "Mathlib/Tactic/NormNum/Basic.lean", "Mathlib/CategoryTheory/Shift/SingleFunctors.lean", "Mathlib/NumberTheory/DirichletCharacter/GaussSum.lean", "Mathlib/Data/Finset/Option.lean", "Mathlib/GroupTheory/Coprod/Basic.lean", "Mathlib/ModelTheory/LanguageMap.lean", "Mathlib/CategoryTheory/Sites/SheafHom.lean", "Mathlib/Algebra/Group/Basic.lean", "Mathlib/Algebra/Order/Monoid/Basic.lean", "Mathlib/Analysis/Normed/Group/Lemmas.lean", "Mathlib/CategoryTheory/Preadditive/AdditiveFunctor.lean", "Mathlib/Init/Data/Nat/Lemmas.lean", "Mathlib/Data/Finsupp/ToDFinsupp.lean", "Mathlib/MeasureTheory/Group/Measure.lean", "Mathlib/CategoryTheory/Monoidal/Preadditive.lean", "Mathlib/Data/PEquiv.lean", "Mathlib/GroupTheory/Perm/Support.lean", "Mathlib/Topology/Gluing.lean", "Mathlib/LinearAlgebra/Matrix/Diagonal.lean", "Mathlib/Topology/Order/Basic.lean", "Mathlib/Tactic/Widget/CongrM.lean", "Mathlib/Algebra/Order/Group/Defs.lean", "Mathlib/CategoryTheory/Functor/Trifunctor.lean", "Mathlib/Order/Heyting/Hom.lean", "Mathlib/CategoryTheory/Shift/Opposite.lean", "Mathlib/Data/Set/Pointwise/Iterate.lean", "Mathlib/Mathport/Attributes.lean", "Mathlib/SetTheory/Cardinal/Basic.lean", "Mathlib/Tactic/Linarith/Parsing.lean", "Mathlib/Data/Finite/Basic.lean", "Mathlib/CategoryTheory/Limits/Shapes/ZeroMorphisms.lean", "Mathlib/Order/Category/Frm.lean", "Mathlib/CategoryTheory/Abelian/FunctorCategory.lean", "Mathlib/Tactic/Basic.lean", "Mathlib/Logic/Equiv/PartialEquiv.lean", "Mathlib/Order/UpperLower/Hom.lean", "Mathlib/Analysis/InnerProductSpace/Positive.lean", "Mathlib/FieldTheory/Minpoly/IsIntegrallyClosed.lean", "Mathlib/Geometry/RingedSpace/Basic.lean", "Mathlib/MeasureTheory/Function/LpSeminorm/Trim.lean", "Mathlib/Tactic/FunProp/Elab.lean", "Mathlib/AlgebraicGeometry/GammaSpecAdjunction.lean", "Mathlib/RingTheory/Ideal/QuotientOperations.lean", "Mathlib/Topology/UniformSpace/Ascoli.lean", "Mathlib/Geometry/Manifold/PoincareConjecture.lean", "Mathlib/CategoryTheory/Category/Cat.lean", "Mathlib/MeasureTheory/Integral/Asymptotics.lean", "Mathlib/Tactic/Congr!.lean", "Mathlib/Algebra/Group/Submonoid/Basic.lean", "Mathlib/LinearAlgebra/Charpoly/ToMatrix.lean", "Mathlib/Algebra/Ring/Rat.lean", "Mathlib/RingTheory/IsAdjoinRoot.lean", "Mathlib/Analysis/Quaternion.lean", "Mathlib/Analysis/InnerProductSpace/Spectrum.lean", "Mathlib/Dynamics/Ergodic/AddCircle.lean", "Mathlib/Topology/Sheaves/LocalPredicate.lean", "Mathlib/Algebra/Algebra/Subalgebra/Directed.lean", "Mathlib/CategoryTheory/Abelian/Transfer.lean", "Mathlib/CategoryTheory/Quotient.lean", "Mathlib/Tactic/FieldSimp.lean", "Mathlib/Algebra/Order/CauSeq/Completion.lean", "Mathlib/Data/Finset/PiInduction.lean", "Mathlib/LinearAlgebra/TensorProduct/Finiteness.lean", "Mathlib/Topology/Algebra/Nonarchimedean/Basic.lean", "Mathlib/Algebra/Lie/Character.lean", "Mathlib/Algebra/Module/Submodule/Equiv.lean", "Mathlib/Analysis/Convex/SpecificFunctions/Basic.lean", "Mathlib/LinearAlgebra/ExteriorAlgebra/OfAlternating.lean", "Mathlib/Analysis/NormedSpace/OperatorNorm/NormedSpace.lean", "Mathlib/LinearAlgebra/JordanChevalley.lean", "Mathlib/CategoryTheory/Groupoid/VertexGroup.lean", "Mathlib/Algebra/Group/AddChar.lean", "Mathlib/Topology/Sheaves/SheafCondition/EqualizerProducts.lean", "Mathlib/GroupTheory/Perm/Fin.lean", "Mathlib/Algebra/Homology/TotalComplexSymmetry.lean", "Mathlib/LinearAlgebra/TensorAlgebra/Basis.lean", "Mathlib/Tactic/Nontriviality/Core.lean", "Mathlib/Data/Quot.lean", "Mathlib/MeasureTheory/Integral/CircleTransform.lean", "Mathlib/Order/SupIndep.lean", "Mathlib/Control/ULiftable.lean", "Mathlib/GroupTheory/Frattini.lean", "Mathlib/NumberTheory/Zsqrtd/GaussianInt.lean", "Mathlib/Analysis/NormedSpace/Multilinear/Basic.lean", "Mathlib/CategoryTheory/Action.lean", "Mathlib/Order/Basic.lean", "Mathlib/Combinatorics/SimpleGraph/IncMatrix.lean", "Mathlib/Data/LazyList/Basic.lean", "Mathlib/Data/Rat/Cast/Order.lean", "Mathlib/Algebra/Homology/ConcreteCategory.lean", "Mathlib/CategoryTheory/Preadditive/Opposite.lean", "Mathlib/CategoryTheory/Sites/CoverPreserving.lean", "Mathlib/Algebra/Star/CHSH.lean", "Mathlib/Order/SetNotation.lean", "Mathlib/Algebra/Ring/Action/Subobjects.lean", "Mathlib/Topology/Category/LightProfinite/Limits.lean", "Mathlib/Topology/FiberBundle/Trivialization.lean", "Mathlib/CategoryTheory/Shift/Induced.lean", "Mathlib/Data/DFinsupp/Order.lean", "Mathlib/Analysis/SpecialFunctions/Gamma/Beta.lean", "Mathlib/CategoryTheory/Abelian/Projective.lean", "Mathlib/MeasureTheory/Group/Convolution.lean", "Mathlib/AlgebraicGeometry/Morphisms/FiniteType.lean", "Mathlib/Data/Multiset/Nodup.lean", "Mathlib/Tactic/Widget/CommDiag.lean", "Mathlib/Topology/Algebra/Ring/Ideal.lean", "Mathlib/LinearAlgebra/Basis/Bilinear.lean", "Mathlib/Algebra/Polynomial/Div.lean", "Mathlib/Topology/Algebra/ValuedField.lean", "Mathlib/Algebra/Order/Interval/Multiset.lean", "Mathlib/FieldTheory/SplittingField/IsSplittingField.lean", "Mathlib/LinearAlgebra/SesquilinearForm.lean", "Mathlib/CategoryTheory/Limits/ConeCategory.lean", "Mathlib/Algebra/Periodic.lean", "Mathlib/CategoryTheory/Subobject/MonoOver.lean", "Mathlib/Geometry/Manifold/Instances/UnitsOfNormedAlgebra.lean", "Mathlib/RingTheory/Polynomial/Cyclotomic/Basic.lean", "Mathlib/Algebra/Category/MonCat/FilteredColimits.lean", "Mathlib/Algebra/Divisibility/Units.lean", "Mathlib/Init/Data/Nat/GCD.lean", "Mathlib/NumberTheory/LSeries/Basic.lean", "Mathlib/Tactic/PushNeg.lean", "Mathlib/Data/Nat/Cast/Basic.lean", "Mathlib/CategoryTheory/Groupoid/Subgroupoid.lean", "Mathlib/Algebra/Lie/Weights/Linear.lean", "Mathlib/Data/Fintype/Basic.lean", "Mathlib/Algebra/Ring/Commute.lean", "Mathlib/Analysis/BoxIntegral/Partition/Tagged.lean", "Mathlib/Algebra/Ring/MinimalAxioms.lean", "Mathlib/Analysis/SpecialFunctions/Pow/Continuity.lean", "Mathlib/Analysis/Matrix.lean", "Mathlib/MeasureTheory/Measure/NullMeasurable.lean", "Mathlib/Algebra/Module/Defs.lean", "Mathlib/Geometry/Manifold/Sheaf/Basic.lean", "Mathlib/Lean/Elab/Term.lean", "Mathlib/MeasureTheory/Measure/DiracProba.lean", "Mathlib/Algebra/Order/Ring/Canonical.lean", "Mathlib/LinearAlgebra/TensorProduct/Tower.lean", "Mathlib/Init/Classes/Order.lean", "Mathlib/Order/Category/HeytAlg.lean", "Mathlib/CategoryTheory/MorphismProperty/Limits.lean", "Mathlib/CategoryTheory/Triangulated/Subcategory.lean", "Mathlib/Order/Monotone/Union.lean", "Mathlib/Geometry/Manifold/VectorBundle/FiberwiseLinear.lean", "Mathlib/Condensed/Equivalence.lean", "Mathlib/Topology/Order/DenselyOrdered.lean", "Mathlib/Data/Fintype/Vector.lean", "Mathlib/Tactic/Convert.lean", "Mathlib/CategoryTheory/Monoidal/Discrete.lean", "Mathlib/CategoryTheory/Products/Bifunctor.lean", "Mathlib/RingTheory/ChainOfDivisors.lean", "Mathlib/LinearAlgebra/QuadraticForm/Isometry.lean", "Mathlib/Tactic/Widget/SelectPanelUtils.lean", "Mathlib/Analysis/Calculus/IteratedDeriv/Lemmas.lean", "Mathlib/Geometry/Manifold/Sheaf/Smooth.lean", "Mathlib/CategoryTheory/Limits/Constructions/LimitsOfProductsAndEqualizers.lean", "Mathlib/CategoryTheory/Preadditive/Projective.lean", "Mathlib/Algebra/Homology/HomotopyCategory/Triangulated.lean", "Mathlib/Analysis/Analytic/RadiusLiminf.lean", "Mathlib/Algebra/Ring/Centralizer.lean", "Mathlib/CategoryTheory/GradedObject/Trifunctor.lean", "Mathlib/MeasureTheory/Category/MeasCat.lean", "Mathlib/Algebra/Homology/HomotopyCofiber.lean", "Mathlib/Algebra/Homology/HomologicalBicomplex.lean", "Mathlib/FieldTheory/Galois.lean", "Mathlib/CategoryTheory/Abelian/NonPreadditive.lean", "Mathlib/AlgebraicGeometry/Morphisms/Constructors.lean", "Mathlib/Topology/MetricSpace/ProperSpace.lean", "Mathlib/Algebra/Jordan/Basic.lean", "Mathlib/RepresentationTheory/Action/Monoidal.lean", "Mathlib/Algebra/Order/Positive/Field.lean", "Mathlib/Order/Filter/ZeroAndBoundedAtFilter.lean", "Mathlib/Data/Set/Sigma.lean", "Mathlib/Data/List/Iterate.lean", "Mathlib/Order/PartialSups.lean", "Mathlib/Topology/Instances/Discrete.lean", "Mathlib/Topology/Compactness/Compact.lean", "Mathlib/Algebra/Group/Subsemigroup/Basic.lean", "Mathlib/LinearAlgebra/Dimension/LinearMap.lean", "Mathlib/Combinatorics/HalesJewett.lean", "Mathlib/Algebra/Lie/Solvable.lean", "Mathlib/GroupTheory/GroupAction/BigOperators.lean", "Mathlib/NumberTheory/Liouville/Measure.lean", "Mathlib/Lean/Expr/Basic.lean", "Mathlib/GroupTheory/Perm/Sign.lean", "Mathlib/MeasureTheory/Function/StronglyMeasurable/Lp.lean", "Mathlib/Tactic/Lift.lean", "Mathlib/GroupTheory/GroupAction/FixingSubgroup.lean", "Mathlib/Algebra/Algebra/Opposite.lean", "Mathlib/CategoryTheory/Limits/Constructions/FiniteProductsOfBinaryProducts.lean", "Mathlib/Algebra/Group/Centralizer.lean", "Mathlib/Algebra/Algebra/Bilinear.lean", "Mathlib/Algebra/BigOperators/Group/Finset.lean", "Mathlib/Data/Sigma/Lex.lean", "Mathlib/Tactic/CC/Lemmas.lean", "Mathlib/Topology/Algebra/Group/TopologicalAbelianization.lean", "Mathlib/RingTheory/Localization/AsSubring.lean", "Mathlib/Algebra/Polynomial/Derivative.lean", "Mathlib/GroupTheory/Perm/ViaEmbedding.lean", "Mathlib/LinearAlgebra/Dimension/Localization.lean", "Mathlib/Data/QPF/Univariate/Basic.lean", "Mathlib/Algebra/Homology/Homotopy.lean", "Mathlib/Analysis/Normed/Group/ControlledClosure.lean", "Mathlib/Algebra/Order/BigOperators/Group/Finset.lean", "Mathlib/CategoryTheory/Preadditive/Injective.lean", "Mathlib/GroupTheory/Subsemigroup/Centralizer.lean", "Mathlib/Order/Filter/Extr.lean", "Mathlib/RingTheory/Ideal/Quotient.lean", "Mathlib/Algebra/Polynomial/HasseDeriv.lean", "Mathlib/CategoryTheory/Limits/Filtered.lean", "Mathlib/Algebra/GroupWithZero/Units/Equiv.lean", "Mathlib/Analysis/Calculus/LocalExtr/Basic.lean", "Mathlib/Combinatorics/Quiver/Covering.lean", "Mathlib/LinearAlgebra/Matrix/FiniteDimensional.lean", "Mathlib/MeasureTheory/Constructions/BorelSpace/ContinuousLinearMap.lean", "Mathlib/RingTheory/Adjoin/Basic.lean", "Mathlib/RingTheory/DedekindDomain/Dvr.lean", "Mathlib/Analysis/Fourier/Inversion.lean", "Mathlib/Topology/MetricSpace/Polish.lean", "Mathlib/Data/Rat/Defs.lean", "Mathlib/LinearAlgebra/CliffordAlgebra/BaseChange.lean", "Mathlib/CategoryTheory/Sites/Coherent/CoherentTopology.lean", "Mathlib/Data/QPF/Multivariate/Constructions/Prj.lean", "Mathlib/Util/Time.lean", "Mathlib/Topology/Order/LeftRightNhds.lean", "Mathlib/Topology/Instances/TrivSqZeroExt.lean", "Mathlib/Analysis/Normed/Group/InfiniteSum.lean", "Mathlib/AlgebraicGeometry/AffineScheme.lean", "Mathlib/Analysis/Normed/MulAction.lean", "Mathlib/LinearAlgebra/Matrix/MvPolynomial.lean", "Mathlib/NumberTheory/LSeries/Deriv.lean", "Mathlib/Topology/ContinuousFunction/UniqueCFC.lean", "Mathlib/Algebra/MonoidAlgebra/Degree.lean", "Mathlib/Algebra/QuadraticDiscriminant.lean", "Mathlib/CategoryTheory/Abelian/Refinements.lean", "Mathlib/Analysis/Calculus/TangentCone.lean", "Mathlib/Algebra/MonoidAlgebra/Grading.lean", "Mathlib/Data/Real/Pi/Bounds.lean", "Mathlib/Data/Set/Pointwise/SMul.lean", "Mathlib/Geometry/Manifold/VectorBundle/Basic.lean", "Mathlib/Order/CountableDenseLinearOrder.lean", "Mathlib/Probability/Variance.lean", "Mathlib/Algebra/Polynomial/Splits.lean", "Mathlib/Algebra/Module/LocalizedModuleIntegers.lean", "Mathlib/Data/MLList/DepthFirst.lean", "Mathlib/NumberTheory/Cyclotomic/CyclotomicCharacter.lean", "Mathlib/Topology/Inseparable.lean", "Mathlib/Logic/Relator.lean", "Mathlib/Data/Int/Log.lean", "Mathlib/Dynamics/OmegaLimit.lean", "Mathlib/Analysis/NormedSpace/Star/Spectrum.lean", "Mathlib/GroupTheory/FiniteAbelian.lean", "Mathlib/Order/Hom/Basic.lean", "Mathlib/LinearAlgebra/Eigenspace/Basic.lean", "Mathlib/Data/Rbtree/Basic.lean", "Mathlib/FieldTheory/Normal.lean", "Mathlib/Geometry/Euclidean/PerpBisector.lean", "Mathlib/Algebra/Algebra/Operations.lean", "Mathlib/Topology/Metrizable/Urysohn.lean", "Mathlib/Algebra/Lie/UniversalEnveloping.lean", "Mathlib/Topology/UniformSpace/Separation.lean", "Mathlib/MeasureTheory/Integral/Average.lean", "Mathlib/Analysis/Complex/HalfPlane.lean", "Mathlib/Combinatorics/SimpleGraph/Trails.lean", "Mathlib/Data/Finset/Sups.lean", "Mathlib/Data/Vector/MapLemmas.lean", "Mathlib/MeasureTheory/Function/UniformIntegrable.lean", "Mathlib/Tactic/NoncommRing.lean", "Mathlib/Algebra/Homology/Localization.lean", "Mathlib/Combinatorics/Additive/Energy.lean", "Mathlib/LinearAlgebra/Multilinear/FiniteDimensional.lean", "Mathlib/NumberTheory/Bertrand.lean", "Mathlib/NumberTheory/Liouville/Residual.lean", "Mathlib/CategoryTheory/Limits/Constructions/BinaryProducts.lean", "Mathlib/RingTheory/FractionalIdeal/Operations.lean", "Mathlib/Probability/Kernel/Invariance.lean", "Mathlib/Order/Filter/Subsingleton.lean", "Mathlib/SetTheory/Ordinal/CantorNormalForm.lean", "Mathlib/CategoryTheory/Limits/Shapes/RegularMono.lean", "Mathlib/RingTheory/Prime.lean", "Mathlib/LinearAlgebra/Matrix/Charpoly/Univ.lean", "Mathlib/Topology/Defs/Basic.lean", "Mathlib/Algebra/Category/ModuleCat/Kernels.lean", "Mathlib/Data/Int/Lemmas.lean", "Mathlib/Analysis/RCLike/Lemmas.lean", "Mathlib/RingTheory/Polynomial/GaussLemma.lean", "Mathlib/Analysis/Convex/Strong.lean", "Mathlib/FieldTheory/Minpoly/MinpolyDiv.lean", "Mathlib/CategoryTheory/Limits/Shapes/Pullbacks.lean", "Mathlib/RingTheory/Derivation/ToSquareZero.lean", "Mathlib/Order/Category/PartOrd.lean", "Mathlib/Algebra/Algebra/NonUnitalSubalgebra.lean", "Mathlib/CategoryTheory/Closed/Ideal.lean", "Mathlib/Tactic/LiftLets.lean", "Mathlib/CategoryTheory/Limits/Constructions/Pullbacks.lean", "Mathlib/Tactic/Check.lean", "Mathlib/RingTheory/IntegralDomain.lean", "Mathlib/Algebra/Category/Grp/Zero.lean", "Mathlib/Algebra/GroupWithZero/ULift.lean", "Mathlib/Tactic/Observe.lean", "Mathlib/Algebra/Category/MonCat/Colimits.lean", "Mathlib/LinearAlgebra/RootSystem/Defs.lean", "Mathlib/Algebra/Order/Ring/Basic.lean", "Mathlib/Order/GaloisConnection.lean", "Mathlib/LinearAlgebra/CliffordAlgebra/CategoryTheory.lean", "Mathlib/RingTheory/Ideal/Norm.lean", "Mathlib/InformationTheory/Hamming.lean", "Mathlib/Algebra/Module/Zlattice/Covolume.lean", "Mathlib/Topology/Algebra/Group/Compact.lean", "Mathlib/GroupTheory/Perm/DomMulAct.lean", "Mathlib/MeasureTheory/Function/ContinuousMapDense.lean", "Mathlib/MeasureTheory/Constructions/BorelSpace/Metrizable.lean", "Mathlib/Topology/Homotopy/HomotopyGroup.lean", "Mathlib/Analysis/NormedSpace/AddTorsorBases.lean", "Mathlib/Analysis/Analytic/CPolynomial.lean", "Mathlib/Topology/Algebra/InfiniteSum/Ring.lean", "Mathlib/CategoryTheory/Bicategory/SingleObj.lean", "Mathlib/Deprecated/Subfield.lean", "Mathlib/SetTheory/Cardinal/PartENat.lean", "Mathlib/Init/Logic.lean", "Mathlib/Analysis/Convex/KreinMilman.lean", "Mathlib/CategoryTheory/Adjunction/Evaluation.lean", "Mathlib/MeasureTheory/Function/SpecialFunctions/Inner.lean", "Mathlib/Topology/Instances/AddCircle.lean", "Mathlib/CategoryTheory/EffectiveEpi/Comp.lean", "Mathlib/Algebra/Category/Ring/Limits.lean", "Mathlib/CategoryTheory/Shift/Quotient.lean", "Mathlib/Data/Nat/ChineseRemainder.lean", "Mathlib/LinearAlgebra/Matrix/Block.lean", "Mathlib/Analysis/SpecialFunctions/Trigonometric/Basic.lean", "Mathlib/Order/ULift.lean", "Mathlib/Topology/MetricSpace/Isometry.lean", "Mathlib/Util/TermBeta.lean", "Mathlib/Data/Nat/Factorization/Basic.lean", "Mathlib/Topology/Order/MonotoneContinuity.lean", "Mathlib/Algebra/Order/Hom/Monoid.lean", "Mathlib/CategoryTheory/Limits/Shapes/SingleObj.lean", "Mathlib/Topology/MetricSpace/PartitionOfUnity.lean", "Mathlib/Tactic/ArithMult/Init.lean", "Mathlib/CategoryTheory/Galois/Basic.lean", "Mathlib/CategoryTheory/Sites/Coverage.lean", "Mathlib/Data/Matrix/PEquiv.lean", "Mathlib/Topology/MetricSpace/Pseudo/Constructions.lean", "Mathlib/Algebra/Module/Torsion.lean", "Mathlib/Topology/Order/MonotoneConvergence.lean", "Mathlib/RingTheory/ZMod.lean", "Mathlib/Analysis/SpecialFunctions/Exponential.lean", "Mathlib/RingTheory/Kaehler/Polynomial.lean", "Mathlib/Tactic/MoveAdd.lean", "Mathlib/RingTheory/Ideal/Operations.lean", "Mathlib/Topology/LocallyConstant/Basic.lean", "Mathlib/RingTheory/HahnSeries/PowerSeries.lean", "Mathlib/LinearAlgebra/TensorProduct/Basis.lean", "Mathlib/GroupTheory/GroupAction/Defs.lean", "Mathlib/Topology/Category/Profinite/EffectiveEpi.lean", "Mathlib/Tactic/FunProp/Decl.lean", "Mathlib/Order/Filter/CardinalInter.lean", "Mathlib/Data/DList/Basic.lean", "Mathlib/AlgebraicGeometry/ProjectiveSpectrum/StructureSheaf.lean", "Mathlib/Data/Num/Basic.lean", "Mathlib/Data/List/Cycle.lean", "Mathlib/Algebra/Star/Module.lean", "Mathlib/Geometry/Manifold/ChartedSpace.lean", "Mathlib/RingTheory/GradedAlgebra/HomogeneousLocalization.lean", "Mathlib/GroupTheory/Perm/Cycle/PossibleTypes.lean", "Mathlib/Data/Set/Image.lean", "Mathlib/CategoryTheory/Monoidal/Center.lean", "Mathlib/CategoryTheory/Category/Preorder.lean", "Mathlib/LinearAlgebra/Matrix/Charpoly/Basic.lean", "Mathlib/MeasureTheory/Function/L1Space.lean", "Mathlib/Order/Category/FinBoolAlg.lean", "Mathlib/Algebra/Group/Equiv/Basic.lean", "Mathlib/Tactic/ReduceModChar/Ext.lean", "Mathlib/Algebra/Group/Int.lean", "Mathlib/CategoryTheory/Adjunction/Reflective.lean", "Mathlib/CategoryTheory/Closed/FunctorCategory.lean", "Mathlib/Combinatorics/Quiver/ConnectedComponent.lean", "Mathlib/Data/Int/Cast/Basic.lean", "Mathlib/LinearAlgebra/QuadraticForm/QuadraticModuleCat.lean", "Mathlib/Analysis/NormedSpace/IndicatorFunction.lean", "Mathlib/Topology/Instances/Int.lean", "Mathlib/GroupTheory/GroupAction/Support.lean", "Mathlib/ModelTheory/ElementarySubstructures.lean", "Mathlib/Order/Category/LinOrd.lean", "Mathlib/Init/Core.lean", "Mathlib/Topology/MetricSpace/Infsep.lean", "Mathlib/Data/List/NatAntidiagonal.lean", "Mathlib/Tactic/Continuity.lean", "Mathlib/CategoryTheory/Localization/LocalizerMorphism.lean", "Mathlib/CategoryTheory/Preadditive/Yoneda/Projective.lean", "Mathlib/Algebra/TrivSqZeroExt.lean", "Mathlib/RingTheory/Coprime/Basic.lean", "Mathlib/Geometry/RingedSpace/PresheafedSpace/Gluing.lean", "Mathlib/Analysis/Convex/Cone/Closure.lean", "Mathlib/Tactic/NormNum/NatFib.lean", "Mathlib/CategoryTheory/ConcreteCategory/EpiMono.lean", "Mathlib/CategoryTheory/Limits/Final.lean", "Mathlib/CategoryTheory/Localization/CalculusOfFractions/Fractions.lean", "Mathlib/LinearAlgebra/Prod.lean", "Mathlib/Computability/Ackermann.lean", "Mathlib/Algebra/Ring/ULift.lean", "Mathlib/CategoryTheory/DifferentialObject.lean", "Mathlib/Topology/Sets/Compacts.lean", "Mathlib/Data/Nat/GCD/Basic.lean", "Mathlib/Data/Rel.lean", "Mathlib/AlgebraicGeometry/Modules/Sheaf.lean", "Mathlib/Analysis/BoxIntegral/Partition/Additive.lean", "Mathlib/CategoryTheory/PathCategory.lean", "Mathlib/Analysis/Convex/SpecificFunctions/Deriv.lean", "Mathlib/CategoryTheory/EffectiveEpi/Preserves.lean", "Mathlib/Algebra/Group/Subgroup/ZPowers.lean", "Mathlib/Algebra/Field/ULift.lean", "Mathlib/Algebra/Homology/ShortComplex/Abelian.lean", "Mathlib/RingTheory/Ideal/MinimalPrime.lean", "Mathlib/Data/Nat/Cast/Commute.lean", "Mathlib/Combinatorics/Enumerative/Catalan.lean", "Mathlib/LinearAlgebra/AffineSpace/AffineMap.lean", "Mathlib/Algebra/Homology/ShortComplex/Basic.lean", "Mathlib/CategoryTheory/ConcreteCategory/Basic.lean", "Mathlib/Topology/Order/ProjIcc.lean", "Mathlib/Algebra/Star/Pointwise.lean", "Mathlib/CategoryTheory/Sites/Sheafification.lean", "Mathlib/RingTheory/MvPowerSeries/Trunc.lean", "Mathlib/Computability/ContextFreeGrammar.lean", "Mathlib/SetTheory/Game/Nim.lean", "Mathlib/Analysis/BoxIntegral/Integrability.lean", "Mathlib/Topology/Algebra/Order/Field.lean", "Mathlib/LinearAlgebra/CliffordAlgebra/Even.lean", "Mathlib/Control/Monad/Cont.lean", "Mathlib/Topology/ContinuousFunction/Polynomial.lean", "Mathlib/Algebra/Category/ModuleCat/Projective.lean", "Mathlib/Data/Multiset/Powerset.lean", "Mathlib/Algebra/Ring/Subring/Pointwise.lean", "Mathlib/RingTheory/WittVector/Isocrystal.lean", "Mathlib/Data/Nat/SqrtNormNum.lean", "Mathlib/RingTheory/Localization/Basic.lean", "Mathlib/CategoryTheory/Monoidal/Subcategory.lean", "Mathlib/CategoryTheory/Monoidal/OfHasFiniteProducts.lean", "Mathlib/Topology/Bornology/Basic.lean", "Mathlib/Topology/Algebra/InfiniteSum/Module.lean", "Mathlib/Topology/EMetricSpace/Paracompact.lean", "Mathlib/CategoryTheory/GradedObject/Bifunctor.lean", "Mathlib/Data/ZMod/Module.lean", "Mathlib/Order/Bounded.lean", "Mathlib/RingTheory/Nakayama.lean", "Mathlib/Analysis/Normed/Order/UpperLower.lean", "Mathlib/CategoryTheory/Monoidal/Rigid/Basic.lean", "Mathlib/Probability/Kernel/WithDensity.lean", "Mathlib/Analysis/SpecialFunctions/Trigonometric/Arctan.lean", "Mathlib/Tactic/IrreducibleDef.lean", "Mathlib/Algebra/Group/Submonoid/MulOpposite.lean", "Mathlib/Tactic/GeneralizeProofs.lean", "Mathlib/Topology/Defs/Filter.lean", "Mathlib/Order/Filter/FilterProduct.lean", "Mathlib/Data/Nat/Choose/Dvd.lean", "Mathlib/Algebra/Category/Ring/Instances.lean", "Mathlib/Data/List/EditDistance/Estimator.lean", "Mathlib/Algebra/Homology/QuasiIso.lean", "Mathlib/Algebra/Algebra/Tower.lean", "Mathlib/FieldTheory/Extension.lean", "Mathlib/Computability/AkraBazzi/GrowsPolynomially.lean", "Mathlib/Data/Set/Pointwise/Basic.lean", "Mathlib/Analysis/NormedSpace/Star/Unitization.lean", "Mathlib/Algebra/Order/CompleteField.lean", "Mathlib/Analysis/SpecialFunctions/Complex/Log.lean", "Mathlib/MeasureTheory/Measure/Haar/NormedSpace.lean", "Mathlib/Algebra/Category/ModuleCat/Monoidal/Basic.lean", "Mathlib/Topology/Algebra/Nonarchimedean/Completion.lean", "Mathlib/Order/ModularLattice.lean", "Mathlib/Data/Nat/Cast/Defs.lean", "Mathlib/Data/Bool/AllAny.lean", "Mathlib/CategoryTheory/Sites/IsSheafFor.lean", "Mathlib/CategoryTheory/PUnit.lean", "Mathlib/Data/ENNReal/Real.lean", "Mathlib/RingTheory/GradedAlgebra/Noetherian.lean", "Mathlib/Condensed/Basic.lean", "Mathlib/Data/Finset/NatAntidiagonal.lean", "Mathlib/Data/List/Permutation.lean", "Mathlib/Algebra/BigOperators/NatAntidiagonal.lean", "Mathlib/Data/FunLike/Equiv.lean", "Mathlib/Data/Set/Accumulate.lean", "Mathlib/GroupTheory/Perm/Subgroup.lean", "Mathlib/RingTheory/Multiplicity.lean", "Mathlib/RingTheory/Valuation/Basic.lean", "Mathlib/LinearAlgebra/TensorProduct/Vanishing.lean", "Mathlib/Topology/Category/UniformSpace.lean", "Mathlib/LinearAlgebra/Dimension/Basic.lean", "Mathlib/MeasureTheory/Integral/SetIntegral.lean", "Mathlib/Topology/Algebra/Module/UniformConvergence.lean", "Mathlib/Algebra/Homology/ModuleCat.lean", "Mathlib/CategoryTheory/Shift/Localization.lean", "Mathlib/Topology/Order/Bounded.lean", "Mathlib/CategoryTheory/Monad/Monadicity.lean", "Mathlib/CategoryTheory/Monad/Algebra.lean", "Mathlib/Order/LatticeIntervals.lean", "Mathlib/Order/MinMax.lean", "Mathlib/MeasureTheory/Integral/VitaliCaratheodory.lean", "Mathlib/MeasureTheory/Measure/Lebesgue/VolumeOfBalls.lean", "Mathlib/Topology/Sheaves/LocallySurjective.lean", "Mathlib/MeasureTheory/Measure/WithDensityFinite.lean", "Mathlib/Logic/Denumerable.lean", "Mathlib/GroupTheory/SemidirectProduct.lean", "Mathlib/CategoryTheory/Comma/StructuredArrow.lean", "Mathlib/Analysis/Analytic/Uniqueness.lean", "Mathlib/AlgebraicTopology/DoldKan/Compatibility.lean", "Mathlib/Analysis/NormedSpace/ContinuousLinearMap.lean", "Mathlib/CategoryTheory/Abelian/Basic.lean", "Mathlib/CategoryTheory/Monoidal/Skeleton.lean", "Mathlib/Data/Set/Semiring.lean", "Mathlib/CategoryTheory/Limits/Preserves/Limits.lean", "Mathlib/Order/Antisymmetrization.lean", "Mathlib/Analysis/Calculus/BumpFunction/InnerProduct.lean", "Mathlib/CategoryTheory/GradedObject/Monoidal.lean", "Mathlib/Data/MLList/Split.lean", "Mathlib/Algebra/ContinuedFractions/ContinuantsRecurrence.lean", "Mathlib/CategoryTheory/Preadditive/Schur.lean", "Mathlib/Analysis/NormedSpace/QuaternionExponential.lean", "Mathlib/NumberTheory/ModularForms/EisensteinSeries/Basic.lean", "Mathlib/Analysis/Convex/StrictConvexSpace.lean", "Mathlib/RingTheory/WittVector/StructurePolynomial.lean", "Mathlib/Analysis/NormedSpace/AddTorsor.lean", "Mathlib/Data/Rbmap/Basic.lean", "Mathlib/GroupTheory/Coset.lean", "Mathlib/Init/Data/List/Instances.lean", "Mathlib/Data/Set/Pairwise/Basic.lean", "Mathlib/Analysis/NormedSpace/OperatorNorm/Completeness.lean", "Mathlib/Analysis/SpecialFunctions/Trigonometric/ArctanDeriv.lean", "Mathlib/Computability/Partrec.lean", "Mathlib/Topology/Algebra/Module/Cardinality.lean", "Mathlib/Combinatorics/SimpleGraph/Ends/Properties.lean", "Mathlib/Order/Filter/Archimedean.lean", "Mathlib/Algebra/BigOperators/Pi.lean", "Mathlib/AlgebraicTopology/FundamentalGroupoid/Basic.lean", "Mathlib/Logic/Equiv/Pairwise.lean", "Mathlib/Probability/Kernel/Disintegration/Density.lean", "Mathlib/Topology/DiscreteQuotient.lean", "Mathlib/Data/Set/Pointwise/Interval.lean", "Mathlib/Topology/MetricSpace/IsometricSMul.lean", "Mathlib/Combinatorics/SimpleGraph/Triangle/Basic.lean", "Mathlib/Algebra/Order/Monoid/OrderDual.lean", "Mathlib/Analysis/NormedSpace/DualNumber.lean", "Mathlib/Topology/Sheaves/SheafCondition/Sites.lean", "Mathlib/Geometry/Manifold/VectorBundle/Hom.lean", "Mathlib/Analysis/Calculus/LineDeriv/IntegrationByParts.lean", "Mathlib/Condensed/Light/Explicit.lean", "Mathlib/RingTheory/OreLocalization/Basic.lean", "Mathlib/Data/Nat/Pairing.lean", "Mathlib/Condensed/Light/Basic.lean", "Mathlib/CategoryTheory/Thin.lean", "Mathlib/Tactic/Linarith/Frontend.lean", "Mathlib/Analysis/Calculus/FDeriv/Basic.lean", "Mathlib/Combinatorics/SimpleGraph/ConcreteColorings.lean", "Mathlib/Data/List/EditDistance/Bounds.lean", "Mathlib/Data/PNat/Basic.lean", "Mathlib/GroupTheory/CommutingProbability.lean", "Mathlib/RingTheory/Polynomial/SeparableDegree.lean", "Mathlib/Tactic/Relation/Trans.lean", "Mathlib/Data/List/OfFn.lean", "Mathlib/LinearAlgebra/Matrix/Spectrum.lean", "Mathlib/Order/Interval/Set/Monotone.lean", "Mathlib/Init/Data/Buffer/Parser.lean", "Mathlib/Data/Complex/Order.lean", "Mathlib/Algebra/Module/Submodule/Localization.lean", "Mathlib/CategoryTheory/Monad/Coequalizer.lean", "Mathlib/RingTheory/IntegralRestrict.lean", "Mathlib/Algebra/Homology/ShortComplex/Preadditive.lean", "Mathlib/Data/Complex/Orientation.lean", "Mathlib/AlgebraicGeometry/Properties.lean", "Mathlib/Data/Fintype/Array.lean", "Mathlib/Data/Matrix/Invertible.lean", "Mathlib/Data/DFinsupp/Encodable.lean", "Mathlib/GroupTheory/PGroup.lean", "Mathlib/Util/GetAllModules.lean", "Mathlib/Algebra/Lie/CartanSubalgebra.lean", "Mathlib/Analysis/NormedSpace/BoundedLinearMaps.lean", "Mathlib/RingTheory/Nilpotent/Defs.lean", "Mathlib/NumberTheory/MaricaSchoenheim.lean", "Mathlib/Data/Bracket.lean", "Mathlib/Analysis/BoxIntegral/Partition/Basic.lean", "Mathlib/CategoryTheory/Idempotents/FunctorCategories.lean", "Mathlib/Tactic/AdaptationNote.lean", "Mathlib/CategoryTheory/Limits/Constructions/Over/Connected.lean", "Mathlib/CategoryTheory/LiftingProperties/Basic.lean", "Mathlib/RingTheory/PolynomialAlgebra.lean", "Mathlib/CategoryTheory/Limits/Preserves/Shapes/BinaryProducts.lean", "Mathlib/Topology/Tactic.lean", "Mathlib/Init/Meta/WellFoundedTactics.lean", "Mathlib/Algebra/Polynomial/UnitTrinomial.lean", "Mathlib/Analysis/Convex/Cone/Basic.lean", "Mathlib/CategoryTheory/Bicategory/Kan/IsKan.lean", "Mathlib/LinearAlgebra/Matrix/LDL.lean", "Mathlib/Data/Nat/Factorial/SuperFactorial.lean", "Mathlib/NumberTheory/LegendreSymbol/ZModChar.lean", "Mathlib/Topology/ContinuousFunction/Units.lean", "Mathlib/CategoryTheory/Limits/Shapes/FiniteLimits.lean", "Mathlib/CategoryTheory/Preadditive/LeftExact.lean", "Mathlib/Analysis/InnerProductSpace/Adjoint.lean", "Mathlib/LinearAlgebra/BilinearForm/Orthogonal.lean", "Mathlib/Algebra/Homology/Refinements.lean", "Mathlib/Tactic/ReduceModChar.lean", "Mathlib/RingTheory/Binomial.lean", "Mathlib/Topology/Category/CompHaus/EffectiveEpi.lean", "Mathlib/Tactic/Set.lean", "Mathlib/GroupTheory/SpecificGroups/Cyclic.lean", "Mathlib/Analysis/SpecialFunctions/Trigonometric/Chebyshev.lean", "Mathlib/CategoryTheory/Limits/Shapes/WideEqualizers.lean", "Mathlib/Algebra/GradedMulAction.lean", "Mathlib/Analysis/SpecificLimits/Basic.lean", "Mathlib/Computability/Halting.lean", "Mathlib/CategoryTheory/Functor/KanExtension/Basic.lean", "Mathlib/Data/Nat/Factorial/BigOperators.lean", "Mathlib/Data/Array/Lemmas.lean", "Mathlib/LinearAlgebra/TensorProduct/Graded/Internal.lean", "Mathlib/Topology/Compactification/OnePoint.lean", "Mathlib/Probability/Distributions/Exponential.lean", "Mathlib/CategoryTheory/Bicategory/End.lean", "Mathlib/Algebra/Homology/ShortComplex/ExactFunctor.lean", "Mathlib/RingTheory/GradedAlgebra/HomogeneousIdeal.lean", "Mathlib/Algebra/Group/Units/Equiv.lean", "Mathlib/Algebra/GCDMonoid/Basic.lean", "Mathlib/FieldTheory/Minpoly/Basic.lean", "Mathlib/RingTheory/Localization/BaseChange.lean", "Mathlib/Analysis/Calculus/LocalExtr/Polynomial.lean", "Mathlib/Data/Int/Sqrt.lean", "Mathlib/Tactic/NormNum/IsCoprime.lean", "Mathlib/Algebra/Polynomial/Basic.lean", "Mathlib/Combinatorics/Quiver/Cast.lean", "Mathlib/Algebra/Symmetrized.lean", "Mathlib/Algebra/MvPolynomial/Derivation.lean", "Mathlib/Analysis/Calculus/SmoothSeries.lean", "Mathlib/Data/Real/StarOrdered.lean", "Mathlib/Data/Nat/Dist.lean", "Mathlib/MeasureTheory/Measure/Hausdorff.lean", "Mathlib/ModelTheory/Types.lean", "Mathlib/Algebra/GroupWithZero/Center.lean", "Mathlib/Probability/ProbabilityMassFunction/Basic.lean", "Mathlib/Data/List/Basic.lean", "Mathlib/Analysis/Calculus/FDeriv/Prod.lean", "Mathlib/Data/Int/Defs.lean", "Mathlib/Topology/Sheaves/Presheaf.lean", "Mathlib/Algebra/Lie/Sl2.lean", "Mathlib/Data/Complex/Determinant.lean", "Mathlib/Algebra/Regular/Pow.lean", "Mathlib/Computability/TuringMachine.lean", "Mathlib/CategoryTheory/Extensive.lean", "Mathlib/Combinatorics/Young/YoungDiagram.lean", "Mathlib/Init/Data/Ordering/Basic.lean", "Mathlib/Logic/Equiv/Nat.lean", "Mathlib/Analysis/Calculus/BumpFunction/Normed.lean", "Mathlib/Analysis/Normed/Order/Lattice.lean", "Mathlib/Computability/AkraBazzi/AkraBazzi.lean", "Mathlib/NumberTheory/Padics/PadicIntegers.lean", "Mathlib/Algebra/FreeAlgebra.lean", "Mathlib/Algebra/Order/Group/WithTop.lean", "Mathlib/MeasureTheory/Group/MeasurableEquiv.lean", "Mathlib/NumberTheory/SumTwoSquares.lean", "Mathlib/Geometry/Euclidean/MongePoint.lean", "Mathlib/CategoryTheory/Limits/Shapes/CommSq.lean", "Mathlib/Analysis/Convex/Exposed.lean", "Mathlib/CategoryTheory/Galois/GaloisObjects.lean", "Mathlib/Algebra/Exact.lean", "Mathlib/Data/ZMod/Basic.lean", "Mathlib/Topology/EMetricSpace/Lipschitz.lean", "Mathlib/Algebra/Homology/ImageToKernel.lean", "Mathlib/Data/Nat/Factorial/Cast.lean", "Mathlib/Analysis/Convex/Intrinsic.lean", "Mathlib/CategoryTheory/Triangulated/TStructure/Basic.lean", "Mathlib/Analysis/Calculus/Deriv/Prod.lean", "Mathlib/Data/String/Defs.lean", "Mathlib/CategoryTheory/Preadditive/Mat.lean", "Mathlib/RingTheory/WittVector/Truncated.lean", "Mathlib/Data/Seq/Seq.lean", "Mathlib/LinearAlgebra/QuadraticForm/IsometryEquiv.lean", "Mathlib/Algebra/Group/Support.lean", "Mathlib/Order/Interval/Multiset.lean", "Mathlib/Data/Matrix/Auto.lean", "Mathlib/CategoryTheory/Monoidal/Internal/Limits.lean", "Mathlib/Data/Rat/Init.lean", "Mathlib/Control/Functor.lean", "Mathlib/Dynamics/Ergodic/MeasurePreserving.lean", "Mathlib/Algebra/Lie/Killing.lean", "Mathlib/Combinatorics/Additive/Corner/Defs.lean", "Mathlib/Mathport/Notation.lean", "Mathlib/Tactic/Core.lean", "Mathlib/Data/Option/Defs.lean", "Mathlib/Data/Sym/Card.lean", "Mathlib/Algebra/Homology/Embedding/Extend.lean", "Mathlib/Analysis/NormedSpace/OperatorNorm/Bilinear.lean", "Mathlib/Topology/Order/LowerUpperTopology.lean", "Mathlib/Algebra/FreeNonUnitalNonAssocAlgebra.lean", "Mathlib/CategoryTheory/Sites/Coherent/RegularTopology.lean", "Mathlib/Init/Data/Bool/Lemmas.lean", "Mathlib/Topology/Algebra/Equicontinuity.lean", "Mathlib/Algebra/Ring/Center.lean", "Mathlib/CategoryTheory/Adhesive.lean", "Mathlib/Data/Nat/Prime.lean", "Mathlib/Algebra/Category/BoolRing.lean", "Mathlib/MeasureTheory/Measure/Lebesgue/Integral.lean", "Mathlib/Algebra/Category/Grp/ForgetCorepresentable.lean", "Mathlib/Algebra/Category/ModuleCat/Abelian.lean", "Mathlib/Combinatorics/SimpleGraph/Clique.lean", "Mathlib/Control/ULift.lean", "Mathlib/FieldTheory/Finite/Trace.lean", "Mathlib/GroupTheory/GroupAction/Blocks.lean", "Mathlib/Analysis/Normed/Group/SemiNormedGrp.lean", "Mathlib/Data/Nat/Multiplicity.lean", "Mathlib/Data/Multiset/Sort.lean", "Mathlib/Algebra/Order/BigOperators/Group/List.lean", "Mathlib/Algebra/Module/DedekindDomain.lean", "Mathlib/RingTheory/WittVector/Frobenius.lean", "Mathlib/Analysis/SpecialFunctions/Trigonometric/Angle.lean", "Mathlib/Analysis/InnerProductSpace/ProdL2.lean", "Mathlib/Algebra/Order/Hom/Ring.lean", "Mathlib/Combinatorics/SimpleGraph/Girth.lean", "Mathlib/Combinatorics/SimpleGraph/Maps.lean", "Mathlib/Geometry/Euclidean/Angle/Unoriented/Conformal.lean", "Mathlib/GroupTheory/Complement.lean", "Mathlib/Algebra/Order/Ring/Cone.lean", "Mathlib/Data/SetLike/Basic.lean", "Mathlib/FieldTheory/AxGrothendieck.lean", "Mathlib/LinearAlgebra/Ray.lean", "Mathlib/Algebra/Lie/Classical.lean", "Mathlib/Topology/RestrictGenTopology.lean", "Mathlib/Tactic.lean", "Mathlib/CategoryTheory/Sites/CompatiblePlus.lean", "Mathlib/Algebra/MvPolynomial/Supported.lean", "Mathlib/Util/LongNames.lean", "Mathlib/CategoryTheory/EssentialImage.lean", "Mathlib/Tactic/Linarith/Oracle/SimplexAlgorithm/PositiveVector.lean", "Mathlib/Combinatorics/Quiver/Path.lean", "Mathlib/NumberTheory/NumberField/Basic.lean", "Mathlib/Tactic/CategoryTheory/Reassoc.lean", "Mathlib/Topology/Homotopy/Basic.lean", "Mathlib/Topology/Order/ExtendFrom.lean", "Mathlib/Order/Filter/Cofinite.lean", "Mathlib/Analysis/SpecialFunctions/Trigonometric/Deriv.lean", "Mathlib/Analysis/InnerProductSpace/Basic.lean", "Mathlib/RingTheory/Nullstellensatz.lean", "Mathlib/Algebra/MvPolynomial/Counit.lean", "Mathlib/Deprecated/Ring.lean", "Mathlib/CategoryTheory/Limits/TypesFiltered.lean", "Mathlib/Order/Birkhoff.lean", "Mathlib/Order/Interval/Set/IsoIoo.lean", "Mathlib/Tactic/Peel.lean", "Mathlib/Topology/Instances/CantorSet.lean", "Mathlib/Algebra/Ring/Subring/Basic.lean", "Mathlib/Topology/FiberBundle/Basic.lean", "Mathlib/SetTheory/Cardinal/ENat.lean", "Mathlib/Algebra/Homology/DerivedCategory/HomologySequence.lean", "Mathlib/CategoryTheory/Noetherian.lean", "Mathlib/Topology/Sets/Order.lean", "Mathlib/CategoryTheory/ConnectedComponents.lean", "Mathlib/Probability/Martingale/OptionalStopping.lean", "Mathlib/Algebra/Order/Group/Action.lean", "Mathlib/CategoryTheory/Monoidal/Bimod.lean", "Mathlib/Algebra/Homology/ShortComplex/Homology.lean", "Mathlib/Tactic/Linarith/Oracle/SimplexAlgorithm/Gauss.lean", "Mathlib/Analysis/Convex/Basic.lean", "Mathlib/Tactic/Change.lean", "Mathlib/GroupTheory/Perm/Cycle/Basic.lean", "Mathlib/MeasureTheory/Integral/SetToL1.lean", "Mathlib/Algebra/Ring/Hom/Defs.lean", "Mathlib/Algebra/FreeMonoid/Basic.lean", "Mathlib/Algebra/EuclideanDomain/Defs.lean", "Mathlib/Algebra/Lie/InvariantForm.lean", "Mathlib/CategoryTheory/Limits/Final/ParallelPair.lean", "Mathlib/Order/Category/DistLat.lean", "Mathlib/LinearAlgebra/AffineSpace/Matrix.lean", "Mathlib/MeasureTheory/MeasurableSpace/Basic.lean", "Mathlib/Data/Multiset/Sections.lean", "Mathlib/Data/Finsupp/Encodable.lean", "Mathlib/Init/Data/Nat/Div.lean", "Mathlib/MeasureTheory/Decomposition/Jordan.lean", "Mathlib/Analysis/NormedSpace/CompactOperator.lean", "Mathlib/GroupTheory/Coxeter/Basic.lean", "Mathlib/Combinatorics/Quiver/SingleObj.lean", "Mathlib/Analysis/SpecialFunctions/Log/Monotone.lean", "Mathlib/ModelTheory/Quotients.lean", "Mathlib/LinearAlgebra/Dimension/Finite.lean", "Mathlib/CategoryTheory/Adjunction/Basic.lean", "Mathlib/Probability/Martingale/Convergence.lean", "Mathlib/Algebra/Polynomial/Taylor.lean", "Mathlib/Algebra/Lie/Derivation/AdjointAction.lean", "Mathlib/CategoryTheory/Subobject/Types.lean", "Mathlib/Order/PiLex.lean", "Mathlib/Topology/Algebra/Affine.lean", "Mathlib/Order/UpperLower/Basic.lean", "Mathlib/GroupTheory/FreeGroup/Basic.lean", "Mathlib/MeasureTheory/MeasurableSpace/Instances.lean", "Mathlib/Order/Booleanisation.lean", "Mathlib/Logic/Small/Module.lean", "Mathlib/Algebra/Lie/Rank.lean", "Mathlib/Topology/Sets/Opens.lean", "Mathlib/Algebra/Ring/Subring/Order.lean", "Mathlib/Analysis/SpecialFunctions/Bernstein.lean", "Mathlib/Order/Interval/Set/Disjoint.lean", "Mathlib/SetTheory/Game/PGame.lean", "Mathlib/AlgebraicTopology/DoldKan/GammaCompN.lean", "Mathlib/Analysis/Complex/LocallyUniformLimit.lean", "Mathlib/CategoryTheory/Skeletal.lean", "Mathlib/Analysis/SpecialFunctions/Pow/Deriv.lean", "Mathlib/Analysis/InnerProductSpace/GramSchmidtOrtho.lean", "Mathlib/NumberTheory/Basic.lean", "Mathlib/Order/Interval/Set/Infinite.lean", "Mathlib/Data/QPF/Multivariate/Constructions/Cofix.lean", "Mathlib/ModelTheory/Fraisse.lean", "Mathlib/Topology/MetricSpace/Kuratowski.lean", "Mathlib/Util/Export.lean", "Mathlib/Algebra/Module/Submodule/RestrictScalars.lean", "Mathlib/Analysis/NormedSpace/Span.lean", "Mathlib/Data/Set/BoolIndicator.lean", "Mathlib/NumberTheory/ClassNumber/AdmissibleAbsoluteValue.lean", "Mathlib/Topology/Algebra/UniformFilterBasis.lean", "Mathlib/Algebra/Homology/BifunctorShift.lean", "Mathlib/CategoryTheory/Sites/EqualizerSheafCondition.lean", "Mathlib/Topology/Sequences.lean", "Mathlib/Algebra/Order/Ring/Finset.lean", "Mathlib/CategoryTheory/Preadditive/Basic.lean", "Mathlib/CategoryTheory/Functor/Flat.lean", "Mathlib/RingTheory/Henselian.lean", "Mathlib/Algebra/Group/Hom/Instances.lean", "Mathlib/LinearAlgebra/Matrix/Basis.lean", "Mathlib/CategoryTheory/Countable.lean", "Mathlib/GroupTheory/GroupAction/SubMulAction/Pointwise.lean", "Mathlib/MeasureTheory/Integral/Layercake.lean", "Mathlib/Algebra/Order/GroupWithZero/WithZero.lean", "Mathlib/MeasureTheory/Constructions/Prod/Integral.lean", "Mathlib/CategoryTheory/Equivalence.lean", "Mathlib/Computability/TMComputable.lean", "Mathlib/Algebra/Order/Sum.lean", "Mathlib/MeasureTheory/Measure/AddContent.lean", "Mathlib/Combinatorics/Young/SemistandardTableau.lean", "Mathlib/Combinatorics/SimpleGraph/DegreeSum.lean", "Mathlib/AlgebraicGeometry/PrimeSpectrum/Noetherian.lean", "Mathlib/AlgebraicTopology/DoldKan/HomotopyEquivalence.lean", "Mathlib/MeasureTheory/Group/Arithmetic.lean", "Mathlib/Order/Compare.lean", "Mathlib/NumberTheory/ClassNumber/AdmissibleCardPowDegree.lean", "Mathlib/Dynamics/Flow.lean", "Mathlib/Tactic/DefEqTransformations.lean", "Mathlib/MeasureTheory/Measure/Complex.lean", "Mathlib/CategoryTheory/Shift/InducedShiftSequence.lean", "Mathlib/Order/Heyting/Basic.lean", "Mathlib/Analysis/BoxIntegral/Partition/SubboxInduction.lean", "Mathlib/Order/Interval/Set/Pi.lean", "Mathlib/RingTheory/Trace.lean", "Mathlib/CategoryTheory/Localization/Prod.lean", "Mathlib/Data/Set/List.lean", "Mathlib/Algebra/Ring/Basic.lean", "Mathlib/Algebra/Lie/Derivation/Killing.lean", "Mathlib/Data/List/DropRight.lean", "Mathlib/Data/Set/Enumerate.lean", "Mathlib/Topology/Sheaves/PUnit.lean", "Mathlib/Topology/Spectral/Hom.lean", "Mathlib/FieldTheory/PurelyInseparable.lean", "Mathlib/Data/List/Indexes.lean", "Mathlib/Data/Set/MemPartition.lean", "Mathlib/Tactic/Linarith/Preprocessing.lean", "Mathlib/CategoryTheory/Monoidal/Rigid/FunctorCategory.lean", "Mathlib/Data/Real/Cardinality.lean", "Mathlib/MeasureTheory/Integral/RieszMarkovKakutani.lean", "Mathlib/NumberTheory/Cyclotomic/PrimitiveRoots.lean", "Mathlib/LinearAlgebra/UnitaryGroup.lean", "Mathlib/Algebra/Order/Sub/Canonical.lean", "Mathlib/AlgebraicTopology/CechNerve.lean", "Mathlib/Analysis/Complex/RealDeriv.lean", "Mathlib/Algebra/Ring/Divisibility/Basic.lean", "Mathlib/Analysis/LocallyConvex/StrongTopology.lean", "Mathlib/CategoryTheory/Limits/Unit.lean", "Mathlib/CategoryTheory/Sites/Pullback.lean", "Mathlib/GroupTheory/Submonoid/Center.lean", "Mathlib/LinearAlgebra/Multilinear/Basic.lean", "Mathlib/Algebra/Group/Pi/Lemmas.lean", "Mathlib/CategoryTheory/Sites/Pretopology.lean", "Mathlib/Algebra/Homology/Linear.lean", "Mathlib/Topology/Germ.lean", "Mathlib/Analysis/SpecialFunctions/Complex/LogBounds.lean", "Mathlib/Data/Nat/Choose/Factorization.lean", "Mathlib/Geometry/Manifold/Metrizable.lean", "Mathlib/Tactic/FunProp/FunctionData.lean", "Mathlib/Tactic/TFAE.lean", "Mathlib/RingTheory/OreLocalization/OreSet.lean", "Mathlib/Data/Int/Bitwise.lean", "Mathlib/Mathport/Rename.lean", "Mathlib/AlgebraicTopology/AlternatingFaceMapComplex.lean", "Mathlib/RingTheory/WittVector/Domain.lean", "Mathlib/LinearAlgebra/LinearIndependent.lean", "Mathlib/Topology/Algebra/PontryaginDual.lean", "Mathlib/LinearAlgebra/TensorProduct/Prod.lean", "Mathlib/RingTheory/MvPolynomial/Basic.lean", "Mathlib/Data/Multiset/Interval.lean", "Mathlib/LinearAlgebra/Matrix/Circulant.lean", "Mathlib/Combinatorics/Pigeonhole.lean", "Mathlib/Order/SemiconjSup.lean", "Mathlib/Analysis/Normed/Field/InfiniteSum.lean", "Mathlib/Algebra/Group/Units.lean", "Mathlib/Control/Functor/Multivariate.lean", "Mathlib/Data/Analysis/Filter.lean", "Mathlib/RingTheory/Localization/NumDen.lean", "Mathlib/Data/Countable/Basic.lean", "Mathlib/LinearAlgebra/Dimension/Free.lean", "Mathlib/Analysis/Complex/Asymptotics.lean", "Mathlib/Data/Fin/Tuple/Finset.lean", "Mathlib/Tactic/Tauto.lean", "Mathlib/AlgebraicTopology/Quasicategory.lean", "Mathlib/Algebra/AddTorsor.lean", "Mathlib/LinearAlgebra/QuadraticForm/QuadraticModuleCat/Symmetric.lean", "Mathlib/Order/Hom/CompleteLattice.lean", "Mathlib/Analysis/Normed/Group/Quotient.lean", "Mathlib/FieldTheory/KummerExtension.lean", "Mathlib/Geometry/Euclidean/Angle/Oriented/Rotation.lean", "Mathlib/Init/Data/Sigma/Basic.lean", "Mathlib/NumberTheory/Zsqrtd/QuadraticReciprocity.lean", "Mathlib/CategoryTheory/Limits/Preserves/Shapes/Zero.lean", "Mathlib/Tactic/Explode.lean", "Mathlib/Algebra/Ring/Hom/Basic.lean", "Mathlib/Analysis/Normed/Group/Rat.lean", "Mathlib/Algebra/Free.lean", "Mathlib/CategoryTheory/WithTerminal.lean", "Mathlib/Tactic/Linarith/Oracle/FourierMotzkin.lean", "Mathlib/Tactic/Propose.lean", "Mathlib/LinearAlgebra/AffineSpace/Combination.lean", "Mathlib/Topology/Compactness/PseudometrizableLindelof.lean", "Mathlib/Control/Fold.lean", "Mathlib/Algebra/Homology/HomotopyCategory/Pretriangulated.lean", "Mathlib/Algebra/ContinuedFractions/Translations.lean", "Mathlib/Algebra/Regular/Basic.lean", "Mathlib/CategoryTheory/SmallObject/Construction.lean", "Mathlib/Topology/Order/NhdsSet.lean", "Mathlib/Algebra/MvPolynomial/Invertible.lean", "Mathlib/Order/Interval/Finset/Box.lean", "Mathlib/Data/Tree/Get.lean", "Mathlib/Data/Tree/Basic.lean", "Mathlib/Order/Category/Lat.lean", "Mathlib/CategoryTheory/Sites/CoversTop.lean", "Mathlib/Algebra/DirectLimit.lean", "Mathlib/Algebra/Order/Group/InjSurj.lean", "Mathlib/Data/Finsupp/Pointwise.lean", "Mathlib/GroupTheory/Divisible.lean", "Mathlib/LinearAlgebra/AffineSpace/AffineSubspace.lean", "Mathlib/Logic/Relation.lean", "Mathlib/Algebra/Homology/HomotopyCategory/HomComplexShift.lean", "Mathlib/Topology/Connected/Basic.lean", "Mathlib/Algebra/Group/Hom/Basic.lean", "Mathlib/Analysis/Convex/Combination.lean", "Mathlib/Analysis/SpecialFunctions/Gamma/Basic.lean", "Mathlib/CategoryTheory/Sites/Whiskering.lean", "Mathlib/Data/DFinsupp/Interval.lean", "Mathlib/Dynamics/FixedPoints/Topology.lean", "Mathlib/FieldTheory/RatFunc/Degree.lean", "Mathlib/Algebra/Polynomial/Inductions.lean", "Mathlib/Analysis/Calculus/Deriv/Mul.lean", "Mathlib/Algebra/Group/PNatPowAssoc.lean", "Mathlib/NumberTheory/NumberField/CanonicalEmbedding/ConvexBody.lean", "Mathlib/Topology/Category/Profinite/Nobeling.lean", "Mathlib/Tactic/FailIfNoProgress.lean", "Mathlib/Data/Nat/Choose/Cast.lean", "Mathlib/Data/Nat/Lattice.lean", "Mathlib/LinearAlgebra/CliffordAlgebra/Star.lean", "Mathlib/Util/IncludeStr.lean", "Mathlib/MeasureTheory/Function/SpecialFunctions/Arctan.lean", "Mathlib/Data/ENNReal/Basic.lean", "Mathlib/FieldTheory/PerfectClosure.lean", "Mathlib/SetTheory/Game/State.lean", "Mathlib/MeasureTheory/Function/ConditionalExpectation/CondexpL2.lean", "Mathlib/Tactic/Monotonicity.lean", "Mathlib/CategoryTheory/Monad/Adjunction.lean", "Mathlib/CategoryTheory/Monoidal/Tor.lean", "Mathlib/Algebra/Group/Subgroup/Actions.lean", "Mathlib/Algebra/Algebra/Prod.lean", "Mathlib/Probability/Kernel/Disintegration/CondCdf.lean", "Mathlib/Data/PFunctor/Multivariate/M.lean", "Mathlib/MeasureTheory/Decomposition/Lebesgue.lean", "Mathlib/CategoryTheory/Triangulated/Triangulated.lean", "Mathlib/Combinatorics/Enumerative/Composition.lean", "Mathlib/Data/Matrix/CharP.lean", "Mathlib/RingTheory/AdicCompletion/Algebra.lean", "Mathlib/Algebra/Ring/Fin.lean", "Mathlib/Data/ZMod/Units.lean", "Mathlib/CategoryTheory/Monoidal/Rigid/OfEquivalence.lean", "Mathlib/Data/PNat/Find.lean", "Mathlib/Algebra/Category/ModuleCat/Images.lean", "Mathlib/CategoryTheory/Limits/Shapes/Images.lean", "Mathlib/ModelTheory/FinitelyGenerated.lean", "Mathlib/NumberTheory/LegendreSymbol/JacobiSymbol.lean", "Mathlib/Testing/SlimCheck/Sampleable.lean", "Mathlib/Topology/Algebra/UniformMulAction.lean", "Mathlib/Topology/Algebra/UniformRing.lean", "Mathlib/MeasureTheory/Measure/MeasureSpace.lean", "Mathlib/MeasureTheory/Integral/MeanInequalities.lean", "Mathlib/Analysis/NormedSpace/Unitization.lean", "Mathlib/Probability/Martingale/OptionalSampling.lean", "Mathlib/MeasureTheory/Measure/MeasureSpaceDef.lean", "Mathlib/Analysis/Distribution/FourierSchwartz.lean", "Mathlib/Data/Finsupp/Indicator.lean", "Mathlib/Analysis/Normed/Ring/Seminorm.lean", "Mathlib/Data/Matroid/Constructions.lean", "Mathlib/MeasureTheory/Function/ConditionalExpectation/Indicator.lean", "Mathlib/MeasureTheory/Function/SpecialFunctions/RCLike.lean", "Mathlib/Algebra/Order/Sub/WithTop.lean", "Mathlib/GroupTheory/GroupAction/Basic.lean", "Mathlib/Algebra/Lie/Quotient.lean", "Mathlib/Data/Rbmap/Default.lean", "Mathlib/CategoryTheory/Category/Basic.lean", "Mathlib/Tactic/FunProp/Differentiable.lean", "Mathlib/Analysis/Convex/Complex.lean", "Mathlib/Analysis/SpecificLimits/Normed.lean", "Mathlib/NumberTheory/PythagoreanTriples.lean", "Mathlib/RepresentationTheory/Basic.lean", "Mathlib/Data/Rat/Cast/Defs.lean", "Mathlib/Data/ZMod/Factorial.lean", "Mathlib/Topology/Compactness/Paracompact.lean", "Mathlib/NumberTheory/Padics/Hensel.lean", "Mathlib/Algebra/Lie/Weights/Basic.lean", "Mathlib/Topology/Order/LawsonTopology.lean", "Mathlib/Topology/Instances/NNReal.lean", "Mathlib/LinearAlgebra/Matrix/Symmetric.lean", "Mathlib/Algebra/Homology/BifunctorHomotopy.lean", "Mathlib/Analysis/SpecialFunctions/JapaneseBracket.lean", "Mathlib/AlgebraicTopology/DoldKan/Decomposition.lean", "Mathlib/Algebra/Ring/InjSurj.lean", "Mathlib/CategoryTheory/Sites/CompatibleSheafification.lean", "Mathlib/LinearAlgebra/FreeModule/Basic.lean", "Mathlib/CategoryTheory/Functor/Hom.lean", "Mathlib/GroupTheory/Nilpotent.lean", "Mathlib/Algebra/Order/Monoid/WithTop.lean", "Mathlib/Topology/Algebra/InfiniteSum/GroupCompletion.lean", "Mathlib/Tactic/GCongr/Core.lean", "Mathlib/Analysis/NormedSpace/MazurUlam.lean", "Mathlib/RingTheory/AdicCompletion/Functoriality.lean", "Mathlib/Topology/Algebra/Module/CharacterSpace.lean", "Mathlib/Tactic/Widget/GCongr.lean", "Mathlib/Algebra/Module/LocalizedModule.lean", "Mathlib/Geometry/Manifold/MFDeriv/Basic.lean", "Mathlib/Algebra/Algebra/Subalgebra/Operations.lean", "Mathlib/Order/SymmDiff.lean", "Mathlib/Data/Int/Star.lean", "Mathlib/NumberTheory/LegendreSymbol/Basic.lean", "Mathlib/NumberTheory/RamificationInertia.lean", "Mathlib/CategoryTheory/Localization/Construction.lean", "Mathlib/NumberTheory/PrimeCounting.lean", "Mathlib/RingTheory/Valuation/Integers.lean", "Mathlib/Order/CompactlyGenerated/Intervals.lean", "Mathlib/Algebra/Ring/Invertible.lean", "Mathlib/RingTheory/RootsOfUnity/Basic.lean", "Mathlib/Analysis/Complex/Tietze.lean", "Mathlib/CategoryTheory/Limits/Constructions/EpiMono.lean", "Mathlib/Analysis/Calculus/Deriv/Add.lean", "Mathlib/GroupTheory/Commensurable.lean", "Mathlib/Algebra/Order/Field/Canonical/Basic.lean", "Mathlib/Data/Finset/Pairwise.lean", "Mathlib/Topology/Category/TopCat/Limits/Cofiltered.lean", "Mathlib/Analysis/SpecialFunctions/Polynomials.lean", "Mathlib/RingTheory/LittleWedderburn.lean", "Mathlib/MeasureTheory/Measure/Portmanteau.lean", "Mathlib/NumberTheory/Harmonic/Defs.lean", "Mathlib/RingTheory/AlgebraTower.lean", "Mathlib/Data/ByteArray.lean", "Mathlib/Algebra/Category/ModuleCat/Presheaf/Colimits.lean", "Mathlib/Data/Matrix/Basic.lean", "Mathlib/Tactic/Qify.lean", "Mathlib/Topology/Sheaves/SheafOfFunctions.lean", "Mathlib/AlgebraicTopology/FundamentalGroupoid/FundamentalGroup.lean", "Mathlib/Analysis/Convex/Strict.lean", "Mathlib/Algebra/Homology/ShortComplex/ModuleCat.lean", "Mathlib/Data/TypeVec.lean", "Mathlib/RingTheory/TensorProduct/Basic.lean", "Mathlib/Analysis/NormedSpace/Star/ContinuousFunctionalCalculus.lean", "Mathlib/Topology/Algebra/InfiniteSum/Nonarchimedean.lean", "Mathlib/Topology/Instances/RatLemmas.lean", "Mathlib/GroupTheory/HNNExtension.lean", "Mathlib/AlgebraicGeometry/EllipticCurve/Affine.lean", "Mathlib/LinearAlgebra/FreeModule/Determinant.lean", "Mathlib/CategoryTheory/Monoidal/Free/Coherence.lean", "Mathlib/Algebra/Category/ModuleCat/Presheaf/ChangeOfRings.lean", "Mathlib/CategoryTheory/Sites/PreservesLocallyBijective.lean", "Mathlib/Data/Rat/Sqrt.lean", "Mathlib/Algebra/MvPolynomial/Equiv.lean", "Mathlib/Algebra/Homology/Homology.lean", "Mathlib/Algebra/Module/LinearMap/Prod.lean", "Mathlib/Analysis/NormedSpace/Connected.lean", "Mathlib/Data/Rbtree/MinMax.lean", "Mathlib/Data/Sigma/Interval.lean", "Mathlib/CategoryTheory/Limits/Shapes/Kernels.lean", "Mathlib/Dynamics/BirkhoffSum/NormedSpace.lean", "Mathlib/RingTheory/DedekindDomain/Factorization.lean", "Mathlib/Algebra/Polynomial/GroupRingAction.lean", "Mathlib/CategoryTheory/Localization/Triangulated.lean", "Mathlib/MeasureTheory/Group/Action.lean", "Mathlib/MeasureTheory/SetAlgebra.lean", "Mathlib/RingTheory/NonUnitalSubsemiring/Basic.lean", "Mathlib/Algebra/MvPolynomial/Variables.lean", "Mathlib/Tactic/Hint.lean", "Mathlib/Algebra/Order/Interval/Set/Instances.lean", "Mathlib/Data/PFunctor/Multivariate/W.lean", "Mathlib/Algebra/Quotient.lean", "Mathlib/Algebra/Homology/HomotopyCategory/HomologicalFunctor.lean", "Mathlib/Combinatorics/SimpleGraph/Turan.lean", "Mathlib/Analysis/Convex/Topology.lean", "Mathlib/Dynamics/FixedPoints/Basic.lean", "Mathlib/Algebra/BigOperators/Module.lean", "Mathlib/NumberTheory/PellMatiyasevic.lean", "Mathlib/Data/Bool/Count.lean", "Mathlib/NumberTheory/Cyclotomic/Embeddings.lean", "Mathlib/Tactic/Linarith/Oracle/SimplexAlgorithm/Datatypes.lean", "Mathlib/Algebra/GCDMonoid/Nat.lean", "Mathlib/Algebra/GroupWithZero/Commute.lean", "Mathlib/CategoryTheory/Monoidal/OfChosenFiniteProducts/Basic.lean", "Mathlib/CategoryTheory/Limits/Shapes/Terminal.lean", "Mathlib/Combinatorics/SimpleGraph/Subgraph.lean", "Mathlib/Algebra/Algebra/Unitization.lean", "Mathlib/MeasureTheory/Function/ConvergenceInMeasure.lean", "Mathlib/Analysis/Convex/Body.lean", "Mathlib/Topology/Algebra/Group/OpenMapping.lean", "Mathlib/GroupTheory/Exponent.lean", "Mathlib/MeasureTheory/Integral/DivergenceTheorem.lean", "Mathlib/Algebra/Homology/DerivedCategory/Basic.lean", "Mathlib/Algebra/Polynomial/Smeval.lean", "Mathlib/MeasureTheory/Measure/OpenPos.lean", "Mathlib/Algebra/Algebra/Subalgebra/Tower.lean", "Mathlib/MeasureTheory/Measure/Restrict.lean", "Mathlib/Analysis/SpecialFunctions/Pow/Complex.lean", "Mathlib/NumberTheory/EllipticDivisibilitySequence.lean", "Mathlib/Combinatorics/Enumerative/DoubleCounting.lean", "Mathlib/Tactic/FunProp/ToBatteries.lean", "Mathlib/RingTheory/Polynomial/ScaleRoots.lean", "Mathlib/CategoryTheory/Limits/Opposites.lean", "Mathlib/Geometry/Euclidean/Sphere/Basic.lean", "Mathlib/Topology/Category/TopCat/Limits/Pullbacks.lean", "Mathlib/Data/Vector/Basic.lean", "Mathlib/RingTheory/OreLocalization/Ring.lean", "Mathlib/CategoryTheory/EqToHom.lean", "Mathlib/Algebra/Group/Aut.lean", "Mathlib/Init/Order/Defs.lean", "Mathlib/Tactic/ProdAssoc.lean", "Mathlib/Data/Holor.lean", "Mathlib/Algebra/Homology/ShortComplex/QuasiIso.lean", "Mathlib/Data/Matroid/Init.lean", "Mathlib/ModelTheory/Substructures.lean", "Mathlib/Data/Real/Sqrt.lean", "Mathlib/Algebra/Category/ModuleCat/Presheaf/Abelian.lean", "Mathlib/Geometry/Manifold/Algebra/Monoid.lean", "Mathlib/LinearAlgebra/Matrix/Permutation.lean", "Mathlib/Data/List/Defs.lean", "Mathlib/Analysis/Complex/UpperHalfPlane/Basic.lean", "Mathlib/Data/Nat/PrimeNormNum.lean", "Mathlib/Topology/Algebra/Valuation.lean", "Mathlib/Data/Set/Pointwise/Support.lean", "Mathlib/Analysis/Calculus/Deriv/Shift.lean", "Mathlib/Analysis/NormedSpace/Spectrum.lean", "Mathlib/Algebra/Group/Indicator.lean", "Mathlib/RepresentationTheory/GroupCohomology/Basic.lean", "Mathlib/Analysis/InnerProductSpace/MeanErgodic.lean", "Mathlib/Order/OrdContinuous.lean", "Mathlib/Testing/SlimCheck/Gen.lean", "Mathlib/Topology/MetricSpace/GromovHausdorff.lean", "Mathlib/Topology/MetricSpace/GromovHausdorffRealized.lean", "Mathlib/Analysis/NormedSpace/MatrixExponential.lean", "Mathlib/Topology/Algebra/Nonarchimedean/AdicTopology.lean", "Mathlib/Analysis/SpecialFunctions/Trigonometric/Bounds.lean", "Mathlib/Data/Nat/Factorization/PrimePow.lean", "Mathlib/Probability/Kernel/CondDistrib.lean", "Mathlib/Tactic/SuccessIfFailWithMsg.lean", "Mathlib/Data/String/Basic.lean", "Mathlib/NumberTheory/Cyclotomic/Discriminant.lean", "Mathlib/LinearAlgebra/Matrix/DotProduct.lean", "Mathlib/Algebra/GroupWithZero/InjSurj.lean", "Mathlib/Data/Fintype/Fin.lean", "Mathlib/Tactic/ExtractLets.lean", "Mathlib/Data/Sym/Sym2.lean", "Mathlib/Topology/UniformSpace/Compact.lean", "Mathlib/Topology/UniformSpace/UniformConvergenceTopology.lean", "Mathlib/MeasureTheory/Function/Jacobian.lean", "Mathlib/Algebra/RingQuot.lean", "Mathlib/Analysis/InnerProductSpace/EuclideanDist.lean", "Mathlib/Algebra/Homology/Augment.lean", "Mathlib/CategoryTheory/Limits/IsConnected.lean", "Mathlib/RingTheory/Filtration.lean", "Mathlib/Analysis/Complex/Convex.lean", "Mathlib/Geometry/Manifold/InteriorBoundary.lean", "Mathlib/Algebra/Homology/Factorizations/Basic.lean" ]
[]
.lake/packages/proofwidgets/ProofWidgets/Demos/Conv.lean
[ ".lake/packages/lean4/src/lean/Lean/Meta/ExprLens.lean", ".lake/packages/proofwidgets/ProofWidgets/Component/MakeEditLink.lean", ".lake/packages/lean4/src/lean/Init.lean", ".lake/packages/proofwidgets/ProofWidgets/Component/Panel/Basic.lean", ".lake/packages/proofwidgets/ProofWidgets/Component/OfRpcMethod.lean", ".lake/packages/proofwidgets/ProofWidgets/Data/Html.lean" ]
[ { "full_name": "NewCursorPos", "code": "structure NewCursorPos where\n newCursorPos? : Option Lsp.Position\n uri? : Option String\n deriving ToJson, FromJson", "start": [ 17, 1 ], "end": [ 20, 28 ], "kind": "commanddeclaration" }, { "full_name": "SolveReturn", "code": "private structure SolveReturn where\n expr : Expr\n val? : Option String\n listRest : List Nat", "start": [ 22, 1 ], "end": [ 25, 22 ], "kind": "commanddeclaration" }, { "full_name": "solveLevel", "code": "private def solveLevel (expr : Expr) (path : List Nat) : MetaM SolveReturn := match expr with\n | Expr.app _ _ => do\n let mut descExp := expr\n let mut count := 0\n let mut explicitList := []\n\n while descExp.isApp do\n if (←Lean.Meta.inferType descExp.appFn!).bindingInfo!.isExplicit then\n explicitList := true::explicitList\n count := count + 1\n else\n explicitList := false::explicitList\n descExp := descExp.appFn!\n\n let mut mutablePath := path\n let mut length := count\n explicitList := List.reverse explicitList\n while !mutablePath.isEmpty && mutablePath.head! == 0 do\n if explicitList.head! == true then\n count := count - 1\n explicitList := explicitList.tail!\n mutablePath := mutablePath.tail!\n\n let mut nextExp := expr\n while length > count do\n nextExp := nextExp.appFn!\n length := length - 1\n nextExp := nextExp.appArg!\n\n let pathRest := if mutablePath.isEmpty then [] else mutablePath.tail!\n\n return { expr := nextExp, val? := toString count , listRest := pathRest }\n\n | Expr.lam n _ b _ => do\n let name := match n with\n | Name.str _ s => s\n | _ => panic! \"no name found\"\n return { expr := b, val? := name, listRest := path.tail! }\n\n | Expr.forallE n _ b _ => do\n let name := match n with\n | Name.str _ s => s\n | _ => panic! \"no name found\"\n return { expr := b, val? := name, listRest := path.tail! }\n\n | Expr.mdata _ b => do\n match b with\n | Expr.mdata _ _ => return { expr := b, val? := none, listRest := path }\n | _ => return { expr := b.appFn!.appArg!, val? := none, listRest := path.tail!.tail! }\n\n | _ => do\n return { expr := ←(Lean.Core.viewSubexpr path.head! expr), val? := toString (path.head! + 1), listRest := path.tail! }", "start": [ 27, 1 ], "end": [ 81, 123 ], "kind": "commanddeclaration" }, { "full_name": "reprint!", "code": "def reprint! (stx : Syntax) : String :=\n match stx.reprint with\n | some x => x\n | none => panic! \"Could not reprint syntax\"", "start": [ 84, 1 ], "end": [ 87, 49 ], "kind": "commanddeclaration" }, { "full_name": "LocateReturn", "code": "structure LocateReturn where\n pathBeforeConv : List Nat\n pathAfterConv : List Nat\n deriving Inhabited", "start": [ 89, 1 ], "end": [ 92, 21 ], "kind": "commanddeclaration" }, { "full_name": "locate", "code": "private def locate (stx : Syntax) (pos : String.Pos) : LocateReturn := Id.run do\n let mut t := Syntax.Traverser.fromSyntax stx\n let mut path := []\n let mut rangeList := []\n\n while !t.cur.getArgs.isEmpty do\n let mut args := t.cur.getArgs\n let mut i := 0\n let mut newT := t\n let mut found := false\n rangeList := []\n for arg in args do\n let mut range := match arg.getRange? with\n | some x => x\n | none => { start := 0, stop := 0 }\n rangeList := range::rangeList\n if range.start < pos && pos <= range.stop then do\n newT := t.down i\n path := i::path\n found := true\n i := i + 1\n if !found then break\n t := newT\n\n let mut pathAfterConv := []\n while !(t.cur.getKind == `Lean.Parser.Tactic.Conv.conv\n || t.cur.getKind == `Lean.Parser.Tactic.Conv.convConvSeq\n || t.cur.getKind == `Lean.Widget.conv!)\n && path.length > 0 do\n t := t.up\n pathAfterConv := path.head!::pathAfterConv\n path := path.tail!\n\n if pathAfterConv == [] || pathAfterConv.length == 1 then\n pathAfterConv := [t.cur.getArgs.size - 2]\n\n else if pathAfterConv.length == 3 then\n let mut rangeList' := rangeList.reverse\n let mut ctr := 0\n while rangeList'.head!.stop < pos do\n ctr := ctr + 1\n rangeList' := rangeList'.tail!\n pathAfterConv := List.append pathAfterConv ((ctr-2)::[0])\n\n return {pathBeforeConv := path.reverse, pathAfterConv := pathAfterConv }", "start": [ 94, 1 ], "end": [ 142, 75 ], "kind": "commanddeclaration" }, { "full_name": "extractIndentation", "code": "private partial def extractIndentation (input : String) : String := match \" \".isPrefixOf input with\n | true => \" \" ++ extractIndentation (input.drop 2)\n | false => \"\"", "start": [ 144, 1 ], "end": [ 146, 16 ], "kind": "commanddeclaration" }, { "full_name": "InsertReturn", "code": "private structure InsertReturn where\n stx : Syntax\n newPath : List Nat\n newCursorPos : Lsp.Position", "start": [ 148, 1 ], "end": [ 151, 30 ], "kind": "commanddeclaration" }, { "full_name": "insertAfterArrow", "code": "private def insertAfterArrow (stx : Syntax) (pathBeforeConvParam : List Nat) (pathAfterConvParam : List Nat) (value : String) (text : FileMap) : InsertReturn := Id.run do\n let mut t := Syntax.Traverser.fromSyntax stx\n let mut pathBeforeConv := pathBeforeConvParam\n while pathBeforeConv.length > 0 do\n t := t.down pathBeforeConv.head!\n pathBeforeConv := pathBeforeConv.tail!\n let mut pathAfterConv := pathAfterConvParam\n\nlet mut pathBeforeConv' := pathBeforeConvParam.reverse\n let mut returnPath := []\n for _ in [:4] do\n t := t.up\n returnPath := pathBeforeConv'.head!::returnPath\n pathBeforeConv' := pathBeforeConv'.tail!\n t := t.up\n\n let argNr := pathBeforeConv'.head! - 1\n let prevArg := reprint! t.cur.getArgs[argNr]!\n let mut previousIndentation := extractIndentation (prevArg.splitOn \"\\n\").reverse.head!\n\n t := t.down pathBeforeConv'.head!\n while returnPath.length > 0 do\n t := t.down returnPath.head!\n returnPath := returnPath.tail!\n\n let arrow := reprint! t.cur.getArgs[pathAfterConv.head!]!\n let mut arrowIndentation := extractIndentation (arrow.splitOn \"\\n\").reverse.head!\n let mut newCursorPos := match t.cur.getArgs[pathAfterConv.head!]!.getRange? with\n | some range => text.utf8PosToLspPos range.stop\n | none => text.utf8PosToLspPos 0\n\n let mut newNode := Syntax.missing\n if reprint! t.cur.getArgs[pathAfterConv.head! + 1]! == \"\" || previousIndentation == arrowIndentation then\n let newArrow := Syntax.atom (SourceInfo.original \"\".toSubstring 0 \"\".toSubstring 0) \"=>\\n\"\n t := t.setCur (t.cur.setArgs (List.append (t.cur.getArgs.toList.take pathAfterConv.head!) (newArrow::t.cur.getArgs.toList.drop (pathAfterConv.head! + 1))).toArray)\n newNode := Syntax.atom (SourceInfo.original \"\".toSubstring 0 \"\".toSubstring 0) (\" \" ++ previousIndentation ++ value ++ \"\\n\" ++ arrowIndentation)\n newCursorPos := { line := newCursorPos.line + 1, character := 2 + previousIndentation.length + value.length }\n else\n newNode := Syntax.atom (SourceInfo.original \"\".toSubstring 0 \"\".toSubstring 0) (value ++ \"\\n\" ++ arrowIndentation)\n newCursorPos := { line := newCursorPos.line + 1, character := arrowIndentation.length + value.length }\n\n t := t.down (pathAfterConv.head! + 1)\n t := t.down 0\n t := t.down 0\n\n let newArgList := newNode::t.cur.getArgs.toList\n t := t.setCur (t.cur.setArgs newArgList.toArray)\n while t.parents.size > 0 do\n t := t.up\n\n let newPath := pathBeforeConvParam ++ (pathAfterConv.head! + 1)::0::0::[0]\n\n return { stx := t.cur, newPath := newPath, newCursorPos }", "start": [ 153, 1 ], "end": [ 212, 60 ], "kind": "commanddeclaration" }, { "full_name": "insertAnywhereElse", "code": "private def insertAnywhereElse (stx : Syntax) (pathBeforeConvParam : List Nat) (pathAfterConvParam : List Nat) (value : String) (text : FileMap): InsertReturn := Id.run do\n let mut t := Syntax.Traverser.fromSyntax stx\n let mut pathBeforeConv := pathBeforeConvParam\n while pathBeforeConv.length > 0 do\n t := t.down pathBeforeConv.head!\n pathBeforeConv := pathBeforeConv.tail!\n let mut pathAfterConv := pathAfterConvParam\n\nlet nothingAfterConv := t.up.cur.getArgs.size - 1 == pathBeforeConvParam.reverse.head!\n\n for _ in [:3] do\n t := t.down pathAfterConv.head!\n pathAfterConv := pathAfterConv.tail!\n\n let argAsString := reprint! t.cur.getArgs[pathAfterConv.head!]!\n let mut newval := value\n let mut entersMerged := false\n if toString t.cur.getArgs[pathAfterConv.head!]!.getKind == \"Lean.Parser.Tactic.Conv.Β«convEnter[__]Β»\" then\n let mut additionalArgs := (argAsString.splitOn \"\\n\").head!\n additionalArgs := (additionalArgs.drop \"enter [\".length).dropRight 1\n\n let left := value.take \"enter [\".length\n let right := value.drop \"enter [\".length\n newval := left ++ additionalArgs ++ \", \" ++ right\n entersMerged := true\n\n let mut newCursorPos := match t.cur.getArgs[pathAfterConv.head!]!.getRange? with\n | some range => text.utf8PosToLspPos range.stop\n | none => text.utf8PosToLspPos 0\n\n let mut argNr := pathAfterConv.head!\n let mut indentation := \"\"\n if argNr == 0 then\n indentation := extractIndentation ((reprint! t.up.up.up.cur).splitOn \"\\n\").tail!.head!\n else\n argNr := argNr - 2\n let mut prevArg := reprint! t.cur.getArgs[argNr]!\n let mut split := prevArg.splitOn \"\\n\"\n while split.length == 1 do\n argNr := argNr + 2\n prevArg := reprint! t.cur.getArgs[argNr]!\n split := prevArg.splitOn \"\\n\"\n\n let mut indentationLine := split.reverse.head!\n indentation := extractIndentation indentationLine\n\n newCursorPos := match entersMerged with\n | true => { line := newCursorPos.line, character := indentation.length + newval.length }\n | false => { line := newCursorPos.line + 1, character := indentation.length + newval.length }\n\n let mut frontIndentation := \"\"\n if pathAfterConv.head! == t.cur.getArgs.size - 1 then\n let lastArg := reprint! t.cur.getArgs[ t.cur.getArgs.size - 1]!\n let mut lastArgIndentation := extractIndentation (lastArg.splitOn \"\\n\").reverse.head!\n let numOfWhitespace := indentation.length - lastArgIndentation.length\n for _ in [:numOfWhitespace] do\n frontIndentation := frontIndentation ++ \" \"\n indentation := indentation.drop numOfWhitespace\n\n let mut argList := []\n if nothingAfterConv then\n let mut adjustedLastLine := reprint! t.cur.getArgs[t.cur.getArgs.size - 1]!\n while adjustedLastLine.takeRight 1 == \"\\n\" do\n adjustedLastLine := adjustedLastLine.dropRight 1\n adjustedLastLine := adjustedLastLine ++ \"\\n\"\n let adjustedLastNode := Syntax.atom (SourceInfo.original \"\".toSubstring 0 \"\".toSubstring 0) adjustedLastLine\n argList := (adjustedLastNode::t.cur.getArgs.toList.reverse.tail!).reverse\n else\n argList := t.cur.getArgs.toList\n\n let newNode := match entersMerged with\n | true => Syntax.atom (SourceInfo.original \"\".toSubstring 0 \"\".toSubstring 0) (newval ++ \"\\n\" ++ indentation)\n | false => Syntax.atom (SourceInfo.original \"\".toSubstring 0 \"\".toSubstring 0) (frontIndentation ++ newval ++ \"\\n\" ++ indentation)\n let newArgList := match entersMerged with\n | true => List.append (argList.take (pathAfterConv.head!) ) (newNode::(argList.drop (pathAfterConv.head! + 1)))\n | false => List.append (argList.take (pathAfterConv.head! + 1) ) (newNode::(argList.drop (pathAfterConv.head! + 1)))\n let newPath := match entersMerged with\n | true => pathBeforeConvParam ++ (pathAfterConvParam.take 4)\n | false => pathBeforeConvParam ++ (pathAfterConvParam.take 3) ++ [(pathAfterConvParam.get! 3) + 2]\n\n t := t.setCur (t.cur.setArgs newArgList.toArray)\n while t.parents.size > 0 do\n t := t.up\n\n return { stx := t.cur, newPath := newPath, newCursorPos := newCursorPos }", "start": [ 214, 1 ], "end": [ 309, 76 ], "kind": "commanddeclaration" }, { "full_name": "syntaxInsert", "code": "private def syntaxInsert (stx : Syntax) (pathBeforeConvParam : List Nat) (pathAfterConvParam : List Nat) (value : String) (text : FileMap): InsertReturn := Id.run do\n if value == \"\" then return { stx := stx, newPath := pathBeforeConvParam ++ pathAfterConvParam, newCursorPos := {line := 0, character := 0} }\n if pathAfterConvParam.length == 1 then\n return insertAfterArrow stx pathBeforeConvParam pathAfterConvParam value text\n else\n return insertAnywhereElse stx pathBeforeConvParam pathAfterConvParam value text", "start": [ 311, 1 ], "end": [ 316, 84 ], "kind": "commanddeclaration" }, { "full_name": "InsertEnterResponse", "code": "structure InsertEnterResponse where\n \n label : String\n edit : Lsp.TextDocumentEdit\n \n newCursorPos : Lsp.Position\n deriving FromJson, ToJson", "start": [ 318, 1 ], "end": [ 324, 28 ], "kind": "commanddeclaration" }, { "full_name": "insertEnter", "code": "def insertEnter (subexprPos : SubExpr.Pos) (goalType : Expr) (cmdStx : Syntax)\n (cursorPos : String.Pos) (doc : Lean.Server.FileWorker.EditableDocument) : MetaM InsertEnterResponse := do\n let mut list := (SubExpr.Pos.toArray subexprPos).toList\n let mut expr := goalType\n let mut retList := []\n while !list.isEmpty do\n let res ← solveLevel expr list\n expr := res.expr\n retList := match res.val? with\n | none => retList\n | some val => val::retList\n list := res.listRest\n\n retList := List.reverse retList\n let mut enterval := \"enter \" ++ toString retList\n if enterval.contains '0' then enterval := \"Error: Not a valid conv target\"\n if retList.isEmpty then enterval := \"\"\n\n let range := match cmdStx.getRange? with\n | some x => x\n | none => panic! \"could not get range\"\n\n let text := doc.meta.text\n\n let located := locate cmdStx { byteIdx := (min cursorPos.byteIdx range.stop.byteIdx) }\n let inserted := syntaxInsert cmdStx located.pathBeforeConv located.pathAfterConv enterval text\n let mut newSyntax := reprint! inserted.stx\n\n let mut syntaxAsList := newSyntax.data.reverse\n while syntaxAsList.head! == '\\n' || syntaxAsList.head! == ' ' do\n newSyntax := newSyntax.dropRight 1\n syntaxAsList := syntaxAsList.tail!\n\n let textEdit : Lsp.TextEdit := { range := { start := text.utf8PosToLspPos range.start, Β«endΒ» := text.utf8PosToLspPos { byteIdx := range.stop.byteIdx } }, newText := newSyntax }\n let edit : Lsp.TextDocumentEdit := { textDocument := { uri := doc.meta.uri, version? := doc.meta.version }, edits := [textEdit].toArray }\n\n return { label := enterval, edit, newCursorPos := inserted.newCursorPos }", "start": [ 326, 1 ], "end": [ 367, 76 ], "kind": "commanddeclaration" }, { "full_name": "ConvButtonProps", "code": "structure ConvButtonProps where\n pos : Lsp.Position\n goal : Widget.InteractiveGoal\n loc : SubExpr.GoalLocation\n deriving RpcEncodable", "start": [ 373, 1 ], "end": [ 377, 24 ], "kind": "commanddeclaration" }, { "full_name": "ConvButton.rpc", "code": "@[server_rpc_method]\ndef ConvButton.rpc (props : ConvButtonProps) : RequestM (RequestTask Html) :=\n RequestM.withWaitFindSnapAtPos props.pos fun snap => do\n if props.goal.goalPrefix != \"| \" then\n throw $ .invalidParams s!\"The current goal is not a conv goal.\"\n let .target subexprPos := props.loc\n | throw $ .invalidParams s!\"Select something in the target type.\"\n let doc ← RequestM.readDoc\n let cursorPos := doc.meta.text.lspPosToUtf8Pos props.pos\n props.goal.ctx.val.runMetaM {} do\n let md ← props.goal.mvarId.getDecl\n let lctx := md.lctx |>.sanitizeNames.run' {options := (← getOptions)}\n Meta.withLCtx lctx md.localInstances do\n let resp ← insertEnter subexprPos md.type snap.stx cursorPos doc\n return <div><MakeEditLink\n edit={resp.edit}\n newSelection?={some ⟨resp.newCursorPos, resp.newCursorPos⟩}\n title?={resp.label}\n >\n {.text resp.label}\n </MakeEditLink></div>", "start": [ 380, 1 ], "end": [ 400, 32 ], "kind": "commanddeclaration" }, { "full_name": "ConvButton", "code": "@[widget_module]\ndef ConvButton : Component ConvButtonProps :=\n mk_rpc_widget% ConvButton.rpc", "start": [ 402, 1 ], "end": [ 404, 32 ], "kind": "commanddeclaration" }, { "full_name": "findGoalForLocation", "code": "def findGoalForLocation (goals : Array Widget.InteractiveGoal) (loc : SubExpr.GoalsLocation) :\n Option Widget.InteractiveGoal :=\n goals.find? (Β·.mvarId == loc.mvarId)", "start": [ 406, 1 ], "end": [ 408, 39 ], "kind": "commanddeclaration" }, { "full_name": "ConvPanel.rpc", "code": "@[server_rpc_method]\ndef ConvPanel.rpc (props : PanelWidgetProps) : RequestM (RequestTask Html) :=\n RequestM.asTask do\n let inner : Html ← (do\n if props.selectedLocations.isEmpty then\n return <span>No actions available. You can use shift-click to select an expression in the goal state.</span>\n let buttons : Array Html ← props.selectedLocations.mapM fun loc => do\n let some g := findGoalForLocation props.goals loc\n | throw $ .invalidParams s!\"could not find goal for location {toJson loc}\"\n return <ConvButton pos={props.pos} goal={g} loc={loc.loc} />\n return Html.element \"div\" #[] buttons)\n return <details Β«openΒ»={true}>\n <summary className=\"mv2 pointer\">Conv πŸ”</summary>\n <div className=\"ml1\">{inner}</div>\n </details>", "start": [ 411, 1 ], "end": [ 425, 17 ], "kind": "commanddeclaration" }, { "full_name": "ConvPanel", "code": "@[widget_module]\ndef ConvPanel : Component PanelWidgetProps :=\n mk_rpc_widget% ConvPanel.rpc", "start": [ 427, 1 ], "end": [ 429, 31 ], "kind": "commanddeclaration" }, { "full_name": "test_sorry", "code": "axiom test_sorry {Ξ±} : Ξ±", "start": [ 434, 1 ], "end": [ 434, 25 ], "kind": "commanddeclaration" } ]
.lake/packages/proofwidgets/ProofWidgets/Demos/SelectInsertConv.lean
[ ".lake/packages/lean4/src/lean/Lean/Meta/ExprLens.lean", ".lake/packages/proofwidgets/ProofWidgets/Component/MakeEditLink.lean", ".lake/packages/batteries/Batteries/Lean/Position.lean", ".lake/packages/lean4/src/lean/Init.lean", ".lake/packages/proofwidgets/ProofWidgets/Component/Panel/Basic.lean", ".lake/packages/proofwidgets/ProofWidgets/Component/OfRpcMethod.lean", ".lake/packages/proofwidgets/ProofWidgets/Data/Html.lean" ]
[ { "full_name": "SolveReturn", "code": "private structure SolveReturn where\n expr : Expr\n val? : Option String\n listRest : List Nat", "start": [ 23, 1 ], "end": [ 26, 22 ], "kind": "commanddeclaration" }, { "full_name": "solveLevel", "code": "private def solveLevel (expr : Expr) (path : List Nat) : MetaM SolveReturn := match expr with\n | Expr.app _ _ => do\n let mut descExp := expr\n let mut count := 0\n let mut explicitList := []\n\n while descExp.isApp do\n if (←Lean.Meta.inferType descExp.appFn!).bindingInfo!.isExplicit then\n explicitList := true::explicitList\n count := count + 1\n else\n explicitList := false::explicitList\n descExp := descExp.appFn!\n\n let mut mutablePath := path\n let mut length := count\n explicitList := List.reverse explicitList\n while !mutablePath.isEmpty && mutablePath.head! == 0 do\n if explicitList.head! == true then\n count := count - 1\n explicitList := explicitList.tail!\n mutablePath := mutablePath.tail!\n\n let mut nextExp := expr\n while length > count do\n nextExp := nextExp.appFn!\n length := length - 1\n nextExp := nextExp.appArg!\n\n let pathRest := if mutablePath.isEmpty then [] else mutablePath.tail!\n\n return { expr := nextExp, val? := toString count , listRest := pathRest }\n\n | Expr.lam n _ b _ => do\n let name := match n with\n | Name.str _ s => s\n | _ => panic! \"no name found\"\n return { expr := b, val? := name, listRest := path.tail! }\n\n | Expr.forallE n _ b _ => do\n let name := match n with\n | Name.str _ s => s\n | _ => panic! \"no name found\"\n return { expr := b, val? := name, listRest := path.tail! }\n\n | Expr.mdata _ b => do\n match b with\n | Expr.mdata _ _ => return { expr := b, val? := none, listRest := path }\n | _ => return { expr := b.appFn!.appArg!, val? := none, listRest := path.tail!.tail! }\n\n | _ => do\n return {\n expr := ←(Lean.Core.viewSubexpr path.head! expr)\n val? := toString (path.head! + 1)\n listRest := path.tail!\n }", "start": [ 28, 1 ], "end": [ 86, 6 ], "kind": "commanddeclaration" }, { "full_name": "insertEnter", "code": "def insertEnter (locations : Array Lean.SubExpr.GoalsLocation) (goalType : Expr) : MetaM String := do\n let some pos := locations[0]? | throwError \"You must select something.\"\n let ⟨_, .target subexprPos⟩ := pos | throwError \"You must select something in the goal.\"\n let mut list := (SubExpr.Pos.toArray subexprPos).toList\n let mut expr := goalType\n let mut retList := []\n while !list.isEmpty do\n let res ← solveLevel expr list\n expr := res.expr\n retList := match res.val? with\n | none => retList\n | some val => val::retList\n list := res.listRest\n\n retList := List.reverse retList\n let mut enterval := \"conv => enter \" ++ toString retList\n if enterval.contains '0' then enterval := \"Error: Not a valid conv target\"\n if retList.isEmpty then enterval := \"\"\n return enterval", "start": [ 89, 1 ], "end": [ 109, 18 ], "kind": "commanddeclaration" }, { "full_name": "findGoalForLocation", "code": "def findGoalForLocation (goals : Array Widget.InteractiveGoal) (loc : SubExpr.GoalsLocation) :\n Option Widget.InteractiveGoal :=\n goals.find? (Β·.mvarId == loc.mvarId)", "start": [ 111, 1 ], "end": [ 113, 39 ], "kind": "commanddeclaration" }, { "full_name": "ConvSelectionPanelProps", "code": "structure ConvSelectionPanelProps extends PanelWidgetProps where\n \n replaceRange : Lsp.Range\n deriving RpcEncodable", "start": [ 115, 1 ], "end": [ 118, 24 ], "kind": "commanddeclaration" }, { "full_name": "ConvSelectionPanel.rpc", "code": "@[server_rpc_method]\ndef ConvSelectionPanel.rpc (props : ConvSelectionPanelProps) : RequestM (RequestTask Html) :=\n RequestM.asTask do\n let doc ← RequestM.readDoc\n let inner : Html ← (do\n if props.selectedLocations.isEmpty then\n return <span>Use shift-click to select one sub-expression in the goal that you want to zoom on.</span>\n let some selectedLoc := props.selectedLocations[0]? | unreachable!\n\n let some g := findGoalForLocation props.goals selectedLoc\n | throw $ .invalidParams\n s!\"could not find goal for location {toJson selectedLoc}\"\n g.ctx.val.runMetaM {} do\n let md ← g.mvarId.getDecl\n let lctx := md.lctx |>.sanitizeNames.run' {options := (← getOptions)}\n Meta.withLCtx lctx md.localInstances do\n let newCode ← insertEnter props.selectedLocations md.type\n return .ofComponent\n MakeEditLink\n (.ofReplaceRange doc.meta props.replaceRange newCode)\n #[ .text newCode ])\n return <details Β«openΒ»={true}>\n <summary className=\"mv2 pointer\">Conv πŸ”</summary>\n <div className=\"ml1\">{inner}</div>\n </details>", "start": [ 121, 1 ], "end": [ 145, 17 ], "kind": "commanddeclaration" }, { "full_name": "ConvSelectionPanel", "code": "@[widget_module]\ndef ConvSelectionPanel : Component ConvSelectionPanelProps :=\n mk_rpc_widget% ConvSelectionPanel.rpc", "start": [ 147, 1 ], "end": [ 149, 40 ], "kind": "commanddeclaration" }, { "full_name": "test_sorry", "code": "axiom test_sorry {Ξ±} : Ξ±", "start": [ 158, 1 ], "end": [ 158, 25 ], "kind": "commanddeclaration" } ]
.lake/packages/proofwidgets/ProofWidgets/Demos/Plot.lean
[ ".lake/packages/lean4/src/lean/Init.lean", ".lake/packages/proofwidgets/ProofWidgets/Component/HtmlDisplay.lean", ".lake/packages/proofwidgets/ProofWidgets/Component/Recharts.lean" ]
[ { "full_name": "fn", "code": "def fn (t : Float) (x : Float): Float :=\n 50 * (x - 0.25) * (x - 0.5) * (x - 0.7) + 0.1 * (x * 40 - t * 2 * 3.141).sin", "start": [ 6, 1 ], "end": [ 7, 80 ], "kind": "commanddeclaration" }, { "full_name": "Plot", "code": "def Plot (fn : Float β†’ Float) (steps := 100) : Html :=\n let jsonData : Array Json :=\n Nat.fold (flip Array.push) (steps + 1) #[]\n |> Array.map (fun (x : Nat) => let x : Float := x.toFloat / steps.toFloat; (x, fn x))\n |> Array.map (fun (x,y) => json% {x: $(toJson x) , y: $(toJson y)});\n <LineChart width={400} height={400} data={jsonData}>\n <XAxis domain?={#[toJson 0, toJson 1]} dataKey?=\"x\" />\n <YAxis domain?={#[toJson (-1), toJson 1]} allowDataOverflow={Bool.false} />\n <Line type={.monotone} dataKey=\"y\" stroke=\"#8884d8\" dot?={Bool.false} />\n </LineChart>", "start": [ 10, 1 ], "end": [ 19, 15 ], "kind": "commanddeclaration" }, { "full_name": "mkFrames", "code": "def mkFrames (fn : Float β†’ Float β†’ Float) (steps := 100) : Array Html:=\n List.range (steps + 1) |>.toArray |>.map (fun t => Plot (fn (t.toFloat / steps.toFloat)))", "start": [ 30, 1 ], "end": [ 31, 92 ], "kind": "commanddeclaration" }, { "full_name": "AnimatedHtmlProps", "code": "structure AnimatedHtmlProps where\n frames : Array Html\n framesPerSecond? : Option Nat := none\n deriving Server.RpcEncodable", "start": [ 33, 1 ], "end": [ 36, 31 ], "kind": "commanddeclaration" }, { "full_name": "AnimatedHtml", "code": "@[widget_module]\ndef AnimatedHtml : Component AnimatedHtmlProps where\n javascript := include_str \"..\" / \"..\" / \".lake\" / \"build\" / \"js\" / \"animatedHtml.js\"", "start": [ 38, 1 ], "end": [ 40, 87 ], "kind": "commanddeclaration" } ]
.lake/packages/proofwidgets/ProofWidgets/Demos/InteractiveSvg.lean
[ ".lake/packages/lean4/src/lean/Init.lean", ".lake/packages/proofwidgets/ProofWidgets/Component/HtmlDisplay.lean", ".lake/packages/proofwidgets/ProofWidgets/Component/InteractiveSvg.lean" ]
[ { "full_name": "State", "code": "abbrev State := Array (Float Γ— Float)", "start": [ 7, 1 ], "end": [ 7, 38 ], "kind": "commanddeclaration" }, { "full_name": "isvg", "code": "def isvg : InteractiveSvg State where\n init := #[(-0.5, -0.5), (0.5, -0.5), (0.5, 0.5), (-0.5, 0.5)]\n\n frame :=\n { xmin := -1\n ymin := -1\n xSize := 2\n width := 400\n height := 400 }\n\n update _time _Ξ”t _action _mouseStart mouseEnd _selected getData state :=\n match getData Nat, mouseEnd with\n | some id, some p => state.set! id p.toAbsolute\n | _, _ => state\n\n render _time mouseStart mouseEnd state :=\n {\n elements :=\n let mousePointer :=\n match mouseStart, mouseEnd with\n | some s, some e =>\n #[\n Svg.circle e (.px 5) |>.setFill (1.,1.,1.),\n Svg.line s e |>.setStroke (1.,1.,1.) (.px 2)\n ]\n | _, _ => #[]\n let circles := (state.mapIdx fun idx (p : Float Γ— Float) =>\n Svg.circle p (.abs 0.2) |>.setFill (0.7,0.7,0.7) |>.setId s!\"circle{idx}\" |>.setData idx.1\n )\n mousePointer.append circles\n }", "start": [ 9, 1 ], "end": [ 39, 6 ], "kind": "commanddeclaration" }, { "full_name": "updateSvg", "code": "@[server_rpc_method]\ndef updateSvg (params : UpdateParams State) : RequestM (RequestTask (UpdateResult State)) := isvg.serverRpcMethod params", "start": [ 42, 1 ], "end": [ 43, 121 ], "kind": "commanddeclaration" }, { "full_name": "SvgWidget", "code": "@[widget_module]\ndef SvgWidget : Component (UpdateResult State) where\n javascript := include_str \"..\" / \"..\" / \".lake\" / \"build\" / \"js\" / \"interactiveSvg.js\"", "start": [ 45, 1 ], "end": [ 47, 89 ], "kind": "commanddeclaration" }, { "full_name": "init", "code": "def init : UpdateResult State := {\n html := <div>Init!!!</div>,\n state := { state := isvg.init\n time := 0\n selected := none\n mousePos := none\n idToData := isvg.render 0 none none isvg.init |>.idToDataList}\n}", "start": [ 49, 1 ], "end": [ 56, 2 ], "kind": "commanddeclaration" } ]
.lake/packages/proofwidgets/ProofWidgets/Demos/Venn.lean
[ ".lake/packages/proofwidgets/ProofWidgets/Component/PenroseDiagram.lean", ".lake/packages/proofwidgets/ProofWidgets/Component/HtmlDisplay.lean", ".lake/packages/lean4/src/lean/Lean/Data/HashMap.lean", ".lake/packages/lean4/src/lean/Lean/Elab/Tactic.lean", ".lake/packages/lean4/src/lean/Init.lean", ".lake/packages/proofwidgets/ProofWidgets/Component/Panel/Basic.lean", ".lake/packages/proofwidgets/ProofWidgets/Component/OfRpcMethod.lean" ]
[ { "full_name": "Set", "code": "def Set (Ξ± : Type u) := Ξ± β†’ Prop", "start": [ 12, 1 ], "end": [ 12, 33 ], "kind": "commanddeclaration" }, { "full_name": "Set.Mem", "code": "protected def Mem (a : Ξ±) (s : Set Ξ±) : Prop :=\n s a", "start": [ 16, 1 ], "end": [ 18, 6 ], "kind": "commanddeclaration" }, { "full_name": "Set.ext", "code": "theorem ext {a b : Set Ξ±} (h : βˆ€ (x : Ξ±), x ∈ a ↔ x ∈ b) : a = b", "start": [ 23, 1 ], "end": [ 24, 33 ], "kind": "commanddeclaration" }, { "full_name": "Set.Subset", "code": "protected def Subset (s₁ sβ‚‚ : Set Ξ±) :=\n βˆ€ ⦃a⦄, a ∈ s₁ β†’ a ∈ sβ‚‚", "start": [ 26, 1 ], "end": [ 27, 25 ], "kind": "commanddeclaration" }, { "full_name": "isSubsetPred?", "code": "def isSubsetPred? (e : Expr) : Option (Expr Γ— Expr) := do\n let some (_, _, S, T) := e.app4? ``HasSubset.Subset | none\n return (S, T)", "start": [ 41, 1 ], "end": [ 44, 16 ], "kind": "commanddeclaration" }, { "full_name": "ExprEmbeds", "code": "abbrev ExprEmbeds := Array (String Γ— Expr)", "start": [ 46, 1 ], "end": [ 47, 43 ], "kind": "commanddeclaration" }, { "full_name": "mkSetDiag", "code": "def mkSetDiag (sub : String) (embeds : ExprEmbeds) : MetaM Html := do\n let embeds ← embeds.mapM fun (s, h) =>\n return (s, <InteractiveCode fmt={← Widget.ppExprTagged h} />)\n return <PenroseDiagram\n embeds={embeds}\n dsl={include_str \"..\"/\"..\"/\"widget\"/\"penrose\"/\"setTheory.dsl\"}\n sty={include_str \"..\"/\"..\"/\"widget\"/\"penrose\"/\"venn.sty\"}\n sub={sub} />", "start": [ 50, 1 ], "end": [ 57, 19 ], "kind": "commanddeclaration" }, { "full_name": "isSetGoal?", "code": "def isSetGoal? (hyps : Array LocalDecl) : MetaM (Option Html) := do\n let mut sub := \"AutoLabel All\\n\"\n let mut sets : HashMap String Expr := .empty\n for assm in hyps do\n let tp ← instantiateMVars assm.type\n if let some (S, T) := isSubsetPred? tp then\n let sS ← toString <$> Lean.Meta.ppExpr S\n let sT ← toString <$> Lean.Meta.ppExpr T\n let (sets', cS) := sets.insert' sS S\n let (sets', cT) := sets'.insert' sT T\n sets := sets'\n if !cS then\n sub := sub ++ s!\"Set {sS}\\n\"\n if !cT then\n sub := sub ++ s!\"Set {sT}\\n\"\n sub := sub ++ s!\"IsSubset({sS}, {sT})\\n\"\n if sets.isEmpty then return none\n some <$> mkSetDiag sub sets.toArray", "start": [ 59, 1 ], "end": [ 76, 38 ], "kind": "commanddeclaration" }, { "full_name": "findGoalForLocation", "code": "def findGoalForLocation (goals : Array Widget.InteractiveGoal) (loc : SubExpr.GoalsLocation) :\n Option Widget.InteractiveGoal :=\n goals.find? (Β·.mvarId == loc.mvarId)", "start": [ 80, 1 ], "end": [ 82, 39 ], "kind": "commanddeclaration" }, { "full_name": "VennDisplay.rpc", "code": "@[server_rpc_method]\ndef VennDisplay.rpc (props : PanelWidgetProps) : RequestM (RequestTask Html) :=\n RequestM.asTask do\n let inner : Html ← (do\n if props.selectedLocations.isEmpty then\n return <span>Use shift-click to select hypotheses to include in the diagram.</span>\n let some selectedLoc := props.selectedLocations[0]? | unreachable!\n\n let some g := findGoalForLocation props.goals selectedLoc\n | throw $ .invalidParams\n s!\"could not find goal for location {toJson selectedLoc}\"\n g.ctx.val.runMetaM {} do\n let md ← g.mvarId.getDecl\n let lctx := md.lctx |>.sanitizeNames.run' {options := (← getOptions)}\n Meta.withLCtx lctx md.localInstances do\n let locs : Array LocalDecl ← props.selectedLocations.filterMapM fun\n | ⟨mv, .hyp fv⟩ | ⟨mv, .hypType fv _⟩ =>\n if mv == g.mvarId then return some (← fv.getDecl) else return none\n | _ => return none\n match ← isSetGoal? locs with\n | some html => return html\n | none => return <span>No set goal.</span>)\n return <details Β«openΒ»={true}>\n <summary className=\"mv2 pointer\">Venn diagram</summary>\n <div className=\"ml1\">{inner}</div>\n </details>", "start": [ 85, 1 ], "end": [ 110, 17 ], "kind": "commanddeclaration" }, { "full_name": "VennDisplay", "code": "@[widget_module]\ndef VennDisplay : Component PanelWidgetProps :=\n mk_rpc_widget% VennDisplay.rpc", "start": [ 112, 1 ], "end": [ 114, 33 ], "kind": "commanddeclaration" } ]
.lake/packages/proofwidgets/ProofWidgets/Demos/Euclidean.lean
[ ".lake/packages/proofwidgets/ProofWidgets/Component/PenroseDiagram.lean", ".lake/packages/proofwidgets/ProofWidgets/Component/MakeEditLink.lean", ".lake/packages/proofwidgets/ProofWidgets/Component/HtmlDisplay.lean", ".lake/packages/lean4/src/lean/Lean/Data/HashMap.lean", ".lake/packages/lean4/src/lean/Lean/Elab/Tactic.lean", ".lake/packages/lean4/src/lean/Init.lean", ".lake/packages/proofwidgets/ProofWidgets/Component/Panel/Basic.lean", ".lake/packages/proofwidgets/ProofWidgets/Component/OfRpcMethod.lean" ]
[ { "full_name": "IncidenceGeometry", "code": "class IncidenceGeometry where\n Point : Type u₁\n Line : Type uβ‚‚\n Circle : Type u₃\n\n between : Point β†’ Point β†’ Point β†’ Prop onLine : Point β†’ Line β†’ Prop\n onCircle : Point β†’ Circle β†’ Prop\n inCircle : Point β†’ Circle β†’ Prop\n centerCircle : Point β†’ Circle β†’ Prop\n circlesInter : Circle β†’ Circle β†’ Prop\n\n ne_23_of_between : βˆ€ {a b c : Point}, between a b c β†’ b β‰  c\n line_unique_of_pts : βˆ€ {a b : Point}, βˆ€ {L M : Line},\n a β‰  b β†’ onLine a L β†’ onLine b L β†’ onLine a M β†’ onLine b M β†’ L = M\n onLine_2_of_between : βˆ€ {a b c : Point}, βˆ€ {L : Line},\n between a b c β†’ onLine a L β†’ onLine c L β†’ onLine b L\n line_of_pts : βˆ€ a b, βˆƒ L, onLine a L ∧ onLine b L\n circle_of_ne : βˆ€ a b, a β‰  b β†’ βˆƒ C, centerCircle a C ∧ onCircle b C\n circlesInter_of_onCircle_inCircle :\n βˆ€ {a b Ξ± Ξ²}, onCircle b Ξ± β†’ onCircle a Ξ² β†’ inCircle a Ξ± β†’\n inCircle b Ξ² β†’ circlesInter Ξ± Ξ²\n pts_of_circlesInter : βˆ€ {Ξ± Ξ²}, circlesInter Ξ± Ξ² β†’\n βˆƒ a b, a β‰  b ∧ onCircle a Ξ± ∧ onCircle a Ξ² ∧ onCircle b Ξ± ∧ onCircle b Ξ²\n inCircle_of_centerCircle : βˆ€ {a Ξ±}, centerCircle a Ξ± β†’ inCircle a Ξ±", "start": [ 25, 1 ], "end": [ 49, 70 ], "kind": "commanddeclaration" }, { "full_name": "isBetweenPred?", "code": "def isBetweenPred? (e : Expr) : Option (Expr Γ— Expr Γ— Expr) := do\n let some (_, a, b, c) := e.app4? ``between | none\n return (a, b, c)", "start": [ 55, 1 ], "end": [ 58, 19 ], "kind": "commanddeclaration" }, { "full_name": "isOnLinePred?", "code": "def isOnLinePred? (e : Expr) : Option (Expr Γ— Expr) := do\n let some (_, a, L) := e.app3? ``onLine | none\n return (a, L)", "start": [ 60, 1 ], "end": [ 63, 16 ], "kind": "commanddeclaration" }, { "full_name": "isOnCirclePred?", "code": "def isOnCirclePred? (e : Expr) : Option (Expr Γ— Expr) := do\n let some (_, a, C) := e.app3? ``onCircle | none\n return (a, C)", "start": [ 65, 1 ], "end": [ 68, 16 ], "kind": "commanddeclaration" }, { "full_name": "isInCirclePred?", "code": "def isInCirclePred? (e : Expr) : Option (Expr Γ— Expr) := do\n let some (_, a, C) := e.app3? ``inCircle | none\n return (a, C)", "start": [ 70, 1 ], "end": [ 73, 16 ], "kind": "commanddeclaration" }, { "full_name": "isCenterCirclePred?", "code": "def isCenterCirclePred? (e : Expr) : Option (Expr Γ— Expr) := do\n let some (_, a, C) := e.app3? ``centerCircle | none\n return (a, C)", "start": [ 75, 1 ], "end": [ 78, 16 ], "kind": "commanddeclaration" }, { "full_name": "isCirclesInterPred?", "code": "def isCirclesInterPred? (e : Expr) : Option (Expr Γ— Expr) := do\n let some (_, a, C) := e.app3? ``circlesInter | none\n return (a, C)", "start": [ 80, 1 ], "end": [ 83, 16 ], "kind": "commanddeclaration" }, { "full_name": "isPoint?", "code": "def isPoint? (e : Expr) : Bool :=\n e.isAppOf ``Point", "start": [ 85, 1 ], "end": [ 86, 20 ], "kind": "commanddeclaration" }, { "full_name": "isLine?", "code": "def isLine? (e : Expr) : Bool :=\n e.isAppOf ``Line", "start": [ 88, 1 ], "end": [ 89, 19 ], "kind": "commanddeclaration" }, { "full_name": "addHypotheses", "code": "def addHypotheses (hyps : Array LocalDecl) : DiagramBuilderM Unit := do\n for h in hyps do\n let tp ← instantiateMVars h.type\n if isPoint? tp then\n discard $ addExpr \"Point\" h.toExpr\n if isLine? tp then\n discard $ addExpr \"Line\" h.toExpr\n if let some (a, b, c) := isBetweenPred? tp then\n let sa ← addExpr \"Point\" a\n let sb ← addExpr \"Point\" b\n let sc ← addExpr \"Point\" c\n addInstruction s!\"Between({sa}, {sb}, {sc})\"\n if let some (a, L) := isOnLinePred? tp then\n let sa ← addExpr \"Point\" a\n let sL ← addExpr \"Line\" L\n addInstruction s!\"OnLine({sa}, {sL})\"\n if let some (a, C) := isOnCirclePred? tp then\n let sa ← addExpr \"Point\" a\n let sC ← addExpr \"Circle\" C\n addInstruction s!\"OnCircle({sa}, {sC})\"\n if let some (a, C) := isInCirclePred? tp then\n let sa ← addExpr \"Point\" a\n let sC ← addExpr \"Circle\" C\n addInstruction s!\"InCircle({sa}, {sC})\"\n if let some (a, C) := isCenterCirclePred? tp then\n let sa ← addExpr \"Point\" a\n let sC ← addExpr \"Circle\" C\n addInstruction s!\"CenterCircle({sa}, {sC})\"\n if let some (C, D) := isCirclesInterPred? tp then\n let sC ← addExpr \"Circle\" C\n let sD ← addExpr \"Circle\" D\n addInstruction s!\"CirclesInter({sC}, {sD})\"", "start": [ 94, 1 ], "end": [ 125, 50 ], "kind": "commanddeclaration" }, { "full_name": "EuclideanDisplay.dsl", "code": "def EuclideanDisplay.dsl :=\n include_str \"..\"/\"..\"/\"widget\"/\"penrose\"/\"euclidean.dsl\"", "start": [ 129, 1 ], "end": [ 130, 59 ], "kind": "commanddeclaration" }, { "full_name": "EuclideanDisplay.sty", "code": "def EuclideanDisplay.sty :=\n include_str \"..\"/\"..\"/\"widget\"/\"penrose\"/\"euclidean.sty\"", "start": [ 132, 1 ], "end": [ 133, 59 ], "kind": "commanddeclaration" }, { "full_name": "EuclideanDisplay.rpc", "code": "@[server_rpc_method]\ndef EuclideanDisplay.rpc (props : PanelWidgetProps) : RequestM (RequestTask Html) :=\n RequestM.asTask do\n let inner : Html ← (do\n if props.goals.isEmpty then\n return <span>No goals.</span>\n let some g := props.goals[0]? | unreachable!\n\n g.ctx.val.runMetaM {} do\n let md ← g.mvarId.getDecl\n let lctx := md.lctx |>.sanitizeNames.run' {options := (← getOptions)}\n Meta.withLCtx lctx md.localInstances do\n let mut hiddenLocs : HashSet FVarId := mkHashSet props.selectedLocations.size\n for l in props.selectedLocations do\n match l with\n | ⟨mv, .hyp fv⟩ | ⟨mv, .hypType fv _⟩ =>\n if mv == g.mvarId then\n hiddenLocs := hiddenLocs.insert fv\n | _ => continue\n let locs := (← getLCtx).decls.toArray.filterMap (fun d? =>\n if let some d := d? then\n if !hiddenLocs.contains d.fvarId then some d else none\n else\n none)\n DiagramBuilderM.run do\n addHypotheses locs\n match ← DiagramBuilderM.buildDiagram dsl sty with\n | some html => return html\n | none => return <span>No Euclidean goal.</span>)\n\n return <details Β«openΒ»={true}>\n <summary className=\"mv2 pointer\">Euclidean diagram</summary>\n <div className=\"ml1\">{inner}</div>\n </details>", "start": [ 136, 1 ], "end": [ 175, 17 ], "kind": "commanddeclaration" }, { "full_name": "EuclideanDisplay", "code": "@[widget_module]\ndef EuclideanDisplay : Component PanelWidgetProps :=\n mk_rpc_widget% EuclideanDisplay.rpc", "start": [ 177, 1 ], "end": [ 179, 38 ], "kind": "commanddeclaration" }, { "full_name": "constructLines", "code": "def constructLines (hyps : Array LocalDecl) (meta : Server.DocumentMeta) (cursorPos : Lsp.Position)\n : DiagramBuilderM Unit := do\n let mut points : Array LocalDecl := {}\n let mut circleInters : Array (LocalDecl Γ— LocalDecl Γ— LocalDecl) := {}\n for h in hyps do\n let tp ← instantiateMVars h.type\n if isPoint? tp then\n points := points.push h\n if let some (.fvar C, .fvar D) := isCirclesInterPred? tp then\n circleInters := circleInters.push (h, ← C.getDecl, ← D.getDecl)\n\n let addConstruction (nm tp ctr : String) : DiagramBuilderM Unit := do\n addEmbed nm tp (\n <span>\n <b>{.text nm}</b> ({\n .ofComponent MakeEditLink\n (MakeEditLinkProps.ofReplaceRange meta ⟨cursorPos, cursorPos⟩ ctr)\n #[.text \"insert\"]\n })\n </span>)\n addInstruction s!\"Emphasize({nm})\"\n\n for hi : i in [0:points.size] do\n let p := points[i]\n let sp ← addExpr \"Point\" p.toExpr\n for hj : j in [i+1:points.size] do\n let q := points[j]\n let sq ← addExpr \"Point\" q.toExpr\n\n let nm := s!\"{sp}{sq}\"\n addConstruction nm \"Line\" s!\"let ⟨{nm}, _, _⟩ := line_of_pts {sp} {sq}\"\n addInstruction s!\"OnLine({sp}, {nm})\"\n addInstruction s!\"OnLine({sq}, {nm})\"\n\n let nm := s!\"C{sp}{sq}\"\n addConstruction nm \"Circle\" s!\"let ⟨{nm}, _, _⟩ := circle_of_ne {sp} {sq} (by assumption)\"\n addInstruction s!\"CenterCircle({sp}, {nm})\"\n addInstruction s!\"OnCircle({sq}, {nm})\"\n\n let nm := s!\"C{sq}{sp}\"\n addConstruction nm \"Circle\" s!\"let ⟨{nm}, _, _⟩ := circle_of_ne {sq} {sp} (by assumption)\"\n addInstruction s!\"CenterCircle({sq}, {nm})\"\n addInstruction s!\"OnCircle({sp}, {nm})\"\n\n for hi : i in [0:circleInters.size] do\n let (h, C, D) := circleInters[i]\n let sC ← addExpr \"Circle\" C.toExpr\n let sD ← addExpr \"Circle\" D.toExpr\n let nm := s!\"{sC}{sD}\"\n let nm' := s!\"{sD}{sC}\"\n addConstruction nm \"Point\" s!\"let ⟨{nm}, {nm'}, _, _, _, _, _⟩ := pts_of_circlesInter {h.userName}\"\n addEmbed nm' \"Point\" <b>{.text nm'}</b>\n addInstruction s!\"OnCircle({nm'}, {sC})\"\n addInstruction s!\"OnCircle({nm}, {sD})\"\n addInstruction s!\"OnCircle({nm}, {sC})\"\n addInstruction s!\"OnCircle({nm'}, {sD})\"", "start": [ 197, 1 ], "end": [ 261, 45 ], "kind": "commanddeclaration" }, { "full_name": "EuclideanConstructions.rpc", "code": "@[server_rpc_method]\ndef EuclideanConstructions.rpc (props : PanelWidgetProps) : RequestM (RequestTask Html) :=\n RequestM.asTask do\n let doc ← RequestM.readDoc\n let inner : Html ← (do\n if props.goals.isEmpty then\n return <span>No goals.</span>\n let some g := props.goals[0]? | unreachable!\n\n g.ctx.val.runMetaM {} do\n let md ← g.mvarId.getDecl\n let lctx := md.lctx |>.sanitizeNames.run' {options := (← getOptions)}\n Meta.withLCtx lctx md.localInstances do\n\n let allHyps := (← getLCtx).decls.toArray.filterMap id\n\n let selectedHyps ← props.selectedLocations.filterMapM fun\n | ⟨mv, .hyp fv⟩ | ⟨mv, .hypType fv _⟩ =>\n if mv == g.mvarId then return some (← fv.getDecl) else return none\n | _ =>\n return none\n\n DiagramBuilderM.run do\n addHypotheses allHyps\n constructLines selectedHyps doc.meta props.pos\n match ← DiagramBuilderM.buildDiagram EuclideanDisplay.dsl EuclideanDisplay.sty 1500 with\n | some html => return html\n | none => return <span>No Euclidean goal.</span>)\n\n return <details Β«openΒ»={true}>\n <summary className=\"mv2 pointer\">Euclidean constructions</summary>\n <div className=\"ml1\">{inner}</div>\n </details>", "start": [ 264, 1 ], "end": [ 302, 17 ], "kind": "commanddeclaration" }, { "full_name": "EuclideanConstructions", "code": "@[widget_module]\ndef EuclideanConstructions : Component PanelWidgetProps :=\n mk_rpc_widget% EuclideanConstructions.rpc", "start": [ 304, 1 ], "end": [ 306, 44 ], "kind": "commanddeclaration" }, { "full_name": "test_sorry", "code": "axiom test_sorry {Ξ±} : Ξ±", "start": [ 308, 1 ], "end": [ 308, 25 ], "kind": "commanddeclaration" } ]
.lake/packages/proofwidgets/ProofWidgets/Demos/Rubiks.lean
[ ".lake/packages/lean4/src/lean/Init.lean", ".lake/packages/proofwidgets/ProofWidgets/Component/HtmlDisplay.lean" ]
[ { "full_name": "RubiksProps", "code": "structure RubiksProps where\n seq : Array String := #[]\n deriving ToJson, FromJson, Inhabited", "start": [ 6, 1 ], "end": [ 8, 39 ], "kind": "commanddeclaration" }, { "full_name": "Rubiks", "code": "@[widget_module]\ndef Rubiks : Component RubiksProps where\n javascript := include_str \"..\" / \"..\" / \".lake\" / \"build\" / \"js\" / \"rubiks.js\"", "start": [ 10, 1 ], "end": [ 12, 81 ], "kind": "commanddeclaration" }, { "full_name": "eg", "code": "def eg := #[\"L\", \"L\", \"D⁻¹\", \"U⁻¹\", \"L\", \"D\", \"D\", \"L\", \"U⁻¹\", \"R\", \"D\", \"F\", \"F\", \"D\"]", "start": [ 14, 1 ], "end": [ 14, 88 ], "kind": "commanddeclaration" } ]
.lake/packages/proofwidgets/ProofWidgets/Demos/Macro.lean
[ ".lake/packages/lean4/src/lean/Init.lean", ".lake/packages/proofwidgets/ProofWidgets/Component/HtmlDisplay.lean" ]
[ { "full_name": "Lean.SourceInfo.mkCanonical", "code": "def Lean.SourceInfo.mkCanonical : SourceInfo β†’ SourceInfo\n | .synthetic s e _ => .synthetic s e true\n | si => si", "start": [ 13, 1 ], "end": [ 15, 13 ], "kind": "commanddeclaration" }, { "full_name": "Lean.Syntax.mkInfoCanonical", "code": "def Lean.Syntax.mkInfoCanonical : Syntax β†’ Syntax\n | .missing => .missing\n | .node i k a => .node i.mkCanonical k a\n | .atom i v => .atom i.mkCanonical v\n | .ident i r v p => .ident i.mkCanonical r v p", "start": [ 17, 1 ], "end": [ 21, 49 ], "kind": "commanddeclaration" }, { "full_name": "Lean.TSyntax.mkInfoCanonical", "code": "def Lean.TSyntax.mkInfoCanonical : TSyntax k β†’ TSyntax k :=\n (.mk Β·.raw.mkInfoCanonical)", "start": [ 23, 1 ], "end": [ 24, 30 ], "kind": "commanddeclaration" } ]
.lake/packages/proofwidgets/ProofWidgets/Demos/Jsx.lean
[ ".lake/packages/lean4/src/lean/Init.lean", ".lake/packages/proofwidgets/ProofWidgets/Component/HtmlDisplay.lean" ]
[ { "full_name": "htmlLetters", "code": "def htmlLetters : Array ProofWidgets.Html := #[\n <span style={json% {color: \"red\"}}>H</span>,\n <span style={json% {color: \"yellow\"}}>T</span>,\n <span style={json% {color: \"green\"}}>M</span>,\n <span style={json% {color: \"blue\"}}>L</span>\n ]", "start": [ 13, 1 ], "end": [ 18, 4 ], "kind": "commanddeclaration" }, { "full_name": "x", "code": "def x := <b>You can use {...htmlLetters} in Lean {.text s!\"{1 + 3}\"}! <hr/> </b>", "start": [ 21, 1 ], "end": [ 21, 81 ], "kind": "commanddeclaration" } ]
.lake/packages/proofwidgets/ProofWidgets/Demos/LazyComputation.lean
[ ".lake/packages/lean4/src/lean/Init.lean", ".lake/packages/proofwidgets/ProofWidgets/Component/Basic.lean" ]
[ { "full_name": "MetaMStringCont", "code": "structure MetaMStringCont where\n ci : Elab.ContextInfo\n lctx : LocalContext\n k : MetaM String\n deriving TypeName", "start": [ 6, 1 ], "end": [ 12, 20 ], "kind": "commanddeclaration" }, { "full_name": "RunnerWidgetProps", "code": "structure RunnerWidgetProps where\n \n k : WithRpcRef MetaMStringCont\n deriving RpcEncodable", "start": [ 14, 1 ], "end": [ 18, 24 ], "kind": "commanddeclaration" }, { "full_name": "runMetaMStringCont", "code": "@[server_rpc_method]\ndef runMetaMStringCont : RunnerWidgetProps β†’ RequestM (RequestTask String)\n | {k := ⟨{ci, lctx, k}⟩} => RequestM.asTask do\n ci.runMetaM lctx k", "start": [ 20, 1 ], "end": [ 23, 23 ], "kind": "commanddeclaration" }, { "full_name": "runnerWidget", "code": "@[widget_module]\ndef runnerWidget : Component RunnerWidgetProps where\n javascript := \"\n import { RpcContext, mapRpcError } from '@leanprover/infoview'\n import * as React from 'react';\n const e = React.createElement;\n\n export default function(props) {\n const [contents, setContents] = React.useState('Run!')\n const rs = React.useContext(RpcContext)\n return e('button', { onClick: () => {\n setContents('Running..')\n rs.call('runMetaMStringCont', props)\n .then(setContents)\n .catch(e => { setContents(mapRpcError(e).message) })\n }}, contents)\n }\n \"", "start": [ 25, 1 ], "end": [ 42, 4 ], "kind": "commanddeclaration" }, { "full_name": "makeRunner", "code": "@[tactic makeRunnerTac] def makeRunner : Tactic\n | `(tactic| make_runner%$tk) => do\n let x : MetaM String := do\n return \"Hello, world!\"\n let props : RunnerWidgetProps := {\n k := ⟨{\n ci := { ← CommandContextInfo.save with }\n lctx := (← getLCtx)\n k := x\n }⟩}\n Widget.savePanelWidgetInfo runnerWidget.javascriptHash (rpcEncode props) tk\n | _ => throwUnsupportedSyntax", "start": [ 46, 1 ], "end": [ 59, 32 ], "kind": "commanddeclaration" } ]
.lake/packages/proofwidgets/ProofWidgets/Demos/Dynkin.lean
[ ".lake/packages/lean4/src/lean/Init.lean", ".lake/packages/proofwidgets/ProofWidgets/Component/HtmlDisplay.lean" ]
[ { "full_name": "List.product", "code": "def List.product : List Ξ± β†’ List Ξ² β†’ List (Ξ± Γ— Ξ²)\n | [], _ => []\n | a::as, bs => bs.map ((a, Β·)) ++ as.product bs", "start": [ 6, 1 ], "end": [ 8, 50 ], "kind": "commanddeclaration" }, { "full_name": "Matrix", "code": "def Matrix (n m Ξ± : Type) := n β†’ m β†’ Ξ±", "start": [ 10, 1 ], "end": [ 10, 39 ], "kind": "commanddeclaration" }, { "full_name": "Matrix.nat_index", "code": "def nat_index (i j : Nat) : Int :=\n if h : i < n ∧ j < n then A ⟨i, h.1⟩ ⟨j, h.2⟩ else 999", "start": [ 19, 1 ], "end": [ 20, 57 ], "kind": "commanddeclaration" }, { "full_name": "Matrix.get_node_pos_E", "code": "def get_node_pos_E : Nat β†’ Nat Γ— Nat\n | 0 => ⟨0, 0⟩\n | 1 => ⟨2, 1⟩\n | (i+1) => ⟨i, 0⟩", "start": [ 22, 1 ], "end": [ 26, 20 ], "kind": "commanddeclaration" }, { "full_name": "Matrix.get_node_pos", "code": "def get_node_pos (n : Nat) : Nat β†’ Nat Γ— Nat := if n < 6 then ((Β·, 0)) else get_node_pos_E", "start": [ 28, 1 ], "end": [ 29, 91 ], "kind": "commanddeclaration" }, { "full_name": "Matrix.get_node_cx", "code": "def get_node_cx (n i : Nat) : Int := 20 + (get_node_pos n i).1 * 40", "start": [ 31, 1 ], "end": [ 31, 68 ], "kind": "commanddeclaration" }, { "full_name": "Matrix.get_node_cy", "code": "def get_node_cy (n i : Nat) : Int := 20 + (get_node_pos n i).2 * 40", "start": [ 33, 1 ], "end": [ 33, 68 ], "kind": "commanddeclaration" }, { "full_name": "Matrix.get_node_html", "code": "def get_node_html (n i : Nat) : Html :=\n <circle\n cx={toString <| get_node_cx n i}\n cy={toString <| get_node_cy n i}\n r=\"10\"\n fill=\"white\"\n stroke=\"black\" />", "start": [ 35, 1 ], "end": [ 41, 22 ], "kind": "commanddeclaration" }, { "full_name": "Matrix.get_edge_html", "code": "def get_edge_html : Nat Γ— Nat β†’ List Html\n | (i, j) => if A.nat_index i j = 0 then [] else\n [<line\n x1={toString <| get_node_cx n i}\n y1={toString <| get_node_cy n i}\n x2={toString <| get_node_cx n j}\n y2={toString <| get_node_cy n j}\n fill=\"black\"\n stroke=\"black\" />]", "start": [ 43, 1 ], "end": [ 56, 24 ], "kind": "commanddeclaration" }, { "full_name": "Matrix.get_nodes_html", "code": "def get_nodes_html (n : Nat) : List Html :=\n (List.range n).map (get_node_html n)", "start": [ 58, 1 ], "end": [ 59, 39 ], "kind": "commanddeclaration" }, { "full_name": "Matrix.get_edges_html", "code": "def get_edges_html : List Html := Id.run do\n let mut out := []\n for j in [:n] do\n for i in [:j] do\n out := A.get_edge_html (i, j) ++ out\n return out", "start": [ 61, 1 ], "end": [ 66, 13 ], "kind": "commanddeclaration" }, { "full_name": "Matrix.toHtml", "code": "def toHtml (M : Matrix (Fin n) (Fin n) Int) : Html :=\n <div style={json% { height: \"100px\", width: \"300px\", background: \"grey\" }}>\n {Html.element \"svg\" #[] (M.get_edges_html ++ Matrix.get_nodes_html n).toArray}\n </div>", "start": [ 68, 1 ], "end": [ 71, 9 ], "kind": "commanddeclaration" }, { "full_name": "cartanMatrix.Eβ‚ˆ", "code": "def cartanMatrix.Eβ‚ˆ : Matrix (Fin 8) (Fin 8) Int :=\n fun i j =>\n [[ 2, 0, -1, 0, 0, 0, 0, 0],\n [ 0, 2, 0, -1, 0, 0, 0, 0],\n [-1, 0, 2, -1, 0, 0, 0, 0],\n [ 0, -1, -1, 2, -1, 0, 0, 0],\n [ 0, 0, 0, -1, 2, -1, 0, 0],\n [ 0, 0, 0, 0, -1, 2, -1, 0],\n [ 0, 0, 0, 0, 0, -1, 2, -1],\n [ 0, 0, 0, 0, 0, 0, -1, 2]].get! i |>.get! j", "start": [ 75, 1 ], "end": [ 84, 56 ], "kind": "commanddeclaration" } ]
.lake/packages/proofwidgets/ProofWidgets/Demos/ExprPresentation.lean
[ ".lake/packages/proofwidgets/ProofWidgets/Component/Panel/SelectionPanel.lean", ".lake/packages/lean4/src/lean/Init.lean", ".lake/packages/proofwidgets/ProofWidgets/Component/Panel/GoalTypePanel.lean" ]
[ { "full_name": "presenter", "code": "@[expr_presenter]\ndef presenter : ExprPresenter where\n userName := \"With octopodes\"\n layoutKind := .inline\n present e :=\n return <span>\n {.text \"πŸ™ \"}<InteractiveCode fmt={← Lean.Widget.ppExprTagged e} />{.text \" πŸ™\"}\n </span>", "start": [ 6, 1 ], "end": [ 13, 14 ], "kind": "commanddeclaration" } ]
.lake/packages/proofwidgets/ProofWidgets/Demos/RbTree.lean
[ ".lake/packages/proofwidgets/ProofWidgets/Component/Panel/SelectionPanel.lean", ".lake/packages/lean4/src/lean/Init.lean", ".lake/packages/proofwidgets/ProofWidgets/Presentation/Expr.lean" ]
[ { "full_name": "RBColour", "code": "inductive RBColour where\n | red | black", "start": [ 7, 1 ], "end": [ 8, 16 ], "kind": "commanddeclaration" }, { "full_name": "RBTree", "code": "inductive RBTree (Ξ± : Type u) where\n | empty : RBTree Ξ±\n | node (color : RBColour) (l : RBTree Ξ±) (a : Ξ±) (r : RBTree Ξ±) : RBTree Ξ±", "start": [ 10, 1 ], "end": [ 12, 77 ], "kind": "commanddeclaration" }, { "full_name": "RBTree.contains", "code": "def contains [Ord Ξ±] (a : Ξ±) : RBTree Ξ± β†’ Bool\n | empty => false\n | node _ l b r => match compare a b with\n | .lt => l.contains a\n | .eq => true\n | .gt => r.contains a", "start": [ 16, 1 ], "end": [ 21, 26 ], "kind": "commanddeclaration" }, { "full_name": "RBTree.balance", "code": "def balance : RBColour β†’ RBTree Ξ± β†’ Ξ± β†’ RBTree Ξ± β†’ RBTree Ξ±\n | .black, (node .red (node .red a x b) y c), z, d\n | .black, (node .red a x (node .red b y c)), z, d\n | .black, a, x, (node .red (node .red b y c) z d)\n | .black, a, x, (node .red b y (node .red c z d)) =>\n node .red (node .black a x b) y (node .black c z d)\n | color, a, x, b => node color a x b", "start": [ 23, 1 ], "end": [ 29, 39 ], "kind": "commanddeclaration" }, { "full_name": "RBTree.insert", "code": "def insert [Ord Ξ±] (a : Ξ±) (s : RBTree Ξ±) : RBTree Ξ± :=\n makeBlack (ins s)\nwhere\n ins : RBTree Ξ± β†’ RBTree Ξ±\n | empty => node .red empty a empty\n | node c l b r => match compare a b with\n | .lt => balance c (ins l) b r\n | .eq => node c l b r\n | .gt => balance c l b (ins r)\n makeBlack : RBTree Ξ± β†’ RBTree Ξ±\n | empty => empty\n | node _ l b r => node .black l b r", "start": [ 31, 1 ], "end": [ 42, 40 ], "kind": "commanddeclaration" }, { "full_name": "empty?", "code": "def empty? (e : Expr) : Bool :=\n e.app1? ``RBTree.empty matches some _", "start": [ 50, 1 ], "end": [ 51, 40 ], "kind": "commanddeclaration" }, { "full_name": "Lean.Expr.app5?", "code": "@[inline] def Lean.Expr.app5? (e : Expr) (fName : Name) : Option (Expr Γ— Expr Γ— Expr Γ— Expr Γ— Expr) :=\n if e.isAppOfArity fName 5 then\n some (\n e.appFn!.appFn!.appFn!.appFn!.appArg!,\n e.appFn!.appFn!.appFn!.appArg!,\n e.appFn!.appFn!.appArg!,\n e.appFn!.appArg!,\n e.appArg!)\n else\n none", "start": [ 53, 1 ], "end": [ 62, 9 ], "kind": "commanddeclaration" }, { "full_name": "node?", "code": "def node? (e : Expr) : Option (Expr Γ— Expr Γ— Expr Γ— Expr) := do\n let some (_, color, l, a, r) := e.app5? ``RBTree.node | none\n return (color, l, a, r)", "start": [ 64, 1 ], "end": [ 66, 26 ], "kind": "commanddeclaration" }, { "full_name": "evalColourUnsafe", "code": "unsafe def evalColourUnsafe (e : Expr) : MetaM RBColour :=\n Lean.Meta.evalExpr' RBColour ``RBColour e", "start": [ 68, 1 ], "end": [ 69, 44 ], "kind": "commanddeclaration" }, { "full_name": "evalColour", "code": "@[implemented_by evalColourUnsafe]\nopaque evalColour (e : Expr) : MetaM RBColour", "start": [ 71, 1 ], "end": [ 72, 46 ], "kind": "commanddeclaration" }, { "full_name": "RBTreeVarsColour", "code": "inductive RBTreeVarsColour where\n | red | black | blue\n deriving FromJson, ToJson", "start": [ 74, 1 ], "end": [ 77, 28 ], "kind": "commanddeclaration" }, { "full_name": "RBTreeVars", "code": "inductive RBTreeVars where\n | empty : RBTreeVars\n | var : CodeWithInfos β†’ RBTreeVars\n | node (color : RBTreeVarsColour) (l : RBTreeVars) (a : CodeWithInfos) (r : RBTreeVars) : RBTreeVars\n deriving Server.RpcEncodable", "start": [ 80, 1 ], "end": [ 89, 31 ], "kind": "commanddeclaration" }, { "full_name": "RBDisplayProps", "code": "structure RBDisplayProps where\n tree : RBTreeVars\n deriving Server.RpcEncodable", "start": [ 93, 1 ], "end": [ 95, 31 ], "kind": "commanddeclaration" }, { "full_name": "RBDisplay", "code": "@[widget_module]\ndef RBDisplay : Component RBDisplayProps where\n javascript := include_str \"..\" / \"..\" / \".lake\" / \"build\" / \"js\" / \"rbTree.js\"", "start": [ 99, 1 ], "end": [ 101, 81 ], "kind": "commanddeclaration" }, { "full_name": "drawTree?", "code": "partial def drawTree? (e : Expr) : MetaM (Option Html) := do\n if let some _ := node? e then\n return some <RBDisplay tree={← go e}/>\n else if empty? e then\n return some <RBDisplay tree={← go e}/>\n else\n return none\nwhere go (e : Expr) : MetaM RBTreeVars := do\n if let some (color, l, a, r) := node? e then\n let color ← try\n match ← evalColour color with\n | .red => pure .red\n | .black => pure .black\n catch _ => pure .blue\n return .node color (← go l) (← Widget.ppExprTagged a) (← go r)\n else if empty? e then\n return .empty\n else\n return .var (← Widget.ppExprTagged e)", "start": [ 104, 1 ], "end": [ 122, 42 ], "kind": "commanddeclaration" }, { "full_name": "RBTree.presenter", "code": "@[expr_presenter]\ndef RBTree.presenter : ExprPresenter where\n userName := \"Red-black tree\"\n present e := do\n let some t ← drawTree? e\n | throwError \"not a tree :(\"\n return t", "start": [ 124, 1 ], "end": [ 130, 13 ], "kind": "commanddeclaration" } ]
.lake/packages/proofwidgets/ProofWidgets/Demos/Svg.lean
[ ".lake/packages/lean4/src/lean/Init.lean", ".lake/packages/proofwidgets/ProofWidgets/Component/HtmlDisplay.lean", ".lake/packages/proofwidgets/ProofWidgets/Data/Svg.lean" ]
[ { "full_name": "frame", "code": "private def frame : Frame where\n xmin := -2\n ymin := -2\n xSize := 4\n width := 400\n height := 400", "start": [ 6, 1 ], "end": [ 11, 16 ], "kind": "commanddeclaration" }, { "full_name": "svg", "code": "private def svg : Svg frame :=\n { elements :=\n #[line (0.,0.) (1.,0.) |>.setStroke (1.,0.,0.) (.px 2),\n line (1.,0.) (0.,1.) |>.setStroke (0.,1.,0.) (.px 2),\n line (0.,1.) (0.,0.) |>.setStroke (0.,0.,1.) (.px 2),\n circle (0.,0.) (.abs 0.1) |>.setStroke (0.,0.,0.) (.px 2) |>.setFill (0.,1.,1.) |>.setId \"point1\",\n circle (1.,0.) (.abs 0.1) |>.setStroke (0.,0.,0.) (.px 2) |>.setFill (1.,0.,1.) |>.setId \"point2\",\n circle (0.,1.) (.abs 0.1) |>.setStroke (0.,0.,0.) (.px 2) |>.setFill (1.,1.,0.) |>.setId \"point3\"] }", "start": [ 13, 1 ], "end": [ 20, 109 ], "kind": "commanddeclaration" } ]
.lake/packages/lean4/src/lean/Lean/Compiler/IR/EmitLLVM.lean
[ ".lake/packages/lean4/src/lean/Lean/Compiler/ExportAttr.lean", ".lake/packages/lean4/src/lean/Lean/Runtime.lean", ".lake/packages/lean4/src/lean/Lean/Compiler/IR/EmitUtil.lean", ".lake/packages/lean4/src/lean/Lean/Compiler/IR/ResetReuse.lean", ".lake/packages/lean4/src/lean/Lean/Compiler/IR/Boxing.lean", ".lake/packages/lean4/src/lean/Lean/Compiler/IR/SimpCase.lean", ".lake/packages/lean4/src/lean/Lean/Compiler/NameMangling.lean", ".lake/packages/lean4/src/lean/Lean/Data/HashMap.lean", ".lake/packages/lean4/src/lean/Lean/Compiler/InitAttr.lean", ".lake/packages/lean4/src/lean/Lean/Compiler/IR/NormIds.lean", ".lake/packages/lean4/src/lean/Lean/Compiler/IR/CompilerM.lean", ".lake/packages/lean4/src/lean/Lean/Compiler/IR/LLVMBindings.lean" ]
[ { "full_name": "Lean.IR.leanMainFn", "code": "def leanMainFn := \"_lean_main\"", "start": [ 24, 1 ], "end": [ 24, 31 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.LLVM.size_tType", "code": "def size_tType (llvmctx : LLVM.Context) : BaseIO (LLVM.LLVMType llvmctx) :=\n LLVM.i64Type llvmctx", "start": [ 28, 1 ], "end": [ 29, 23 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.LLVM.unsignedType", "code": "def unsignedType (llvmctx : LLVM.Context) : BaseIO (LLVM.LLVMType llvmctx) :=\n LLVM.i32Type llvmctx", "start": [ 32, 1 ], "end": [ 33, 23 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.LLVM.getOrAddFunction", "code": "def getOrAddFunction (m : LLVM.Module ctx) (name : String) (type : LLVM.LLVMType ctx) : BaseIO (LLVM.Value ctx) := do\n match (← LLVM.getNamedFunction m name) with\n | some fn => return fn\n | none =>\n \n let fn ← LLVM.addFunction m name type\n let attr ← LLVM.createStringAttribute \"probe-stack\" \"inline-asm\"\n LLVM.addAttributeAtIndex fn LLVM.AttributeIndex.AttributeFunctionIndex attr\n return fn", "start": [ 36, 1 ], "end": [ 48, 14 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.LLVM.getOrAddGlobal", "code": "def getOrAddGlobal (m : LLVM.Module ctx) (name : String) (type : LLVM.LLVMType ctx) : BaseIO (LLVM.Value ctx) := do\n match (← LLVM.getNamedGlobal m name) with\n | .some fn => return fn\n | .none => LLVM.addGlobal m name type", "start": [ 50, 1 ], "end": [ 53, 40 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.Context", "code": "structure Context (llvmctx : LLVM.Context) where\n env : Environment\n modName : Name\n jpMap : JPParamsMap := {}\n mainFn : FunId := default\n mainParams : Array Param := #[]\n llvmmodule : LLVM.Module llvmctx", "start": [ 59, 1 ], "end": [ 65, 35 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.State", "code": "structure State (llvmctx : LLVM.Context) where\n var2val : HashMap VarId (LLVM.LLVMType llvmctx Γ— LLVM.Value llvmctx)\n jp2bb : HashMap JoinPointId (LLVM.BasicBlock llvmctx)", "start": [ 67, 1 ], "end": [ 69, 58 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.Error", "code": "abbrev Error := String", "start": [ 71, 1 ], "end": [ 71, 23 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.M", "code": "abbrev M (llvmctx : LLVM.Context) :=\n StateRefT (State llvmctx) (ReaderT (Context llvmctx) (ExceptT Error IO))", "start": [ 73, 1 ], "end": [ 74, 75 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.addVartoState", "code": "def addVartoState (x : VarId) (v : LLVM.Value llvmctx) (ty : LLVM.LLVMType llvmctx) : M llvmctx Unit := do\n modify (fun s => { s with var2val := s.var2val.insert x (ty, v) })", "start": [ 79, 1 ], "end": [ 80, 69 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.addJpTostate", "code": "def addJpTostate (jp : JoinPointId) (bb : LLVM.BasicBlock llvmctx) : M llvmctx Unit :=\n modify (fun s => { s with jp2bb := s.jp2bb.insert jp bb })", "start": [ 82, 1 ], "end": [ 83, 61 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitJp", "code": "def emitJp (jp : JoinPointId) : M llvmctx (LLVM.BasicBlock llvmctx) := do\n let state ← get\n match state.jp2bb.find? jp with\n | .some bb => return bb\n | .none => throw s!\"unable to find join point {jp}\"", "start": [ 85, 1 ], "end": [ 89, 54 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.getLLVMModule", "code": "def getLLVMModule : M llvmctx (LLVM.Module llvmctx) := Context.llvmmodule <$> read", "start": [ 91, 1 ], "end": [ 91, 83 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.getEnv", "code": "def getEnv : M llvmctx Environment := Context.env <$> read", "start": [ 93, 1 ], "end": [ 93, 59 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.getModName", "code": "def getModName : M llvmctx Name := Context.modName <$> read", "start": [ 95, 1 ], "end": [ 95, 61 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.getDecl", "code": "def getDecl (n : Name) : M llvmctx Decl := do\n let env ← getEnv\n match findEnvDecl env n with\n | some d => pure d\n | none => throw s!\"unknown declaration {n}\"", "start": [ 97, 1 ], "end": [ 101, 48 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.constInt8", "code": "def constInt8 (n : Nat) : M llvmctx (LLVM.Value llvmctx) := do\n LLVM.constInt8 llvmctx (UInt64.ofNat n)", "start": [ 103, 1 ], "end": [ 104, 44 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.constInt64", "code": "def constInt64 (n : Nat) : M llvmctx (LLVM.Value llvmctx) := do\n LLVM.constInt64 llvmctx (UInt64.ofNat n)", "start": [ 106, 1 ], "end": [ 107, 45 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.constIntSizeT", "code": "def constIntSizeT (n : Nat) : M llvmctx (LLVM.Value llvmctx) := do\n LLVM.constIntSizeT llvmctx (UInt64.ofNat n)", "start": [ 109, 1 ], "end": [ 110, 48 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.constIntUnsigned", "code": "def constIntUnsigned (n : Nat) : M llvmctx (LLVM.Value llvmctx) := do\n LLVM.constIntUnsigned llvmctx (UInt64.ofNat n)", "start": [ 112, 1 ], "end": [ 113, 51 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.getOrCreateFunctionPrototype", "code": "def getOrCreateFunctionPrototype (mod : LLVM.Module llvmctx)\n (retty : LLVM.LLVMType llvmctx) (name : String) (args : Array (LLVM.LLVMType llvmctx)) : M llvmctx (LLVM.Value llvmctx) := do\n LLVM.getOrAddFunction mod name $ ← LLVM.functionType retty args (isVarArg := false)", "start": [ 115, 1 ], "end": [ 117, 86 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.callLeanBox", "code": "def callLeanBox (builder : LLVM.Builder llvmctx)\n (arg : LLVM.Value llvmctx) (name : String := \"\") : M llvmctx (LLVM.Value llvmctx) := do\n let fnName := \"lean_box\"\n let retty ← LLVM.voidPtrType llvmctx\n let argtys := #[ ← LLVM.size_tType llvmctx ]\n let fn ← getOrCreateFunctionPrototype (← getLLVMModule) retty fnName argtys\n let fnty ← LLVM.functionType retty argtys\n LLVM.buildCall2 builder fnty fn #[arg] name", "start": [ 119, 1 ], "end": [ 126, 47 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.callLeanMarkPersistentFn", "code": "def callLeanMarkPersistentFn (builder : LLVM.Builder llvmctx) (arg : LLVM.Value llvmctx) : M llvmctx Unit := do\n let fnName := \"lean_mark_persistent\"\n let retty ← LLVM.voidType llvmctx\n let argtys := #[ ← LLVM.voidPtrType llvmctx ]\n let fn ← getOrCreateFunctionPrototype (← getLLVMModule) retty fnName argtys\n let fnty ← LLVM.functionType retty argtys\n let _ ← LLVM.buildCall2 builder fnty fn #[arg]", "start": [ 128, 1 ], "end": [ 134, 52 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.RefcountKind", "code": "inductive RefcountKind where\n | inc | dec", "start": [ 137, 1 ], "end": [ 138, 14 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.callLeanRefcountFn", "code": "def callLeanRefcountFn (builder : LLVM.Builder llvmctx)\n (kind : RefcountKind) (checkRef? : Bool) (arg : LLVM.Value llvmctx)\n (delta : Option (LLVM.Value llvmctx) := Option.none) : M llvmctx Unit := do\n let fnName := s!\"lean_{kind}{if checkRef? then \"\" else \"_ref\"}{if delta.isNone then \"\" else \"_n\"}\"\n let retty ← LLVM.voidType llvmctx\n let argtys ← if delta.isNone then pure #[← LLVM.voidPtrType llvmctx] else pure #[← LLVM.voidPtrType llvmctx, ← LLVM.size_tType llvmctx]\n let fn ← getOrCreateFunctionPrototype (← getLLVMModule) retty fnName argtys\n let fnty ← LLVM.functionType retty argtys\n match delta with\n | .none => do\n let _ ← LLVM.buildCall2 builder fnty fn #[arg]\n | .some n => do\n let _ ← LLVM.buildCall2 builder fnty fn #[arg, n]", "start": [ 145, 1 ], "end": [ 158, 54 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.callLeanDecRef", "code": "def callLeanDecRef (builder : LLVM.Builder llvmctx) (res : LLVM.Value llvmctx) : M llvmctx Unit := do\n let fnName := \"lean_dec_ref\"\n let retty ← LLVM.voidType llvmctx\n let argtys := #[ ← LLVM.i8PtrType llvmctx ]\n let fn ← getOrCreateFunctionPrototype (← getLLVMModule) retty fnName argtys\n let fnty ← LLVM.functionType retty argtys\n let _ ← LLVM.buildCall2 builder fnty fn #[res]", "start": [ 163, 1 ], "end": [ 169, 50 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.callLeanUnsignedToNatFn", "code": "def callLeanUnsignedToNatFn (builder : LLVM.Builder llvmctx)\n (n : Nat) (name : String := \"\") : M llvmctx (LLVM.Value llvmctx) := do\n let mod ← getLLVMModule\n let argtys := #[← LLVM.i32Type llvmctx]\n let retty ← LLVM.voidPtrType llvmctx\n let f ← getOrCreateFunctionPrototype mod retty \"lean_unsigned_to_nat\" argtys\n let fnty ← LLVM.functionType retty argtys\n let nv ← constIntUnsigned n\n LLVM.buildCall2 builder fnty f #[nv] name", "start": [ 171, 1 ], "end": [ 179, 44 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.callLeanMkStringUncheckedFn", "code": "def callLeanMkStringUncheckedFn (builder : LLVM.Builder llvmctx)\n (strPtr nBytes nChars : LLVM.Value llvmctx) (name : String) : M llvmctx (LLVM.Value llvmctx) := do\n let fnName := \"lean_mk_string_unchecked\"\n let retty ← LLVM.voidPtrType llvmctx\n let argtys := #[← LLVM.voidPtrType llvmctx, ← LLVM.size_tType llvmctx, ← LLVM.size_tType llvmctx]\n let fn ← getOrCreateFunctionPrototype (← getLLVMModule) retty fnName argtys\n let fnty ← LLVM.functionType retty argtys\n LLVM.buildCall2 builder fnty fn #[strPtr, nBytes, nChars] name", "start": [ 181, 1 ], "end": [ 188, 65 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.callLeanMkString", "code": "def callLeanMkString (builder : LLVM.Builder llvmctx)\n (strPtr : LLVM.Value llvmctx) (name : String) : M llvmctx (LLVM.Value llvmctx) := do\n let retty ← LLVM.voidPtrType llvmctx\n let argtys := #[← LLVM.voidPtrType llvmctx]\n let fn ← getOrCreateFunctionPrototype (← getLLVMModule) retty \"lean_mk_string\" argtys\n let fnty ← LLVM.functionType retty argtys\n LLVM.buildCall2 builder fnty fn #[strPtr] name", "start": [ 190, 1 ], "end": [ 196, 49 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.callLeanCStrToNatFn", "code": "def callLeanCStrToNatFn (builder : LLVM.Builder llvmctx)\n (n : Nat) (name : String := \"\") : M llvmctx (LLVM.Value llvmctx) := do\n let fnName := \"lean_cstr_to_nat\"\n let retty ← LLVM.voidPtrType llvmctx\n let argtys := #[← LLVM.voidPtrType llvmctx]\n let fn ← getOrCreateFunctionPrototype (← getLLVMModule) retty fnName argtys\n let fnty ← LLVM.functionType retty argtys\n let s ← LLVM.buildGlobalString builder (value := toString n)\n LLVM.buildCall2 builder fnty fn #[s] name", "start": [ 198, 1 ], "end": [ 206, 44 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.callLeanIOMkWorld", "code": "def callLeanIOMkWorld (builder : LLVM.Builder llvmctx) : M llvmctx (LLVM.Value llvmctx) := do\n let fnName := \"lean_io_mk_world\"\n let retty ← LLVM.voidPtrType llvmctx\n let argtys := #[]\n let fn ← getOrCreateFunctionPrototype (← getLLVMModule) retty fnName argtys\n let fnty ← LLVM.functionType retty argtys\n LLVM.buildCall2 builder fnty fn #[] \"mk_io_out\"", "start": [ 208, 1 ], "end": [ 214, 50 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.callLeanIOResultIsError", "code": "def callLeanIOResultIsError (builder : LLVM.Builder llvmctx)\n (arg : LLVM.Value llvmctx) (name : String := \"\") : M llvmctx (LLVM.Value llvmctx) := do\n let fnName := \"lean_io_result_is_error\"\n let retty ← LLVM.i1Type llvmctx\n let argtys := #[← LLVM.voidPtrType llvmctx]\n let fn ← getOrCreateFunctionPrototype (← getLLVMModule) retty fnName argtys\n let fnty ← LLVM.functionType retty argtys\n LLVM.buildCall2 builder fnty fn #[arg] name", "start": [ 216, 1 ], "end": [ 223, 46 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.callLeanAllocCtor", "code": "def callLeanAllocCtor (builder : LLVM.Builder llvmctx)\n (tag num_objs scalar_sz : Nat) (name : String := \"\") : M llvmctx (LLVM.Value llvmctx) := do\n let fnName := \"lean_alloc_ctor\"\n let retty ← LLVM.voidPtrType llvmctx\n let i32 ← LLVM.i32Type llvmctx\n let argtys := #[i32, i32, i32]\n let fn ← getOrCreateFunctionPrototype (← getLLVMModule) retty fnName argtys\n let fnty ← LLVM.functionType retty argtys\n\n let tag ← constIntUnsigned tag\n let num_objs ← constIntUnsigned num_objs\n let scalar_sz ← constIntUnsigned scalar_sz\n LLVM.buildCall2 builder fnty fn #[tag, num_objs, scalar_sz] name", "start": [ 225, 1 ], "end": [ 237, 67 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.callLeanCtorSet", "code": "def callLeanCtorSet (builder : LLVM.Builder llvmctx)\n (o i v : LLVM.Value llvmctx) : M llvmctx Unit := do\n let fnName := \"lean_ctor_set\"\n let retty ← LLVM.voidType llvmctx\n let voidptr ← LLVM.voidPtrType llvmctx\n let unsigned ← LLVM.unsignedType llvmctx\n let argtys := #[voidptr, unsigned, voidptr]\n let fn ← getOrCreateFunctionPrototype (← getLLVMModule) retty fnName argtys\n let fnty ← LLVM.functionType retty argtys\n _ <- LLVM.buildCall2 builder fnty fn #[o, i, v]", "start": [ 239, 1 ], "end": [ 248, 51 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.callLeanIOResultMKOk", "code": "def callLeanIOResultMKOk (builder : LLVM.Builder llvmctx)\n (v : LLVM.Value llvmctx) (name : String := \"\") : M llvmctx (LLVM.Value llvmctx) := do\n let fnName := \"lean_io_result_mk_ok\"\n let voidptr ← LLVM.voidPtrType llvmctx\n let retty := voidptr\n let argtys := #[voidptr]\n let fn ← getOrCreateFunctionPrototype (← getLLVMModule) retty fnName argtys\n let fnty ← LLVM.functionType retty argtys\n LLVM.buildCall2 builder fnty fn #[v] name", "start": [ 250, 1 ], "end": [ 258, 44 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.callLeanAllocClosureFn", "code": "def callLeanAllocClosureFn (builder : LLVM.Builder llvmctx)\n (f arity nys : LLVM.Value llvmctx) (retName : String := \"\") : M llvmctx (LLVM.Value llvmctx) := do\n let fnName := \"lean_alloc_closure\"\n let retty ← LLVM.voidPtrType llvmctx\n let argtys := #[ ← LLVM.voidPtrType llvmctx, ← LLVM.unsignedType llvmctx, ← LLVM.unsignedType llvmctx]\n let fn ← getOrCreateFunctionPrototype (← getLLVMModule) retty fnName argtys\n let fnty ← LLVM.functionType retty argtys\n LLVM.buildCall2 builder fnty fn #[f, arity, nys] retName", "start": [ 260, 1 ], "end": [ 267, 60 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.callLeanClosureSetFn", "code": "def callLeanClosureSetFn (builder : LLVM.Builder llvmctx)\n (closure ix arg : LLVM.Value llvmctx) (retName : String := \"\") : M llvmctx Unit := do\n let fnName := \"lean_closure_set\"\n let retty ← LLVM.voidType llvmctx\n let argtys := #[ ← LLVM.voidPtrType llvmctx, ← LLVM.unsignedType llvmctx, ← LLVM.voidPtrType llvmctx]\n let fn ← getOrCreateFunctionPrototype (← getLLVMModule) retty fnName argtys\n let fnty ← LLVM.functionType retty argtys\n let _ ← LLVM.buildCall2 builder fnty fn #[closure, ix, arg] retName", "start": [ 269, 1 ], "end": [ 276, 71 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.callLeanObjTag", "code": "def callLeanObjTag (builder : LLVM.Builder llvmctx)\n (closure : LLVM.Value llvmctx) (retName : String := \"\") : M llvmctx (LLVM.Value llvmctx) := do\n let fnName := \"lean_obj_tag\"\n let retty ← LLVM.i32Type llvmctx\n let argtys := #[ ← LLVM.voidPtrType llvmctx]\n let fn ← getOrCreateFunctionPrototype (← getLLVMModule) retty fnName argtys\n let fnty ← LLVM.functionType retty argtys\n let out ← LLVM.buildCall2 builder fnty fn #[closure] retName\n LLVM.buildSextOrTrunc builder out (← LLVM.i64Type llvmctx)", "start": [ 278, 1 ], "end": [ 286, 61 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.callLeanIOResultGetValue", "code": "def callLeanIOResultGetValue (builder : LLVM.Builder llvmctx)\n (v : LLVM.Value llvmctx) (name : String := \"\") : M llvmctx (LLVM.Value llvmctx) := do\n let fnName := \"lean_io_result_get_value\"\n let retty ← LLVM.voidPtrType llvmctx\n let argtys := #[ ← LLVM.voidPtrType llvmctx]\n let fn ← getOrCreateFunctionPrototype (← getLLVMModule) retty fnName argtys\n let fnty ← LLVM.functionType retty argtys\n LLVM.buildCall2 builder fnty fn #[v] name", "start": [ 288, 1 ], "end": [ 295, 44 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.callLeanCtorRelease", "code": "def callLeanCtorRelease (builder : LLVM.Builder llvmctx)\n (closure i : LLVM.Value llvmctx) (retName : String := \"\") : M llvmctx Unit := do\n let fnName := \"lean_ctor_release\"\n let retty ← LLVM.voidType llvmctx\n let argtys := #[ ← LLVM.voidPtrType llvmctx, ← LLVM.unsignedType llvmctx]\n let fn ← getOrCreateFunctionPrototype (← getLLVMModule) retty fnName argtys\n let fnty ← LLVM.functionType retty argtys\n let _ ← LLVM.buildCall2 builder fnty fn #[closure, i] retName", "start": [ 297, 1 ], "end": [ 304, 65 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.callLeanCtorSetTag", "code": "def callLeanCtorSetTag (builder : LLVM.Builder llvmctx)\n (closure i : LLVM.Value llvmctx) (retName : String := \"\") : M llvmctx Unit := do\n let fnName := \"lean_ctor_set_tag\"\n let retty ← LLVM.voidType llvmctx\n let argtys := #[ ← LLVM.voidPtrType llvmctx, ← LLVM.i8Type llvmctx]\n let fn ← getOrCreateFunctionPrototype (← getLLVMModule) retty fnName argtys\n let fnty ← LLVM.functionType retty argtys\n let _ ← LLVM.buildCall2 builder fnty fn #[closure, i] retName", "start": [ 306, 1 ], "end": [ 313, 65 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.toLLVMType", "code": "def toLLVMType (t : IRType) : M llvmctx (LLVM.LLVMType llvmctx) := do\n match t with\n | IRType.float => LLVM.doubleTypeInContext llvmctx\n | IRType.uint8 => LLVM.intTypeInContext llvmctx 8\n | IRType.uint16 => LLVM.intTypeInContext llvmctx 16\n | IRType.uint32 => LLVM.intTypeInContext llvmctx 32\n | IRType.uint64 => LLVM.intTypeInContext llvmctx 64\n | IRType.usize => LLVM.size_tType llvmctx\n | IRType.object => do LLVM.pointerType (← LLVM.i8Type llvmctx)\n | IRType.tobject => do LLVM.pointerType (← LLVM.i8Type llvmctx)\n | IRType.irrelevant => do LLVM.pointerType (← LLVM.i8Type llvmctx)\n | IRType.struct _ _ => panic! \"not implemented yet\"\n | IRType.union _ _ => panic! \"not implemented yet\"", "start": [ 315, 1 ], "end": [ 328, 54 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.throwInvalidExportName", "code": "def throwInvalidExportName {Ξ± : Type} (n : Name) : M llvmctx Ξ± := do\n throw s!\"invalid export name {n.toString}\"", "start": [ 330, 1 ], "end": [ 331, 45 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.toCName", "code": "def toCName (n : Name) : M llvmctx String := do\n match getExportNameFor? (← getEnv) n with\n | some (.str .anonymous s) => pure s\n | some _ => throwInvalidExportName n\n | none => if n == `main then pure leanMainFn else pure n.mangle", "start": [ 333, 1 ], "end": [ 337, 86 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.toCInitName", "code": "def toCInitName (n : Name) : M llvmctx String := do\n match getExportNameFor? (← getEnv) n with\n | some (.str .anonymous s) => return \"_init_\" ++ s\n | some _ => throwInvalidExportName n\n | none => pure (\"_init_\" ++ n.mangle)", "start": [ 339, 1 ], "end": [ 343, 60 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.ShouldForwardControlFlow", "code": "inductive ShouldForwardControlFlow where\n| yes | no", "start": [ 345, 1 ], "end": [ 352, 11 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.builderGetInsertionFn", "code": "def builderGetInsertionFn (builder : LLVM.Builder llvmctx) : M llvmctx (LLVM.Value llvmctx) := do\n let builderBB ← LLVM.getInsertBlock builder\n LLVM.getBasicBlockParent builderBB", "start": [ 355, 1 ], "end": [ 357, 37 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.builderAppendBasicBlock", "code": "def builderAppendBasicBlock (builder : LLVM.Builder llvmctx) (name : String) : M llvmctx (LLVM.BasicBlock llvmctx) := do\n let fn ← builderGetInsertionFn builder\n LLVM.appendBasicBlockInContext llvmctx fn name", "start": [ 359, 1 ], "end": [ 361, 49 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.buildPrologueAlloca", "code": "def buildPrologueAlloca (builder : LLVM.Builder llvmctx) (ty : LLVM.LLVMType llvmctx) (name : @&String := \"\") : M llvmctx (LLVM.Value llvmctx) := do\n let origBB ← LLVM.getInsertBlock builder\n\n let fn ← builderGetInsertionFn builder\n if (← LLVM.countBasicBlocks fn) == 0 then\n throw \"Attempt to obtain first BB of function without BBs\"\n\n let entryBB ← LLVM.getEntryBasicBlock fn\n match ← LLVM.getFirstInstruction entryBB with\n | some instr => LLVM.positionBuilderBefore builder instr\n | none => LLVM.positionBuilderAtEnd builder entryBB\n\n let alloca ← LLVM.buildAlloca builder ty name\n LLVM.positionBuilderAtEnd builder origBB\n return alloca", "start": [ 363, 1 ], "end": [ 385, 16 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.buildWhile_", "code": "def buildWhile_ (builder : LLVM.Builder llvmctx) (name : String)\n (condcodegen : LLVM.Builder llvmctx β†’ M llvmctx (LLVM.Value llvmctx))\n (bodycodegen : LLVM.Builder llvmctx β†’ M llvmctx Unit) : M llvmctx Unit := do\n let fn ← builderGetInsertionFn builder\n\n let nameHeader := name ++ \"header\"\n let nameBody := name ++ \"body\"\n let nameMerge := name ++ \"merge\"\n\n let headerbb ← LLVM.appendBasicBlockInContext llvmctx fn nameHeader\n let _ ← LLVM.buildBr builder headerbb\n\n let bodybb ← LLVM.appendBasicBlockInContext llvmctx fn nameBody\n let mergebb ← LLVM.appendBasicBlockInContext llvmctx fn nameMerge\n\n LLVM.positionBuilderAtEnd builder headerbb\n let cond ← condcodegen builder\n let _ ← LLVM.buildCondBr builder cond bodybb mergebb\n\n LLVM.positionBuilderAtEnd builder bodybb\n bodycodegen builder\n let _ ← LLVM.buildBr builder headerbb\n\n LLVM.positionBuilderAtEnd builder mergebb", "start": [ 388, 1 ], "end": [ 415, 44 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.buildIfThen_", "code": "def buildIfThen_ (builder : LLVM.Builder llvmctx) (name : String) (brval : LLVM.Value llvmctx)\n (thencodegen : LLVM.Builder llvmctx β†’ M llvmctx ShouldForwardControlFlow) : M llvmctx Unit := do\n let fn ← builderGetInsertionFn builder\n\n let nameThen := name ++ \"Then\"\n let nameElse := name ++ \"Else\"\n let nameMerge := name ++ \"Merge\"\n\n let thenbb ← LLVM.appendBasicBlockInContext llvmctx fn nameThen\n let elsebb ← LLVM.appendBasicBlockInContext llvmctx fn nameElse\n let mergebb ← LLVM.appendBasicBlockInContext llvmctx fn nameMerge\n let _ ← LLVM.buildCondBr builder brval thenbb elsebb\n LLVM.positionBuilderAtEnd builder thenbb\n let fwd? ← thencodegen builder\n match fwd? with\n | .yes => let _ ← LLVM.buildBr builder mergebb\n | .no => pure ()\n LLVM.positionBuilderAtEnd builder elsebb\n let _ ← LLVM.buildBr builder mergebb\n LLVM.positionBuilderAtEnd builder mergebb", "start": [ 419, 1 ], "end": [ 441, 44 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.buildIfThenElse_", "code": "def buildIfThenElse_ (builder : LLVM.Builder llvmctx) (name : String) (brval : LLVM.Value llvmctx)\n (thencodegen : LLVM.Builder llvmctx β†’ M llvmctx ShouldForwardControlFlow)\n (elsecodegen : LLVM.Builder llvmctx β†’ M llvmctx ShouldForwardControlFlow) : M llvmctx Unit := do\n let fn ← LLVM.getBasicBlockParent (← LLVM.getInsertBlock builder)\n let thenbb ← LLVM.appendBasicBlockInContext llvmctx fn (name ++ \"Then\")\n let elsebb ← LLVM.appendBasicBlockInContext llvmctx fn (name ++ \"Else\")\n let mergebb ← LLVM.appendBasicBlockInContext llvmctx fn (name ++ \"Merge\")\n let _ ← LLVM.buildCondBr builder brval thenbb elsebb\n LLVM.positionBuilderAtEnd builder thenbb\n let fwd? ← thencodegen builder\n match fwd? with\n | .yes => let _ ← LLVM.buildBr builder mergebb\n | .no => pure ()\n LLVM.positionBuilderAtEnd builder elsebb\n let fwd? ← elsecodegen builder\n match fwd? with\n | .yes => let _ ← LLVM.buildBr builder mergebb\n | .no => pure ()\n LLVM.positionBuilderAtEnd builder mergebb", "start": [ 443, 1 ], "end": [ 464, 44 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.buildLeanBoolTrue?", "code": "def buildLeanBoolTrue? (builder : LLVM.Builder llvmctx)\n (b : LLVM.Value llvmctx) (name : String := \"\") : M llvmctx (LLVM.Value llvmctx) := do\n LLVM.buildICmp builder LLVM.IntPredicate.NE b (← constInt8 0) name", "start": [ 467, 1 ], "end": [ 469, 69 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitFnDeclAux", "code": "def emitFnDeclAux (mod : LLVM.Module llvmctx)\n (decl : Decl) (cppBaseName : String) (isExternal : Bool) : M llvmctx (LLVM.Value llvmctx) := do\n let ps := decl.params\n let env ← getEnv\n let global ←\n if ps.isEmpty then\n let retty ← (toLLVMType decl.resultType)\n let global ← LLVM.getOrAddGlobal mod cppBaseName retty\n if !isExternal then\n LLVM.setInitializer global (← LLVM.getUndef retty)\n pure global\n else\n let retty ← (toLLVMType decl.resultType)\n let mut argtys := #[]\n for p in ps do\n if !(isExternC env decl.name) || !p.ty.isIrrelevant then\n argtys := argtys.push (← toLLVMType p.ty)\n if argtys.size > closureMaxArgs && isBoxedName decl.name then\n argtys := #[← LLVM.pointerType (← LLVM.voidPtrType llvmctx)]\n let fnty ← LLVM.functionType retty argtys (isVarArg := false)\n LLVM.getOrAddFunction mod cppBaseName fnty\n if ps.isEmpty then\n if isClosedTermName env decl.name then LLVM.setVisibility global LLVM.Visibility.hidden else if isExternal then pure () else LLVM.setDLLStorageClass global LLVM.DLLStorageClass.export else if !isExternal\n then LLVM.setDLLStorageClass global LLVM.DLLStorageClass.export\n return global", "start": [ 471, 1 ], "end": [ 507, 16 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitFnDecl", "code": "def emitFnDecl (decl : Decl) (isExternal : Bool) : M llvmctx Unit := do\n let cppBaseName ← toCName decl.name\n let _ ← emitFnDeclAux (← getLLVMModule) decl cppBaseName isExternal", "start": [ 510, 1 ], "end": [ 512, 70 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitExternDeclAux", "code": "def emitExternDeclAux (decl : Decl) (cNameStr : String) : M llvmctx Unit := do\n let env ← getEnv\n let extC := isExternC env decl.name\n let _ ← emitFnDeclAux (← getLLVMModule) decl cNameStr extC", "start": [ 514, 1 ], "end": [ 517, 61 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitFnDecls", "code": "def emitFnDecls : M llvmctx Unit := do\n let env ← getEnv\n let decls := getDecls env\n let modDecls : NameSet := decls.foldl (fun s d => s.insert d.name) {}\n let usedDecls : NameSet := decls.foldl (fun s d => collectUsedDecls env d (s.insert d.name)) {}\n let usedDecls := usedDecls.toList\n for n in usedDecls do\n let decl ← getDecl n\n match getExternNameFor env `c decl.name with\n | some cName => emitExternDeclAux decl cName\n | none => emitFnDecl decl (!modDecls.contains n)\n return ()", "start": [ 519, 1 ], "end": [ 530, 12 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitLhsSlot_", "code": "def emitLhsSlot_ (x : VarId) : M llvmctx (LLVM.LLVMType llvmctx Γ— LLVM.Value llvmctx) := do\n let state ← get\n match state.var2val.find? x with\n | .some v => return v\n | .none => throw s!\"unable to find variable {x}\"", "start": [ 532, 1 ], "end": [ 536, 51 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitLhsVal", "code": "def emitLhsVal (builder : LLVM.Builder llvmctx)\n (x : VarId) (name : String := \"\") : M llvmctx (LLVM.Value llvmctx) := do\n let (xty, xslot) ← emitLhsSlot_ x\n LLVM.buildLoad2 builder xty xslot name", "start": [ 538, 1 ], "end": [ 541, 41 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitLhsSlotStore", "code": "def emitLhsSlotStore (builder : LLVM.Builder llvmctx)\n (x : VarId) (v : LLVM.Value llvmctx) : M llvmctx Unit := do\n let (_, slot) ← emitLhsSlot_ x\n LLVM.buildStore builder v slot", "start": [ 543, 1 ], "end": [ 546, 33 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitArgSlot_", "code": "def emitArgSlot_ (builder : LLVM.Builder llvmctx)\n (x : Arg) : M llvmctx (LLVM.LLVMType llvmctx Γ— LLVM.Value llvmctx) := do\n match x with\n | Arg.var x => emitLhsSlot_ x\n | _ => do\n let slotty ← LLVM.voidPtrType llvmctx\n let slot ← buildPrologueAlloca builder slotty \"irrelevant_slot\"\n let v ← callLeanBox builder (← constIntSizeT 0) \"irrelevant_val\"\n let _ ← LLVM.buildStore builder v slot\n return (slotty, slot)", "start": [ 548, 1 ], "end": [ 557, 26 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitArgVal", "code": "def emitArgVal (builder : LLVM.Builder llvmctx)\n (x : Arg) (name : String := \"\") : M llvmctx (LLVM.LLVMType llvmctx Γ— LLVM.Value llvmctx) := do\n let (xty, xslot) ← emitArgSlot_ builder x\n let xval ← LLVM.buildLoad2 builder xty xslot name\n return (xty, xval)", "start": [ 559, 1 ], "end": [ 563, 21 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitAllocCtor", "code": "def emitAllocCtor (builder : LLVM.Builder llvmctx)\n (c : CtorInfo) : M llvmctx (LLVM.Value llvmctx) := do\n let hackSizeofVoidPtr := 8\n let scalarSize := hackSizeofVoidPtr * c.usize + c.ssize\n callLeanAllocCtor builder c.cidx c.size scalarSize \"lean_alloc_ctor_out\"", "start": [ 565, 1 ], "end": [ 570, 75 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitCtorSetArgs", "code": "def emitCtorSetArgs (builder : LLVM.Builder llvmctx)\n (z : VarId) (ys : Array Arg) : M llvmctx Unit := do\n ys.size.forM fun i => do\n let zv ← emitLhsVal builder z\n let (_yty, yv) ← emitArgVal builder ys[i]!\n let iv ← constIntUnsigned i\n callLeanCtorSet builder zv iv yv\n emitLhsSlotStore builder z zv\n pure ()", "start": [ 572, 1 ], "end": [ 580, 12 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitCtor", "code": "def emitCtor (builder : LLVM.Builder llvmctx)\n (z : VarId) (c : CtorInfo) (ys : Array Arg) : M llvmctx Unit := do\n let (_llvmty, slot) ← emitLhsSlot_ z\n if c.size == 0 && c.usize == 0 && c.ssize == 0 then do\n let v ← callLeanBox builder (← constIntSizeT c.cidx) \"lean_box_outv\"\n let _ ← LLVM.buildStore builder v slot\n else do\n let v ← emitAllocCtor builder c\n let _ ← LLVM.buildStore builder v slot\n emitCtorSetArgs builder z ys", "start": [ 582, 1 ], "end": [ 591, 33 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitInc", "code": "def emitInc (builder : LLVM.Builder llvmctx)\n (x : VarId) (n : Nat) (checkRef? : Bool) : M llvmctx Unit := do\n let xv ← emitLhsVal builder x\n if n != 1\n then do\n let nv ← constIntSizeT n\n callLeanRefcountFn builder (kind := RefcountKind.inc) (checkRef? := checkRef?) (delta := nv) xv\n else callLeanRefcountFn builder (kind := RefcountKind.inc) (checkRef? := checkRef?) xv", "start": [ 593, 1 ], "end": [ 600, 89 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitDec", "code": "def emitDec (builder : LLVM.Builder llvmctx)\n (x : VarId) (n : Nat) (checkRef? : Bool) : M llvmctx Unit := do\n let xv ← emitLhsVal builder x\n if n != 1\n then throw \"expected n = 1 for emitDec\"\n else callLeanRefcountFn builder (kind := RefcountKind.dec) (checkRef? := checkRef?) xv", "start": [ 602, 1 ], "end": [ 607, 89 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitNumLit", "code": "def emitNumLit (builder : LLVM.Builder llvmctx)\n (t : IRType) (v : Nat) : M llvmctx (LLVM.Value llvmctx) := do\n if t.isObj then\n if v < UInt32.size then\n callLeanUnsignedToNatFn builder v\n else\n callLeanCStrToNatFn builder v\n else\n LLVM.constInt (← toLLVMType t) (UInt64.ofNat v)", "start": [ 609, 1 ], "end": [ 617, 52 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.toHexDigit", "code": "def toHexDigit (c : Nat) : String :=\n String.singleton c.digitChar", "start": [ 619, 1 ], "end": [ 620, 31 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.quoteString", "code": "def quoteString (s : String) : String :=\n let q := \"\\\"\";\n let q := s.foldl\n (fun q c => q ++\n if c == '\\n' then \"\\\\n\"\n else if c == '\\r' then \"\\\\r\"\n else if c == '\\t' then \"\\\\t\"\n else if c == '\\\\' then \"\\\\\\\\\"\n else if c == '\\\"' then \"\\\\\\\"\"\n else if c.toNat <= 31 then\n \"\\\\x\" ++ toHexDigit (c.toNat / 16) ++ toHexDigit (c.toNat % 16)\n else String.singleton c)\n q;\n q ++ \"\\\"\"", "start": [ 623, 1 ], "end": [ 637, 12 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitSimpleExternalCall", "code": "def emitSimpleExternalCall (builder : LLVM.Builder llvmctx)\n (f : String)\n (ps : Array Param)\n (ys : Array Arg)\n (retty : IRType)\n (name : String) : M llvmctx (LLVM.Value llvmctx) := do\n let mut args := #[]\n let mut argTys := #[]\n for (p, y) in ps.zip ys do\n if !p.ty.isIrrelevant then\n let (_yty, yv) ← emitArgVal builder y \"\"\n argTys := argTys.push (← toLLVMType p.ty)\n args := args.push yv\n let fnty ← LLVM.functionType (← toLLVMType retty) argTys\n let fn ← LLVM.getOrAddFunction (← getLLVMModule) f fnty\n LLVM.buildCall2 builder fnty fn args name", "start": [ 639, 1 ], "end": [ 654, 44 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitExternCall", "code": "def emitExternCall (builder : LLVM.Builder llvmctx)\n (f : FunId)\n (ps : Array Param)\n (extData : ExternAttrData)\n (ys : Array Arg) (retty : IRType)\n (name : String := \"\") : M llvmctx (LLVM.Value llvmctx) :=\n match getExternEntryFor extData `c with\n | some (ExternEntry.standard _ extFn) => emitSimpleExternalCall builder extFn ps ys retty name\n | some (ExternEntry.inline `llvm _pat) => throw \"Unimplemented codegen of inline LLVM\"\n | some (ExternEntry.inline _ pat) => throw s!\"Cannot codegen non-LLVM inline code '{pat}'.\"\n | some (ExternEntry.foreign _ extFn) => emitSimpleExternalCall builder extFn ps ys retty name\n | _ => throw s!\"Failed to emit extern application '{f}'.\"", "start": [ 658, 1 ], "end": [ 669, 60 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.getFunIdTy", "code": "def getFunIdTy (f : FunId) : M llvmctx (LLVM.LLVMType llvmctx) := do\n let decl ← getDecl f\n let retty ← toLLVMType decl.resultType\n let argtys ← decl.params.mapM (fun p => do toLLVMType p.ty)\n LLVM.functionType retty argtys", "start": [ 671, 1 ], "end": [ 675, 33 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.getOrAddFunIdValue", "code": "def getOrAddFunIdValue (builder : LLVM.Builder llvmctx) (f : FunId) : M llvmctx (LLVM.Value llvmctx) := do\n let decl ← getDecl f\n let fcname ← toCName f\n let retty ← toLLVMType decl.resultType\n if decl.params.isEmpty then\n let gslot ← LLVM.getOrAddGlobal (← getLLVMModule) fcname retty\n LLVM.buildLoad2 builder retty gslot\n else\n let argtys ← decl.params.mapM (fun p => do toLLVMType p.ty)\n let fnty ← LLVM.functionType retty argtys\n LLVM.getOrAddFunction (← getLLVMModule) fcname fnty", "start": [ 677, 1 ], "end": [ 694, 56 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitPartialApp", "code": "def emitPartialApp (builder : LLVM.Builder llvmctx) (z : VarId) (f : FunId) (ys : Array Arg) : M llvmctx Unit := do\n let decl ← getDecl f\n let fv ← getOrAddFunIdValue builder f\n let arity := decl.params.size\n let (_zty, zslot) ← emitLhsSlot_ z\n let zval ← callLeanAllocClosureFn builder fv\n (← constIntUnsigned arity)\n (← constIntUnsigned ys.size)\n LLVM.buildStore builder zval zslot\n ys.size.forM fun i => do\n let (yty, yslot) ← emitArgSlot_ builder ys[i]!\n let yval ← LLVM.buildLoad2 builder yty yslot\n callLeanClosureSetFn builder zval (← constIntUnsigned i) yval", "start": [ 696, 1 ], "end": [ 708, 66 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitApp", "code": "def emitApp (builder : LLVM.Builder llvmctx) (z : VarId) (f : VarId) (ys : Array Arg) : M llvmctx Unit := do\n if ys.size > closureMaxArgs then do\n let aargs ← buildPrologueAlloca builder (← LLVM.arrayType (← LLVM.voidPtrType llvmctx) (UInt64.ofNat ys.size)) \"aargs\"\n for i in List.range ys.size do\n let (yty, yv) ← emitArgVal builder ys[i]!\n let aslot ← LLVM.buildInBoundsGEP2 builder yty aargs #[← constIntUnsigned 0, ← constIntUnsigned i] s!\"param_{i}_slot\"\n LLVM.buildStore builder yv aslot\n let fnName := s!\"lean_apply_m\"\n let retty ← LLVM.voidPtrType llvmctx\n let args := #[← emitLhsVal builder f, ← constIntUnsigned ys.size, aargs]\n let argtys := #[← LLVM.voidPtrType llvmctx, ← LLVM.unsignedType llvmctx, ← LLVM.voidPtrType llvmctx]\n let fn ← getOrCreateFunctionPrototype (← getLLVMModule) retty fnName argtys\n let fnty ← LLVM.functionType retty argtys\n let zv ← LLVM.buildCall2 builder fnty fn args\n emitLhsSlotStore builder z zv\n else do\n\n let fnName := s!\"lean_apply_{ys.size}\"\n let retty ← LLVM.voidPtrType llvmctx\n let args : Array (LLVM.Value llvmctx) := #[← emitLhsVal builder f] ++ (← ys.mapM (fun y => Prod.snd <$> (emitArgVal builder y)))\n let argtys := (List.replicate (1 + ys.size) (← LLVM.voidPtrType llvmctx)).toArray\n let fn ← getOrCreateFunctionPrototype (← getLLVMModule) retty fnName argtys\n let fnty ← LLVM.functionType retty argtys\n let zv ← LLVM.buildCall2 builder fnty fn args\n emitLhsSlotStore builder z zv", "start": [ 710, 1 ], "end": [ 736, 34 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitFullApp", "code": "def emitFullApp (builder : LLVM.Builder llvmctx)\n (z : VarId) (f : FunId) (ys : Array Arg) : M llvmctx Unit := do\n let (__zty, zslot) ← emitLhsSlot_ z\n let decl ← getDecl f\n match decl with\n | Decl.extern _ ps retty extData =>\n let zv ← emitExternCall builder f ps extData ys retty\n LLVM.buildStore builder zv zslot\n | Decl.fdecl .. =>\n if ys.size > 0 then\n let fv ← getOrAddFunIdValue builder f\n let ys ← ys.mapM (fun y => do\n let (yty, yslot) ← emitArgSlot_ builder y\n let yv ← LLVM.buildLoad2 builder yty yslot\n return yv)\n let zv ← LLVM.buildCall2 builder (← getFunIdTy f) fv ys\n LLVM.buildStore builder zv zslot\n else\n let zv ← getOrAddFunIdValue builder f\n LLVM.buildStore builder zv zslot", "start": [ 738, 1 ], "end": [ 757, 40 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitLit", "code": "def emitLit (builder : LLVM.Builder llvmctx)\n (z : VarId) (t : IRType) (v : LitVal) : M llvmctx (LLVM.Value llvmctx) := do\n let llvmty ← toLLVMType t\n let zslot ← buildPrologueAlloca builder llvmty\n addVartoState z zslot llvmty\n let zv ← match v with\n | LitVal.num v => emitNumLit builder t v\n | LitVal.str v =>\n let zero ← constIntUnsigned 0\n let str_global ← LLVM.buildGlobalString builder v\n let strPtr ← LLVM.buildInBoundsGEP2 builder\n (← LLVM.opaquePointerTypeInContext llvmctx)\n str_global #[zero] \"\"\n let nbytes ← constIntSizeT v.utf8ByteSize\n let nchars ← constIntSizeT v.length\n callLeanMkStringUncheckedFn builder strPtr nbytes nchars \"\"\n LLVM.buildStore builder zv zslot\n return zslot", "start": [ 760, 1 ], "end": [ 778, 15 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.callLeanCtorGet", "code": "def callLeanCtorGet (builder : LLVM.Builder llvmctx)\n (x i : LLVM.Value llvmctx) (retName : String) : M llvmctx (LLVM.Value llvmctx) := do\n let fnName := \"lean_ctor_get\"\n let retty ← LLVM.voidPtrType llvmctx\n let argtys := #[ ← LLVM.voidPtrType llvmctx, ← LLVM.i32Type llvmctx]\n let fnty ← LLVM.functionType retty argtys\n let fn ← getOrCreateFunctionPrototype (← getLLVMModule) retty fnName argtys\n let i ← LLVM.buildSextOrTrunc builder i (← LLVM.i32Type llvmctx)\n LLVM.buildCall2 builder fnty fn #[x, i] retName", "start": [ 780, 1 ], "end": [ 788, 51 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitProj", "code": "def emitProj (builder : LLVM.Builder llvmctx) (z : VarId) (i : Nat) (x : VarId) : M llvmctx Unit := do\n let xval ← emitLhsVal builder x\n let zval ← callLeanCtorGet builder xval (← constIntUnsigned i) \"\"\n emitLhsSlotStore builder z zval", "start": [ 790, 1 ], "end": [ 793, 34 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.callLeanCtorGetUsize", "code": "def callLeanCtorGetUsize (builder : LLVM.Builder llvmctx)\n (x i : LLVM.Value llvmctx) (retName : String) : M llvmctx (LLVM.Value llvmctx) := do\n let fnName := \"lean_ctor_get_usize\"\n let retty ← LLVM.size_tType llvmctx\n let argtys := #[ ← LLVM.voidPtrType llvmctx, ← LLVM.unsignedType llvmctx]\n let fnty ← LLVM.functionType retty argtys\n let fn ← getOrCreateFunctionPrototype (← getLLVMModule) retty fnName argtys\n LLVM.buildCall2 builder fnty fn #[x, i] retName", "start": [ 795, 1 ], "end": [ 802, 51 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitUProj", "code": "def emitUProj (builder : LLVM.Builder llvmctx) (z : VarId) (i : Nat) (x : VarId) : M llvmctx Unit := do\n let xval ← emitLhsVal builder x\n let zval ← callLeanCtorGetUsize builder xval (← constIntUnsigned i) \"\"\n emitLhsSlotStore builder z zval", "start": [ 804, 1 ], "end": [ 807, 34 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitOffset", "code": "def emitOffset (builder : LLVM.Builder llvmctx)\n (n : Nat) (offset : Nat) : M llvmctx (LLVM.Value llvmctx) := do\n let out ← constIntUnsigned 8\n let out ← LLVM.buildMul builder out (← constIntUnsigned n) \"\" LLVM.buildAdd builder out (← constIntUnsigned offset) \"\"", "start": [ 809, 1 ], "end": [ 814, 60 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitSProj", "code": "def emitSProj (builder : LLVM.Builder llvmctx)\n (z : VarId) (t : IRType) (n offset : Nat) (x : VarId) : M llvmctx Unit := do\n let (fnName, retty) ←\n match t with\n | IRType.float => pure (\"lean_ctor_get_float\", ← LLVM.doubleTypeInContext llvmctx)\n | IRType.uint8 => pure (\"lean_ctor_get_uint8\", ← LLVM.i8Type llvmctx)\n | IRType.uint16 => pure (\"lean_ctor_get_uint16\", ← LLVM.i16Type llvmctx)\n | IRType.uint32 => pure (\"lean_ctor_get_uint32\", ← LLVM.i32Type llvmctx)\n | IRType.uint64 => pure (\"lean_ctor_get_uint64\", ← LLVM.i64Type llvmctx)\n | _ => throw s!\"Invalid type for lean_ctor_get: '{t}'\"\n let argtys := #[ ← LLVM.voidPtrType llvmctx, ← LLVM.unsignedType llvmctx]\n let fn ← getOrCreateFunctionPrototype (← getLLVMModule) retty fnName argtys\n let xval ← emitLhsVal builder x\n let offset ← emitOffset builder n offset\n let fnty ← LLVM.functionType retty argtys\n let zval ← LLVM.buildCall2 builder fnty fn #[xval, offset]\n emitLhsSlotStore builder z zval", "start": [ 816, 1 ], "end": [ 832, 34 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.callLeanIsExclusive", "code": "def callLeanIsExclusive (builder : LLVM.Builder llvmctx)\n (closure : LLVM.Value llvmctx) (retName : String := \"\") : M llvmctx (LLVM.Value llvmctx) := do\n let fnName := \"lean_is_exclusive\"\n let retty ← LLVM.i1Type llvmctx\n let argtys := #[ ← LLVM.voidPtrType llvmctx]\n let fn ← getOrCreateFunctionPrototype (← getLLVMModule) retty fnName argtys\n let fnty ← LLVM.functionType retty argtys\n let out ← LLVM.buildCall2 builder fnty fn #[closure] retName\n LLVM.buildSextOrTrunc builder out (← LLVM.i8Type llvmctx)", "start": [ 834, 1 ], "end": [ 842, 60 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.callLeanIsScalar", "code": "def callLeanIsScalar (builder : LLVM.Builder llvmctx)\n (closure : LLVM.Value llvmctx) (retName : String := \"\") : M llvmctx (LLVM.Value llvmctx) := do\n let fnName := \"lean_is_scalar\"\n let retty ← LLVM.i8Type llvmctx\n let argtys := #[ ← LLVM.voidPtrType llvmctx]\n let fn ← getOrCreateFunctionPrototype (← getLLVMModule) retty fnName argtys\n let fnty ← LLVM.functionType retty argtys\n LLVM.buildCall2 builder fnty fn #[closure] retName", "start": [ 844, 1 ], "end": [ 851, 54 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitIsShared", "code": "def emitIsShared (builder : LLVM.Builder llvmctx) (z : VarId) (x : VarId) : M llvmctx Unit := do\n let xv ← emitLhsVal builder x\n let exclusive? ← callLeanIsExclusive builder xv\n let exclusive? ← LLVM.buildSextOrTrunc builder exclusive? (← LLVM.i1Type llvmctx)\n let shared? ← LLVM.buildNot builder exclusive?\n let shared? ← LLVM.buildSext builder shared? (← LLVM.i8Type llvmctx)\n emitLhsSlotStore builder z shared?", "start": [ 853, 1 ], "end": [ 859, 39 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitBox", "code": "def emitBox (builder : LLVM.Builder llvmctx) (z : VarId) (x : VarId) (xType : IRType) : M llvmctx Unit := do\n let xv ← emitLhsVal builder x\n let (fnName, argTy, xv) ←\n match xType with\n | IRType.usize => pure (\"lean_box_usize\", ← LLVM.size_tType llvmctx, xv)\n | IRType.uint32 => pure (\"lean_box_uint32\", ← LLVM.i32Type llvmctx, xv)\n | IRType.uint64 => pure (\"lean_box_uint64\", ← LLVM.size_tType llvmctx, xv)\n | IRType.float => pure (\"lean_box_float\", ← LLVM.doubleTypeInContext llvmctx, xv)\n | _ => do\n let xv ← LLVM.buildSext builder xv (← LLVM.size_tType llvmctx)\n pure (\"lean_box\", ← LLVM.size_tType llvmctx, xv)\n let retty ← LLVM.voidPtrType llvmctx\n let argtys := #[argTy]\n let fn ← getOrCreateFunctionPrototype (← getLLVMModule) retty fnName argtys\n let fnty ← LLVM.functionType retty argtys\n let zv ← LLVM.buildCall2 builder fnty fn #[xv]\n emitLhsSlotStore builder z zv", "start": [ 861, 1 ], "end": [ 878, 32 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.IRType.isIntegerType", "code": "def IRType.isIntegerType (t : IRType) : Bool :=\n match t with\n | .uint8 => true\n | .uint16 => true\n | .uint32 => true\n | .uint64 => true\n | .usize => true\n | _ => false", "start": [ 880, 1 ], "end": [ 887, 15 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.callUnboxForType", "code": "def callUnboxForType (builder : LLVM.Builder llvmctx)\n (t : IRType)\n (v : LLVM.Value llvmctx)\n (retName : String := \"\") : M llvmctx (LLVM.Value llvmctx) := do\n let (fnName, retty) ←\n match t with\n | IRType.usize => pure (\"lean_unbox_usize\", ← toLLVMType t)\n | IRType.uint32 => pure (\"lean_unbox_uint32\", ← toLLVMType t)\n | IRType.uint64 => pure (\"lean_unbox_uint64\", ← toLLVMType t)\n | IRType.float => pure (\"lean_unbox_float\", ← toLLVMType t)\n | _ => pure (\"lean_unbox\", ← LLVM.size_tType llvmctx)\n let argtys := #[← LLVM.voidPtrType llvmctx ]\n let fn ← getOrCreateFunctionPrototype (← getLLVMModule) retty fnName argtys\n let fnty ← LLVM.functionType retty argtys\n LLVM.buildCall2 builder fnty fn #[v] retName", "start": [ 889, 1 ], "end": [ 903, 47 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitUnbox", "code": "def emitUnbox (builder : LLVM.Builder llvmctx)\n (z : VarId) (t : IRType) (x : VarId) (retName : String := \"\") : M llvmctx Unit := do\n let zval ← callUnboxForType builder t (← emitLhsVal builder x) retName\n let zval ←\n if IRType.isIntegerType t\n then LLVM.buildSextOrTrunc builder zval (← toLLVMType t)\n else pure zval\n emitLhsSlotStore builder z zval", "start": [ 907, 1 ], "end": [ 916, 34 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitReset", "code": "def emitReset (builder : LLVM.Builder llvmctx) (z : VarId) (n : Nat) (x : VarId) : M llvmctx Unit := do\n let xv ← emitLhsVal builder x\n let isExclusive ← callLeanIsExclusive builder xv\n let isExclusive ← buildLeanBoolTrue? builder isExclusive\n buildIfThenElse_ builder \"isExclusive\" isExclusive\n (fun builder => do\n let xv ← emitLhsVal builder x\n n.forM fun i => do\n callLeanCtorRelease builder xv (← constIntUnsigned i)\n emitLhsSlotStore builder z xv\n return ShouldForwardControlFlow.yes\n )\n (fun builder => do\n let xv ← emitLhsVal builder x\n callLeanDecRef builder xv\n let box0 ← callLeanBox builder (← constIntSizeT 0) \"box0\"\n emitLhsSlotStore builder z box0\n return ShouldForwardControlFlow.yes\n )", "start": [ 918, 1 ], "end": [ 936, 5 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitReuse", "code": "def emitReuse (builder : LLVM.Builder llvmctx)\n (z : VarId) (x : VarId) (c : CtorInfo) (updtHeader : Bool) (ys : Array Arg) : M llvmctx Unit := do\n let xv ← emitLhsVal builder x\n let isScalar ← callLeanIsScalar builder xv\n let isScalar ← buildLeanBoolTrue? builder isScalar\n buildIfThenElse_ builder \"isScalar\" isScalar\n (fun builder => do\n let cv ← emitAllocCtor builder c\n emitLhsSlotStore builder z cv\n return ShouldForwardControlFlow.yes\n )\n (fun builder => do\n let xv ← emitLhsVal builder x\n emitLhsSlotStore builder z xv\n if updtHeader then\n let zv ← emitLhsVal builder z\n callLeanCtorSetTag builder zv (← constInt8 c.cidx)\n return ShouldForwardControlFlow.yes\n )\n emitCtorSetArgs builder z ys", "start": [ 938, 1 ], "end": [ 957, 31 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitVDecl", "code": "def emitVDecl (builder : LLVM.Builder llvmctx) (z : VarId) (t : IRType) (v : Expr) : M llvmctx Unit := do\n match v with\n | Expr.ctor c ys => emitCtor builder z c ys\n | Expr.reset n x => emitReset builder z n x\n | Expr.reuse x c u ys => emitReuse builder z x c u ys\n | Expr.proj i x => emitProj builder z i x\n | Expr.uproj i x => emitUProj builder z i x\n | Expr.sproj n o x => emitSProj builder z t n o x\n | Expr.fap c ys => emitFullApp builder z c ys\n | Expr.pap c ys => emitPartialApp builder z c ys\n | Expr.ap x ys => emitApp builder z x ys\n | Expr.box t x => emitBox builder z x t\n | Expr.unbox x => emitUnbox builder z t x\n | Expr.isShared x => emitIsShared builder z x\n | Expr.lit v => let _ ← emitLit builder z t v", "start": [ 959, 1 ], "end": [ 973, 57 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.declareVar", "code": "def declareVar (builder : LLVM.Builder llvmctx) (x : VarId) (t : IRType) : M llvmctx Unit := do\n let llvmty ← toLLVMType t\n let alloca ← buildPrologueAlloca builder llvmty \"varx\"\n addVartoState x alloca llvmty", "start": [ 975, 1 ], "end": [ 978, 32 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.declareVars", "code": "partial def declareVars (builder : LLVM.Builder llvmctx) (f : FnBody) : M llvmctx Unit := do\n match f with\n | FnBody.vdecl x t _ b => do\n declareVar builder x t\n declareVars builder b\n | FnBody.jdecl _ xs _ b => do\n for param in xs do declareVar builder param.x param.ty\n declareVars builder b\n | e => do\n if e.isTerminal then pure () else declareVars builder e.body", "start": [ 980, 1 ], "end": [ 989, 67 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitTag", "code": "def emitTag (builder : LLVM.Builder llvmctx) (x : VarId) (xType : IRType) : M llvmctx (LLVM.Value llvmctx) := do\n if xType.isObj then do\n let xval ← emitLhsVal builder x\n callLeanObjTag builder xval\n else if xType.isScalar then do\n emitLhsVal builder x\n else\n throw \"Do not know how to `emitTag` in general.\"", "start": [ 991, 1 ], "end": [ 998, 53 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitSet", "code": "def emitSet (builder : LLVM.Builder llvmctx) (x : VarId) (i : Nat) (y : Arg) : M llvmctx Unit := do\n let fnName := \"lean_ctor_set\"\n let retty ← LLVM.voidType llvmctx\n let argtys := #[ ← LLVM.voidPtrType llvmctx, ← LLVM.unsignedType llvmctx , ← LLVM.voidPtrType llvmctx]\n let fn ← getOrCreateFunctionPrototype (← getLLVMModule) retty fnName argtys\n let fnty ← LLVM.functionType retty argtys\n let _ ← LLVM.buildCall2 builder fnty fn #[← emitLhsVal builder x, ← constIntUnsigned i, (← emitArgVal builder y).2]", "start": [ 1000, 1 ], "end": [ 1006, 119 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitUSet", "code": "def emitUSet (builder : LLVM.Builder llvmctx) (x : VarId) (i : Nat) (y : VarId) : M llvmctx Unit := do\n let fnName := \"lean_ctor_set_usize\"\n let retty ← LLVM.voidType llvmctx\n let argtys := #[ ← LLVM.voidPtrType llvmctx, ← LLVM.unsignedType llvmctx, ← LLVM.size_tType llvmctx]\n let fn ← getOrCreateFunctionPrototype (← getLLVMModule) retty fnName argtys\n let fnty ← LLVM.functionType retty argtys\n let _ ← LLVM.buildCall2 builder fnty fn #[← emitLhsVal builder x, ← constIntUnsigned i, (← emitLhsVal builder y)]", "start": [ 1008, 1 ], "end": [ 1014, 117 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitTailCall", "code": "def emitTailCall (builder : LLVM.Builder llvmctx) (f : FunId) (v : Expr) : M llvmctx Unit := do\n match v with\n | Expr.fap _ ys => do\n let llvmctx ← read\n let ps := llvmctx.mainParams\n unless ps.size == ys.size do throw s!\"Invalid tail call. f:'{f}' v:'{v}'\"\n let args ← ys.mapM (fun y => Prod.snd <$> emitArgVal builder y)\n let fn ← builderGetInsertionFn builder\n let call ← LLVM.buildCall2 builder (← getFunIdTy f) fn args\n LLVM.setTailCall call true let _ ← LLVM.buildRet builder call\n | _ => throw s!\"EmitTailCall expects function application, found '{v}'\"", "start": [ 1016, 1 ], "end": [ 1028, 74 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitJmp", "code": "def emitJmp (builder : LLVM.Builder llvmctx) (jp : JoinPointId) (xs : Array Arg) : M llvmctx Unit := do\n let llvmctx ← read\n let ps ← match llvmctx.jpMap.find? jp with\n | some ps => pure ps\n | none => throw s!\"Unknown join point {jp}\"\n unless xs.size == ps.size do throw s!\"Invalid goto, mismatched sizes between arguments, formal parameters.\"\n for (p, x) in ps.zip xs do\n let (_xty, xv) ← emitArgVal builder x\n emitLhsSlotStore builder p.x xv\n let _ ← LLVM.buildBr builder (← emitJp jp)", "start": [ 1030, 1 ], "end": [ 1039, 45 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitSSet", "code": "def emitSSet (builder : LLVM.Builder llvmctx) (x : VarId) (n : Nat) (offset : Nat) (y : VarId) (t : IRType) : M llvmctx Unit := do\n let (fnName, setty) ←\n match t with\n | IRType.float => pure (\"lean_ctor_set_float\", ← LLVM.doubleTypeInContext llvmctx)\n | IRType.uint8 => pure (\"lean_ctor_set_uint8\", ← LLVM.i8Type llvmctx)\n | IRType.uint16 => pure (\"lean_ctor_set_uint16\", ← LLVM.i16Type llvmctx)\n | IRType.uint32 => pure (\"lean_ctor_set_uint32\", ← LLVM.i32Type llvmctx)\n | IRType.uint64 => pure (\"lean_ctor_set_uint64\", ← LLVM.i64Type llvmctx)\n | _ => throw s!\"invalid type for 'lean_ctor_set': '{t}'\"\n let argtys := #[ ← LLVM.voidPtrType llvmctx, ← LLVM.unsignedType llvmctx, setty]\n let retty ← LLVM.voidType llvmctx\n let fn ← getOrCreateFunctionPrototype (← getLLVMModule) retty fnName argtys\n let xv ← emitLhsVal builder x\n let offset ← emitOffset builder n offset\n let yv ← emitLhsVal builder y\n let fnty ← LLVM.functionType retty argtys\n let _ ← LLVM.buildCall2 builder fnty fn #[xv, offset, yv]", "start": [ 1041, 1 ], "end": [ 1057, 61 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitDel", "code": "def emitDel (builder : LLVM.Builder llvmctx) (x : VarId) : M llvmctx Unit := do\n let argtys := #[ ← LLVM.voidPtrType llvmctx]\n let retty ← LLVM.voidType llvmctx\n let fn ← getOrCreateFunctionPrototype (← getLLVMModule) retty \"lean_free_object\" argtys\n let xv ← emitLhsVal builder x\n let fnty ← LLVM.functionType retty argtys\n let _ ← LLVM.buildCall2 builder fnty fn #[xv]", "start": [ 1059, 1 ], "end": [ 1065, 49 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitSetTag", "code": "def emitSetTag (builder : LLVM.Builder llvmctx) (x : VarId) (i : Nat) : M llvmctx Unit := do\n let argtys := #[← LLVM.voidPtrType llvmctx, ← LLVM.i8Type llvmctx]\n let retty ← LLVM.voidType llvmctx\n let fn ← getOrCreateFunctionPrototype (← getLLVMModule) retty \"lean_ctor_set_tag\" argtys\n let xv ← emitLhsVal builder x\n let fnty ← LLVM.functionType retty argtys\n let _ ← LLVM.buildCall2 builder fnty fn #[xv, ← constInt8 i]", "start": [ 1067, 1 ], "end": [ 1073, 64 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.ensureHasDefault'", "code": "def ensureHasDefault' (alts : Array Alt) : Array Alt :=\n if alts.any Alt.isDefault then alts\n else\n let last := alts.back\n let alts := alts.pop\n alts.push (Alt.default last.body)", "start": [ 1075, 1 ], "end": [ 1080, 38 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitCase", "code": "partial def emitCase (builder : LLVM.Builder llvmctx)\n (x : VarId) (xType : IRType) (alts : Array Alt) : M llvmctx Unit := do\n let oldBB ← LLVM.getInsertBlock builder\n let tag ← emitTag builder x xType\n let tag ← LLVM.buildZext builder tag (← LLVM.i64Type llvmctx)\n let alts := ensureHasDefault' alts\n let defaultBB ← builderAppendBasicBlock builder s!\"case_{xType}_default\"\n let numCasesHint := alts.size\n let switch ← LLVM.buildSwitch builder tag defaultBB (UInt64.ofNat numCasesHint)\n alts.forM fun alt => do\n match alt with\n | Alt.ctor c b =>\n let destbb ← builderAppendBasicBlock builder s!\"case_{xType}_{c.name}_{c.cidx}\"\n LLVM.addCase switch (← constIntSizeT c.cidx) destbb\n LLVM.positionBuilderAtEnd builder destbb\n emitFnBody builder b\n | Alt.default b =>\n LLVM.positionBuilderAtEnd builder defaultBB\n emitFnBody builder b\n LLVM.clearInsertionPosition builder\n LLVM.positionBuilderAtEnd builder oldBB", "start": [ 1083, 1 ], "end": [ 1106, 42 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitJDecl", "code": "partial def emitJDecl (builder : LLVM.Builder llvmctx)\n (jp : JoinPointId) (_ps : Array Param) (b : FnBody) : M llvmctx Unit := do\n let oldBB ← LLVM.getInsertBlock builder\n let jpbb ← builderAppendBasicBlock builder s!\"jp_{jp.idx}\"\n addJpTostate jp jpbb\n LLVM.positionBuilderAtEnd builder jpbb\n declareVars builder b\n emitBlock builder b\n LLVM.positionBuilderAtEnd builder oldBB", "start": [ 1109, 1 ], "end": [ 1122, 42 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitUnreachable", "code": "partial def emitUnreachable (builder : LLVM.Builder llvmctx) : M llvmctx Unit := do\n let retty ← LLVM.voidType llvmctx\n let argtys := #[]\n let fn ← getOrCreateFunctionPrototype (← getLLVMModule) retty \"lean_internal_panic_unreachable\" argtys\n let fnty ← LLVM.functionType retty argtys\n let _ ← LLVM.buildCall2 builder fnty fn #[]\n let _ ← LLVM.buildUnreachable builder", "start": [ 1124, 1 ], "end": [ 1130, 40 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitBlock", "code": "partial def emitBlock (builder : LLVM.Builder llvmctx) (b : FnBody) : M llvmctx Unit := do\n match b with\n | FnBody.jdecl j xs v b =>\n emitJDecl builder j xs v\n emitBlock builder b\n | d@(FnBody.vdecl x t v b) => do\n let llvmctx ← read\n if isTailCallTo llvmctx.mainFn d then\n emitTailCall builder llvmctx.mainFn v\n else\n emitVDecl builder x t v\n emitBlock builder b\n | FnBody.inc x n c p b =>\n unless p do emitInc builder x n c\n emitBlock builder b\n | FnBody.dec x n c p b =>\n unless p do emitDec builder x n c\n emitBlock builder b\n | FnBody.del x b => emitDel builder x; emitBlock builder b\n | FnBody.setTag x i b => emitSetTag builder x i; emitBlock builder b\n | FnBody.set x i y b => emitSet builder x i y; emitBlock builder b\n | FnBody.uset x i y b => emitUSet builder x i y; emitBlock builder b\n | FnBody.sset x i o y t b => emitSSet builder x i o y t; emitBlock builder b\n | FnBody.mdata _ b => emitBlock builder b\n | FnBody.ret x => do\n let (_xty, xv) ← emitArgVal builder x \"ret_val\"\n let _ ← LLVM.buildRet builder xv\n | FnBody.case _ x xType alts =>\n emitCase builder x xType alts\n | FnBody.jmp j xs =>\n emitJmp builder j xs\n | FnBody.unreachable => emitUnreachable builder", "start": [ 1132, 1 ], "end": [ 1163, 58 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitFnBody", "code": "partial def emitFnBody (builder : LLVM.Builder llvmctx) (b : FnBody) : M llvmctx Unit := do\n declareVars builder b\n emitBlock builder b", "start": [ 1165, 1 ], "end": [ 1167, 22 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitFnArgs", "code": "def emitFnArgs (builder : LLVM.Builder llvmctx)\n (needsPackedArgs? : Bool) (llvmfn : LLVM.Value llvmctx) (params : Array Param) : M llvmctx Unit := do\n if needsPackedArgs? then do\n let argsp ← LLVM.getParam llvmfn 0 for i in List.range params.size do\n let param := params[i]!\n let argsi ← LLVM.buildGEP2 builder (← LLVM.voidPtrType llvmctx) argsp #[← constIntUnsigned i] s!\"packed_arg_{i}_slot\"\n let llvmty ← toLLVMType param.ty\n let pv ← LLVM.buildLoad2 builder llvmty argsi\n let alloca ← buildPrologueAlloca builder llvmty s!\"arg_{i}\"\n LLVM.buildStore builder pv alloca\n addVartoState params[i]!.x alloca llvmty\n else\n let n ← LLVM.countParams llvmfn\n for i in (List.range n.toNat) do\n let llvmty ← toLLVMType params[i]!.ty\n let alloca ← buildPrologueAlloca builder llvmty s!\"arg_{i}\"\n let arg ← LLVM.getParam llvmfn (UInt64.ofNat i)\n let _ ← LLVM.buildStore builder arg alloca\n addVartoState params[i]!.x alloca llvmty", "start": [ 1171, 1 ], "end": [ 1193, 49 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitDeclAux", "code": "def emitDeclAux (mod : LLVM.Module llvmctx) (builder : LLVM.Builder llvmctx) (d : Decl) : M llvmctx Unit := do\n let env ← getEnv\n let (_, jpMap) := mkVarJPMaps d\n withReader (fun llvmctx => { llvmctx with jpMap := jpMap }) do\n unless hasInitAttr env d.name do\n match d with\n | .fdecl (f := f) (xs := xs) (type := t) (body := b) .. =>\n let baseName ← toCName f\n let name := if xs.size > 0 then baseName else \"_init_\" ++ baseName\n let retty ← toLLVMType t\n let mut argtys := #[]\n let needsPackedArgs? := xs.size > closureMaxArgs && isBoxedName d.name\n if needsPackedArgs? then\n argtys := #[← LLVM.pointerType (← LLVM.voidPtrType llvmctx)]\n else\n for x in xs do\n argtys := argtys.push (← toLLVMType x.ty)\n let fnty ← LLVM.functionType retty argtys (isVarArg := false)\n let llvmfn ← LLVM.getOrAddFunction mod name fnty\n if xs.size == 0 then\n LLVM.setVisibility llvmfn LLVM.Visibility.hidden else\n LLVM.setDLLStorageClass llvmfn LLVM.DLLStorageClass.export withReader (fun llvmctx => { llvmctx with mainFn := f, mainParams := xs }) do\n set { var2val := default, jp2bb := default : EmitLLVM.State llvmctx } let bb ← LLVM.appendBasicBlockInContext llvmctx llvmfn \"entry\"\n LLVM.positionBuilderAtEnd builder bb\n emitFnArgs builder needsPackedArgs? llvmfn xs\n emitFnBody builder b\n pure ()\n | _ => pure ()", "start": [ 1195, 1 ], "end": [ 1229, 19 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitDecl", "code": "def emitDecl (mod : LLVM.Module llvmctx) (builder : LLVM.Builder llvmctx) (d : Decl) : M llvmctx Unit := do\n let d := d.normalizeIds try\n emitDeclAux mod builder d\n return ()\n catch err =>\n throw (s!\"emitDecl:\\ncompiling:\\n{d}\\nerr:\\n{err}\\n\")", "start": [ 1231, 1 ], "end": [ 1237, 58 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitFns", "code": "def emitFns (mod : LLVM.Module llvmctx) (builder : LLVM.Builder llvmctx) : M llvmctx Unit := do\n let env ← getEnv\n let decls := getDecls env\n decls.reverse.forM (emitDecl mod builder)", "start": [ 1239, 1 ], "end": [ 1242, 44 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.callIODeclInitFn", "code": "def callIODeclInitFn (builder : LLVM.Builder llvmctx)\n (initFnName : String)\n (world : LLVM.Value llvmctx): M llvmctx (LLVM.Value llvmctx) := do\n let retty ← LLVM.voidPtrType llvmctx\n let argtys := #[← LLVM.voidPtrType llvmctx]\n let fn ← getOrCreateFunctionPrototype (← getLLVMModule) retty initFnName argtys\n let fnty ← LLVM.functionType retty argtys\n LLVM.buildCall2 builder fnty fn #[world]", "start": [ 1244, 1 ], "end": [ 1251, 43 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.callPureDeclInitFn", "code": "def callPureDeclInitFn (builder : LLVM.Builder llvmctx)\n (initFnName : String)\n (retty : LLVM.LLVMType llvmctx): M llvmctx (LLVM.Value llvmctx) := do\n let argtys := #[]\n let fn ← getOrCreateFunctionPrototype (← getLLVMModule) retty initFnName argtys\n let fnty ← LLVM.functionType retty argtys\n LLVM.buildCall2 builder fnty fn #[]", "start": [ 1253, 1 ], "end": [ 1259, 38 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitDeclInit", "code": "def emitDeclInit (builder : LLVM.Builder llvmctx)\n (parentFn : LLVM.Value llvmctx) (d : Decl) : M llvmctx Unit := do\n let env ← getEnv\n if isIOUnitInitFn env d.name then do\n let world ← callLeanIOMkWorld builder\n let resv ← callIODeclInitFn builder (← toCName d.name) world\n let err? ← callLeanIOResultIsError builder resv \"is_error\"\n buildIfThen_ builder s!\"init_{d.name}_isError\" err?\n (fun builder => do\n let _ ← LLVM.buildRet builder resv\n pure ShouldForwardControlFlow.no)\n else if d.params.size == 0 then\n match getInitFnNameFor? env d.name with\n | some initFn =>\n let llvmty ← toLLVMType d.resultType\n let dslot ← LLVM.getOrAddGlobal (← getLLVMModule) (← toCName d.name) llvmty\n LLVM.setInitializer dslot (← LLVM.getUndef llvmty)\n let initBB ← builderAppendBasicBlock builder s!\"do_{d.name}_init\"\n let restBB ← builderAppendBasicBlock builder s!\"post_{d.name}_init\"\n let checkBuiltin? := getBuiltinInitFnNameFor? env d.name |>.isSome\n if checkBuiltin? then\n let builtinParam ← LLVM.getParam parentFn 0\n let cond ← buildLeanBoolTrue? builder builtinParam \"is_builtin_true\"\n let _ ← LLVM.buildCondBr builder cond initBB restBB\n else\n let _ ← LLVM.buildBr builder initBB\n LLVM.positionBuilderAtEnd builder initBB\n let world ← callLeanIOMkWorld builder\n let resv ← callIODeclInitFn builder (← toCName initFn) world\n let err? ← callLeanIOResultIsError builder resv s!\"{d.name}_is_error\"\n buildIfThen_ builder s!\"init_{d.name}_isError\" err?\n (fun builder => do\n let _ ← LLVM.buildRet builder resv\n pure ShouldForwardControlFlow.no)\n if d.resultType.isScalar then\n let dval ← callLeanIOResultGetValue builder resv s!\"{d.name}_res\"\n let dval ← callUnboxForType builder d.resultType dval\n LLVM.buildStore builder dval dslot\n else\n let dval ← callLeanIOResultGetValue builder resv s!\"{d.name}_res\"\n LLVM.buildStore builder dval dslot\n callLeanMarkPersistentFn builder dval\n let _ ← LLVM.buildBr builder restBB\n LLVM.positionBuilderAtEnd builder restBB\n | none => do\n let llvmty ← toLLVMType d.resultType\n let dslot ← LLVM.getOrAddGlobal (← getLLVMModule) (← toCName d.name) llvmty\n LLVM.setInitializer dslot (← LLVM.getUndef llvmty)\n let dval ← callPureDeclInitFn builder (← toCInitName d.name) (← toLLVMType d.resultType)\n LLVM.buildStore builder dval dslot\n if d.resultType.isObj then\n callLeanMarkPersistentFn builder dval", "start": [ 1261, 1 ], "end": [ 1315, 47 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.callModInitFn", "code": "def callModInitFn (builder : LLVM.Builder llvmctx)\n (modName : Name) (input world : LLVM.Value llvmctx) (retName : String): M llvmctx (LLVM.Value llvmctx) := do\n let fnName := mkModuleInitializationFunctionName modName\n let retty ← LLVM.voidPtrType llvmctx\n let argtys := #[ (← LLVM.i8Type llvmctx), (← LLVM.voidPtrType llvmctx)]\n let fn ← getOrCreateFunctionPrototype (← getLLVMModule) retty fnName argtys\n let fnty ← LLVM.functionType retty argtys\n LLVM.buildCall2 builder fnty fn #[input, world] retName", "start": [ 1317, 1 ], "end": [ 1324, 58 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitInitFn", "code": "def emitInitFn (mod : LLVM.Module llvmctx) (builder : LLVM.Builder llvmctx) : M llvmctx Unit := do\n let env ← getEnv\n let modName ← getModName\n\n let initFnTy ← LLVM.functionType (← LLVM.voidPtrType llvmctx) #[ (← LLVM.i8Type llvmctx), (← LLVM.voidPtrType llvmctx)] (isVarArg := false)\n let initFn ← LLVM.getOrAddFunction mod (mkModuleInitializationFunctionName modName) initFnTy\n LLVM.setDLLStorageClass initFn LLVM.DLLStorageClass.export let entryBB ← LLVM.appendBasicBlockInContext llvmctx initFn \"entry\"\n LLVM.positionBuilderAtEnd builder entryBB\n let ginit?ty := ← LLVM.i1Type llvmctx\n let ginit?slot ← LLVM.getOrAddGlobal mod (modName.mangle ++ \"_G_initialized\") ginit?ty\n LLVM.setVisibility ginit?slot LLVM.Visibility.hidden LLVM.setInitializer ginit?slot (← LLVM.constFalse llvmctx)\n let ginit?v ← LLVM.buildLoad2 builder ginit?ty ginit?slot \"init_v\"\n buildIfThen_ builder \"isGInitialized\" ginit?v\n (fun builder => do\n let box0 ← callLeanBox builder (← constIntSizeT 0) \"box0\"\n let out ← callLeanIOResultMKOk builder box0 \"retval\"\n let _ ← LLVM.buildRet builder out\n pure ShouldForwardControlFlow.no)\n LLVM.buildStore builder (← LLVM.constTrue llvmctx) ginit?slot\n\n env.imports.forM fun import_ => do\n let builtin ← LLVM.getParam initFn 0\n let world ← callLeanIOMkWorld builder\n let res ← callModInitFn builder import_.module builtin world (\"res_\" ++ import_.module.mangle)\n let err? ← callLeanIOResultIsError builder res (\"res_is_error_\" ++ import_.module.mangle)\n buildIfThen_ builder (\"IsError\" ++ import_.module.mangle) err?\n (fun builder => do\n let _ ← LLVM.buildRet builder res\n pure ShouldForwardControlFlow.no)\n callLeanDecRef builder res\n let decls := getDecls env\n decls.reverse.forM (emitDeclInit builder initFn)\n let box0 ← callLeanBox builder (← constIntSizeT 0) \"box0\"\n let out ← callLeanIOResultMKOk builder box0 \"retval\"\n let _ ← LLVM.buildRet builder out", "start": [ 1326, 1 ], "end": [ 1362, 36 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.callLeanInitialize", "code": "def callLeanInitialize (builder : LLVM.Builder llvmctx) : M llvmctx Unit := do\n let fnName := \"lean_initialize\"\n let retty ← LLVM.voidType llvmctx\n let argtys := #[]\n let fnty ← LLVM.functionType retty argtys\n let fn ← getOrCreateFunctionPrototype (← getLLVMModule) retty fnName argtys\n let _ ← LLVM.buildCall2 builder fnty fn #[]", "start": [ 1364, 1 ], "end": [ 1370, 46 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.callLeanInitializeRuntimeModule", "code": "def callLeanInitializeRuntimeModule (builder : LLVM.Builder llvmctx) : M llvmctx Unit := do\n let fnName := \"lean_initialize_runtime_module\"\n let retty ← LLVM.voidType llvmctx\n let argtys := #[]\n let fnty ← LLVM.functionType retty argtys\n let fn ← getOrCreateFunctionPrototype (← getLLVMModule) retty fnName argtys\n let _ ← LLVM.buildCall2 builder fnty fn #[]", "start": [ 1372, 1 ], "end": [ 1378, 46 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.callLeanSetPanicMessages", "code": "def callLeanSetPanicMessages (builder : LLVM.Builder llvmctx)\n (enable? : LLVM.Value llvmctx) : M llvmctx Unit := do\n let fnName := \"lean_set_panic_messages\"\n let retty ← LLVM.voidType llvmctx\n let argtys := #[ ← LLVM.i1Type llvmctx ]\n let fn ← getOrCreateFunctionPrototype (← getLLVMModule) retty fnName argtys\n let fnty ← LLVM.functionType retty argtys\n let _ ← LLVM.buildCall2 builder fnty fn #[enable?]", "start": [ 1380, 1 ], "end": [ 1387, 53 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.callLeanIOMarkEndInitialization", "code": "def callLeanIOMarkEndInitialization (builder : LLVM.Builder llvmctx) : M llvmctx Unit := do\n let fnName := \"lean_io_mark_end_initialization\"\n let retty ← LLVM.voidType llvmctx\n let argtys := #[]\n let fn ← getOrCreateFunctionPrototype (← getLLVMModule) retty fnName argtys\n let fnty ← LLVM.functionType retty argtys\n let _ ← LLVM.buildCall2 builder fnty fn #[]", "start": [ 1389, 1 ], "end": [ 1395, 46 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.callLeanIOResultIsOk", "code": "def callLeanIOResultIsOk (builder : LLVM.Builder llvmctx)\n (arg : LLVM.Value llvmctx) (name : String := \"\") : M llvmctx (LLVM.Value llvmctx) := do\n let fnName := \"lean_io_result_is_ok\"\n let retty ← LLVM.i1Type llvmctx\n let argtys := #[ ← LLVM.voidPtrType llvmctx ]\n let fn ← getOrCreateFunctionPrototype (← getLLVMModule) retty fnName argtys\n let fnty ← LLVM.functionType retty argtys\n LLVM.buildCall2 builder fnty fn #[arg] name", "start": [ 1397, 1 ], "end": [ 1404, 46 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.callLeanInitTaskManager", "code": "def callLeanInitTaskManager (builder : LLVM.Builder llvmctx) : M llvmctx Unit := do\n let fnName := \"lean_init_task_manager\"\n let retty ← LLVM.voidType llvmctx\n let argtys := #[]\n let fn ← getOrCreateFunctionPrototype (← getLLVMModule) retty fnName argtys\n let fnty ← LLVM.functionType retty argtys\n let _ ← LLVM.buildCall2 builder fnty fn #[]", "start": [ 1406, 1 ], "end": [ 1412, 47 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.callLeanFinalizeTaskManager", "code": "def callLeanFinalizeTaskManager (builder : LLVM.Builder llvmctx) : M llvmctx Unit := do\n let fnName := \"lean_finalize_task_manager\"\n let retty ← LLVM.voidPtrType llvmctx\n let argtys := #[]\n let fn ← getOrCreateFunctionPrototype (← getLLVMModule) retty fnName argtys\n let fnty ← LLVM.functionType retty argtys\n let _ ← LLVM.buildCall2 builder fnty fn #[]", "start": [ 1414, 1 ], "end": [ 1420, 47 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.callLeanUnboxUint32", "code": "def callLeanUnboxUint32 (builder : LLVM.Builder llvmctx)\n (v : LLVM.Value llvmctx) (name : String := \"\") : M llvmctx (LLVM.Value llvmctx) := do\n let fnName := \"lean_unbox_uint32\"\n let retty ← LLVM.i32Type llvmctx\n let argtys := #[ ← LLVM.voidPtrType llvmctx ]\n let fn ← getOrCreateFunctionPrototype (← getLLVMModule) retty fnName argtys\n let fnty ← LLVM.functionType retty argtys\n LLVM.buildCall2 builder fnty fn #[v] name", "start": [ 1422, 1 ], "end": [ 1429, 45 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.callLeanIOResultShowError", "code": "def callLeanIOResultShowError (builder : LLVM.Builder llvmctx)\n (v : LLVM.Value llvmctx) (name : String := \"\") : M llvmctx Unit := do\n let fnName := \"lean_io_result_show_error\"\n let retty ← LLVM.voidType llvmctx\n let argtys := #[ ← LLVM.voidPtrType llvmctx ]\n let fn ← getOrCreateFunctionPrototype (← getLLVMModule) retty fnName argtys\n let fnty ← LLVM.functionType retty argtys\n let _ ← LLVM.buildCall2 builder fnty fn #[v] name", "start": [ 1431, 1 ], "end": [ 1438, 52 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.callLeanMainFn", "code": "def callLeanMainFn (builder : LLVM.Builder llvmctx)\n (argv? : Option (LLVM.Value llvmctx))\n (world : LLVM.Value llvmctx)\n (name : String) : M llvmctx (LLVM.Value llvmctx) := do\n let retty ← LLVM.voidPtrType llvmctx\n let voidptr ← LLVM.voidPtrType llvmctx\n let argtys := if argv?.isSome then #[ voidptr, voidptr ] else #[ voidptr ]\n let fn ← getOrCreateFunctionPrototype (← getLLVMModule) retty leanMainFn argtys\n let fnty ← LLVM.functionType retty argtys\n let args := match argv? with\n | .some argv => #[argv, world]\n | .none => #[world]\n LLVM.buildCall2 builder fnty fn args name", "start": [ 1440, 1 ], "end": [ 1452, 44 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitMainFn", "code": "def emitMainFn (mod : LLVM.Module llvmctx) (builder : LLVM.Builder llvmctx) : M llvmctx Unit := do\n let d ← getDecl `main\n let xs ← match d with\n | .fdecl (xs := xs) .. => pure xs\n | _ => throw \"Function declaration expected for 'main'\"\n\n unless xs.size == 2 || xs.size == 1 do throw s!\"Invalid main function, main expected to have '2' or '1' arguments, found '{xs.size}' arguments\"\n let env ← getEnv\n let usesLeanAPI := usesModuleFrom env `Lean\n let mainTy ← LLVM.functionType (← LLVM.i64Type llvmctx)\n #[(← LLVM.i64Type llvmctx), (← LLVM.pointerType (← LLVM.voidPtrType llvmctx))]\n let main ← LLVM.getOrAddFunction mod \"main\" mainTy\n let entry ← LLVM.appendBasicBlockInContext llvmctx main \"entry\"\n LLVM.positionBuilderAtEnd builder entry\n \n let inty ← LLVM.voidPtrType llvmctx\n let inslot ← buildPrologueAlloca builder (← LLVM.pointerType inty) \"in\"\n let resty ← LLVM.voidPtrType llvmctx\n let res ← buildPrologueAlloca builder (← LLVM.pointerType resty) \"res\"\n if usesLeanAPI then callLeanInitialize builder else callLeanInitializeRuntimeModule builder\n \n callLeanSetPanicMessages builder (← LLVM.constFalse llvmctx)\n let world ← callLeanIOMkWorld builder\n let resv ← callModInitFn builder (← getModName) (← constInt8 1) world ((← getModName).toString ++ \"_init_out\")\n let _ ← LLVM.buildStore builder resv res\n\n callLeanSetPanicMessages builder (← LLVM.constTrue llvmctx)\n callLeanIOMarkEndInitialization builder\n\n let resv ← LLVM.buildLoad2 builder resty res \"resv\"\n let res_is_ok ← callLeanIOResultIsOk builder resv \"res_is_ok\"\n buildIfThen_ builder \"resIsOkBranches\" res_is_ok\n (fun builder => do callLeanDecRef builder resv\n callLeanInitTaskManager builder\n if xs.size == 2 then\n let inv ← callLeanBox builder (← constIntSizeT 0) \"inv\"\n let _ ← LLVM.buildStore builder inv inslot\n let ity ← LLVM.size_tType llvmctx\n let islot ← buildPrologueAlloca builder ity \"islot\"\n let argcval ← LLVM.getParam main 0\n let argvval ← LLVM.getParam main 1\n LLVM.buildStore builder argcval islot\n buildWhile_ builder \"argv\"\n (condcodegen := fun builder => do\n let iv ← LLVM.buildLoad2 builder ity islot \"iv\"\n let i_gt_1 ← LLVM.buildICmp builder LLVM.IntPredicate.UGT iv (← constIntSizeT 1) \"i_gt_1\"\n return i_gt_1)\n (bodycodegen := fun builder => do\n let iv ← LLVM.buildLoad2 builder ity islot \"iv\"\n let iv_next ← LLVM.buildSub builder iv (← constIntSizeT 1) \"iv.next\"\n LLVM.buildStore builder iv_next islot\n let nv ← callLeanAllocCtor builder 1 2 0 \"nv\"\n let argv_i_next_slot ← LLVM.buildGEP2 builder (← LLVM.voidPtrType llvmctx) argvval #[iv_next] \"argv.i.next.slot\"\n let argv_i_next_val ← LLVM.buildLoad2 builder (← LLVM.voidPtrType llvmctx) argv_i_next_slot \"argv.i.next.val\"\n let argv_i_next_val_str ← callLeanMkString builder argv_i_next_val \"arg.i.next.val.str\"\n callLeanCtorSet builder nv (← constIntUnsigned 0) argv_i_next_val_str\n let inv ← LLVM.buildLoad2 builder inty inslot \"inv\"\n callLeanCtorSet builder nv (← constIntUnsigned 1) inv\n LLVM.buildStore builder nv inslot)\n let world ← callLeanIOMkWorld builder\n let inv ← LLVM.buildLoad2 builder inty inslot \"inv\"\n let resv ← callLeanMainFn builder (argv? := .some inv) (world := world) \"resv\"\n let _ ← LLVM.buildStore builder resv res\n pure ShouldForwardControlFlow.yes\n else\n let world ← callLeanIOMkWorld builder\n let resv ← callLeanMainFn builder (argv? := .none) (world := world) \"resv\"\n let _ ← LLVM.buildStore builder resv res\n pure ShouldForwardControlFlow.yes\n )\n\n let retTy := env.find? `main |>.get! |>.type |>.getForallBody\n let retTy := retTy.appArg!\n callLeanFinalizeTaskManager builder\n let resv ← LLVM.buildLoad2 builder resty res \"resv\"\n let res_is_ok ← callLeanIOResultIsOk builder resv \"res_is_ok\"\n buildIfThenElse_ builder \"res.is.ok\" res_is_ok\n (fun builder => if retTy.constName? == some ``UInt32 then do\n let resv ← LLVM.buildLoad2 builder resty res \"resv\"\n let retv ← callLeanUnboxUint32 builder (← callLeanIOResultGetValue builder resv \"io_val\") \"retv\"\n let retv ← LLVM.buildSext builder retv (← LLVM.i64Type llvmctx) \"retv_sext\"\n callLeanDecRef builder resv\n let _ ← LLVM.buildRet builder retv\n pure ShouldForwardControlFlow.no\n else do\n callLeanDecRef builder resv\n let _ ← LLVM.buildRet builder (← constInt64 0)\n pure ShouldForwardControlFlow.no\n\n )\n (fun builder => do let resv ← LLVM.buildLoad2 builder resty res \"resv\"\n callLeanIOResultShowError builder resv\n callLeanDecRef builder resv\n let _ ← LLVM.buildRet builder (← constInt64 1)\n pure ShouldForwardControlFlow.no)\n let _ ← LLVM.buildUnreachable builder", "start": [ 1454, 1 ], "end": [ 1562, 40 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.hasMainFn", "code": "def hasMainFn : M llvmctx Bool := do\n let env ← getEnv\n let decls := getDecls env\n return decls.any (fun d => d.name == `main)", "start": [ 1564, 1 ], "end": [ 1567, 46 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.emitMainFnIfNeeded", "code": "def emitMainFnIfNeeded (mod : LLVM.Module llvmctx) (builder : LLVM.Builder llvmctx) : M llvmctx Unit := do\n if (← hasMainFn) then emitMainFn mod builder", "start": [ 1569, 1 ], "end": [ 1570, 47 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.EmitLLVM.main", "code": "def main : M llvmctx Unit := do\n emitFnDecls\n let builder ← LLVM.createBuilderInContext llvmctx\n emitFns (← getLLVMModule) builder\n emitInitFn (← getLLVMModule) builder\n emitMainFnIfNeeded (← getLLVMModule) builder", "start": [ 1572, 1 ], "end": [ 1577, 47 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.getLeanHBcPath", "code": "def getLeanHBcPath : IO System.FilePath := do\n return (← getLibDir (← getBuildDir)) / \"lean.h.bc\"", "start": [ 1580, 1 ], "end": [ 1581, 53 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.getModuleGlobals", "code": "partial def getModuleGlobals (mod : LLVM.Module llvmctx) : IO (Array (LLVM.Value llvmctx)) := do\n let rec go (v : LLVM.Value llvmctx) (acc : Array (LLVM.Value llvmctx)) : IO (Array (LLVM.Value llvmctx)) := do\n if v.isNull then return acc\n else go (← LLVM.getNextGlobal v) (acc.push v)\n go (← LLVM.getFirstGlobal mod) #[]", "start": [ 1583, 1 ], "end": [ 1588, 37 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.getModuleFunctions", "code": "partial def getModuleFunctions (mod : LLVM.Module llvmctx) : IO (Array (LLVM.Value llvmctx)) := do\n let rec go (v : LLVM.Value llvmctx) (acc : Array (LLVM.Value llvmctx)) : IO (Array (LLVM.Value llvmctx)) := do\n if v.isNull then return acc\n else go (← LLVM.getNextFunction v) (acc.push v)\n go (← LLVM.getFirstFunction mod) #[]", "start": [ 1590, 1 ], "end": [ 1595, 39 ], "kind": "commanddeclaration" }, { "full_name": "Lean.IR.emitLLVM", "code": "@[export lean_ir_emit_llvm]\ndef emitLLVM (env : Environment) (modName : Name) (filepath : String) : IO Unit := do\n LLVM.llvmInitializeTargetInfo\n let llvmctx ← LLVM.createContext\n let module ← LLVM.createModule llvmctx modName.toString\n let emitLLVMCtx : EmitLLVM.Context llvmctx := {env := env, modName := modName, llvmmodule := module}\n let initState := { var2val := default, jp2bb := default : EmitLLVM.State llvmctx}\n let out? ← ((EmitLLVM.main (llvmctx := llvmctx)).run initState).run emitLLVMCtx\n match out? with\n | .ok _ => do\n let membuf ← LLVM.createMemoryBufferWithContentsOfFile (← getLeanHBcPath).toString\n let modruntime ← LLVM.parseBitcode llvmctx membuf\n \n let runtimeGlobals ← (← getModuleGlobals modruntime).mapM (Β·.getName)\n let filter func := do\n if (← LLVM.isDeclaration func) then\n return none\n else\n return some (← func.getName)\n let runtimeFunctions ← (← getModuleFunctions modruntime).filterMapM filter\n LLVM.linkModules (dest := emitLLVMCtx.llvmmodule) (src := modruntime)\n for name in runtimeGlobals do\n let some global ← LLVM.getNamedGlobal emitLLVMCtx.llvmmodule name\n | throw <| IO.Error.userError s!\"ERROR: linked module must have global from runtime module: '{name}'\"\n LLVM.setLinkage global LLVM.Linkage.internal\n for name in runtimeFunctions do\n let some fn ← LLVM.getNamedFunction emitLLVMCtx.llvmmodule name\n | throw <| IO.Error.userError s!\"ERROR: linked module must have function from runtime module: '{name}'\"\n LLVM.setLinkage fn LLVM.Linkage.internal\n if let some err ← LLVM.verifyModule emitLLVMCtx.llvmmodule then\n throw <| .userError err\n LLVM.writeBitcodeToFile emitLLVMCtx.llvmmodule filepath\n LLVM.disposeModule emitLLVMCtx.llvmmodule\n | .error err => throw (IO.Error.userError err)", "start": [ 1597, 1 ], "end": [ 1638, 49 ], "kind": "commanddeclaration" } ]
.lake/packages/lean4/src/lean/lake/Lake/Main.lean
[ ".lake/packages/lean4/src/lean/Init.lean", ".lake/packages/lean4/src/lean/lake/Lake/CLI.lean", ".lake/packages/lean4/src/lean/lake/Lake.lean" ]
[ { "full_name": "main", "code": "def main (args : List String) : IO UInt32 := do\n Lake.cli args", "start": [ 9, 1 ], "end": [ 10, 16 ], "kind": "commanddeclaration" } ]
.lake/packages/lean4/src/lean/Lean/Compiler/LCNF/Probing.lean
[ ".lake/packages/lean4/src/lean/Lean/Compiler/LCNF/ForEachExpr.lean", ".lake/packages/lean4/src/lean/Lean/Compiler/LCNF/CompilerM.lean", ".lake/packages/lean4/src/lean/Lean/Compiler/LCNF/PassManager.lean", ".lake/packages/lean4/src/lean/Lean/Compiler/LCNF/PhaseExt.lean" ]
[ { "full_name": "Lean.Compiler.LCNF.Probe", "code": "abbrev Probe Ξ± Ξ² := Array Ξ± β†’ CompilerM (Array Ξ²)", "start": [ 14, 1 ], "end": [ 14, 50 ], "kind": "commanddeclaration" }, { "full_name": "Lean.Compiler.LCNF.Probe.map", "code": "@[inline]\ndef map (f : Ξ± β†’ CompilerM Ξ²) : Probe Ξ± Ξ² := fun data => data.mapM f", "start": [ 18, 1 ], "end": [ 19, 69 ], "kind": "commanddeclaration" }, { "full_name": "Lean.Compiler.LCNF.Probe.filter", "code": "@[inline]\ndef filter (f : Ξ± β†’ CompilerM Bool) : Probe Ξ± Ξ± := fun data => data.filterM f", "start": [ 21, 1 ], "end": [ 22, 78 ], "kind": "commanddeclaration" }, { "full_name": "Lean.Compiler.LCNF.Probe.sorted", "code": "@[inline]\ndef sorted [Inhabited Ξ±] [inst : LT Ξ±] [DecidableRel inst.lt] : Probe Ξ± Ξ± := fun data => return data.qsort (Β· < Β·)", "start": [ 24, 1 ], "end": [ 25, 115 ], "kind": "commanddeclaration" }, { "full_name": "Lean.Compiler.LCNF.Probe.sortedBySize", "code": "@[inline]\ndef sortedBySize : Probe Decl (Nat Γ— Decl) := fun decls =>\n let decls := decls.map fun decl => (decl.size, decl)\n return decls.qsort fun (sz₁, decl₁) (szβ‚‚, declβ‚‚) =>\n if sz₁ == szβ‚‚ then Name.lt decl₁.name declβ‚‚.name else sz₁ < szβ‚‚", "start": [ 27, 1 ], "end": [ 31, 68 ], "kind": "commanddeclaration" }, { "full_name": "Lean.Compiler.LCNF.Probe.countUnique", "code": "def countUnique [ToString Ξ±] [BEq Ξ±] [Hashable Ξ±] : Probe Ξ± (Ξ± Γ— Nat) := fun data => do\n let mut map := HashMap.empty\n for d in data do\n if let some count := map.find? d then\n map := map.insert d (count + 1)\n else\n map := map.insert d 1\n return map.toArray", "start": [ 33, 1 ], "end": [ 40, 21 ], "kind": "commanddeclaration" }, { "full_name": "Lean.Compiler.LCNF.Probe.countUniqueSorted", "code": "@[inline]\ndef countUniqueSorted [ToString Ξ±] [BEq Ξ±] [Hashable Ξ±] [Inhabited Ξ±] : Probe Ξ± (Ξ± Γ— Nat) :=\n countUnique >=> fun data => return data.qsort (fun l r => l.snd < r.snd)", "start": [ 42, 1 ], "end": [ 44, 75 ], "kind": "commanddeclaration" }, { "full_name": "Lean.Compiler.LCNF.Probe.getLetValues", "code": "partial def getLetValues : Probe Decl LetValue := fun decls => do\n let (_, res) ← start decls |>.run #[]\n return res\nwhere\n go (c : Code) : StateRefT (Array LetValue) CompilerM Unit := do\n match c with\n | .let (decl : LetDecl) (k : Code) =>\n modify fun s => s.push decl.value\n go k\n | .fun decl k | .jp decl k =>\n go decl.value\n go k\n | .cases (cases : CasesCore Code) => cases.alts.forM (go Β·.getCode)\n | .jmp .. | .return .. | .unreach .. => return ()\n start (decls : Array Decl) : StateRefT (Array LetValue) CompilerM Unit :=\n decls.forM (go Β·.value)", "start": [ 46, 1 ], "end": [ 61, 28 ], "kind": "commanddeclaration" }, { "full_name": "Lean.Compiler.LCNF.Probe.getJps", "code": "partial def getJps : Probe Decl FunDecl := fun decls => do\n let (_, res) ← start decls |>.run #[]\n return res\nwhere\n go (code : Code) : StateRefT (Array FunDecl) CompilerM Unit := do\n match code with\n | .let _ k => go k\n | .fun decl k => go decl.value; go k\n | .jp decl k => modify (Β·.push decl); go decl.value; go k\n | .cases cs => cs.alts.forM (go Β·.getCode)\n | .jmp .. | .return .. | .unreach .. => return ()\n\n start (decls : Array Decl) : StateRefT (Array FunDecl) CompilerM Unit :=\n decls.forM fun decl => go decl.value", "start": [ 63, 1 ], "end": [ 76, 41 ], "kind": "commanddeclaration" }, { "full_name": "Lean.Compiler.LCNF.Probe.filterByLet", "code": "partial def filterByLet (f : LetDecl β†’ CompilerM Bool) : Probe Decl Decl :=\n filter (fun decl => go decl.value)\nwhere\n go : Code β†’ CompilerM Bool\n | .let decl k => do if (← f decl) then return true else go k\n | .fun decl k | .jp decl k => go decl.value <||> go k\n | .cases cs => cs.alts.anyM (go Β·.getCode)\n | .jmp .. | .return .. | .unreach .. => return false", "start": [ 78, 1 ], "end": [ 85, 55 ], "kind": "commanddeclaration" }, { "full_name": "Lean.Compiler.LCNF.Probe.filterByFun", "code": "partial def filterByFun (f : FunDecl β†’ CompilerM Bool) : Probe Decl Decl :=\n filter (fun decl => go decl.value)\nwhere\n go : Code β†’ CompilerM Bool\n | .let _ k | .jp _ k => go k\n | .fun decl k => do if (← f decl) then return true else go decl.value <||> go k\n | .cases cs => cs.alts.anyM (go Β·.getCode)\n | .jmp .. | .return .. | .unreach .. => return false", "start": [ 87, 1 ], "end": [ 94, 55 ], "kind": "commanddeclaration" }, { "full_name": "Lean.Compiler.LCNF.Probe.filterByJp", "code": "partial def filterByJp (f : FunDecl β†’ CompilerM Bool) : Probe Decl Decl :=\n filter (fun decl => go decl.value)\nwhere\n go : Code β†’ CompilerM Bool\n | .let _ k => go k\n | .fun decl k => go decl.value <||> go k\n | .jp decl k => do if (← f decl) then return true else go decl.value <||> go k\n | .cases cs => cs.alts.anyM (go Β·.getCode)\n | .jmp .. | .return .. | .unreach .. => return false", "start": [ 96, 1 ], "end": [ 104, 55 ], "kind": "commanddeclaration" }, { "full_name": "Lean.Compiler.LCNF.Probe.filterByFunDecl", "code": "partial def filterByFunDecl (f : FunDecl β†’ CompilerM Bool) : Probe Decl Decl :=\n filter (fun decl => go decl.value)\nwhere\n go : Code β†’ CompilerM Bool\n | .let _ k => go k\n | .fun decl k | .jp decl k => do if (← f decl) then return true else go decl.value <||> go k\n | .cases cs => cs.alts.anyM (go Β·.getCode)\n | .jmp .. | .return .. | .unreach .. => return false", "start": [ 106, 1 ], "end": [ 113, 55 ], "kind": "commanddeclaration" }, { "full_name": "Lean.Compiler.LCNF.Probe.filterByCases", "code": "partial def filterByCases (f : Cases β†’ CompilerM Bool) : Probe Decl Decl :=\n filter (fun decl => go decl.value)\nwhere\n go : Code β†’ CompilerM Bool\n | .let _ k => go k\n | .fun decl k | .jp decl k => go decl.value <||> go k\n | .cases cs => do if (← f cs) then return true else cs.alts.anyM (go Β·.getCode)\n | .jmp .. | .return .. | .unreach .. => return false", "start": [ 115, 1 ], "end": [ 122, 55 ], "kind": "commanddeclaration" }, { "full_name": "Lean.Compiler.LCNF.Probe.filterByJmp", "code": "partial def filterByJmp (f : FVarId β†’ Array Arg β†’ CompilerM Bool) : Probe Decl Decl :=\n filter (fun decl => go decl.value)\nwhere\n go : Code β†’ CompilerM Bool\n | .let _ k => go k\n | .fun decl k | .jp decl k => go decl.value <||> go k\n | .cases cs => cs.alts.anyM (go Β·.getCode)\n | .jmp fn var => f fn var\n | .return .. | .unreach .. => return false", "start": [ 124, 1 ], "end": [ 132, 45 ], "kind": "commanddeclaration" }, { "full_name": "Lean.Compiler.LCNF.Probe.filterByReturn", "code": "partial def filterByReturn (f : FVarId β†’ CompilerM Bool) : Probe Decl Decl :=\n filter (fun decl => go decl.value)\nwhere\n go : Code β†’ CompilerM Bool\n | .let _ k => go k\n | .fun decl k | .jp decl k => go decl.value <||> go k\n | .cases cs => cs.alts.anyM (go Β·.getCode)\n | .jmp .. | .unreach .. => return false\n | .return var => f var", "start": [ 134, 1 ], "end": [ 142, 26 ], "kind": "commanddeclaration" }, { "full_name": "Lean.Compiler.LCNF.Probe.filterByUnreach", "code": "partial def filterByUnreach (f : Expr β†’ CompilerM Bool) : Probe Decl Decl :=\n filter (fun decl => go decl.value)\nwhere\n go : Code β†’ CompilerM Bool\n | .let _ k => go k\n | .fun decl k | .jp decl k => go decl.value <||> go k\n | .cases cs => cs.alts.anyM (go Β·.getCode)\n | .jmp .. | .return .. => return false\n | .unreach typ => f typ", "start": [ 144, 1 ], "end": [ 152, 27 ], "kind": "commanddeclaration" }, { "full_name": "Lean.Compiler.LCNF.Probe.declNames", "code": "@[inline]\ndef declNames : Probe Decl Name :=\n Probe.map (fun decl => return decl.name)", "start": [ 154, 1 ], "end": [ 156, 43 ], "kind": "commanddeclaration" }, { "full_name": "Lean.Compiler.LCNF.Probe.toString", "code": "@[inline]\ndef toString [ToString Ξ±] : Probe Ξ± String :=\n Probe.map (return ToString.toString Β·)", "start": [ 158, 1 ], "end": [ 160, 41 ], "kind": "commanddeclaration" }, { "full_name": "Lean.Compiler.LCNF.Probe.count", "code": "@[inline]\ndef count : Probe Ξ± Nat := fun data => return #[data.size]", "start": [ 162, 1 ], "end": [ 163, 59 ], "kind": "commanddeclaration" }, { "full_name": "Lean.Compiler.LCNF.Probe.sum", "code": "@[inline]\ndef sum : Probe Nat Nat := fun data => return #[data.foldl (init := 0) (Β·+Β·)]", "start": [ 165, 1 ], "end": [ 166, 78 ], "kind": "commanddeclaration" }, { "full_name": "Lean.Compiler.LCNF.Probe.tail", "code": "@[inline]\ndef tail (n : Nat) : Probe Ξ± Ξ± := fun data => return data[data.size - n:]", "start": [ 168, 1 ], "end": [ 169, 74 ], "kind": "commanddeclaration" }, { "full_name": "Lean.Compiler.LCNF.Probe.head", "code": "@[inline]\ndef head (n : Nat) : Probe Ξ± Ξ± := fun data => return data[:n]", "start": [ 171, 1 ], "end": [ 172, 62 ], "kind": "commanddeclaration" }, { "full_name": "Lean.Compiler.LCNF.Probe.runOnModule", "code": "def runOnModule (moduleName : Name) (probe : Probe Decl Ξ²) (phase : Phase := Phase.base): CoreM (Array Ξ²) := do\n let ext := getExt phase\n let env ← getEnv\n let some modIdx := env.getModuleIdx? moduleName | throwError \"module `{moduleName}` not found\"\n let decls := ext.getModuleEntries env modIdx\n probe decls |>.run (phase := phase)", "start": [ 174, 1 ], "end": [ 179, 38 ], "kind": "commanddeclaration" }, { "full_name": "Lean.Compiler.LCNF.Probe.runGlobally", "code": "def runGlobally (probe : Probe Decl Ξ²) (phase : Phase := Phase.base) : CoreM (Array Ξ²) := do\n let ext := getExt phase\n let env ← getEnv\n let mut decls := #[]\n for modIdx in [:env.allImportedModuleNames.size] do\n decls := decls.append <| ext.getModuleEntries env modIdx\n probe decls |>.run (phase := phase)", "start": [ 181, 1 ], "end": [ 187, 38 ], "kind": "commanddeclaration" }, { "full_name": "Lean.Compiler.LCNF.Probe.toPass", "code": "def toPass [ToString Ξ²] (probe : Probe Decl Ξ²) (phase : Phase) : Pass where\n phase := phase\n name := `probe\n run := fun decls => do\n let res ← probe decls\n trace[Compiler.probe] s!\"{res}\"\n return decls", "start": [ 189, 1 ], "end": [ 195, 17 ], "kind": "commanddeclaration" } ]
.lake/packages/lean4/src/lean/Lean/Meta/Match/MatcherApp.lean
[ ".lake/packages/lean4/src/lean/Lean/Meta/Match/MatcherApp/Basic.lean", ".lake/packages/lean4/src/lean/Lean/Meta/Match/MatcherApp/Transform.lean" ]
[]
.lake/packages/lean4/src/lean/Lean/Meta/Match/MVarRenaming.lean
[ ".lake/packages/lean4/src/lean/Lean/Util/ReplaceExpr.lean" ]
[ { "full_name": "Lean.Meta.MVarRenaming", "code": "structure MVarRenaming where\n map : MVarIdMap MVarId := {}", "start": [ 11, 1 ], "end": [ 13, 31 ], "kind": "commanddeclaration" }, { "full_name": "Lean.Meta.MVarRenaming.isEmpty", "code": "def MVarRenaming.isEmpty (s : MVarRenaming) : Bool :=\n s.map.isEmpty", "start": [ 15, 1 ], "end": [ 16, 16 ], "kind": "commanddeclaration" }, { "full_name": "Lean.Meta.MVarRenaming.find?", "code": "def MVarRenaming.find? (s : MVarRenaming) (mvarId : MVarId) : Option MVarId :=\n s.map.find? mvarId", "start": [ 18, 1 ], "end": [ 19, 21 ], "kind": "commanddeclaration" }, { "full_name": "Lean.Meta.MVarRenaming.find!", "code": "def MVarRenaming.find! (s : MVarRenaming) (mvarId : MVarId) : MVarId :=\n (s.find? mvarId).get!", "start": [ 21, 1 ], "end": [ 22, 24 ], "kind": "commanddeclaration" }, { "full_name": "Lean.Meta.MVarRenaming.insert", "code": "def MVarRenaming.insert (s : MVarRenaming) (mvarId mvarId' : MVarId) : MVarRenaming :=\n { s with map := s.map.insert mvarId mvarId' }", "start": [ 24, 1 ], "end": [ 25, 48 ], "kind": "commanddeclaration" }, { "full_name": "Lean.Meta.MVarRenaming.apply", "code": "def MVarRenaming.apply (s : MVarRenaming) (e : Expr) : Expr :=\n if !e.hasMVar then e\n else if s.map.isEmpty then e\n else e.replace fun e => match e with\n | Expr.mvar mvarId => match s.map.find? mvarId with\n | none => e\n | some newMVarId => mkMVar newMVarId\n | _ => none", "start": [ 27, 1 ], "end": [ 34, 16 ], "kind": "commanddeclaration" } ]
.lake/packages/lean4/src/lean/Lean/Data/Lsp/Window.lean
[ ".lake/packages/lean4/src/lean/Lean/Data/Json.lean" ]
[ { "full_name": "MessageType", "code": "inductive MessageType where\n | error\n | warning\n | info\n | log", "start": [ 11, 1 ], "end": [ 15, 8 ], "kind": "commanddeclaration" }, { "full_name": "ShowMessageParams", "code": "structure ShowMessageParams where\n type : MessageType\n message : String\n deriving FromJson, ToJson", "start": [ 32, 1 ], "end": [ 35, 28 ], "kind": "commanddeclaration" }, { "full_name": "MessageActionItem", "code": "structure MessageActionItem where\n title : String\n deriving FromJson, ToJson", "start": [ 37, 1 ], "end": [ 39, 28 ], "kind": "commanddeclaration" }, { "full_name": "ShowMessageRequestParams", "code": "structure ShowMessageRequestParams where\n type : MessageType\n message : String\n actions? : Option (Array MessageActionItem)\n deriving FromJson, ToJson", "start": [ 41, 1 ], "end": [ 45, 28 ], "kind": "commanddeclaration" }, { "full_name": "ShowMessageResponse", "code": "def ShowMessageResponse := Option MessageActionItem\n deriving FromJson, ToJson", "start": [ 47, 1 ], "end": [ 48, 28 ], "kind": "commanddeclaration" } ]
.lake/packages/lean4/src/lean/Std.lean
[ ".lake/packages/lean4/src/lean/Init.lean" ]
[]