Skip to content

Commit 88ce099

Browse files
committed
chore: substitute some . with · (#12137)
Co-authored-by: Moritz Firsching <firsching@google.com>
1 parent 7eeaaff commit 88ce099

File tree

13 files changed

+27
-27
lines changed

13 files changed

+27
-27
lines changed

Mathlib/Algebra/GroupPower/Order.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -532,7 +532,7 @@ namespace Nat
532532
variable {n : ℕ} {f : α → ℕ}
533533

534534
/-- See also `pow_left_strictMonoOn`. -/
535-
protected lemma pow_left_strictMono (hn : n ≠ 0) : StrictMono (. ^ n : ℕ → ℕ) :=
535+
protected lemma pow_left_strictMono (hn : n ≠ 0) : StrictMono (· ^ n : ℕ → ℕ) :=
536536
fun _ _ h ↦ Nat.pow_lt_pow_left h hn
537537
#align nat.pow_left_strict_mono Nat.pow_left_strictMono
538538

Mathlib/Algebra/Polynomial/Basic.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -299,7 +299,7 @@ instance semiring : Semiring R[X] :=
299299
toMul := Polynomial.mul'
300300
toZero := Polynomial.zero
301301
toOne := Polynomial.one
302-
nsmul := (..)
302+
nsmul := (··)
303303
npow := fun n x => (x ^ n) }
304304
#align polynomial.semiring Polynomial.semiring
305305

@@ -1190,7 +1190,7 @@ instance ring : Ring R[X] :=
11901190
toIntCast := Polynomial.intCast
11911191
toNeg := Polynomial.neg'
11921192
toSub := Polynomial.sub
1193-
zsmul := ((..) : ℤ → R[X] → R[X]) }
1193+
zsmul := ((··) : ℤ → R[X] → R[X]) }
11941194
#align polynomial.ring Polynomial.ring
11951195

11961196
@[simp]

Mathlib/Data/Fin/Tuple/Curry.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -73,7 +73,7 @@ variable {n : ℕ} {p : Fin n → Type u} {τ : Type u}
7373
theorem curry_uncurry (f : Function.FromTypes p τ) : curry (uncurry f) = f := by
7474
induction n with
7575
| zero => rfl
76-
| succ n ih => exact funext (ih $ f .)
76+
| succ n ih => exact funext (ih $ f ·)
7777

7878
@[simp]
7979
theorem uncurry_curry (f : ((i : Fin n) → p i) → τ) :

Mathlib/Data/Pi/Lex.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -119,15 +119,15 @@ open Function
119119

120120
theorem toLex_monotone : Monotone (@toLex (∀ i, β i)) := fun a b h =>
121121
or_iff_not_imp_left.2 fun hne =>
122-
let ⟨i, hi, hl⟩ := IsWellFounded.wf.has_min (r := (· < · )) { i | a i ≠ b i }
122+
let ⟨i, hi, hl⟩ := IsWellFounded.wf.has_min (r := (· < ·)) { i | a i ≠ b i }
123123
(Function.ne_iff.1 hne)
124124
⟨i, fun j hj => by
125125
contrapose! hl
126126
exact ⟨j, hl, hj⟩, (h i).lt_of_ne hi⟩
127127
#align pi.to_lex_monotone Pi.toLex_monotone
128128

129129
theorem toLex_strictMono : StrictMono (@toLex (∀ i, β i)) := fun a b h =>
130-
let ⟨i, hi, hl⟩ := IsWellFounded.wf.has_min (r := (· < · )) { i | a i ≠ b i }
130+
let ⟨i, hi, hl⟩ := IsWellFounded.wf.has_min (r := (· < ·)) { i | a i ≠ b i }
131131
(Function.ne_iff.1 h.ne)
132132
⟨i, fun j hj => by
133133
contrapose! hl

