Skip to content

Commit

Permalink
remove unneeded lines found by linter
Browse files Browse the repository at this point in the history
  • Loading branch information
dwrensha committed Nov 20, 2024
1 parent a84dd02 commit 5a43d32
Show file tree
Hide file tree
Showing 2 changed files with 0 additions and 33 deletions.
11 changes: 0 additions & 11 deletions Compfiles/Imo1970P4.lean
Original file line number Diff line number Diff line change
Expand Up @@ -452,9 +452,6 @@ lemma subsets_must_overlap_pigeonhole (s s1 s2 : Finset ℕ) (predicate_s1: ℕ
have s1_is_subset: s1 ⊆ s := by
rw[s1_filter]
apply Finset.filter_subset
have s2_is_subset: s2 ⊆ s := by
rw[s2_filter]
apply Finset.filter_subset
have lift_x_in_s1 : ∀ x ∈ s, x ∈ s1 ↔ predicate_s1 x := by
rw[s1_filter]
intro x _
Expand Down Expand Up @@ -634,18 +631,12 @@ lemma contradiction_of_finset_icc_1_6 (s1 s2 : Finset ℕ) (partition : s1 ∪ s
have five_set_in_s2 : {5} ⊆ s2 := by
simp_all only [Finset.singleton_subset_iff]
have set_five_in_empty := s1_s2_disjoint five_set_in_s1 five_set_in_s2
have : Nonempty ({5} : Finset ℕ) := by
simp_all only [Finset.singleton_subset_iff, Finset.mem_singleton, nonempty_subtype, exists_eq]
have : ({5} : Finset ℕ).Nonempty := by
simp_all only [Finset.singleton_subset_iff, Finset.mem_singleton, nonempty_subtype, exists_eq, Finset.singleton_nonempty]
apply not_empty_subst_of_nonempty {5} this
exact set_five_in_empty
have s2_in_interval : s2 ⊆ Finset.Icc 1 6 := by
rw[partition] at s2_in_s1_s2
exact s2_in_s1_s2
have explicit_interval: Finset.Icc 1 6 = {1, 2, 3, 4, 5, 6} := by
rfl
rw [explicit_interval] at s2_in_interval
have := diffs_of_disjoint s2 (s1 ∪ s2) {5} s2_in_s1_s2 five_not_in_s2
rw [partition] at this
rw[explicit_interval] at this
Expand Down Expand Up @@ -683,8 +674,6 @@ lemma contradiction_of_finset_icc_1_6 (s1 s2 : Finset ℕ) (partition : s1 ∪ s
have five_set_in_s2 : {5} ⊆ s2 := by
simp_all only [Finset.singleton_subset_iff]
have set_five_in_empty := s2_s1_disjoint five_set_in_s2 five_set_in_s1
have : Nonempty ({5} : Finset ℕ) := by
simp_all only [Finset.singleton_subset_iff, Finset.mem_singleton, nonempty_subtype, exists_eq]
have : ({5} : Finset ℕ).Nonempty := by
simp_all only [Finset.singleton_subset_iff, Finset.mem_singleton, nonempty_subtype, exists_eq, Finset.singleton_nonempty]
apply not_empty_subst_of_nonempty {5} this
Expand Down
22 changes: 0 additions & 22 deletions Compfiles/Usa1992P1.lean
Original file line number Diff line number Diff line change
Expand Up @@ -114,8 +114,6 @@ lemma Finset.prod_odd {α : Type} [DecidableEq α] {f : α → ℕ} {s : Finset

lemma lemma3 {m : ℕ} (hm : (m % 10) + 1 < 10) :
(Nat.digits 10 (m + 1)).sum = (Nat.digits 10 m).sum + 1 := by
have h1 : 101 := by norm_num
have h2 : 1 < 10 := by norm_num
rw [Nat.digits_eq_cons_digits_div (by norm_num) (by omega)]
by_cases h : m = 0
· simp [h]
Expand Down Expand Up @@ -342,11 +340,6 @@ lemma lemma5 {m n : ℕ} (hm : m < 10^n) :
unfold complement_digits
rw [←h1, ←lemma8, h_sub2]
rw [h_sub]
have h11 : ∀ l ∈ complement_digits, l < 10 := by
intro l hl
unfold complement_digits at hl
simp only [List.mem_map] at hl
omega
have h12 : ∀ l ∈ complement_digits, l < 10 := by
intro x hx
simp only [List.map_append, List.mem_append, List.mem_map, complement_digits, m_digits_padded,
Expand All @@ -362,12 +355,6 @@ lemma lemma5 {m n : ℕ} (hm : m < 10^n) :
simp_all
have h13 := digitsPadded_ofDigits 10 n (by norm_num) complement_digits h12 h14
rw [h13]
have h15 : n -
(List.map (fun d ↦ 9 - d) (Nat.digits 10 m) ++
List.replicate (n - (Nat.digits 10 m).length) 9).length = 0 := by
simp only [Nat.reduceLeDiff, List.length_append, List.length_map, List.length_replicate]
have : (Nat.digits 10 m).length ≤ n := lemma9 hm
simp_all

have h16 : (Nat.digits 10 m).length ≤ n := lemma9 hm
simp [digitsPadded, padList, List.map_append, List.map_replicate, tsub_zero, complement_digits,
Expand All @@ -385,7 +372,6 @@ match l1, l2 with
simp only [List.zipWith_cons_cons, List.sum_cons]
rw [ih.1]
have h3 : hd1 ≥ hd2 := (List.forall₂_cons.mp h2).1
have h4 : tl1.sum ≥ tl2.sum := ih.2
omega

lemma List.sum_map_sub (l1 l2 : List ℕ) (h2 : List.Forall₂ (· ≥ ·) l1 l2) :
Expand All @@ -394,9 +380,6 @@ lemma List.sum_map_sub (l1 l2 : List ℕ) (h2 : List.Forall₂ (· ≥ ·) l1 l2

lemma lemma4 {m n : ℕ} (hm : m < 10^n) :
(Nat.digits 10 (10^n - 1 - m)).sum = 9 * n - (Nat.digits 10 m).sum := by
have h1 : (Nat.digits 10 m).sum =
(Nat.digits 10 m ++ List.replicate (n - (Nat.digits 10 m).length) 0).sum := by
simp
rw [←digitsPadded_sum, lemma5 hm]
have h2 := List.map_eq_zip 9 (digitsPadded 10 m n) (fun x y ↦ x - y)
rw [h2]
Expand Down Expand Up @@ -538,8 +521,6 @@ problem usa1992_p1 (n : ℕ) :
have h10 : (Nat.digits 10 (b n)).head! ≠ 0 := by
rw [Nat.head!_digits (by norm_num)]
intro h11
have h12 : 10 ∣ b n := Nat.dvd_of_mod_eq_zero h11
rw [show 10 = 2 * 5 by norm_num] at h12
have h13 : 2 ∣ b n := by omega
have h14 : ¬ 2 ∣ b n := Odd.not_two_dvd_nat (h9 _)
contradiction
Expand All @@ -553,8 +534,6 @@ problem usa1992_p1 (n : ℕ) :
rw [List.sum_cons, List.sum_cons]
have h13 : b n % 100 := by
intro h11
have h12 : 10 ∣ b n := Nat.dvd_of_mod_eq_zero h11
rw [show 10 = 2 * 5 by norm_num] at h12
have h13 : 2 ∣ b n := by omega
have h14 : ¬ 2 ∣ b n := Odd.not_two_dvd_nat (h9 _)
contradiction
Expand Down Expand Up @@ -602,7 +581,6 @@ problem usa1992_p1 (n : ℕ) :
have h43 : Odd 1 := Nat.odd_iff.mpr rfl
have h44 : 110 ^ 2 ^ (n+1) := Nat.one_le_pow' _ _
have h45 : Odd (10 ^ 2 ^ (n + 1) - 1) := Nat.Even.sub_odd h44 h42 h43
have h46 : b n ≤ 10 ^ 2 ^ (n + 1) - 1 := (Nat.le_sub_one_iff_lt h44).mpr h5
have h47 : Even (10 ^ 2 ^ (n + 1) - 1 - b n) := Nat.Odd.sub_odd h45 (h9 n)
rw [Nat.even_iff] at h47
rw [Nat.odd_iff] at H1
Expand Down

0 comments on commit 5a43d32

Please sign in to comment.