Skip to content

Commit

Permalink
chore: make sure all #align's are on a single line (#8215)
Browse files Browse the repository at this point in the history
We'll need to do this step anyway when it is time to remove them all.

(See #8214 where I'm benchmarking the removal.)



Co-authored-by: Scott Morrison <scott.morrison@gmail.com>
  • Loading branch information
semorrison and semorrison committed Nov 8, 2023
1 parent 9718370 commit 3dc73bd
Show file tree
Hide file tree
Showing 13 changed files with 20 additions and 41 deletions.
6 changes: 2 additions & 4 deletions Mathlib/Analysis/SpecialFunctions/Complex/Arg.lean
Expand Up @@ -583,8 +583,7 @@ theorem tendsto_arg_nhdsWithin_im_neg_of_re_neg_of_im_zero {z : ℂ} (hre : z.re
· simp [him]
· lift z to ℝ using him
simpa using hre.ne
#align complex.tendsto_arg_nhds_within_im_neg_of_re_neg_of_im_zero
Complex.tendsto_arg_nhdsWithin_im_neg_of_re_neg_of_im_zero
#align complex.tendsto_arg_nhds_within_im_neg_of_re_neg_of_im_zero Complex.tendsto_arg_nhdsWithin_im_neg_of_re_neg_of_im_zero

theorem continuousWithinAt_arg_of_re_neg_of_im_zero {z : ℂ} (hre : z.re < 0) (him : z.im = 0) :
ContinuousWithinAt arg { z : ℂ | 0 ≤ z.im } z := by
Expand All @@ -608,8 +607,7 @@ theorem tendsto_arg_nhdsWithin_im_nonneg_of_re_neg_of_im_zero {z : ℂ} (hre : z
(him : z.im = 0) : Tendsto arg (𝓝[{ z : ℂ | 0 ≤ z.im }] z) (𝓝 π) := by
simpa only [arg_eq_pi_iff.2 ⟨hre, him⟩] using
(continuousWithinAt_arg_of_re_neg_of_im_zero hre him).tendsto
#align complex.tendsto_arg_nhds_within_im_nonneg_of_re_neg_of_im_zero
Complex.tendsto_arg_nhdsWithin_im_nonneg_of_re_neg_of_im_zero
#align complex.tendsto_arg_nhds_within_im_nonneg_of_re_neg_of_im_zero Complex.tendsto_arg_nhdsWithin_im_nonneg_of_re_neg_of_im_zero

theorem continuousAt_arg_coe_angle (h : x ≠ 0) : ContinuousAt ((↑) ∘ arg : ℂ → Real.Angle) x := by
by_cases hs : 0 < x.re ∨ x.im ≠ 0
Expand Down
3 changes: 1 addition & 2 deletions Mathlib/Analysis/SpecialFunctions/Complex/Log.lean
Expand Up @@ -199,8 +199,7 @@ theorem continuousWithinAt_log_of_re_neg_of_im_zero {z : ℂ} (hre : z.re < 0) (
tendsto_const_nhds) using 1
· lift z to ℝ using him
simpa using hre.ne
#align complex.continuous_within_at_log_of_re_neg_of_im_zero
Complex.continuousWithinAt_log_of_re_neg_of_im_zero
#align complex.continuous_within_at_log_of_re_neg_of_im_zero Complex.continuousWithinAt_log_of_re_neg_of_im_zero

theorem tendsto_log_nhdsWithin_im_nonneg_of_re_neg_of_im_zero {z : ℂ} (hre : z.re < 0)
(him : z.im = 0) : Tendsto log (𝓝[{ z : ℂ | 0 ≤ z.im }] z) (𝓝 <| Real.log (abs z) + π * I) := by
Expand Down
3 changes: 1 addition & 2 deletions Mathlib/Data/Set/Card.lean
Expand Up @@ -985,8 +985,7 @@ theorem exists_subset_or_subset_of_two_mul_lt_ncard {n : ℕ} (hst : 2 * n < (s
(hu.subset (subset_union_right _ _))] at hst
obtain ⟨r', hnr', hr'⟩ := Finset.exists_subset_or_subset_of_two_mul_lt_card hst
exact ⟨r', by simpa, by simpa using hr'⟩
#align set.exists_subset_or_subset_of_two_mul_lt_ncard
Set.exists_subset_or_subset_of_two_mul_lt_ncard
#align set.exists_subset_or_subset_of_two_mul_lt_ncard Set.exists_subset_or_subset_of_two_mul_lt_ncard

/-! ### Explicit description of a set from its cardinality -/

Expand Down
3 changes: 1 addition & 2 deletions Mathlib/FieldTheory/Adjoin.lean
Expand Up @@ -791,8 +791,7 @@ theorem bot_eq_top_of_finrank_adjoin_le_one [FiniteDimensional F E]
theorem subsingleton_of_finrank_adjoin_le_one [FiniteDimensional F E]
(h : ∀ x : E, finrank F F⟮x⟯ ≤ 1) : Subsingleton (IntermediateField F E) :=
subsingleton_of_bot_eq_top (bot_eq_top_of_finrank_adjoin_le_one h)
#align intermediate_field.subsingleton_of_finrank_adjoin_le_one
IntermediateField.subsingleton_of_finrank_adjoin_le_one
#align intermediate_field.subsingleton_of_finrank_adjoin_le_one IntermediateField.subsingleton_of_finrank_adjoin_le_one

end AdjoinRank

Expand Down
3 changes: 1 addition & 2 deletions Mathlib/GroupTheory/Schreier.lean
Expand Up @@ -198,8 +198,7 @@ theorem card_commutator_le_of_finite_commutatorSet [Finite (commutatorSet G)] :
rw [← pow_succ'] at h2
refine' (Nat.le_of_dvd _ h2).trans (Nat.pow_le_pow_of_le_left h1 _)
exact pow_pos (Nat.pos_of_ne_zero FiniteIndex.finiteIndex) _
#align subgroup.card_commutator_le_of_finite_commutator_set
Subgroup.card_commutator_le_of_finite_commutatorSet
#align subgroup.card_commutator_le_of_finite_commutator_set Subgroup.card_commutator_le_of_finite_commutatorSet

/-- A theorem of Schur: A group with finitely many commutators has finite commutator subgroup. -/
instance [Finite (commutatorSet G)] : Finite (_root_.commutator G) := by
Expand Down
12 changes: 4 additions & 8 deletions Mathlib/MeasureTheory/Function/StronglyMeasurable/Basic.lean
Expand Up @@ -1806,8 +1806,7 @@ theorem aestronglyMeasurable_uIoc_iff [LinearOrder α] [PseudoMetrizableSpace β
AEStronglyMeasurable f (μ.restrict <| Ioc a b) ∧
AEStronglyMeasurable f (μ.restrict <| Ioc b a) :=
by rw [uIoc_eq_union, aestronglyMeasurable_union_iff]
#align measure_theory.ae_strongly_measurable.ae_strongly_measurable_uIoc_iff
MeasureTheory.AEStronglyMeasurable.aestronglyMeasurable_uIoc_iff
#align measure_theory.ae_strongly_measurable.ae_strongly_measurable_uIoc_iff MeasureTheory.AEStronglyMeasurable.aestronglyMeasurable_uIoc_iff

@[measurability]
theorem smul_measure {R : Type*} [Monoid R] [DistribMulAction R ℝ≥0∞] [IsScalarTower R ℝ≥0∞ ℝ≥0∞]
Expand Down Expand Up @@ -1879,8 +1878,7 @@ theorem _root_.ContinuousLinearMap.aestronglyMeasurable_comp₂ (L : E →L[𝕜
{g : α → F} (hf : AEStronglyMeasurable f μ) (hg : AEStronglyMeasurable g μ) :
AEStronglyMeasurable (fun x => L (f x) (g x)) μ :=
L.continuous₂.comp_aestronglyMeasurable <| hf.prod_mk hg
#align continuous_linear_map.ae_strongly_measurable_comp₂
ContinuousLinearMap.aestronglyMeasurable_comp₂
#align continuous_linear_map.ae_strongly_measurable_comp₂ ContinuousLinearMap.aestronglyMeasurable_comp₂

end ContinuousLinearMapNontriviallyNormedField

Expand Down Expand Up @@ -1936,16 +1934,14 @@ theorem finStronglyMeasurable_mk (hf : AEFinStronglyMeasurable f μ) :

theorem ae_eq_mk (hf : AEFinStronglyMeasurable f μ) : f =ᵐ[μ] hf.mk f :=
hf.choose_spec.2
#align measure_theory.ae_fin_strongly_measurable.ae_eq_mk
MeasureTheory.AEFinStronglyMeasurable.ae_eq_mk
#align measure_theory.ae_fin_strongly_measurable.ae_eq_mk MeasureTheory.AEFinStronglyMeasurable.ae_eq_mk

@[aesop 10% apply (rule_sets [Measurable])]
protected theorem aemeasurable {β} [Zero β] [MeasurableSpace β] [TopologicalSpace β]
[PseudoMetrizableSpace β] [BorelSpace β] {f : α → β} (hf : AEFinStronglyMeasurable f μ) :
AEMeasurable f μ :=
⟨hf.mk f, hf.finStronglyMeasurable_mk.measurable, hf.ae_eq_mk⟩
#align measure_theory.ae_fin_strongly_measurable.ae_measurable
MeasureTheory.AEFinStronglyMeasurable.aemeasurable
#align measure_theory.ae_fin_strongly_measurable.ae_measurable MeasureTheory.AEFinStronglyMeasurable.aemeasurable

end Mk

Expand Down
3 changes: 1 addition & 2 deletions Mathlib/NumberTheory/Cyclotomic/Basic.lean
Expand Up @@ -476,8 +476,7 @@ theorem isSplittingField_X_pow_sub_one : IsSplittingField K L (X ^ (n : ℕ) - 1
and_iff_right_iff_imp, Polynomial.map_sub, Polynomial.map_pow, Polynomial.map_one]
exact fun _ => X_pow_sub_C_ne_zero n.pos (1 : L) }
set_option linter.uppercaseLean3 false in
#align is_cyclotomic_extension.splitting_field_X_pow_sub_one
IsCyclotomicExtension.isSplittingField_X_pow_sub_one
#align is_cyclotomic_extension.splitting_field_X_pow_sub_one IsCyclotomicExtension.isSplittingField_X_pow_sub_one

/-- Any two `n`-th cyclotomic extensions are isomorphic. -/
def algEquiv (L' : Type*) [Field L'] [Algebra K L'] [IsCyclotomicExtension {n} K L'] :
Expand Down
5 changes: 1 addition & 4 deletions Mathlib/RepresentationTheory/Action.lean
Expand Up @@ -263,14 +263,11 @@ attribute above
theorem functorCategoryEquivalence.functor_def :
(functorCategoryEquivalence V G).functor = FunctorCategoryEquivalence.functor :=
rfl
set_option linter.uppercaseLean3 false in
#align Action.functor_category_equivalence.functor_def Action.functorCategoryEquivalence.functor_def
theorem functorCategoryEquivalence.inverse_def :
(functorCategoryEquivalence V G).inverse = FunctorCategoryEquivalence.inverse :=
rfl
set_option linter.uppercaseLean3 false in
#align Action.functor_category_equivalence.inverse_def Action.functorCategoryEquivalence.inverse_def-/
-/

instance [HasFiniteProducts V] : HasFiniteProducts (Action V G) where
out _ :=
Expand Down
3 changes: 1 addition & 2 deletions Mathlib/RingTheory/IntegralClosure.lean
Expand Up @@ -1075,8 +1075,7 @@ theorem RingHom.isIntegralElem_of_isIntegralElem_comp {x : T} (h : (g.comp f).Is
g.IsIntegralElem x :=
let ⟨p, ⟨hp, hp'⟩⟩ := h
⟨p.map f, hp.map f, by rwa [← eval₂_map] at hp'⟩
#align ring_hom.is_integral_elem_of_is_integral_elem_comp
RingHom.isIntegralElem_of_isIntegralElem_comp
#align ring_hom.is_integral_elem_of_is_integral_elem_comp RingHom.isIntegralElem_of_isIntegralElem_comp

theorem RingHom.isIntegral_tower_top_of_isIntegral (h : (g.comp f).IsIntegral) : g.IsIntegral :=
fun x => RingHom.isIntegralElem_of_isIntegralElem_comp f g (h x)
Expand Down
6 changes: 2 additions & 4 deletions Mathlib/Topology/Connected/Basic.lean
Expand Up @@ -714,8 +714,7 @@ theorem Continuous.mapsTo_connectedComponent [TopologicalSpace β] {f : α →
theorem irreducibleComponent_subset_connectedComponent {x : α} :
irreducibleComponent x ⊆ connectedComponent x :=
isIrreducible_irreducibleComponent.isConnected.subset_connectedComponent mem_irreducibleComponent
#align irreducible_component_subset_connected_component
irreducibleComponent_subset_connectedComponent
#align irreducible_component_subset_connected_component irreducibleComponent_subset_connectedComponent

@[mono]
theorem connectedComponentIn_mono (x : α) {F G : Set α} (h : F ⊆ G) :
Expand Down Expand Up @@ -1112,8 +1111,7 @@ theorem isPreconnected_iff_subset_of_fully_disjoint_closed {s : Set α} (hs : Is
· rw [← inter_distrib_right]
exact subset_inter hss Subset.rfl
· rwa [disjoint_iff_inter_eq_empty, ← inter_inter_distrib_right, inter_comm]
#align is_preconnected_iff_subset_of_fully_disjoint_closed
isPreconnected_iff_subset_of_fully_disjoint_closed
#align is_preconnected_iff_subset_of_fully_disjoint_closed isPreconnected_iff_subset_of_fully_disjoint_closed

theorem IsClopen.connectedComponent_subset {x} (hs : IsClopen s) (hx : x ∈ s) :
connectedComponent x ⊆ s :=
Expand Down
3 changes: 1 addition & 2 deletions Mathlib/Topology/Connected/LocallyConnected.lean
Expand Up @@ -36,8 +36,7 @@ theorem locallyConnectedSpace_iff_open_connected_basis :
LocallyConnectedSpace α ↔
∀ x, (𝓝 x).HasBasis (fun s : Set α => IsOpen s ∧ x ∈ s ∧ IsConnected s) id :=
⟨@LocallyConnectedSpace.open_connected_basis _ _, LocallyConnectedSpace.mk⟩
#align locally_connected_space_iff_open_connected_basis
locallyConnectedSpace_iff_open_connected_basis
#align locally_connected_space_iff_open_connected_basis locallyConnectedSpace_iff_open_connected_basis

theorem locallyConnectedSpace_iff_open_connected_subsets :
LocallyConnectedSpace α ↔
Expand Down
9 changes: 3 additions & 6 deletions Mathlib/Topology/Connected/TotallyDisconnected.lean
Expand Up @@ -117,8 +117,7 @@ theorem totallyDisconnectedSpace_iff_connectedComponent_subsingleton :
rcases eq_empty_or_nonempty s with (rfl | ⟨x, x_in⟩)
· exact subsingleton_empty
· exact (h x).anti (hs.subset_connectedComponent x_in)
#align totally_disconnected_space_iff_connected_component_subsingleton
totallyDisconnectedSpace_iff_connectedComponent_subsingleton
#align totally_disconnected_space_iff_connected_component_subsingleton totallyDisconnectedSpace_iff_connectedComponent_subsingleton

/-- A space is totally disconnected iff its connected components are singletons. -/
theorem totallyDisconnectedSpace_iff_connectedComponent_singleton :
Expand All @@ -127,8 +126,7 @@ theorem totallyDisconnectedSpace_iff_connectedComponent_singleton :
refine forall_congr' fun x => ?_
rw [subsingleton_iff_singleton]
exact mem_connectedComponent
#align totally_disconnected_space_iff_connected_component_singleton
totallyDisconnectedSpace_iff_connectedComponent_singleton
#align totally_disconnected_space_iff_connected_component_singleton totallyDisconnectedSpace_iff_connectedComponent_singleton

@[simp] theorem connectedComponent_eq_singleton [TotallyDisconnectedSpace α] (x : α) :
connectedComponent x = {x} :=
Expand Down Expand Up @@ -228,8 +226,7 @@ class TotallySeparatedSpace (α : Type u) [TopologicalSpace α] : Prop where
instance (priority := 100) TotallySeparatedSpace.totallyDisconnectedSpace (α : Type u)
[TopologicalSpace α] [TotallySeparatedSpace α] : TotallyDisconnectedSpace α :=
⟨TotallySeparatedSpace.isTotallySeparated_univ.isTotallyDisconnected⟩
#align totally_separated_space.totally_disconnected_space
TotallySeparatedSpace.totallyDisconnectedSpace
#align totally_separated_space.totally_disconnected_space TotallySeparatedSpace.totallyDisconnectedSpace

-- see Note [lower instance priority]
instance (priority := 100) TotallySeparatedSpace.of_discrete (α : Type*) [TopologicalSpace α]
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Topology/ContinuousFunction/Basic.lean
Expand Up @@ -597,7 +597,7 @@ instance : Coe (α ≃ₜ β) C(α, β) :=
-- Porting note: Syntactic tautology
/-theorem toContinuousMap_as_coe : f.toContinuousMap = f :=
rfl
#align homeomorph.to_continuous_map_as_coe Homeomorph.toContinuousMap_as_coe-/
-/
#noalign homeomorph.to_continuous_map_as_coe

@[simp]
Expand Down

0 comments on commit 3dc73bd

Please sign in to comment.