Skip to content

Commit 9c7047a

Browse files
author
Will Bradley
committed
State all parts of the fifth homework problem
1 parent 3d8f714 commit 9c7047a

File tree

1 file changed

+32
-8
lines changed

1 file changed

+32
-8
lines changed
Lines changed: 32 additions & 8 deletions
Original file line numberDiff line numberDiff line change
@@ -1,6 +1,25 @@
11
import LogicFormalization.Chapter2.Section4.Term
2+
import Mathlib.Data.Fin.VecNotation
23

3-
-- TODO: problems 1, 2, 3, 4, 5 (b) (c), rename and organize stuff (see previous `Homework.lean` files)
4+
namespace Homeworks
5+
6+
open Term HasVar
7+
8+
section Problem1
9+
/-! TODO -/
10+
end Problem1
11+
12+
section Problem2
13+
/-! TODO -/
14+
end Problem2
15+
16+
section Problem3
17+
/-! TODO -/
18+
end Problem3
19+
20+
section Problem4
21+
/-! TODO -/
22+
end Problem4
423

524
section Problem5
625

@@ -12,15 +31,20 @@ def 𝒩 : Structure .Rig ℕ where
1231
| .add, a => a 0 + a 1
1332
| .mul, a => a 0 * a 1
1433

15-
open Term
16-
open HasVar
34+
/-- 2.4 #5 (a) -/
35+
theorem not_exists_nat_rig_term₁ : ¬∃ (t: Term .Rig) (x: Var) (hx: AreVarsFor ![x] t),
36+
interp t 𝒩 hx ![0] = 1 ∧ interp t 𝒩 hx ![1] = 0 :=
37+
sorry
1738

39+
/-- 2.4 #5 (b) -/
40+
theorem not_exists_nat_rig_term₂ : ¬∃ (t: Term .Rig) (x: Var) (hx: AreVarsFor ![x] t),
41+
∀ n, interp t 𝒩 hx ![n] = 2^n :=
42+
sorry
1843

19-
theorem a : ¬∃ (t: Term .Rig) (x: Var)
20-
(hx: AreVarsFor (m := 1) (fun | 0 => x) t),
21-
interp t 𝒩 hx (fun _ => 0) = 1 ∧ interp t 𝒩 hx (fun _ => 1) = 0 := by
22-
push_neg
23-
intro t x hx h₀ h₁
44+
open Structure in
45+
/-- 2.4 #5 (c). The only substructure of `𝒩` is `𝒩` itself. -/
46+
theorem 𝒩.substructures: ∀ {A: Set ℕ} [Nonempty A] {𝒜: Structure .Rig A},
47+
𝒜 ⊆ 𝒩 ↔ HEq 𝒜 𝒩 :=
2448
sorry
2549

2650
end Problem5

0 commit comments

Comments
 (0)