Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit 3088264

Browse files
committed
chore(archive/imo): fix some naming inconsistencies and whitespace (#19155)
I realize that this is the third PR concerning namespacing the files in `archive/imo`. These are some simple inconsistencies in naming. There is no rush in merging this PR, but in the long run it might help to have consistent namespacing, so that batch renames can be simpler.
1 parent 533f62f commit 3088264

18 files changed

+27
-19
lines changed

archive/imo/imo1975_q1.lean

Lines changed: 1 addition & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -31,9 +31,7 @@ variables (hx : antitone_on x (finset.Icc 1 n))
3131
variables (hy : antitone_on y (finset.Icc 1 n))
3232
include hx hy hσ
3333

34-
namespace imo1975_q1
35-
36-
theorem IMO_1975_Q1 :
34+
theorem imo1975_q1 :
3735
∑ i in finset.Icc 1 n, (x i - y i) ^ 2 ≤ ∑ i in finset.Icc 1 n, (x i - y (σ i)) ^ 2 :=
3836
begin
3937
simp only [sub_sq, finset.sum_add_distrib, finset.sum_sub_distrib],
@@ -48,5 +46,3 @@ begin
4846
-- them being `decreasing`
4947
exact antitone_on.monovary_on hx hy
5048
end
51-
52-
end imo1975_q1

archive/imo/imo1977_q6.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -36,6 +36,7 @@ begin
3636
end
3737

3838
end imo1977_q6
39+
3940
open imo1977_q6
4041

4142
theorem imo1977_q6 (f : ℕ+ → ℕ+) (h : ∀ n, f (f n) < f (n + 1)) :

archive/imo/imo1988_q6.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -186,6 +186,7 @@ begin
186186
end
187187

188188
end imo1988_q6
189+
189190
open imo1988_q6
190191

191192
/--Question 6 of IMO1988. If a and b are two natural numbers

archive/imo/imo1994_q1.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -46,6 +46,7 @@ begin
4646
end
4747

4848
end imo1994_q1
49+
4950
open imo1994_q1
5051

5152
theorem imo1994_q1 (n : ℕ) (m : ℕ) (A : finset ℕ) (hm : A.card = m + 1)

archive/imo/imo1998_q2.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -198,6 +198,7 @@ lemma clear_denominators {a b k : ℕ} (ha : 0 < a) (hb : 0 < b) :
198198
by rw div_le_div_iff; norm_cast; simp [ha, hb]
199199

200200
end imo1998_q2
201+
201202
open imo1998_q2
202203

203204
theorem imo1998_q2 [fintype J] [fintype C]

archive/imo/imo2001_q2.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -67,6 +67,7 @@ calc _ ≥ _ : add_le_add (add_le_add (bound ha hb hc) (bound hb hc ha)) (bound
6767
... = 1 : by rw [h₁, h₂, ← add_div, ← add_div, div_self $ ne_of_gt $ denom_pos ha hb hc]
6868

6969
end imo2001_q2
70+
7071
open imo2001_q2
7172

7273
theorem imo2001_q2 (ha : 0 < a) (hb : 0 < b) (hc : 0 < c) :

archive/imo/imo2005_q3.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -45,6 +45,7 @@ begin
4545
end
4646

4747
end imo2005_q3
48+
4849
open imo2005_q3
4950

5051
theorem imo2005_q3 (x y z : ℝ) (hx : x > 0) (hy : y > 0) (hz : z > 0) (h : x*y*z ≥ 1) :

archive/imo/imo2005_q4.lean

Lines changed: 5 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -55,8 +55,12 @@ begin
5555
... = 0 : by ring,
5656
end
5757

58+
end imo2005_q4
59+
60+
open imo2005_q4
61+
5862
/-- Main statement: The only positive integer coprime to all terms of the sequence `a` is `1`. -/
59-
example {k : ℕ} (hk : 0 < k) : (∀ n : ℕ, 1 ≤ n → is_coprime (a n) k) ↔ k = 1 :=
63+
theorem imo2005_q4 {k : ℕ} (hk : 0 < k) : (∀ n : ℕ, 1 ≤ n → is_coprime (a n) k) ↔ k = 1 :=
6064
begin
6165
split, rotate,
6266
{ -- The property is clearly true for `k = 1`
@@ -95,5 +99,3 @@ begin
9599
-- Contradiction!
96100
contradiction,
97101
end
98-
99-
end imo2005_q4

archive/imo/imo2006_q3.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -136,6 +136,7 @@ begin
136136
end
137137

138138
end imo2006_q3
139+
139140
open imo2006_q3
140141

141142
theorem imo2006_q3 (M : ℝ) :

archive/imo/imo2006_q5.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -201,6 +201,7 @@ begin
201201
end
202202

203203
end imo2006_q5
204+
204205
open imo2006_q5
205206

206207
/-- The general problem follows easily from the k = 2 case. -/

0 commit comments

Comments
 (0)