Skip to content

Commit a4be976

Browse files
committed
Update Sun Nov 24 11:16:32 EST 2024
1 parent 16067e3 commit a4be976

File tree

1 file changed

+85
-0
lines changed

1 file changed

+85
-0
lines changed

Math2001/Homework/hw9.lean

+85
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,85 @@
1+
/- Copyright (c) Heather Macbeth, 2023-4. All rights reserved. -/
2+
import Mathlib.Data.Real.Basic
3+
import Library.Theory.InjectiveSurjective
4+
import Library.Basic
5+
import AutograderLib
6+
7+
math2001_init
8+
set_option pp.funBinderTypes true
9+
10+
open Function
11+
12+
13+
/-! # Homework 9
14+
15+
Don't forget to compare with the text version,
16+
https://github.com/hrmacbeth/math2001/wiki/Homework-9,
17+
for clearer statements and any special instructions. -/
18+
19+
20+
/- Problem 1: prove one of these, delete the other -/
21+
22+
@[autograded 4]
23+
theorem problem1a : Surjective (fun (x : ℝ) ↦ 2 * x) := by
24+
sorry
25+
26+
@[autograded 4]
27+
theorem problem1b : ¬ Surjective (fun (x : ℝ) ↦ 2 * x) := by
28+
sorry
29+
30+
31+
/- Problem 2: prove one of these, delete the other -/
32+
33+
@[autograded 4]
34+
theorem problem2a : Surjective (fun (x : ℤ) ↦ 2 * x) := by
35+
sorry
36+
37+
@[autograded 4]
38+
theorem problem2b : ¬ Surjective (fun (x : ℤ) ↦ 2 * x) := by
39+
sorry
40+
41+
42+
/- Problem 3: prove one of these, delete the other -/
43+
44+
@[autograded 4]
45+
theorem problem3a : ∀ (f : ℚ → ℚ), Injective f → Injective (fun x ↦ f x + 1) := by
46+
sorry
47+
48+
@[autograded 4]
49+
theorem problem3b : ¬ ∀ (f : ℚ → ℚ), Injective f → Injective (fun x ↦ f x + 1) := by
50+
sorry
51+
52+
53+
/- Problem 4: prove one of these, delete the other -/
54+
55+
@[autograded 4]
56+
theorem problem4a : Bijective (fun (x : ℝ) ↦ 3 - 2 * x) := by
57+
sorry
58+
59+
@[autograded 4]
60+
theorem problem4b : ¬ Bijective (fun (x : ℝ) ↦ 3 - 2 * x) := by
61+
sorry
62+
63+
64+
/- Problem 5: prove one of these, delete the other -/
65+
66+
@[autograded 5]
67+
theorem problem5a :
68+
Injective (fun ((x, y, z) : ℝ × ℝ × ℝ) ↦ (x + y + z, x + 2 * y + 3 * z)) := by
69+
sorry
70+
71+
@[autograded 5]
72+
theorem problem5b :
73+
¬Injective (fun ((x, y, z) : ℝ × ℝ × ℝ) ↦ (x + y + z, x + 2 * y + 3 * z)) := by
74+
sorry
75+
76+
77+
/- Problem 6: prove one of these, delete the other -/
78+
79+
@[autograded 4]
80+
theorem problem6a : Bijective (fun ((r, s) : ℚ × ℚ) ↦ (s, r + 2 * s)) := by
81+
sorry
82+
83+
@[autograded 4]
84+
theorem problem6b : ¬ Bijective (fun ((r, s) : ℚ × ℚ) ↦ (s, r + 2 * s)) := by
85+
sorry

0 commit comments

Comments
 (0)