Shawn Zhong

Shawn Zhong

钟万祥
  • Tutorials
  • Mathematics
    • Math 240
    • Math 375
    • Math 431
    • Math 514
    • Math 521
    • Math 541
    • Math 632
    • Abstract Algebra
    • Linear Algebra
    • Category Theory
  • Computer Sciences
    • CS/ECE 252
    • CS/ECE 352
    • Learn Haskell
  • AP Notes
    • AP Microecon
    • AP Macroecon
    • AP Statistics
    • AP Chemistry
    • AP Physics E&M
    • AP Physics Mech
    • CLEP Psycho

Shawn Zhong

钟万祥
  • Tutorials
  • Mathematics
    • Math 240
    • Math 375
    • Math 431
    • Math 514
    • Math 521
    • Math 541
    • Math 632
    • Abstract Algebra
    • Linear Algebra
    • Category Theory
  • Computer Sciences
    • CS/ECE 252
    • CS/ECE 352
    • Learn Haskell
  • AP Notes
    • AP Microecon
    • AP Macroecon
    • AP Statistics
    • AP Chemistry
    • AP Physics E&M
    • AP Physics Mech
    • CLEP Psycho

Home / 2018 / Page 35

Math 541 – 1/29

  • Jan 30, 2018
  • Shawn
  • Math 541
  • No comments yet
Proposition 2: The Division Algorithm • Statement ○ Let a,b∈Z, where b 0 ○ Then ∃!q,r∈Z s.t. a=qb+r, and 0≤r b • Proof (Existence) ○ Let S≔{a−bq│q∈Za−bq≥0}⊆Z(≥0) ○ S is not empty § Let q∈Z s.t. q≤a/b § Then bq≤a § ⇒0≤a−bq § i.e. a−bq∈S ○ Thus S contains a unique minumum elemtent: call it r ○ Choose q∈Z s.t. § a−bq=r § ⇒a=bq+r ○ We still need to show 0≤r b § We know 0≤r, since r∈S, so we just need to show r b § If r≥b, then a−b(q+1)=a−bq−b=r−b≥0 § But a−b(q+1)∈S, and it is less than r § This is impossible, since r is minimum element of S § Thus, r b ○ Therefore we ve proven the existence of q and r • Proof (Uniqueness) ○ Suppose ∃q,q^′,r,r^′∈Z s.t. § a=bq+r, where 0≤r b § a=bq^′+r^′, where 0≤r^′ b ○ We must show q=q′ and r=r^′ ○ Suppose r≠r^′ § Without loss of generality, assume r^′ r § Then 0 r^′−r=(a−bq^′ )−(a−bq)=b(q−q^′ ) § Thus, ├ b┤|├ (r^′−r)┤, but 0 r^′−r≤r^′ b. § This is impossible, thus r=r^′ ○ We have bq+r=bq^′+r⇒q=q^′ ○ Therefore we ve proven the uniqueness of q and r • Note we can prove the following stronger statement ○ If a,b∈Z, and b≠0, then ∃!q,r∈Z ○ s.t. a=bq+r, and 0≤r |b| • Proof (Existence) ○ Assume b 0 ○ Choose q,r∈Z s.t. a=(−b)q+r, and 0≤r −b ○ Then a=b(−q)+r, and 0≤r |b| ○ This proves existence • Proof (Uniqueness) ○ Assume b 0 ○ Suppose ∃q,q^′,r,r^′∈Z s.t. § a=bq+r, where 0≤r b § a=bq^′+r^′, where 0≤r^′ b ○ Then § a=(−b)(−q)+r, where 0≤r |b|=−b § a=(−b)(−q′)+r^′, where 0≤r^′ |b|=−b ○ Since −b 0, our previous result implies −q=−q^′ ○ ⇒q=q′ and r=r^′ Greatest Common Divisor • If a,b∈Z, where either a≠0 or b≠0 • A greatest common divisor of a and b is a positive integer d s.t. ○ d|a and d|b ○ If e∈Z s.t. e|a and e|b then e|d • We write the g.c.d. of a and b, if it exists, as (a,b) • As a convention (0,0)≔0 Proposition 3: Uniqueness of Greatest Common Divisor • Statement ○ Let a,b∈Z, where either a≠0 or b≠0 ○ Suppose ∃d,d^′∈Z( 0) s.t. (1) d and d′ both divide a and b (2) If e∈Z s.t. e|a and e|b, then e|d and e|d^′ ○ Then d=d^′ • Proof ○ Combining properties (1) and (2), we have d|d′ and d^′ |d ○ Choose q,q^′∈Z s.t. dq=d′ and d^′ q^′=d ○ By substitution, we get dqq^′=d ○ Then qq^′=1⇒q=q^′=±1 ○ If q=q^′=−1, then d=−d^′ 0. ○ This is impossible since d and d′ are both positive ○ Therefore q=q^′=1 and d=d^′ Proposition 4 • Statement ○ Suppose a,b∈Z, where b≠0 ○ Choose q,r∈Z s.t. a=qb+r, and 0≤r |b| ○ If (b,r) exists, then (a,b) exists and (a,b)=(b,r) • Proof ○ Set d≔(b,r) ○ d|a and d|b § Choose q_1,q_2∈Z s.t. dq_1=b and dq_2=r § Then a=qb+r=qq_1 d+q_2 d=d(qq_1+q_2 ), so d|a § And we already know d|b ○ If e∈Z s.t. e|a and e|b, then e|d § Let e∈Z s.t. e|a and e|b § Choose q_3,q_4∈Z s.t. eq_3=a and eq_4=b § a=qb+r § ⇒a−qb=r § ⇒eq_3−qeq_4=r § ⇒e(q_3−qq_4 )=r § Thus e|r § Since e|b and d=(b,r) § We can conclude that e|d ○ By Proposition 3, (a,b)=(b,r) Proposition 5 • Statement ○ (a,0)=|a|,∀a∈Z • Proof ○ If a=0 § This is true by our convention ○ If a≠0 § Certainly ├ |a|┤|├ a┤, and ├ |a|┤|├ 0┤ § If e∈Z s.t. e|a and ├ e┤|├ 0┤, then ├ e┤|├ |a|┤ § Therefore (a,0)=|a|
Read More >>

