Lecture 2: Spectra of Graphs

Size: px
Start display at page:

Download "Lecture 2: Spectra of Graphs"

Transcription

1 Spectral Graph Theory ad Applicatios WS 20/202 Lecture 2: Spectra of Graphs Lecturer: Thomas Sauerwald & He Su Our goal is to use the properties of the adjacecy/laplacia matrix of graphs to first uderstad the structure of the graph ad, based o these isights, to desig efficiet algorithms. The study of algebraic properties of graphs is called algebraic graph theory. Oe of the most useful algebraic properties of graphs are the eigevalues (ad eigevectors) of the adjacecy/laplacia matrix. Defiitios Defiitio 2.. Let G = (V, E) be a udirected graph with vertex set [] := {,..., }. The adjacecy matrix of G is a by matrix A give by { if i ad j are adjacet A i,j = 0 otherwise If G is a multi-graph, the A i,j is the umber of edges betwee vertex i ad vertex j. The sum of elemets i every row/colum equals the degree of the correspodig vertex. If G is udirected, the A is symmetric. Example. The adjacecy matrix of a triagle is Defiitio 2.2. We defie the Laplacia matrix L of graph G as follows: deg(i) if i = j L i,j = if i ad j are adjacet 0 otherwise where deg(i) is the degree of vertex i. Let D be a by diagoal matrix with deg(),..., deg() as diagoal elemets. We ca rewrite L as L = D A. I particular, if G is d-regular, the L = d I A. Give a matrix A, a vector x 0 is defied to be a eigevector of A if ad oly if there is a λ C such that Ax = λx. I this case, λ is called a eigevalue of A.

2 Defiitio 2.3 (graph spectrum). Let A be the adjacecy matrix of a udirected graph G with vertices. The A has real eigevalues, deoted by λ λ. These eigevalues associated with their multiplicities compose the spectrum of G. Here are some basic facts about the graph spectrum. Lemma 2.4. Let G be ay udirected simple graph with vertices. The. i= λ i = i= λ2 i = i= deg(i). 3. If λ = = λ, the E[G] =. 4. deg avg λ deg max. 5. deg max λ deg max. Proof. We oly prove the first three items. () Sice G does ot have self-loops, all the diagoal elemets of A are zero. By the defiitio of trace, we have ı= λ i = tr(a) = i= A i,i = 0. (2) By the properties of matrix trace, we have ı= λ2 i = tr ( A 2) = i= A2 i,i. Sice A2 i,i is the degree of vertex i, tr(a 2 ) equals the sum of every vertex s degree i G. (3) Combig i= λ i = 0 with λ = = λ, we have λ i = 0 for every vertex i. By item (2), we have deg(i) = 0 for ay vertex i. Therefore E[G] =. For a graph G with adjacecy matrix A ad iteger k, A k u,v is the umber of walks of legth k from u to v. Let x p := ( i= x i p ) /p. The for ay p q <, it holds that x q x p /p /q x q. Lemma 2.5. For ay graph G with m edges, the umber of cycles of legth k i G is bouded by O ( m k/2). Proof. Let A be the adjacecy matrix of G with eigevalues λ,..., λ. Thus the umber of C k (cycles of legth k) i G is bouded by tr ( A k) /(2k) = ( ) i= λk i /(2k). For ay k 3, it holds that ( ) /k ( ) /k ( ) /2 λ k i λ i k λ i 2 = (2 m) /2. i= i= Hece tr ( A k) (2m) k/2 ad the umber of C k is at most O ( m k/2). Example. Some examples for differet spectra of graphs: For the complete graph K, the eigevalues are with multiplicity ad with multiplicity. For the complete bipartite graph K m,, the eigevalues are + m, m ad 0 with multiplicity m + 2. For the cycle C, the spectrum is 2 cos(2πj/) (j = 0,,..., ). Two assumptios that we make throughout the course are as follows: i= 2

3 . We oly cosider udirected graphs. Note that if G is ot udirected, the A ad L is ot symmetric ay more ad the eigevalues of A ad L could be complex umbers. A matrix A = (a i,j ) is called a Hermitia matrix if a i,j = a j,i for ay elemet a i,j. Hermitia matrices always have real eigevalues. 2. Uless metioed otherwise, we cosider regular graphs. Lemma 2.6. Cosider ay udirected graph G with adjacecy matrix A.. If G is d-regular, the λ = d ad λ i d for i = 2,...,. 2. G is coected iff λ 2 < d, i.e., the eigevalue d has multiplicity. Moreover, the umber of coected compoets of G equals the multiplicity of eigevalue d. 3. If G is coected, the G is bipartite iff λ = d. Lemma 2.7. All eigevalues of L are o-egative. Proof. Follows from Lemma 2.6 ad the defiitio of L = D A. For studyig regular graphs, it is coveiet to work with the ormalized adjacecy matrix M of graph G. For ay d-regular graph with adjacecy matrix A, defie M := d A. Throughout this course, we use λ λ to deote the eigevalues of matrix M of graph G. For regular graphs, λ = ad we maily cosider the secod largest eigevalue i absolute value. The formal defiitio is as follows. Defiitio 2.8 (spectral expasio). The spectral expasio of graph G is defied by λ := max { λ 2, λ }, i.e. λ = max Ax x =,x u Courat-Fischer Formula. Let B be a by symmetric matrix with eigevalues λ λ ad correspodig eigevectors v,..., v. The x T Bx λ = mi x = xt Bx = mi x 0 x T x, λ 2 = mi x = x v x T x T Bx Bx = mi x 0 x T x, x v x T Bx λ = max x = xt Bx = max x 0 x T x. It is well kow that λ relates to various graph properties. I particular, we shall see that there is a close coectio betwee λ ad the expasio of the graph. Lemma 2.9. d λ d( ). 3

4 Proof. Follows from tr ( M 2) = /d = i= λ2 i + ( )λ2. Theorem 2.0. [Alo86] Ay ifiite family of d-regular graphs {G } N has spectral expasio (as ) at least 2 d /d o(). Defiitio 2. (Ramauja graphs). A family of d-regular graphs with spectral expasio at most 2 d /d is called Ramauja graphs. Although Friedma [Fri9] showed that radom d-regular graphs are close to beig Ramauja i the sese that λ satisfies λ 2 d /d + 2 log(d)/d + o(), costructig families of Ramauja graphs with arbitrary degree is oe of the biggest ope problems i this area. So far, we oly kow the costructio of Ramauja graphs with certai degrees ad these costructios are based o deep algebraic kowledge. See [LPS88] for example. Aother quite importat problem is to fid a combiatorial costructio of Ramauja graphs. At the ed of this sectio, we list some more iterestig facts o eigevalues of graphs:. If graphs G ad H are isomorphic, the there is a permutatio matrix P such that P A(G) P T = A(H) ad hece the matrices A(G) ad A(H) are similar. 2. There are oisomorphic graphs with the same spectrum. See Figure. Figure : A example for two graphs which are ot isomorphic but have the same spectrum. Their commo graph spectrum is 2, 0, 0, 0, 2. 2 Combiatorial Expasio of Graphs For ay d-regular graph G = (V, E), let Γ(v) be the set of eighbors of v, i.e., Γ(v) = {u (u, v) E }. For ay subset S V, let Γ(S) = v S Γ(v) ad Γ (S) = Γ(S) S. Moreoever, for ay set S V we defie S := E(S, S). Defiitio 2.2 (vertex expasio). A graph G with vertices is said to have vertex expasio (K, A) if Γ(S) mi A. S : K If K = /2, the for simplicity we call G a A-expader. Iformally expaders are graphs with the property that every subset (uder some costrait o their size) has may eighbors outside the set. Moreover, we ca use differet ways to study expaders: () Combiatorically, expaders are highly coected graphs, ad to discoect a large part of the graph, oe has to remove may edges; (2) Geometrically, every vertex set has a relatively very large boudary; (3) From the Probabilistic view, expaders are graphs whose behavior is like radom graphs. (4) Algebraically, expaders are the real-symmetric matrix whose first positive eigevalue of the Laplace operator is bouded away from zero. 4

5 Figure 2: Compariso of the vertex expasio ad the edge expasio of a set of vertices of size 5. Defiitio 2.3 (edge expasio). The edge expasio of a graph G = (V, E) is defied by h(g) := S mi S : V /2. To explai edge expasio, let us see two examples. () If G is ot coected, we choose oe coected compoet as S so that E(S, S) = 0. Therefore h(g) = 0. (2) If G is a complete graph K, the E(S, S) = ( ) ad h(g) = /2. Defiitio 2.4 (expaders). Let d N. A sequece of d-regular graphs {G i } i N of size icreasig with i is a family of expaders if there is a costat ɛ > 0 such that h(g i ) ɛ for all i. Usually, whe speakig of a expader G i, we actually mea a family of graphs {G i } i N, where each graph i {G i } i N is d-regular ad its expasio is lower bouded by ɛ > 0. Observatio 2.5. Ay expader graph is a coected graph. 3 Spectral Expasio vs. Combiatorial Expasio The ext result shows that small spectral expasio implies large vertex expasio. Theorem 2.6 (spectral expasio vertex ( expasio). ) If G has spectral expasio λ, the for all 0 < α <, G has vertex expasio α,. ( α)λ 2 +α Before showig the proof, we itroduce some otatios at first. For ay probability distributio π, the support of π is defied by support(π) = {x : π x > 0}. Defiitio 2.7. Give a probability distributio π, the collisio probability of π is defied to be the probability that two idepedet samples from π are equal, i.e. CP(π) = x π2 x. Lemma 2.8. Let u = (/,..., /) be the uiform distributio. The for every probability distributio π [0, ], we have. CP(π) = π 2 = π u 2 + /. 2. CP(π) / support(π). Proof. () We write π as π = u + (π u) where u (π u). By Pythagorea theorem CP(π) = π 2 = π u 2 + u 2 = π u 2 + /. (2) By Cauchy-Schwarz iequality, we get = x support(π) π x 2 5 support(π) x π 2 x

6 ad hece CP(π) = x π 2 x support(π). Let us tur to the proof of Theorem 2.6. Proof. Let α. Choose a probability distributio π that is uiform o S ad 0 o the S, i.e. ( ) π =,,...,, 0,..., 0. Note that M is a real symmetric matrix, the M has orthoormal eigevectors v,..., v, the we ca decompose π as i= π i where π i is a costat multiplicity of v i. The CP(π) = / ad by Lemma 2.8 (2), CP(Mπ) support(mπ) = Γ(S). O the other had, by item () of Lemma 2.8 we have CP(Mπ) = Mπ u 2 = Mu + Mπ Mπ u 2 = λ 2 π λ π 2 ( λ 2 π u 2 = λ 2 CP(π) ) ( = λ 2 ). Hece ad Γ(S) Γ(S) CP(Mπ) ( λ2 ), ( ) λ 2 + λ 2 + ( λ 2 )α = = ( λ 2 α + ( α)λ 2. ) + = λ 2 + ( λ 2 ) / Theorem 2.9 (vertex expasio spectral expasio). Let G be a d-regular graph. For every δ > 0 ad d > 0, there exists γ > 0 such that if G is a d-regular ( + δ)-expader accordig to Defiitio 2.2, the it G has spectral expasio ( γ). Specifically, we ca take γ = Ω(δ 2 /d). Whe talkig about expaders, we ofte mea a family of d-regular graphs satisfyig oe of the followig two equivalet properties: Every graph i the family has spectral expasio λ. Every graph i the family is a ( + δ)-expader for some costat δ. 6

7 Refereces [Alo86] N. Alo. Eigevalues ad expaders. Combiatorica, 6(2):83 96, 986. [Fri9] Joel Friedma. O the secod eigevalue ad radom walks i radom d-regular graphs. Combiatorica, :33 362, 99. [LPS88] A. Lubotzky, R. Phillips, ad P. Sarak. Ramauja graphs. Combiatorica, 8:26 277,

CHAPTER IV: GRAPH THEORY. Section 1: Introduction to Graphs

CHAPTER IV: GRAPH THEORY. Section 1: Introduction to Graphs CHAPTER IV: GRAPH THEORY Sectio : Itroductio to Graphs Sice this class is called Number-Theoretic ad Discrete Structures, it would be a crime to oly focus o umber theory regardless how woderful those topics

More information

1 Graph Sparsfication

1 Graph Sparsfication CME 305: Discrete Mathematics ad Algorithms 1 Graph Sparsficatio I this sectio we discuss the approximatio of a graph G(V, E) by a sparse graph H(V, F ) o the same vertex set. I particular, we cosider

More information

New Results on Energy of Graphs of Small Order

New Results on Energy of Graphs of Small Order Global Joural of Pure ad Applied Mathematics. ISSN 0973-1768 Volume 13, Number 7 (2017), pp. 2837-2848 Research Idia Publicatios http://www.ripublicatio.com New Results o Eergy of Graphs of Small Order

More information

Strong Complementary Acyclic Domination of a Graph

Strong Complementary Acyclic Domination of a Graph Aals of Pure ad Applied Mathematics Vol 8, No, 04, 83-89 ISSN: 79-087X (P), 79-0888(olie) Published o 7 December 04 wwwresearchmathsciorg Aals of Strog Complemetary Acyclic Domiatio of a Graph NSaradha

More information

The Adjacency Matrix and The nth Eigenvalue

The Adjacency Matrix and The nth Eigenvalue Spectral Graph Theory Lecture 3 The Adjacecy Matrix ad The th Eigevalue Daiel A. Spielma September 5, 2012 3.1 About these otes These otes are ot ecessarily a accurate represetatio of what happeed i class.

More information

A RELATIONSHIP BETWEEN BOUNDS ON THE SUM OF SQUARES OF DEGREES OF A GRAPH

A RELATIONSHIP BETWEEN BOUNDS ON THE SUM OF SQUARES OF DEGREES OF A GRAPH J. Appl. Math. & Computig Vol. 21(2006), No. 1-2, pp. 233-238 Website: http://jamc.et A RELATIONSHIP BETWEEN BOUNDS ON THE SUM OF SQUARES OF DEGREES OF A GRAPH YEON SOO YOON AND JU KYUNG KIM Abstract.

More information

Sorting in Linear Time. Data Structures and Algorithms Andrei Bulatov

Sorting in Linear Time. Data Structures and Algorithms Andrei Bulatov Sortig i Liear Time Data Structures ad Algorithms Adrei Bulatov Algorithms Sortig i Liear Time 7-2 Compariso Sorts The oly test that all the algorithms we have cosidered so far is compariso The oly iformatio

More information

condition w i B i S maximum u i

condition w i B i S maximum u i ecture 10 Dyamic Programmig 10.1 Kapsack Problem November 1, 2004 ecturer: Kamal Jai Notes: Tobias Holgers We are give a set of items U = {a 1, a 2,..., a }. Each item has a weight w i Z + ad a utility

More information

Combination Labelings Of Graphs

Combination Labelings Of Graphs Applied Mathematics E-Notes, (0), - c ISSN 0-0 Available free at mirror sites of http://wwwmaththuedutw/ame/ Combiatio Labeligs Of Graphs Pak Chig Li y Received February 0 Abstract Suppose G = (V; E) is

More information

Some cycle and path related strongly -graphs

Some cycle and path related strongly -graphs Some cycle ad path related strogly -graphs I. I. Jadav, G. V. Ghodasara Research Scholar, R. K. Uiversity, Rajkot, Idia. H. & H. B. Kotak Istitute of Sciece,Rajkot, Idia. jadaviram@gmail.com gaurag ejoy@yahoo.co.i

More information

On (K t e)-saturated Graphs

On (K t e)-saturated Graphs Noame mauscript No. (will be iserted by the editor O (K t e-saturated Graphs Jessica Fuller Roald J. Gould the date of receipt ad acceptace should be iserted later Abstract Give a graph H, we say a graph

More information

On Characteristic Polynomial of Directed Divisor Graphs

On Characteristic Polynomial of Directed Divisor Graphs Iter. J. Fuzzy Mathematical Archive Vol. 4, No., 04, 47-5 ISSN: 30 34 (P), 30 350 (olie) Published o April 04 www.researchmathsci.org Iteratioal Joural of V. Maimozhi a ad V. Kaladevi b a Departmet of

More information

The isoperimetric problem on the hypercube

The isoperimetric problem on the hypercube The isoperimetric problem o the hypercube Prepared by: Steve Butler November 2, 2005 1 The isoperimetric problem We will cosider the -dimesioal hypercube Q Recall that the hypercube Q is a graph whose

More information

CS 683: Advanced Design and Analysis of Algorithms

CS 683: Advanced Design and Analysis of Algorithms CS 683: Advaced Desig ad Aalysis of Algorithms Lecture 6, February 1, 2008 Lecturer: Joh Hopcroft Scribes: Shaomei Wu, Etha Feldma February 7, 2008 1 Threshold for k CNF Satisfiability I the previous lecture,

More information

Symmetric Class 0 subgraphs of complete graphs

Symmetric Class 0 subgraphs of complete graphs DIMACS Techical Report 0-0 November 0 Symmetric Class 0 subgraphs of complete graphs Vi de Silva Departmet of Mathematics Pomoa College Claremot, CA, USA Chaig Verbec, Jr. Becer Friedma Istitute Booth

More information

Random Graphs and Complex Networks T

Random Graphs and Complex Networks T Radom Graphs ad Complex Networks T-79.7003 Charalampos E. Tsourakakis Aalto Uiversity Lecture 3 7 September 013 Aoucemet Homework 1 is out, due i two weeks from ow. Exercises: Probabilistic iequalities

More information

Lecture 6. Lecturer: Ronitt Rubinfeld Scribes: Chen Ziv, Eliav Buchnik, Ophir Arie, Jonathan Gradstein

Lecture 6. Lecturer: Ronitt Rubinfeld Scribes: Chen Ziv, Eliav Buchnik, Ophir Arie, Jonathan Gradstein 068.670 Subliear Time Algorithms November, 0 Lecture 6 Lecturer: Roitt Rubifeld Scribes: Che Ziv, Eliav Buchik, Ophir Arie, Joatha Gradstei Lesso overview. Usig the oracle reductio framework for approximatig

More information

A Note on Chromatic Transversal Weak Domination in Graphs

A Note on Chromatic Transversal Weak Domination in Graphs Iteratioal Joural of Mathematics Treds ad Techology Volume 17 Number 2 Ja 2015 A Note o Chromatic Trasversal Weak Domiatio i Graphs S Balamuruga 1, P Selvalakshmi 2 ad A Arivalaga 1 Assistat Professor,

More information

Lecture 1: Introduction and Strassen s Algorithm

Lecture 1: Introduction and Strassen s Algorithm 5-750: Graduate Algorithms Jauary 7, 08 Lecture : Itroductio ad Strasse s Algorithm Lecturer: Gary Miller Scribe: Robert Parker Itroductio Machie models I this class, we will primarily use the Radom Access

More information

Average Connectivity and Average Edge-connectivity in Graphs

Average Connectivity and Average Edge-connectivity in Graphs Average Coectivity ad Average Edge-coectivity i Graphs Jaehoo Kim, Suil O July 1, 01 Abstract Coectivity ad edge-coectivity of a graph measure the difficulty of breakig the graph apart, but they are very

More information

Convergence results for conditional expectations

Convergence results for conditional expectations Beroulli 11(4), 2005, 737 745 Covergece results for coditioal expectatios IRENE CRIMALDI 1 ad LUCA PRATELLI 2 1 Departmet of Mathematics, Uiversity of Bologa, Piazza di Porta Sa Doato 5, 40126 Bologa,

More information

Characterizing graphs of maximum principal ratio

Characterizing graphs of maximum principal ratio Characterizig graphs of maximum pricipal ratio Michael Tait ad Josh Tobi November 9, 05 Abstract The pricipal ratio of a coected graph, deoted γg, is the ratio of the maximum ad miimum etries of its first

More information

The Counterchanged Crossed Cube Interconnection Network and Its Topology Properties

The Counterchanged Crossed Cube Interconnection Network and Its Topology Properties WSEAS TRANSACTIONS o COMMUNICATIONS Wag Xiyag The Couterchaged Crossed Cube Itercoectio Network ad Its Topology Properties WANG XINYANG School of Computer Sciece ad Egieerig South Chia Uiversity of Techology

More information

Relationship between augmented eccentric connectivity index and some other graph invariants

Relationship between augmented eccentric connectivity index and some other graph invariants Iteratioal Joural of Advaced Mathematical Scieces, () (03) 6-3 Sciece Publishig Corporatio wwwsciecepubcocom/idexphp/ijams Relatioship betwee augmeted eccetric coectivity idex ad some other graph ivariats

More information

Recursive Estimation

Recursive Estimation Recursive Estimatio Raffaello D Adrea Sprig 2 Problem Set: Probability Review Last updated: February 28, 2 Notes: Notatio: Uless otherwise oted, x, y, ad z deote radom variables, f x (x) (or the short

More information

Improved Random Graph Isomorphism

Improved Random Graph Isomorphism Improved Radom Graph Isomorphism Tomek Czajka Gopal Paduraga Abstract Caoical labelig of a graph cosists of assigig a uique label to each vertex such that the labels are ivariat uder isomorphism. Such

More information

n n B. How many subsets of C are there of cardinality n. We are selecting elements for such a

n n B. How many subsets of C are there of cardinality n. We are selecting elements for such a 4. [10] Usig a combiatorial argumet, prove that for 1: = 0 = Let A ad B be disjoit sets of cardiality each ad C = A B. How may subsets of C are there of cardiality. We are selectig elemets for such a subset

More information

A study on Interior Domination in Graphs

A study on Interior Domination in Graphs IOSR Joural of Mathematics (IOSR-JM) e-issn: 2278-5728, p-issn: 219-765X. Volume 12, Issue 2 Ver. VI (Mar. - Apr. 2016), PP 55-59 www.iosrjourals.org A study o Iterior Domiatio i Graphs A. Ato Kisley 1,

More information

The size Ramsey number of a directed path

The size Ramsey number of a directed path The size Ramsey umber of a directed path Ido Be-Eliezer Michael Krivelevich Bey Sudakov May 25, 2010 Abstract Give a graph H, the size Ramsey umber r e (H, q) is the miimal umber m for which there is a

More information

On Spectral Theory Of K-n- Arithmetic Mean Idempotent Matrices On Posets

On Spectral Theory Of K-n- Arithmetic Mean Idempotent Matrices On Posets Iteratioal Joural of Sciece, Egieerig ad echology Research (IJSER), Volume 5, Issue, February 016 O Spectral heory Of -- Arithmetic Mea Idempotet Matrices O Posets 1 Dr N Elumalai, ProfRMaikada, 3 Sythiya

More information

CIS 121 Data Structures and Algorithms with Java Fall Big-Oh Notation Tuesday, September 5 (Make-up Friday, September 8)

CIS 121 Data Structures and Algorithms with Java Fall Big-Oh Notation Tuesday, September 5 (Make-up Friday, September 8) CIS 11 Data Structures ad Algorithms with Java Fall 017 Big-Oh Notatio Tuesday, September 5 (Make-up Friday, September 8) Learig Goals Review Big-Oh ad lear big/small omega/theta otatios Practice solvig

More information

Ones Assignment Method for Solving Traveling Salesman Problem

Ones Assignment Method for Solving Traveling Salesman Problem Joural of mathematics ad computer sciece 0 (0), 58-65 Oes Assigmet Method for Solvig Travelig Salesma Problem Hadi Basirzadeh Departmet of Mathematics, Shahid Chamra Uiversity, Ahvaz, Ira Article history:

More information

2 X = 2 X. The number of all permutations of a set X with n elements is. n! = n (n 1) (n 2) nn e n

2 X = 2 X. The number of all permutations of a set X with n elements is. n! = n (n 1) (n 2) nn e n 1 Discrete Mathematics revisited. Facts to remember Give set X, the umber of subsets of X is give by X = X. The umber of all permutatios of a set X with elemets is! = ( 1) ( )... 1 e π. The umber ( ) k

More information

FIGHTING CONSTRAINED FIRES IN GRAPHS

FIGHTING CONSTRAINED FIRES IN GRAPHS FIGHTING CONSTRAINED FIRES IN GRAPHS ANTHONY BONATO, MARGARET-ELLEN MESSINGER, AND PAWE L PRA LAT Abstract The Firefighter Problem is a simplified model for the spread of a fire or disease or computer

More information

Alpha Individual Solutions MAΘ National Convention 2013

Alpha Individual Solutions MAΘ National Convention 2013 Alpha Idividual Solutios MAΘ Natioal Covetio 0 Aswers:. D. A. C 4. D 5. C 6. B 7. A 8. C 9. D 0. B. B. A. D 4. C 5. A 6. C 7. B 8. A 9. A 0. C. E. B. D 4. C 5. A 6. D 7. B 8. C 9. D 0. B TB. 570 TB. 5

More information

Mean cordiality of some snake graphs

Mean cordiality of some snake graphs Palestie Joural of Mathematics Vol. 4() (015), 49 445 Palestie Polytechic Uiversity-PPU 015 Mea cordiality of some sake graphs R. Poraj ad S. Sathish Narayaa Commuicated by Ayma Badawi MSC 010 Classificatios:

More information

Visualization of Gauss-Bonnet Theorem

Visualization of Gauss-Bonnet Theorem Visualizatio of Gauss-Boet Theorem Yoichi Maeda maeda@keyaki.cc.u-tokai.ac.jp Departmet of Mathematics Tokai Uiversity Japa Abstract: The sum of exteral agles of a polygo is always costat, π. There are

More information

Matrix representation of a solution of a combinatorial problem of the group theory

Matrix representation of a solution of a combinatorial problem of the group theory Matrix represetatio of a solutio of a combiatorial problem of the group theory Krasimir Yordzhev, Lilyaa Totia Faculty of Mathematics ad Natural Scieces South-West Uiversity 66 Iva Mihailov Str, 2700 Blagoevgrad,

More information

On Infinite Groups that are Isomorphic to its Proper Infinite Subgroup. Jaymar Talledo Balihon. Abstract

On Infinite Groups that are Isomorphic to its Proper Infinite Subgroup. Jaymar Talledo Balihon. Abstract O Ifiite Groups that are Isomorphic to its Proper Ifiite Subgroup Jaymar Talledo Baliho Abstract Two groups are isomorphic if there exists a isomorphism betwee them Lagrage Theorem states that the order

More information

Perhaps the method will give that for every e > U f() > p - 3/+e There is o o-trivial upper boud for f() ad ot eve f() < Z - e. seems to be kow, where

Perhaps the method will give that for every e > U f() > p - 3/+e There is o o-trivial upper boud for f() ad ot eve f() < Z - e. seems to be kow, where ON MAXIMUM CHORDAL SUBGRAPH * Paul Erdos Mathematical Istitute of the Hugaria Academy of Scieces ad Reu Laskar Clemso Uiversity 1. Let G() deote a udirected graph, with vertices ad V(G) deote the vertex

More information

Lower Bounds for Sorting

Lower Bounds for Sorting Liear Sortig Topics Covered: Lower Bouds for Sortig Coutig Sort Radix Sort Bucket Sort Lower Bouds for Sortig Compariso vs. o-compariso sortig Decisio tree model Worst case lower boud Compariso Sortig

More information

THE COMPETITION NUMBERS OF JOHNSON GRAPHS

THE COMPETITION NUMBERS OF JOHNSON GRAPHS Discussioes Mathematicae Graph Theory 30 (2010 ) 449 459 THE COMPETITION NUMBERS OF JOHNSON GRAPHS Suh-Ryug Kim, Boram Park Departmet of Mathematics Educatio Seoul Natioal Uiversity, Seoul 151 742, Korea

More information

Examples and Applications of Binary Search

Examples and Applications of Binary Search Toy Gog ITEE Uiersity of Queeslad I the secod lecture last week we studied the biary search algorithm that soles the problem of determiig if a particular alue appears i a sorted list of iteger or ot. We

More information

Eigenimages. Digital Image Processing: Bernd Girod, Stanford University -- Eigenimages 1

Eigenimages. Digital Image Processing: Bernd Girod, Stanford University -- Eigenimages 1 Eigeimages Uitary trasforms Karhue-Loève trasform ad eigeimages Sirovich ad Kirby method Eigefaces for geder recogitio Fisher liear discrimat aalysis Fisherimages ad varyig illumiatio Fisherfaces vs. eigefaces

More information

INTERSECTION CORDIAL LABELING OF GRAPHS

INTERSECTION CORDIAL LABELING OF GRAPHS INTERSECTION CORDIAL LABELING OF GRAPHS G Meea, K Nagaraja Departmet of Mathematics, PSR Egieerig College, Sivakasi- 66 4, Virudhuagar(Dist) Tamil Nadu, INDIA meeag9@yahoocoi Departmet of Mathematics,

More information

Some non-existence results on Leech trees

Some non-existence results on Leech trees Some o-existece results o Leech trees László A.Székely Hua Wag Yog Zhag Uiversity of South Carolia This paper is dedicated to the memory of Domiique de Cae, who itroduced LAS to Leech trees.. Abstract

More information

ON A PROBLEM OF C. E. SHANNON IN GRAPH THEORY

ON A PROBLEM OF C. E. SHANNON IN GRAPH THEORY ON A PROBLEM OF C. E. SHANNON IN GRAPH THEORY m. rosefeld1 1. Itroductio. We cosider i this paper oly fiite odirected graphs without multiple edges ad we assume that o each vertex of the graph there is

More information

How do we evaluate algorithms?

How do we evaluate algorithms? F2 Readig referece: chapter 2 + slides Algorithm complexity Big O ad big Ω To calculate ruig time Aalysis of recursive Algorithms Next time: Litterature: slides mostly The first Algorithm desig methods:

More information

arxiv: v2 [cs.ds] 24 Mar 2018

arxiv: v2 [cs.ds] 24 Mar 2018 Similar Elemets ad Metric Labelig o Complete Graphs arxiv:1803.08037v [cs.ds] 4 Mar 018 Pedro F. Felzeszwalb Brow Uiversity Providece, RI, USA pff@brow.edu March 8, 018 We cosider a problem that ivolves

More information

1.2 Binomial Coefficients and Subsets

1.2 Binomial Coefficients and Subsets 1.2. BINOMIAL COEFFICIENTS AND SUBSETS 13 1.2 Biomial Coefficiets ad Subsets 1.2-1 The loop below is part of a program to determie the umber of triagles formed by poits i the plae. for i =1 to for j =

More information

Counting the Number of Minimum Roman Dominating Functions of a Graph

Counting the Number of Minimum Roman Dominating Functions of a Graph Coutig the Number of Miimum Roma Domiatig Fuctios of a Graph SHI ZHENG ad KOH KHEE MENG, Natioal Uiversity of Sigapore We provide two algorithms coutig the umber of miimum Roma domiatig fuctios of a graph

More information

Graphs ORD SFO LAX DFW. Lecture notes adapted from Goodrich and Tomassia. 3/14/18 10:28 AM Graphs 1

Graphs ORD SFO LAX DFW. Lecture notes adapted from Goodrich and Tomassia. 3/14/18 10:28 AM Graphs 1 Graphs 337 1843 1743 1233 802 Lecture otes adapted from Goodrich ad Tomassia 3/14/18 10:28 AM Graphs 1 Graph A graph is a pair (V, E), where V is a set of odes, called vertices E is a collectio of pairs

More information

Octahedral Graph Scaling

Octahedral Graph Scaling Octahedral Graph Scalig Peter Russell Jauary 1, 2015 Abstract There is presetly o strog iterpretatio for the otio of -vertex graph scalig. This paper presets a ew defiitio for the term i the cotext of

More information

Assignment 5; Due Friday, February 10

Assignment 5; Due Friday, February 10 Assigmet 5; Due Friday, February 10 17.9b The set X is just two circles joied at a poit, ad the set X is a grid i the plae, without the iteriors of the small squares. The picture below shows that the iteriors

More information

NTH, GEOMETRIC, AND TELESCOPING TEST

NTH, GEOMETRIC, AND TELESCOPING TEST NTH, GEOMETRIC, AND TELESCOPING TEST Sectio 9. Calculus BC AP/Dual, Revised 08 viet.dag@humbleisd.et /4/08 0:0 PM 9.: th, Geometric, ad Telescopig Test SUMMARY OF TESTS FOR SERIES Lookig at the first few

More information

CS473-Algorithms I. Lecture 2. Asymptotic Notation. CS 473 Lecture 2 1

CS473-Algorithms I. Lecture 2. Asymptotic Notation. CS 473 Lecture 2 1 CS473-Algorithms I Lecture Asymptotic Notatio CS 473 Lecture 1 O-otatio (upper bouds) f() = O(g()) if positive costats c, 0 such that e.g., = O( 3 ) 0 f() cg(), 0 c 3 c c = 1 & 0 = or c = & 0 = 1 Asymptotic

More information

Eigenimages. Digital Image Processing: Bernd Girod, 2013 Stanford University -- Eigenimages 1

Eigenimages. Digital Image Processing: Bernd Girod, 2013 Stanford University -- Eigenimages 1 Eigeimages Uitary trasforms Karhue-Loève trasform ad eigeimages Sirovich ad Kirby method Eigefaces for geder recogitio Fisher liear discrimat aalysis Fisherimages ad varyig illumiatio Fisherfaces vs. eigefaces

More information

Throughput-Delay Scaling in Wireless Networks with Constant-Size Packets

Throughput-Delay Scaling in Wireless Networks with Constant-Size Packets Throughput-Delay Scalig i Wireless Networks with Costat-Size Packets Abbas El Gamal, James Mamme, Balaji Prabhakar, Devavrat Shah Departmets of EE ad CS Staford Uiversity, CA 94305 Email: {abbas, jmamme,

More information

Recursive Procedures. How can you model the relationship between consecutive terms of a sequence?

Recursive Procedures. How can you model the relationship between consecutive terms of a sequence? 6. Recursive Procedures I Sectio 6.1, you used fuctio otatio to write a explicit formula to determie the value of ay term i a Sometimes it is easier to calculate oe term i a sequece usig the previous terms.

More information

Module 8-7: Pascal s Triangle and the Binomial Theorem

Module 8-7: Pascal s Triangle and the Binomial Theorem Module 8-7: Pascal s Triagle ad the Biomial Theorem Gregory V. Bard April 5, 017 A Note about Notatio Just to recall, all of the followig mea the same thig: ( 7 7C 4 C4 7 7C4 5 4 ad they are (all proouced

More information

Big-O Analysis. Asymptotics

Big-O Analysis. Asymptotics Big-O Aalysis 1 Defiitio: Suppose that f() ad g() are oegative fuctios of. The we say that f() is O(g()) provided that there are costats C > 0 ad N > 0 such that for all > N, f() Cg(). Big-O expresses

More information

Hash Tables. Presentation for use with the textbook Algorithm Design and Applications, by M. T. Goodrich and R. Tamassia, Wiley, 2015.

Hash Tables. Presentation for use with the textbook Algorithm Design and Applications, by M. T. Goodrich and R. Tamassia, Wiley, 2015. Presetatio for use with the textbook Algorithm Desig ad Applicatios, by M. T. Goodrich ad R. Tamassia, Wiley, 2015 Hash Tables xkcd. http://xkcd.com/221/. Radom Number. Used with permissio uder Creative

More information

THE DIAMETER GAME JÓZSEF BALOGH, RYAN MARTIN, AND ANDRÁS PLUHÁR

THE DIAMETER GAME JÓZSEF BALOGH, RYAN MARTIN, AND ANDRÁS PLUHÁR THE DIAMETER GAME JÓZSEF BALOGH, RYAN MARTIN, AND ANDRÁS PLUHÁR Abstract. A large class of the so-called Positioal Games are defied o the complete graph o vertices. The players, Maker ad Breaker, take

More information

Compactness of Fuzzy Sets

Compactness of Fuzzy Sets Compactess of uzzy Sets Amai E. Kadhm Departmet of Egieerig Programs, Uiversity College of Madeat Al-Elem, Baghdad, Iraq. Abstract The objective of this paper is to study the compactess of fuzzy sets i

More information

Big-O Analysis. Asymptotics

Big-O Analysis. Asymptotics Big-O Aalysis 1 Defiitio: Suppose that f() ad g() are oegative fuctios of. The we say that f() is O(g()) provided that there are costats C > 0 ad N > 0 such that for all > N, f() Cg(). Big-O expresses

More information

Name of the Student: Unit I (Logic and Proofs) 1) Truth Table: Conjunction Disjunction Conditional Biconditional

Name of the Student: Unit I (Logic and Proofs) 1) Truth Table: Conjunction Disjunction Conditional Biconditional SUBJECT NAME : Discrete Mathematics SUBJECT CODE : MA 2265 MATERIAL NAME : Formula Material MATERIAL CODE : JM08ADM009 (Sca the above QR code for the direct dowload of this material) Name of the Studet:

More information

An Efficient Algorithm for Graph Bisection of Triangularizations

An Efficient Algorithm for Graph Bisection of Triangularizations A Efficiet Algorithm for Graph Bisectio of Triagularizatios Gerold Jäger Departmet of Computer Sciece Washigto Uiversity Campus Box 1045 Oe Brookigs Drive St. Louis, Missouri 63130-4899, USA jaegerg@cse.wustl.edu

More information

Super Vertex Magic and E-Super Vertex Magic. Total Labelling

Super Vertex Magic and E-Super Vertex Magic. Total Labelling Proceedigs of the Iteratioal Coferece o Applied Mathematics ad Theoretical Computer Sciece - 03 6 Super Vertex Magic ad E-Super Vertex Magic Total Labellig C.J. Deei ad D. Atoy Xavier Abstract--- For a

More information

Protected points in ordered trees

Protected points in ordered trees Applied Mathematics Letters 008 56 50 www.elsevier.com/locate/aml Protected poits i ordered trees Gi-Sag Cheo a, Louis W. Shapiro b, a Departmet of Mathematics, Sugkyukwa Uiversity, Suwo 440-746, Republic

More information

Lecture Notes 6 Introduction to algorithm analysis CSS 501 Data Structures and Object-Oriented Programming

Lecture Notes 6 Introduction to algorithm analysis CSS 501 Data Structures and Object-Oriented Programming Lecture Notes 6 Itroductio to algorithm aalysis CSS 501 Data Structures ad Object-Orieted Programmig Readig for this lecture: Carrao, Chapter 10 To be covered i this lecture: Itroductio to algorithm aalysis

More information

ENGI 4421 Probability and Statistics Faculty of Engineering and Applied Science Problem Set 1 Descriptive Statistics

ENGI 4421 Probability and Statistics Faculty of Engineering and Applied Science Problem Set 1 Descriptive Statistics ENGI 44 Probability ad Statistics Faculty of Egieerig ad Applied Sciece Problem Set Descriptive Statistics. If, i the set of values {,, 3, 4, 5, 6, 7 } a error causes the value 5 to be replaced by 50,

More information

Sum-connectivity indices of trees and unicyclic graphs of fixed maximum degree

Sum-connectivity indices of trees and unicyclic graphs of fixed maximum degree 1 Sum-coectivity idices of trees ad uicyclic graphs of fixed maximum degree Zhibi Du a, Bo Zhou a *, Nead Triajstić b a Departmet of Mathematics, South Chia Normal Uiversity, uagzhou 510631, Chia email:

More information

CSE 417: Algorithms and Computational Complexity

CSE 417: Algorithms and Computational Complexity Time CSE 47: Algorithms ad Computatioal Readig assigmet Read Chapter of The ALGORITHM Desig Maual Aalysis & Sortig Autum 00 Paul Beame aalysis Problem size Worst-case complexity: max # steps algorithm

More information

Bezier curves. Figure 2 shows cubic Bezier curves for various control points. In a Bezier curve, only

Bezier curves. Figure 2 shows cubic Bezier curves for various control points. In a Bezier curve, only Edited: Yeh-Liag Hsu (998--; recommeded: Yeh-Liag Hsu (--9; last updated: Yeh-Liag Hsu (9--7. Note: This is the course material for ME55 Geometric modelig ad computer graphics, Yua Ze Uiversity. art of

More information

CSC165H1 Worksheet: Tutorial 8 Algorithm analysis (SOLUTIONS)

CSC165H1 Worksheet: Tutorial 8 Algorithm analysis (SOLUTIONS) CSC165H1, Witer 018 Learig Objectives By the ed of this worksheet, you will: Aalyse the ruig time of fuctios cotaiig ested loops. 1. Nested loop variatios. Each of the followig fuctios takes as iput a

More information

Chapter 3 Classification of FFT Processor Algorithms

Chapter 3 Classification of FFT Processor Algorithms Chapter Classificatio of FFT Processor Algorithms The computatioal complexity of the Discrete Fourier trasform (DFT) is very high. It requires () 2 complex multiplicatios ad () complex additios [5]. As

More information

Lecture 5. Counting Sort / Radix Sort

Lecture 5. Counting Sort / Radix Sort Lecture 5. Coutig Sort / Radix Sort T. H. Corme, C. E. Leiserso ad R. L. Rivest Itroductio to Algorithms, 3rd Editio, MIT Press, 2009 Sugkyukwa Uiversity Hyuseug Choo choo@skku.edu Copyright 2000-2018

More information

15-859E: Advanced Algorithms CMU, Spring 2015 Lecture #2: Randomized MST and MST Verification January 14, 2015

15-859E: Advanced Algorithms CMU, Spring 2015 Lecture #2: Randomized MST and MST Verification January 14, 2015 15-859E: Advaced Algorithms CMU, Sprig 2015 Lecture #2: Radomized MST ad MST Verificatio Jauary 14, 2015 Lecturer: Aupam Gupta Scribe: Yu Zhao 1 Prelimiaries I this lecture we are talkig about two cotets:

More information

The digraph drop polynomial

The digraph drop polynomial The digraph drop polyomial Fa Chug Ro Graham Abstract For a weighted directed graph (or digraph, for short), deoted by D = (V, E, w), we defie a two-variable polyomial B D (x, y), called the drop polyomial

More information

Area As A Limit & Sigma Notation

Area As A Limit & Sigma Notation Area As A Limit & Sigma Notatio SUGGESTED REFERENCE MATERIAL: As you work through the problems listed below, you should referece Chapter 5.4 of the recommeded textbook (or the equivalet chapter i your

More information

Thompson s Group F (p + 1) is not Minimally Almost Convex

Thompson s Group F (p + 1) is not Minimally Almost Convex Thompso s Group F (p + ) is ot Miimally Almost Covex Claire Wladis Thompso s Group F (p + ). A Descriptio of F (p + ) Thompso s group F (p + ) ca be defied as the group of piecewiseliear orietatio-preservig

More information

4-Prime cordiality of some cycle related graphs

4-Prime cordiality of some cycle related graphs Available at http://pvamu.edu/aam Appl. Appl. Math. ISSN: 193-9466 Vol. 1, Issue 1 (Jue 017), pp. 30 40 Applicatios ad Applied Mathematics: A Iteratioal Joural (AAM) 4-Prime cordiality of some cycle related

More information

Pattern Recognition Systems Lab 1 Least Mean Squares

Pattern Recognition Systems Lab 1 Least Mean Squares Patter Recogitio Systems Lab 1 Least Mea Squares 1. Objectives This laboratory work itroduces the OpeCV-based framework used throughout the course. I this assigmet a lie is fitted to a set of poits usig

More information

Matrix Partitions of Split Graphs

Matrix Partitions of Split Graphs Matrix Partitios of Split Graphs Tomás Feder, Pavol Hell, Ore Shklarsky Abstract arxiv:1306.1967v2 [cs.dm] 20 Ju 2013 Matrix partitio problems geeralize a umber of atural graph partitio problems, ad have

More information

Normal Distributions

Normal Distributions Normal Distributios Stacey Hacock Look at these three differet data sets Each histogram is overlaid with a curve : A B C A) Weights (g) of ewly bor lab rat pups B) Mea aual temperatures ( F ) i A Arbor,

More information

An Efficient Algorithm for Graph Bisection of Triangularizations

An Efficient Algorithm for Graph Bisection of Triangularizations Applied Mathematical Scieces, Vol. 1, 2007, o. 25, 1203-1215 A Efficiet Algorithm for Graph Bisectio of Triagularizatios Gerold Jäger Departmet of Computer Sciece Washigto Uiversity Campus Box 1045, Oe

More information

The Platonic solids The five regular polyhedra

The Platonic solids The five regular polyhedra The Platoic solids The five regular polyhedra Ole Witt-Hase jauary 7 www.olewitthase.dk Cotets. Polygos.... Topologically cosideratios.... Euler s polyhedro theorem.... Regular ets o a sphere.... The dihedral

More information

On Ryser s conjecture for t-intersecting and degree-bounded hypergraphs arxiv: v2 [math.co] 9 Dec 2017

On Ryser s conjecture for t-intersecting and degree-bounded hypergraphs arxiv: v2 [math.co] 9 Dec 2017 O Ryser s cojecture for t-itersectig ad degree-bouded hypergraphs arxiv:1705.1004v [math.co] 9 Dec 017 Zoltá Király Departmet of Computer Sciece ad Egerváry Research Group (MTA-ELTE) Eötvös Uiversity Pázmáy

More information

c-dominating Sets for Families of Graphs

c-dominating Sets for Families of Graphs c-domiatig Sets for Families of Graphs Kelsie Syder Mathematics Uiversity of Mary Washigto April 6, 011 1 Abstract The topic of domiatio i graphs has a rich history, begiig with chess ethusiasts i the

More information

An (or ) is a sequence in which each term after the first differs from the preceding term by a fixed constant, called the.

An (or ) is a sequence in which each term after the first differs from the preceding term by a fixed constant, called the. Sectio.2 Arithmetic Sequeces ad Series -.2 Arithmetic Sequeces ad Series Arithmetic Sequeces Arithmetic Series Key Terms: arithmetic sequece (arithmetic progressio), commo differece, arithmetic series

More information

ON MATHIEU-BERG S INEQUALITY

ON MATHIEU-BERG S INEQUALITY ON MATHIEU-BERG S INEQUALITY BICHENG YANG DEPARTMENT OF MATHEMATICS, GUANGDONG EDUCATION COLLEGE, GUANGZHOU, GUANGDONG 533, PEOPLE S REPUBLIC OF CHINA. bcyag@pub.guagzhou.gd.c ABSTRACT. I this paper, by

More information

Analysis Metrics. Intro to Algorithm Analysis. Slides. 12. Alg Analysis. 12. Alg Analysis

Analysis Metrics. Intro to Algorithm Analysis. Slides. 12. Alg Analysis. 12. Alg Analysis Itro to Algorithm Aalysis Aalysis Metrics Slides. Table of Cotets. Aalysis Metrics 3. Exact Aalysis Rules 4. Simple Summatio 5. Summatio Formulas 6. Order of Magitude 7. Big-O otatio 8. Big-O Theorems

More information

Some New Results on Prime Graphs

Some New Results on Prime Graphs Ope Joural of Discrete Mathematics, 202, 2, 99-04 http://dxdoiorg/0426/ojdm202209 Published Olie July 202 (http://wwwscirporg/joural/ojdm) Some New Results o Prime Graphs Samir Vaidya, Udaya M Prajapati

More information

Algorithms Chapter 3 Growth of Functions

Algorithms Chapter 3 Growth of Functions Algorithms Chapter 3 Growth of Fuctios Istructor: Chig Chi Li 林清池助理教授 chigchi.li@gmail.com Departmet of Computer Sciece ad Egieerig Natioal Taiwa Ocea Uiversity Outlie Asymptotic otatio Stadard otatios

More information

EVALUATION OF TRIGONOMETRIC FUNCTIONS

EVALUATION OF TRIGONOMETRIC FUNCTIONS EVALUATION OF TRIGONOMETRIC FUNCTIONS Whe first exposed to trigoometric fuctios i high school studets are expected to memorize the values of the trigoometric fuctios of sie cosie taget for the special

More information

. Perform a geometric (ray-optics) construction (i.e., draw in the rays on the diagram) to show where the final image is formed.

. Perform a geometric (ray-optics) construction (i.e., draw in the rays on the diagram) to show where the final image is formed. MASSACHUSETTS INSTITUTE of TECHNOLOGY Departmet of Electrical Egieerig ad Computer Sciece 6.161 Moder Optics Project Laboratory 6.637 Optical Sigals, Devices & Systems Problem Set No. 1 Geometric optics

More information

What are we going to learn? CSC Data Structures Analysis of Algorithms. Overview. Algorithm, and Inputs

What are we going to learn? CSC Data Structures Analysis of Algorithms. Overview. Algorithm, and Inputs What are we goig to lear? CSC316-003 Data Structures Aalysis of Algorithms Computer Sciece North Carolia State Uiversity Need to say that some algorithms are better tha others Criteria for evaluatio Structure

More information

MAXIMUM MATCHINGS IN COMPLETE MULTIPARTITE GRAPHS

MAXIMUM MATCHINGS IN COMPLETE MULTIPARTITE GRAPHS Fura Uiversity Electroic Joural of Udergraduate Matheatics Volue 00, 1996 6-16 MAXIMUM MATCHINGS IN COMPLETE MULTIPARTITE GRAPHS DAVID SITTON Abstract. How ay edges ca there be i a axiu atchig i a coplete

More information

Graph operations and synchronization of complex networks

Graph operations and synchronization of complex networks PHYSICAL REVIEW E 72, 016217 2005 Graph operatios ad sychroizatio of complex etworks Fatihca M. Atay* ad Türker Bıyıkoğlu Max Plack Istitute for Mathematics i the Scieces, Iselstr. 22, D-04103 Leipzig,

More information

COMP 558 lecture 6 Sept. 27, 2010

COMP 558 lecture 6 Sept. 27, 2010 Radiometry We have discussed how light travels i straight lies through space. We would like to be able to talk about how bright differet light rays are. Imagie a thi cylidrical tube ad cosider the amout

More information