Skip to content

Commit 6534503

Browse files
committed
chore: fix some indentation (#24874)
1 parent 1bd7adb commit 6534503

File tree

4 files changed

+7
-7
lines changed

4 files changed

+7
-7
lines changed

Mathlib/Analysis/SpecialFunctions/Pow/Continuity.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -217,7 +217,7 @@ theorem continuousAt_rpow (p : ℝ × ℝ) (h : p.1 ≠ 0 ∨ 0 < p.2) :
217217
@[fun_prop]
218218
theorem continuousAt_rpow_const (x : ℝ) (q : ℝ) (h : x ≠ 00 ≤ q) :
219219
ContinuousAt (fun x : ℝ => x ^ q) x := by
220-
· rw [le_iff_lt_or_eq, ← or_assoc] at h
220+
rw [le_iff_lt_or_eq, ← or_assoc] at h
221221
obtain h|rfl := h
222222
· exact (continuousAt_rpow (x, q) h).comp₂ continuousAt_id continuousAt_const
223223
· simp_rw [rpow_zero]; exact continuousAt_const

Mathlib/Deprecated/Cardinal/Finite.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -77,7 +77,7 @@ theorem _root_.Cardinal.natCast_eq_toPartENat_iff {n : ℕ} {c : Cardinal} :
7777
@[simp]
7878
theorem _root_.Cardinal.toPartENat_eq_natCast_iff {c : Cardinal} {n : ℕ} :
7979
Cardinal.toPartENat c = n ↔ c = n := by
80-
rw [eq_comm, Cardinal.natCast_eq_toPartENat_iff, eq_comm]
80+
rw [eq_comm, Cardinal.natCast_eq_toPartENat_iff, eq_comm]
8181

8282
@[simp]
8383
theorem _root_.Cardinal.natCast_lt_toPartENat_iff {n : ℕ} {c : Cardinal} :

Mathlib/LinearAlgebra/Lagrange.lean

Lines changed: 4 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -471,10 +471,10 @@ theorem natDegree_nodal [Nontrivial R] : (nodal s v).natDegree = #s := by
471471
natDegree_X_sub_C, sum_const, smul_eq_mul, mul_one]
472472

473473
theorem nodal_ne_zero [Nontrivial R] : nodal s v ≠ 0 := by
474-
rcases s.eq_empty_or_nonempty with (rfl | h)
475-
· exact one_ne_zero
476-
· apply ne_zero_of_natDegree_gt (n := 0)
477-
simp only [natDegree_nodal, h.card_pos]
474+
rcases s.eq_empty_or_nonempty with (rfl | h)
475+
· exact one_ne_zero
476+
· apply ne_zero_of_natDegree_gt (n := 0)
477+
simp only [natDegree_nodal, h.card_pos]
478478

479479
@[simp]
480480
theorem degree_nodal [Nontrivial R] : (nodal s v).degree = #s := by

Mathlib/Logic/Relation.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -482,7 +482,7 @@ theorem TransGen.lift {p : β → β → Prop} {a b : α} (f : α → β) (h :
482482
theorem TransGen.lift' {p : β → β → Prop} {a b : α} (f : α → β)
483483
(h : ∀ a b, r a b → TransGen p (f a) (f b)) (hab : TransGen r a b) :
484484
TransGen p (f a) (f b) := by
485-
simpa [transGen_idem] using hab.lift f h
485+
simpa [transGen_idem] using hab.lift f h
486486

487487
theorem TransGen.closed {p : α → α → Prop} :
488488
(∀ a b, r a b → TransGen p a b) → TransGen r a b → TransGen p a b :=

0 commit comments

Comments
 (0)