Math 541 – 1/26

  • Jan 30, 2018
  • Shawn
  • Math 541
  • No comments yet
Induction • Prove that ∑_(i=1)^n▒i=n(n+1)/2, ∀n≥1 • Base case, n=1 ○ ∑_(i=1)^i▒i=1=(1×2)/2 • Induction step ○ For n 1 ○ Assume ∀k s.t. 1≤kn, ∑_(i=1)^k▒i=k(k+1)/2 ○ Then∑_(i=1)^n▒i=(∑_(i=1)^(n−1)▒i)+n=(n−1)(n)/2+n=n(n+1)/2 Proposition 1: Well-ordering of Z • Statement ○ Every nonempty set S of Z(≥0) has a unique minimum element ○ That is, ∃!m∈S s.t. m≤s, ∀s∈S • Proof (Existence) ○ Assume S is finite § We will argue by induction on |S| § Base case: |S|=1 □ This is clear § Assume |S| 1 □ Choose x∈S, then |S∖{x}|=|S|−1 □ By induction S∖\{x} has a minimum value: call it m □ Case 1: xm, then x is a minimum value of S □ Case 2: mx, then m is a minimum value of S ○ Now we prove the general case § Choose x∈S § Let S^′≔{s∈S│s≤x} § Then |S^′ |≤x+1∞ § Choose a minimum element of S: call it m § Let s∈S □ If s∈S^′, then m≤s □ If s∉S′, then m≤xs § In either case, m≤s, so m is a minimum element of S ○ This proves existence • Proof (Uniqueness) ○ Suppose m and m′ are both minimum elements of S ○ m≤m′, and m^′≤m ○ Thus, m=m^′ ○ This proves uniqueness Proposition 2: The Division Algorithm • Statement ○ Let a,b∈Z, where b 0 ○ Then ∃!q,r∈Z s.t. a=qb+r, and 0≤rb • Proof (Existence) ○ Let S≔{a−bq│q∈Za−bq≥0}⊆Z(≥0) ○ S is not empty § Let q∈Z s.t. q≤a/b § Then bq≤a § ⇒0≤a−bq § i.e. a−bq∈S ○ Thus S contains a unique minumum elemtent: call it r ○ Choose q∈Z s.t. § a−bq=r § ⇒a=bq+r ○ We still need to show 0≤rb § We know 0≤r, since r∈S, so we just need to show rb § If r≥b, then a−b(q+1)=a−bq−b=r−b≥0 § But a−b(q+1)∈S, and it is less than r § This is impossible, since r is minimum element of S § Thus, rb ○ Therefore we ve proven the existence of q and r
Read More >>

