bookshelf/Bookshelf/Fraleigh/Chapter_1.lean

24 lines
440 B
Plaintext
Raw Permalink Normal View History

2023-05-04 22:37:54 +00:00
import Mathlib.Data.Complex.Basic
2023-05-08 19:43:54 +00:00
/-! # Fraleign.Chapter1
2023-04-02 14:57:58 +00:00
Introduction and Examples
-/
2023-05-08 19:43:54 +00:00
namespace Fraleign.Chapter1
open Complex
open HPow
2023-05-04 22:37:54 +00:00
/-! ## Exercises 1 Through 9
2023-05-04 22:37:54 +00:00
In Exercises 1 through 9 compute the given arithmetic expression and give the
answer in the form `a + bi` for `a, b ∈ `.
-/
theorem exercise1 : I^3 = 0 + (-1) * I := calc
I^3
= I * (I * hPow I 1) := rfl
2023-04-02 14:57:58 +00:00
_ = 0 + (-1) * I := by simp
2023-05-04 22:37:54 +00:00
2023-05-08 19:43:54 +00:00
end Fraleign.Chapter1