Skip to content

Commit d3599bd

Browse files
committed
chore: more adaptations for lean4#5542 (#17655)
In [lean4#5542](leanprover/lean4#5542) we are deprecating `inductive ... :=`, `structure ... :=`, and `class ... :=` for their `... where` counterparts. Continuation of #17564.
1 parent ee31f16 commit d3599bd

File tree

4 files changed

+6
-6
lines changed

4 files changed

+6
-6
lines changed

Diff for: Mathlib/Analysis/NormedSpace/HahnBanach/SeparatingDual.lean

+1-1
Original file line numberDiff line numberDiff line change
@@ -26,7 +26,7 @@ equivalences acts transitively on the set of nonzero vectors.
2626
registers that continuous linear forms on `E` separate points of `E`. -/
2727
@[mk_iff separatingDual_def]
2828
class SeparatingDual (R V : Type*) [Ring R] [AddCommGroup V] [TopologicalSpace V]
29-
[TopologicalSpace R] [Module R V] : Prop :=
29+
[TopologicalSpace R] [Module R V] : Prop where
3030
/-- Any nonzero vector can be mapped by a continuous linear map to a nonzero scalar. -/
3131
exists_ne_zero' : ∀ (x : V), x ≠ 0 → ∃ f : V →L[R] R, f x ≠ 0
3232

Diff for: Mathlib/Probability/Kernel/Disintegration/CDFToKernel.lean

+2-2
Original file line numberDiff line numberDiff line change
@@ -235,7 +235,7 @@ variable {f : α × β → ℚ → ℝ}
235235
conditions are the same, but the limit properties of `IsRatCondKernelCDF` are replaced by
236236
limits of integrals. -/
237237
structure IsRatCondKernelCDFAux (f : α × β → ℚ → ℝ) (κ : Kernel α (β × ℝ)) (ν : Kernel α β) :
238-
Prop :=
238+
Prop where
239239
measurable : Measurable f
240240
mono' (a : α) {q r : ℚ} (_hqr : q ≤ r) : ∀ᵐ c ∂(ν a), f (a, c) q ≤ f (a, c) r
241241
nonneg' (a : α) (q : ℚ) : ∀ᵐ c ∂(ν a), 0 ≤ f (a, c) q
@@ -425,7 +425,7 @@ respect to `ν` if it is measurable, tends to 0 at -∞ and to 1 at +∞ for all
425425
`fun b ↦ f (a, b) x` is `(ν a)`-integrable for all `a : α` and `x : ℝ` and for all
426426
measurable sets `s : Set β`, `∫ b in s, f (a, b) x ∂(ν a) = (κ a (s ×ˢ Iic x)).toReal`. -/
427427
structure IsCondKernelCDF (f : α × β → StieltjesFunction) (κ : Kernel α (β × ℝ)) (ν : Kernel α β) :
428-
Prop :=
428+
Prop where
429429
measurable (x : ℝ) : Measurable fun p ↦ f p x
430430
integrable (a : α) (x : ℝ) : Integrable (fun b ↦ f (a, b) x) (ν a)
431431
tendsto_atTop_one (p : α × β) : Tendsto (f p) atTop (𝓝 1)

Diff for: Mathlib/RingTheory/Algebraic.lean

+2-2
Original file line numberDiff line numberDiff line change
@@ -48,11 +48,11 @@ def Subalgebra.IsAlgebraic (S : Subalgebra R A) : Prop :=
4848
variable (R A)
4949

5050
/-- An algebra is algebraic if all its elements are algebraic. -/
51-
protected class Algebra.IsAlgebraic : Prop :=
51+
protected class Algebra.IsAlgebraic : Prop where
5252
isAlgebraic : ∀ x : A, IsAlgebraic R x
5353

5454
/-- An algebra is transcendental if some element is transcendental. -/
55-
protected class Algebra.Transcendental : Prop :=
55+
protected class Algebra.Transcendental : Prop where
5656
transcendental : ∃ x : A, Transcendental R x
5757

5858
variable {R A}

Diff for: Mathlib/RingTheory/IntegralClosure/Algebra/Defs.lean

+1-1
Original file line numberDiff line numberDiff line change
@@ -29,7 +29,7 @@ variable [Algebra R A] (R)
2929
variable (A)
3030

3131
/-- An algebra is integral if every element of the extension is integral over the base ring. -/
32-
protected class Algebra.IsIntegral : Prop :=
32+
protected class Algebra.IsIntegral : Prop where
3333
isIntegral : ∀ x : A, IsIntegral R x
3434

3535
variable {R A}

0 commit comments

Comments
 (0)