Math 541 – 1/24

  • Jan 30, 2018
  • Shawn
  • Math 541
  • No comments yet
Introduction • Course Plan ○ Frist 2/3 - Groups ("Sets with a multiplication rule") ○ Last 1/3 - Rings ("Set with notions of addition and multiplication") • Office Hours ○ Tuesdays 2:30 p.m. - 4:00 p.m. ○ Wednesdays 12:30 p.m. - 2:00 p.m. Notations • "□(≔) " means "equals, by definition" • Z≔{0,±1,±2,±3,…} the set of integers • Q≔{a/b│a,b∈Zb≠0} • R≔ the set of all real numbers • ℂ≔{a+bi│a,b∈Ri^2=−1} • Z(≥0)≔{a∈Za≥0} • S∖{x}≔{s∈S│s≠x} • Denote a function f from a set A to set B by f:A→B • Denote the image of f by im(f)≔{b∈B│∃a∈A s.t. f(a)=b} Injective, Surjective and Bijective • Definition ○ Let f:A→B be a function, then ○ f is injective if ∀a,a^′∈A, a≠a^′, f(a)≠f(a′) ○ f is surjective if ∀b∈B, ∃a∈A s.t. f(a)=b (i.e. im(f)=B) ○ f is bijective if f is both injective and surjective. • Example 1 ○ For f:Z→Z, f(a)=2a ○ f is injective § Let a,a^′∈Z § Suppose f(a)=f(a′) § ⇒2a=2a^′ § ⇒2a−2a^′=0 § ⇒2(a−a^′ )=0 § ⇒a−a^′=0 § ⇒a=a^′ § Therefore f is injective ○ f is not surjective § Because the image of f does not contain any odd integers § im(f)={even integer} • Example 2 ○ Let f:Q→Q is given by f(a)=2a ○ f is injective § By the same proof as before ○ f is surjective § Let b∈Q, then b/2∈Q § And f(b/2)=2(b/2)=b∈Q § Therefore f is surjective ○ f is bijective § Since f is both injective and surjective. Divides • Definition ○ If x,y∈Z, and x≠0 ○ We say x divides y and write x|y, if ∃q∈Z s.t. xq=y • Examples ○ ∀x∈Z\\{0}, x|0, since x⋅0=0 ○ ∀x∈Z, 1|x, since 1⋅x=x ○ ∀x∈Z, −1|x, since (−1)⋅(−x)=x Equivalence Relations • Product of Two Sets ○ If A and B are sets, then the product of A and B is ○ A×B≔{(a,b)│a∈A, b∈B} • Relations ○ A relation on a set A is a subset R of A×A ○ We write a~a′ if (a,a^′ )∈R • Equivalence Relations ○ A equivalence relation is a relation R on A such that R is ○ Reflexive § if a∈A, a~a § i.e. (a,a)∈R ○ Symmetric § if a~a′, then a^′~a § i.e. (a,a′)∈R⇒(a′,a)∈R ○ Transitive § if a~a^′, a^′~a^′′, then a~a′′ § i.e. if (a,a′)∈R and (a^′,a^′′ )∈R, then (a,a^′′ )∈R • Example 1 ○ Let R be a relation on set A such that R≔{(a,a)│a∈A} ○ Then R is an equivalence relation (a~a^′⟺a=a^′) ○ Reflexive § If a∈A,(a,a)∈R ○ Symmetric § If a~a′,a=a^′ § Thus a^′=a, hence a^′~a ○ Transitive § If a~a^′,a^′~a′′ then a=a′ and a=a′′ § Thus a=a^′′, hence a~a^′′ • Example 2 ○ Let n be a positive integer ○ Then R≔{(a,b)∈ZZn|(a−b) } is an equivalence relation ○ Reflexive § Recall that n|0 § Thus, n|(a−a), ∀a∈Z § It follows that a~a,∀a∈Z ○ Symmetric § Let a,b∈Z, and suppose n|(a−b) (i.e. a~b) § Choose q∈Z s.t. nq=a−b § Then n(−q)=−(a−b)=b−a § Thus, n|(b−a), and so b~a ○ Transitive § Suppose a,b,c∈Z, and we have a~b, b~c § Then n|(a−b) and n|(b−c) § Choose q,q^′∈Z s.t. nq=a−b, nq^′=b−c § Then n(q+q^′ )=(a−b)+(b−c)=a−c § Thus, n|(a−c), and so a~c
Read More >>

