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 / February / Page 3

Math 541 – 2/16

  • Feb 21, 2018
  • Shawn
  • Math 541
  • No comments yet
Proposition 16 • Let f:G→H be an isomorphism • G is abelian if and only if H is abelian ○ (⟹) Suppose G is abelian ○ Let h,h′∈H ○ Choose g,g^′∈G s.t. f(g)=h,f(g′)=h′ ○ Then hh′=f(g)f(g^′ )=f(gg^′ )=f(g^′ g)=f(g^′ )f(g)=h′ h ○ (⟸) Apply the same argument with f^(−1):H→G • ∀g∈G, |g|=|f(g)| ○ Proof: f(1_G )=1_H § Let g∈G, then § f(g)=f(1_G⋅g)=f(1_G )⋅f(g) § By Cancellation Law, f(1_G )=1_H ○ Proof: When |g| ∞ § Let n≔|g|, then § 1_H=f(1_G )=f(g^n )=f(g)^n § (This last equality follows from an induction argument) § Therefore, |f(g)|≤n § Now, apply this same argument with f replaced by f^(−1) § So we can conclude that |f(g)|=n ○ Proof: When |g|=∞ § If |f(g)| ∞ § The above argument shows |g| ∞ § This is impossible § Thus, |f(g)|=∞ ○ Note § This result also holds if we only assume f is injective Order and Homomorphism • G,H are groups, and |G|=|H|, is it the case that G≅H? No • Counterexample 1 ○ Z and Q ○ |Z=|Q, but Z≇Q • Fact: Any homomorphism f:Z→Q is not surjective ○ Let f:Z→Q be a homomorphism ○ If f(a)=0,∀a∈Z § Obviously f is not surjective ○ Assume otherwise § By induction, f(a)=f ⏟((1+1+…+1) )┬(n copies)=a⋅f(1) § By assumption, f(1)≠0; otherwise f=0 § We know that f(1)/2∈Q § But ∄a∈Z s.t. f(1)/2=af(1) § i.e. f(1)/2∉im(f) § Thus f is not surjective • Counterexample 2 ○ Z\/6Z and S_3 ○ |Z6Z=|S_3 |, but Z\/6Z≇S_3 ○ Because Z\/6Z is abelian, but S_3 is not ○ Also |1 ̅ |=6 in Z\/6Z, but S_3 have no element of order 6 Orders of elements in S_n • Let σ∈S_n • If σ=σ_1⋯σ_m, where σ_1⋯σ_m are disjoint cycles • Then |σ|=lcm(|σ_1 |,…,|σ_m |) • Also, if τ is a t-cycle, then |τ|=t Subgroup • Definition ○ Let G be a group, and let H⊆G ○ H is a subgroup if § H≠∅ (nonempty) § If h,h′∈H, then hh′∈H (closure under the operation) § If h∈H, then h(−1)∈H (closure under inverse) ○ We will write H≤G • Note ○ Subgroups of a group are also groups • Example 1 ○ If G is a group, then G≤G and {1}≤G • Example 2 ○ If m,n∈Z( 0), and n≥m, then S_m≤S_n • Example 3 ○ Let G be a group, and let g∈G ○ Then ⟨g⟩≔{g^n│n∈Z≤G ○ ⟨g⟩ is called the cyclic subsgroup generated by g ○ ⟨g⟩≠∅, since g∈⟨g⟩ ○ Let g^i,g^j∈⟨g⟩, then g^i g^j=g^ij∈⟨g⟩ ○ If g^i∈⟨g⟩, then (g^i )^(−1)=g^(−i)∈⟨g⟩ Regular n\-gon • A regular n\-gon is a polygon with all sides and angles equal
Read More >>

2.6 Matrices

  • Feb 21, 2018
  • Shawn
  • Math 240
  • No comments yet
Matrices • Matrices are useful discrete structures that can be used in many ways. • For example, they are used to: ○ describe certain types of functions known as linear transformations. ○ Express which vertices of a graph are connected by edges (see Chapter 10). • Here we cover the aspect of matrix arithmetic that will be needed later. • Definition ○ A matrix is a rectangular array of numbers. ○ A matrix with m rows and n columns is called an m×n matrix. ○ The plural of matrix is matrices. ○ A matrix with the same number of rows as columns is called square. ○ Two matrices are equal if they have the same number of rows and the same number of columns and the corresponding entries in every position are equal. • Example: 3×2 matrix ○ [■8(1&1@0&2@1&3)] • Notation ○ Let m and n be positive integers and let § A=[■8(a_11&a_12&…&a_1n@a_21&a_22&…&a_2n@⋮&⋮&⋱&⋮@a_m1&a_m2&…&a_mn )] ○ The ith row of A is the 1×n matrix § [a_i1, a_i2,…,a_in]. ○ The jth column of A is the m×1 matrix: § [█(a_1j@a_2j@⋮@a_mj )] ○ The (i,j)th element or entry of A is the element a_ij ○ We can use A = [a_ij] to denote the matrix with its (i,j)th element equal to a_ij Matrix Arithmetic: Addition • Let A = [a_ij] and B = [b_ij] be m×n matrices. • The sum of A and B, denoted by A + B, is the m×n matrix that has a_ij + b_ij as its (i,j)th element. • In other words, A + B = [a_ij + bij]. • Example ○ [■8(1&0&−1@2&2&−3@3&4&0)]+[■8(3&4&−1@1&−3&0@−1&1&2)]=[■8(4&4&−2@3&−1&−3@2&5&2)] • Note that matrices of different sizes cannot be added. Matrix Multiplication • Let A be an m×k matrix and B be a k×n matrix. • The product of A and B, denoted by AB, is the m×n matrix that has its (i,j)th element equal to the sum of the products of the corresponding elements from the ith row of A and the jth column of B. • In other words, if AB = [c_ij] then c_ij=a_i1 b_1j+a_i2 b_2j+⋯+a_kj b_kj. • Example ○ [■8(1&0&4@2&1&1@3&1&0@0&2&2)][■8(2&4@1&1@3&0)]=[■8(14&4@8&9@7&13@8&2)] Matrix Multiplication is not Commutative • Let A=[■8(1&1@2&1)],B=[■8(2&1@1&1)], then • AB=[■8(3&2@5&3)],BA=[■8(4&3@3&2)] • Thus AB≠BA Identity Matrix and Powers of Matrices • The identity matrix of order n is the m×n matrix I_n=[δ_ij ], where ○ δ_ij = 1 if i = j ○ δ_ij = 0 if i≠j • I_n=[■(1&&@&⋱&@&&1)] • AI_n=I_m A=A when A is an m×n matrix • Powers of square matrices can be defined. When A is an n×n matrix, we have: ○ A^0=I_n ○ A^r=⏟(AA⋯A)┬(r times) Transposes of Matrices • Let A = [a_ij] be an m×n matrix. • The transpose of A, denoted by A^t ,is • the n×n matrix obtained by interchanging the rows and columns of A. • If A^t = [b_ij], then b_ij=a_ji for i =1,2,…,n and j = 1,2, …,m • The transpose of the matrix [■8(1&2&3@4&5&6)] is the matrix [■8(1&4@2&5@3&6)] Symmetric Matrices • A square matrix A is called symmetric if A=A^t. • Thus A = [a_ij] is symmetric if a_ij=a_ji for i and j with 1≤i≤n and 1≤j≤n. • The matrix [■8(1&1&0@1&0&0@0&1&0)] is square • Symmetric matrices do not change when their rows and columns are interchanged Zero-One Matrices • A matrix all of whose entries are either 0 or 1 is called a zero-one matrix. • Algorithms operating on discrete structures represented by zero-one matrices are based on Boolean arithmetic defined by the following Boolean operations: ○ b_1∧b_2={■8(1&if b_1=b_2=1@0&otherwise)┤ ○ b_1∨b_2={■8(1&if b_1=1 or b_2=1@0&otherwise)┤ Joint and Meet of Zero-One Matrices • Definition: Let A = [a_ij] and B = [b_ij] be an m×n zero-one matrices. • The join of A and B is the zero-one matrix with (i,j)th entry a_ij∨b_ij. • The join of A and B is denoted by A ∨ B. • The meet of of A and B is the zero-one matrix with (i,j)th entry a_ij∧b_ij. • The meet of A and B is denoted by A ∧ B. • Example ○ Find the join and meet of the zero-one matrices § A=[■8(1&0&1@0&1&0)] § B=[■8(0&1&0@1&1&0)] ○ The joint of A and B is § A∨B=[■8(1&1&1@1&1&0)] ○ The meet of A and B is § A∧B=[■8(0&0&0@0&1&0)] Boolean Product of Zero-One Matrices • Definition: ○ Let A = [a_ij] be an m×k zero-one matrix and B = [b_ij] be a k×n zero-one matrix. ○ The Boolean product of A and B, denoted by A⨀B, is the m×n zero-one matrix with (i,j)th entry c_ij=(a_i1∧b_1j )∨(a_i2∧b_2j )∨⋯∨(a_ik∧b_kj ). • Example: Find the Boolean product of A and B, where ○ A=[■8(1&0@0&1@1&0)],B=[■8(1&1&0@0&1&1)] ○ A⨀B=[■8(1&1&0@0&1&1@1&1&0)] Boolean Powers of Zero-One Matrices • Let A be a square zero-one matrix and let r be a positive integer. • The rth Boolean power of A is the Boolean product of r factors of A, denoted by A^[r] . • Hence, A^[r] =⏟(A⨀A⨀⋯⨀A)┬(r times) • We define A^[0] =I_n • The Boolean product is well defined because the Boolean product of matrices is associative • Example ○ Let A=[■8(0&0&1@1&0&0@1&1&0)] ○ Find A^[n] for all positive integers n ○ A^[2] =[■8(1&1&0@0&0&1@1&0&1)] ○ A^[3] =[■8(1&0&1@1&1&0@1&1&1)] ○ A^[4] =[■8(1&1&1@1&0&1@1&1&1)] ○ A^[5] =[■8(1&1&1@1&1&1@1&1&1)]
Read More >>

2.5 Cardinality of Sets

  • Feb 21, 2018
  • Shawn
  • Math 240
  • No comments yet
Cardinality • The cardinality of a set A is equal to the cardinality of a set B, denoted |A|=|B|, • if and only if there is a one-to-one correspondence (i.e., a bijection) from A to B • If there is a one-to-one function (i.e., an injection) from A to B, then • the cardinality of A is less than or equal to the cardinality of B and we write |A|≤|B| • When |A|≤|B| and A and B have different cardinality, • we say that the cardinality of A is less than the cardinality of B and write |A||B| Countable and Uncountable • A set that is either finite or has the same cardinality as Z+ is called countable. • A set that is not countable is uncountable. • The set of real numbers R is an uncountable set. • When an infinite set is countable (countably infinite) its cardinality is ℵ_0 • (where ℵ is aleph, the 1st letter of the Hebrew alphabet). • We write |S|=ℵ_0 and say that S has cardinality “aleph null.” Showing that a Set is Countable • An infinite set is countable iff it is possible to list the elements of the set in a sequence. • A 1-1 correspondence f from the set of positive integers to a set S can be expressed • in terms of a sequence a_1,a_2,…,a_n where a_1=f(1), a_2=f(2),…,a_n=f(n) • Example 1: The set of positive even integers E is countable set. ○ Let f(x)=2x ○ ■8(1&2&3&4&…@↕&↕&↕&↕&↕@2&4&6&8&…) ○ Then f is a bijection from N to E since f is both one-to-one and onto. ○ To show that it is one-to-one, suppose that f(n)=f(m). ○ Then 2n=2m, and so n=m. ○ To see that it is onto, suppose that t is an even positive integer. ○ Then t=2k for some positive integer k and f(k)=t. • Example 2: The set of integers Z is countable. ○ Can list in a sequence: 0, 1, − 1, 2, − 2, 3, − 3,… ○ Or can define a bijection from N to Z: § f(2n)=−n § f(2n+1)=n+1 • Example 3: The positive rational numbers are countable. § A rational number can be expressed as p/1 where p,q∈Z and q≠0. ○ Note: § p and q such that q≠0. ○ The positive rational numbers are countable since they can be arranged in a sequence • Example 4: Union of countable sets is countable ○ A={a_1,a_2,…,a_n,…} ○ B={b_1,b_2,…,b_n,…} ○ A∪B={a_1,b_1,a_2,b_2,…,a_n,b_n,…} • Example 5: The set of all rationals is countable ○ Q={0}∪Q+∪Q− ○ f(−p/q)=p/q is a bijiection from Q− to Q+ • Example 6: The set of finite string S over a finite alphabet A is counitable infinite ○ A={a,b} ○ List all strings with length § 0: λ § 1: a, b § 2: aa,ab,ba,bb § 3: aaa,aab,aba,abb,baa,bab,bba,bbb § ⋯ • Example 7: Show that the set of all Java program is countable ○ Just list all the strings Hilbert’s Grand Hotel • The Grand Hotel has countably infinite number of rooms, each occupied by a guest. • We can always accommodate a new guest at this hotel. • How is this possible? • Because the rooms of Grand Hotel are countable • We can list them as Room 1, Room 2, Room 3, and so on. • When a new guest arrives, we move the guest in Room n to Room n+1 • This frees up Room 1, which we assign to the new guest, and all the current guests still have rooms. • The hotel can also accommodate a countable number of new guests, all the guests on a countable number of buses where each bus contains a countable number of guests The Real Numbers are Uncountable • The method is called the Cantor diagnalization argument • Suppose R is countable. Then the real numbers between 0 and 1 are also countable • The real numbers between 0 and 1 can be listed in order r1 , r2 , r3 ,… . • Let the decimal representation of this listing be ○ r_1=0.d_11 d_12 d_13… ○ r_2=0.d_21 d_22 d_23… ○ r_3=0.d_31 d_32 d_33… • Form a new real number with the decimal expansion r=0.s_1 s_2 s_3… where ○ s_n={■8(4&d_nn=4@3&d_nn≠3)┤ • r is not equal to any of the r_1,r_2,r_3,… • Because it differs from r_i in its i-th position after the decimal point. • Therefore there is a real number between 0 and 1 that is not on the list • since every real number has a unique decimal expansion. • Hence, all the real numbers between 0 and 1 cannot be listed • so the set of real numbers between 0 and 1 is uncountable. • Since a set with an uncountable subset is uncountable • the set of real numbers is uncountable. Computability • We say that a function is computable if there is a computer program in some programming language that finds the values of this function. • If a function is not computable we say it is uncomputable. • There are uncomputable functions. • We have shown that the set of Java programs is countable. • We can show that the set of functions f:N→N is uncountable • Therefore there must be uncomputable functions
Read More >>

Math 521 – 2/19

  • Feb 19, 2018
  • Shawn
  • Math 521
  • No comments yet
Metric Space • Definition ○ A set X of points is called a metric space if ○ there exists a metric or distance function d(p,q):X×X→R such that § Positivity □ d(p,q)0 if p,q∈X and p≠q □ d(p,p)=0 for all p∈X § Symmetry □ d(p,q)=d(q,p) for all p,q∈X § Triangle Inequality □ d(p,q)≤d(p,r)+d(r,q) for all p,q,r∈X • Example 1 ○ X=Rk ○ d(p ⃗,q ⃗ )=|p ⃗−q ⃗ | ○ If k=1, this is just standard numerical absolute value ○ and d is distance on the number line • Example 2 (Taxicab metric) ○ X=R2 ○ d((p_1,p_2 ),(q_1,q_2 ))=|p_1−q_1 |+|p_2−q_2 | where p_1,p_2,q_1,q_2∈R ○ Is this a true metric space? ○ Positivity § Clearly d((p_1,p_2 ),(q_1,q_2 ))≥0 since it is a sum of absolute values § Suppose d((p_1,p_2 ),(q_1,q_2 ))=0 □ |p_1−q_1 |+|p_2−q_2 |=0 □ |p_1−q_1 |=−|p_2−q_2 | □ {█(|p_1−q_1 |=0@|p_2−q_2 |=0)┤⇒{█(p_1=q_1@p_2=q_2 )┤ □ i.e. (p_1,p_2 )=(q_1,q_2 ) § Suppose (p_1,p_2 )=(q_1,q_2 ) □ d((p_1,p_2 ),(q_1,q_2 ))=|p_1−q_1 |+|p_2−q_2 |=|0|+|0|=0 § Thus d((p_1,p_2 ),(q_1,q_2 ))=0 iff (p_1,p_2 )=(q_1,q_2 ) ○ Symmetry § d((p_1,p_2 ),(q_1,q_2 ))=|p_1−q_1 |+|p_2−q_2 | § =|q_1−p_1 |+|q_2−p_2 |=d((q_1,q_2 ),(p_1,p_2 )) ○ Triangular Inequality § d((p_1,p_2 ),(r_1,r_2 ))+d((r_1,r_2 ),(q_1,q_2 )) § =|p_1−r_1 |+|p_2−r_2 |+|r_1−q_1 |+|r_2−q_2 | § =(|p_1−r_1 |+|r_1−q_1 |)+(|p_2−r_2 |+|r_2−q_2 |) § ≥|p_1−r_2+r_1−q_1 |+|p_2−r_2+r_2−q_2 | by Triangle Inequality of R § =|p_1−q_1 |+|p_2−q_2 | § =d((p_1,p_2 ),(q_1,q_2 )) Definition 2.17 • Interval ○ Segment (a,b) is {x∈Raxb} (open interval) ○ Interval [a,b] is {x∈Ra≤x≤b} (closed interval) ○ We can also have half-open intervals: (a,b] and [a,b) • k-cell ○ If a_ib_i for i=1,2,…,k ○ The set of points x ⃗=(x_1,x_2,…,x_k ) in Rk ○ that satisfy a_i≤x_i≤b_i (1≤i≤k) is called a k-cell • Ball ○ If x ⃗∈Rk and r0 ○ the open ball with center x ⃗ with radius r is {y ⃗∈Rk│|x ⃗−y ⃗ |r} ○ the closed ball with center x ⃗ with radius r is {y ⃗∈Rk│|x ⃗−y ⃗ |≤r} • Convex ○ We call a set E⊂Rk convex if ○ λx ⃗+(1−λ) y ⃗∈E, ∀x ⃗,y ⃗∈E, 0λ1 ○ i.e. All points along a straight line from x ⃗ to y ⃗ and between x ⃗ and y ⃗ is in E • Example: Balls are convex ○ Given an open ball with center x ⃗ and radius r ○ If y ⃗,z ⃗∈B, then |y ⃗−x ⃗ |r and |z ⃗−x ⃗ |r ○ |λz ⃗+(1−λ) y ⃗−x ⃗ | ○ =|λz ⃗+(1−λ) y ⃗−(λ+1−λ) x ⃗ | ○ =|λz ⃗−λx ⃗+(1−λ) y ⃗−(1−λ) x ⃗ | ○ ≤|λz ⃗−λx ⃗ |+|(1−λ) y ⃗−(1−λ) x ⃗ | by Triangle Inequality ○ =λ|z ⃗−x ⃗ |+(1−λ)|y ⃗−x ⃗ | ○ λr+(1−λ)r=r ○ Thus |λz ⃗+(1−λ) y ⃗−x ⃗ |r ○ i.e. λz ⃗+(1−λ) y ⃗∈B Definition 2.18 (a) Neighborhood (b) Limit point (c) Isolated point (d) Closed (e) Interior point (f) Open (g) Complement (h) Perfect (i) Bounded (j) Dense
Read More >>

Math 521 – 2/16

  • Feb 19, 2018
  • Shawn
  • Math 521
  • No comments yet
Set-Theoretic Operations • Set theoretic union ○ ⋃24_(n=1)^∞▒A_n =A_1∪A_2∪A_3∪⋯ • Set theoretic intersection ○ ⋂24_(n=1)^∞▒A_n =A_1∩A_2∩A_3∩⋯ • Indexing set ○ ⋃8_(α∈A)▒E_α , where ○ A is an indexing set ○ E_α is a specific set that depends on A • Example ○ Let A={x∈R0x≤1} ○ Let E_α={x∈R0xa} ○ Then⋃8_(α∈A)▒E_α =(0,1) and ⋂8_(α∈A)▒E_α =∅ Theorem 2.12 • Statement ○ Let {E_n }_(n∈N be a sequence of countable sets, then ○ S=⋃24_(n=1)^∞▒E_n is also countable • Proof ○ Just like the proof that Q is countable ○ E_n={〖x_n〗_k }={〖x_n〗_1,〖x_n〗_2,〖x_n〗_3,…} ○ ■(x_11&x_12&x_13&x_14&…&@x_21&x_22&x_23&⋱&&@x_31&x_32&⋱&&&@x_41&⋱&&&&@⋮&&&&&) ○ Go along the diagonal, we have ○ S={x_11,x_21,x_12,x_31,x_22,x_13…} • Corollary ○ Suppose A is at most countable ○ If for α∈A, B_α is at most countable, then ○ T=⋃8_(α∈A)▒B_α is also at most countable Theorem 2.13 • Statement ○ Let A be a countable set ○ Let B_n be the set of all n-tuples (a_1,a_2,…a_n ) where a_k∈A for 1≤k≤n ○ And a_k may not be distinct, then B_n is countable • Proof ○ We proof by induction on n ○ Base case: n=2 § ■((a_1,a_1 )&(a_1,a_2 )&(a_1,a_3 )&(a_1,a_4 )&…&@(a_2,a_1 )&(a_2,a_2 )&(a_2,a_3 )&⋱&&@(a_3,a_1 )&(a_3,a_2 )&⋱&&&@(a_4,a_1 )&⋱&&&&@⋮&&&&&) § Here a_i are all the elements of A with possible repetition ○ Now assume for n=m (m≥2) § The set of m-tuples (a_1,a_2,…a_m ) are countable § Now we treat the (m+1)\-tuples as ordered pairs § (a_1,a_2,…a_(m+1) )=((a_1,a_2,…a_m ),a_(m+1) ) § By n=2 case, the set of (m+1)\-tuples is still countable Theorem 2.14 • Statement ○ Let A be the set of all sequqnecse whose digits are 0 and 1 ○ Then A is uncountable • Proof: Cantor
Read More >>
  • 1
  • 2
  • 3
  • 4
  • 5
  • …
  • 7

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