File tree 1 file changed +49
-0
lines changed
1 file changed +49
-0
lines changed Original file line number Diff line number Diff line change
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
+ @[autograded 3]
20
+ theorem problem1 {f : X → Y} (hf : Injective f) {g : Y → Z} (hg : Injective g) :
21
+ Injective (g ∘ f) := by
22
+ sorry
23
+
24
+ @[autograded 4]
25
+ theorem problem2a : Bijective (fun (x : ℝ) ↦ 5 + 3 * x) := by
26
+ sorry
27
+
28
+ @[autograded 4]
29
+ theorem problem2b : ¬ Bijective (fun (x : ℝ) ↦ 5 + 3 * x) := by
30
+ sorry
31
+
32
+ @[autograded 5]
33
+ theorem problem3 :
34
+ ¬Injective (fun ((x, y, z) : ℝ × ℝ × ℝ) ↦ (x + y + z, x - 2 * y + z)) := by
35
+ sorry
36
+
37
+ @[autograded 4]
38
+ theorem problem4 : Bijective (fun ((r, s) : ℚ × ℚ) ↦ (s, r + 2 * s)) := by
39
+ rw [bijective_iff_exists_inverse]
40
+ use fun (a, b) ↦ (sorry , sorry )
41
+ sorry
42
+
43
+ @[autograded 4]
44
+ theorem problem5 : ¬ Surjective (fun ((x, y) : ℚ × ℚ) ↦ x ^ 2 + y ^ 2 ) := by
45
+ sorry
46
+
47
+ @[autograded 5]
48
+ theorem problem6 : Surjective (fun ((x, y) : ℚ × ℚ) ↦ x ^ 2 - y ^ 2 ) := by
49
+ sorry
You can’t perform that action at this time.
0 commit comments