Math 521 – 1/29

  • Jan 30, 2018
  • Shawn
  • Math 521
  • No comments yet
Proposition 1.14 • Given a field F, for x,y,z∈F (1) If x+y=x+z, then y=z (2) If x+y=x, then y=0 (3) If x+y=0, then y=−x (4) −(−x)=x • Proof (1) ○ x+y=x+z ○ (x+y)+(−x)=(x+z)+(−x) by (A5) ○ x+y+(−x)=x+z+(−x) by (A3) ○ x+(−x)+y=x+(−x)+z by (A2) ○ 0+y=0+z by (A6) ○ y=z∎ by (A4) • Proof (2) ○ x+y=x=x+0 ○ ⇒y=0∎ • Proof (3) ○ x+y=0=x+(−x) ○ ⇒y=−x∎ • Proof (4) ○ (−x)+(−(−x))=0 ○ x+(−x)+(−(−x))=x+0 ○ 0+(−(−x))=x+0 ○ −(−x)=x∎ Proposition 1.15 • Given a field F, for x,y,z∈F (1) If x≠0 and xy=xz, then y=z (2) If x≠0 and xy=x, then y=1 (3) If x≠0 and xy=1, then y=1/x (4) If x≠0, then 1/(1/x)=x • Proof similar to Proposition 1.14 Proposition 1.16 • Given a field F, for x,y∈F (1) 0x=0 (2) If x≠0 and y≠0, then xy≠0 (3) (−x)y=−(xy)=x(−y) (4) (−x)(−y)=xy • Proof (1) ○ 0+0=0 ○ (0+0)x=0x ○ 0x+0x=0x ○ 0x+0x+(−(0x))=0x+(−(0x)) ○ 0x=0∎ • Proof (2) ○ Suppose x≠0, y≠0, but xy=0 ○ x≠0, so 1/x exists ○ 1/x (xy)=1/x⋅0 ○ (1/x⋅x)y=1/x⋅0 ○ 1⋅y=0 ○ y=0 ○ This is a contradiction, so xy≠0∎ • Proof (3) ○ (−x)y+xy=((−x)+x)y=0⋅y=0 ○ (−x)y+xy+(−xy)=0+(−xy) ○ (−x)y=−xy ○ And the rest is similar • Proof (4) ○ Use (3), (−x)(−y)=−(x(−y))=−(−xy)=xy∎ Order • Intuition ○ The real number line • Definition ○ Let S be a set. ○ An order on S is a relation, denoted by ,with the following two properties: § If x∈S and y∈S, then one and only one of the statements xy, x=y, yx is true § If x,y,z∈S, if xy and yz, then xz (Transitivity) ○ x≤y means either xy or x=y ○ x≥y means either xy or x=y ○ An ordered set is a set for which an order is defined. • Example ○ Q is an ordered set under the definition that ○ For r,s∈Q, rs, if and only if s−r is positive Upper Bound and Lower Bound • Definition ○ Suppose S is an ordered set and E⊂S. ○ If there exists β∈S such that x≤β, ∀x∈E ○ We say that x is bounded above and call β an upper bound for E ○ Similarly, if x≥β, ∀x∈E. ○ We say that x is bonded below by β, and β is a lower bound for E
Read More >>

Math 521 – 1/26

  • Jan 30, 2018
  • Shawn
  • Math 521
  • No comments yet