Mathlib/Data/Set/Subset.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -74,7 +74,7 @@ lemma preimage_val_sInter : A ↓∩ (⋂₀ S) = ⋂₀ { (A ↓∩ B) | B ∈
7474
erw [sInter_image]
7575
simp_rw [sInter_eq_biInter, preimage_iInter]
7676

77-
lemma preimage_val_sInter_eq_sInter : A ↓∩ (⋂₀ S) = ⋂₀ ((A ↓∩ .) '' S) := by
77+
lemma preimage_val_sInter_eq_sInter : A ↓∩ (⋂₀ S) = ⋂₀ ((A ↓∩ ·) '' S) := by
7878
simp only [preimage_sInter, sInter_image]
7979

8080
lemma eq_of_preimage_val_eq_of_subset (hB : B ⊆ A) (hC : C ⊆ A) (h : A ↓∩ B = A ↓∩ C) : B = C := by

Mathlib/GroupTheory/Exponent.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -93,7 +93,7 @@ open MulOpposite in
9393
theorem _root_.MulOpposite.exponent : exponent (MulOpposite G) = exponent G := by
9494
simp only [Monoid.exponent, ExponentExists]
9595
congr!
96-
all_goals exact ⟨(op_injective <| · <| op ·), (unop_injective <| . <| unop .)⟩
96+
all_goals exact ⟨(op_injective <| · <| op ·), (unop_injective <| · <| unop ·)⟩
9797

9898
@[to_additive]
9999
theorem ExponentExists.isOfFinOrder (h : ExponentExists G) {g : G} : IsOfFinOrder g :=

Mathlib/GroupTheory/HNNExtension.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -591,7 +591,7 @@ open NormalWord
591591
theorem of_injective : Function.Injective (of : G → HNNExtension G A B φ) := by
592592
rcases TransversalPair.nonempty G A B with ⟨d⟩
593593
refine Function.Injective.of_comp
594-
(f := ((..) : HNNExtension G A B φ → NormalWord d → NormalWord d)) ?_
594+
(f := ((··) : HNNExtension G A B φ → NormalWord d → NormalWord d)) ?_
595595
intros _ _ h
596596
exact eq_of_smul_eq_smul (fun w : NormalWord d =>
597597
by simp_all [Function.funext_iff, of_smul_eq_smul])

Mathlib/GroupTheory/PushoutI.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -596,7 +596,7 @@ theorem of_injective (hφ : ∀ i, Function.Injective (φ i)) (i : ι) :
596596
let _ := Classical.decEq ι
597597
let _ := fun i => Classical.decEq (G i)
598598
refine Function.Injective.of_comp
599-
(f := ((..) : PushoutI φ → NormalWord d → NormalWord d)) ?_
599+
(f := ((··) : PushoutI φ → NormalWord d → NormalWord d)) ?_
600600
intros _ _ h
601601
exact eq_of_smul_eq_smul (fun w : NormalWord d =>
602602
by simp_all [Function.funext_iff, of_smul_eq_smul])
@@ -607,7 +607,7 @@ theorem base_injective (hφ : ∀ i, Function.Injective (φ i)) :
607607
let _ := Classical.decEq ι
608608
let _ := fun i => Classical.decEq (G i)
609609
refine Function.Injective.of_comp
610-
(f := ((..) : PushoutI φ → NormalWord d → NormalWord d)) ?_
610+
(f := ((··) : PushoutI φ → NormalWord d → NormalWord d)) ?_
611611
intros _ _ h
612612
exact eq_of_smul_eq_smul (fun w : NormalWord d =>
613613
by simp_all [Function.funext_iff, base_smul_eq_smul])

Mathlib/ModelTheory/Definability.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -60,7 +60,7 @@ theorem Definable.map_expansion {L' : FirstOrder.Language} [L'.Structure M] (h :
6060
theorem definable_iff_exists_formula_sum :
6161
A.Definable L s ↔ ∃ φ : L.Formula (A ⊕ α), s = {v | φ.Realize (Sum.elim (↑) v)} := by
6262
rw [Definable, Equiv.exists_congr_left (BoundedFormula.constantsVarsEquiv)]
63-
refine exists_congr (fun φ => iff_iff_eq.2 (congr_arg (s = .) ?_))
63+
refine exists_congr (fun φ => iff_iff_eq.2 (congr_arg (s = ·) ?_))
6464
ext
6565
simp only [Formula.Realize, BoundedFormula.constantsVarsEquiv, constantsOn, mk₂_Relations,
6666
BoundedFormula.mapTermRelEquiv_symm_apply, mem_setOf_eq]

Mathlib/ModelTheory/Syntax.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -667,11 +667,11 @@ def toFormula : ∀ {n : ℕ}, L.BoundedFormula α n → L.Formula (Sum α (Fin
667667

668668
/-- take the disjunction of a finite set of formulas -/
669669
noncomputable def iSup (s : Finset β) (f : β → L.BoundedFormula α n) : L.BoundedFormula α n :=
670-
(s.toList.map f).foldr (..) ⊥
670+
(s.toList.map f).foldr (··) ⊥
671671

672672
/-- take the conjunction of a finite set of formulas -/
673673
noncomputable def iInf (s : Finset β) (f : β → L.BoundedFormula α n) : L.BoundedFormula α n :=
674-
(s.toList.map f).foldr (..) ⊤
674+
(s.toList.map f).foldr (··) ⊤
675675

676676

677677
variable {l : ℕ} {φ ψ : L.BoundedFormula α l} {θ : L.BoundedFormula α l.succ}

0 commit comments

Comments
 (0)