Sets • Contains ○ If A is a set and x is an element of A (an object of A), then we write x∈A ○ Otherwise, we write x∉A • Set ○ The empty set or null set is a set with no elements, and is denoted as ∅ ○ If a set has at least one element, it is called nonempty • Subset ○ If A and B are sets and every element of A is an element of B ○ Then A is a subset of B ○ Rubin write this A⊂B, or B⊃A ○ A⊂A for all sets A • Proper subset ○ If B contain something not in A, then A is a proper subset of B • Equal ○ If A⊂B and B⊂A then A=B. ○ Otherwise A≠B √2 is Not Rational • We proved that √2 is not rational • i.e. there is no rational number p such that p^2=2 • Let A={p∈Qp^2<2}, B={p∈Qp^2>2} • Prove: A has no largest element, and B has no smallest element ○ Let p∈Q, and p>0 ○ Let q≔p−(p^2−2)/(p+2)=(2p+2)/(p+2),then q^2−2=((2p+2)/(p+2))^2−2=2(p^2−2)/(p+2)^2 ○ If p∈A § then p^2−2<0 § ⇒q^2−2=2(p^2−2)/(p+2)^2 <0 § ⇒q^2<2 § ⇒q∈A § ⇒q>p § i.e. A has no largest element ○ If p∈B § then p^2−2>0 § ⇒q^2−2=2(p^2−2)/(p+2)^2 >0 § ⇒q^2>2 § ⇒q∈B § ⇒q</p> <p § i.e. B has no smallest element What is R? • The real numbers are an example of field. • A field is a set F with two binary operations called addition and multiplication that satisfy that following axioms: • Axioms for addition (+) ○ (A1) If x∈F and y∈F, then x+y∈F ○ (A2) Addition is communicate: x+y=y+x,∀x,y∈F ○ (A3) Addition is associative: (x+y)+z=x+(y+z),∀x,y,z∈F ○ (A4) There exists 0∈F s.t. x+0=x, ∀x∈F ○ (A5) ∀x∈F, there exists an additive inverse −x∈F s.t. x+(−x)=0 • Axioms for multiplication (× or ⋅) ○ (M1) If x∈F and y∈F, then xy∈F ○ (M2) Addition is communicate: xy=yx,∀x,y∈F ○ (M3) Addition is associative: (xy)z=x(yz),∀x,y,z∈F ○ (M4) F contains an element 1≠0 s.t. 1⋅x=x, ∀x∈F ○ (M5) If x∈F and x≠0, then there exists 1/x∈F s.t. x⋅1/x=1 • (D) The distributive law: x(y+z)=xy+xz, ∀x,y,z∈F
Read More >>
  • 1
  • …
  • 33
  • 34
  • 35
  • 36
  • 37
  • …
  • 41

Search

  • Home Page
  • Tutorials
  • Mathematics
    • Math 240 – Discrete Math
    • Math 375 – Linear Algebra
    • Math 431 – Intro to Probability
    • Math 514 – Numerical Analysis
    • Math 521 – Analysis I
    • Math 541 – Abstract Algebra
    • Math 632 – Stochastic Processes
    • Abstract Algebra @ 万门大学
    • Linear Algebra @ 万门大学
    • Category Theory
  • Computer Sciences
    • CS/ECE 252 – Intro to Computer Engr.
    • CS/ECE 352 – Digital System Fund.
    • Learn Haskell
  • Course Notes
    • AP Macroeconomics
    • AP Microeconomics
    • AP Chemistry
    • AP Statistics
    • AP Physics C: E&M
    • AP Physics C: Mechanics
    • CLEP Psychology
  • 2048 Game
  • HiMCM 2016
  • 登峰杯 MCM

WeChat Account

Categories

  • Notes (418)
    • AP (115)
      • AP Macroeconomics (20)
      • AP Microeconomics (23)
      • AP Physics C E&M (25)
      • AP Physics C Mechanics (28)
      • AP Statistics (19)
    • Computer Sciences (2)
    • Mathematics (300)
      • Abstract Algebra (29)
      • Category Theory (7)
      • Linear Algebra (29)
      • Math 240 (42)
      • Math 375 (71)
      • Math 514 (18)
      • Math 521 (39)
      • Math 541 (39)
      • Math 632 (26)
  • Projects (2)
  • Tutorials (11)

Archives

  • October 2019
  • May 2019
  • April 2019
  • March 2019
  • February 2019
  • December 2018
  • November 2018
  • October 2018
  • September 2018
  • July 2018
  • May 2018
  • April 2018
  • March 2018
  • February 2018
  • January 2018
  • December 2017
  • November 2017
  • October 2017
  • September 2017
  • August 2017
  • July 2017
  • June 2017

WeChat Account

Links

RobeZH's thoughts on Algorithms - Ziyi Zhang
Copyright © 2018.      
TOP