Non-Regular Languages and The Pumping Lemma

Size: px
Start display at page:

Download "Non-Regular Languages and The Pumping Lemma"

Transcription

1 CS240 Lnguge Theory nd Automt Fll 2011 Non-Regulr Lnguges nd The Pumping Lemm Non-Regulr Lnguges Not every lnguge is regulr lnguge. However, there re some rules tht sy "if these lnguges re regulr, so is this one derived from them" There is lso powerful technique -- the pumping lemm -- tht helps us prove lnguge not to e regulr. Key tool: Since we know RE's, DFA's, NFA's, NFAε's ll define exctly the regulr lnguges, we cn use whichever representtion suits us when proving something out regulr lnguge. The Pumping Lemm If L is regulr lnguge, then there exists constnt n such tht every string w in L, of length n or more, cn e written s w = xyz, where: 0 < y xy <= n For ll i 0, xy i z is lso in L Note y i = y repeted i times; y 0 = ε. Intuitive Explntion The utomton elow hs n sttes nd no loops. Expressed in terms of n, wht is the longest string this utomton cn ccept? Generlly, in n utomton (grph) with n sttes (vertices), ny "wlk" of length n or greter must repet some stte (vertex)--tht is, it must contin cycle 1

2 Proof of Pumping Lemm Since we clim L is regulr, there must e DFA A such tht L = L(A). Let A hve n sttes; choose this n for the pumping lemm Let w e string of length n in L, sy w = 1 2 m, where m n. Let q i e the stte A is in fter reding the first i symols of w. q 0 = strt stte, q 1 = δ(q 0, 1 ), q 2 = ˆ δ (q 0, 1 2 ), etc. Since there re only n different sttes, two of q 0, q 1, q n must e the sme; sy q i = q j, where 0 <= i < j <= n. Let x = 1 i ; y = i+1 j ; z = j +1 m. Then y repeting the loop from q i to q j with lel i +1 j zero times, once, or more, we cn show tht xy i z is ccepted y A. y! i+1 j! 1! q j!. i q i! j +1 m! z! x! Exmple DFA with 6 sttes tht ccepts n infinite lnguge , Any string of length 6 or more contins circuit Some strings with length < 6 lso contin circuit (), Pth tht this string tkes through the DFA cn e decomposed into three stges: 1. x prt : goes from strt stte to eginning of the first circuit 2. y prt : circuit 3. z prt : the rest x y z 2

3 PL gets its nme ecuse the repeted string is "pumped" Note tht ecuse of the nture of FAs, we cnnot control the numer of times it is pumped So, regulr lnguge with strings of length n is lwys infinite! PL is only interesting for infinite lnguges ut works for finite lnguges, which re lwys regulr--for finite lnguges n is lrger thn the longest string, so nothing cn e pumped PL Use We use the PL to show lnguge L is not regulr. Strt y ssuming L is regulr. Then there must e some n tht serves s the PL constnt. We my not know wht n is, ut we cn work the rest of the "gme" with n s prmeter. We choose some w tht is known to e in L. Typiclly, w depends on n. Applying the PL, we know w cn e roken into xyz, stisfying the PL properties. Agin, we my not know how to rek w, so we use x, y, z s prmeters. We derive contrdiction y picking i (which might depend on n, x, y, nd/or z) such tht xy i z is not in L. Exmple Consider the lnguge i i This lnguge is not regulr! Intuitive explntion: Imgine n FA to ccept this lnguge Since the numer of s must e equl to the numer of s, must hve some wy to rememer how mny s were seen, nd ccept if the rest of the string contins the sme numer of s 3

4 How mny sttes re needed? 1 2 s etc. 1, 1 2 s, 2 s Using the PL to prove L = i i is not regulr Suppose L is regulr. Then there is constnt n stisfying the PL conditions. Consider the string w = n n Then w = xyz, where xy <= n nd y ε, nd we cn rek this string into xyz where for ny j 0 xy j z is in L But ecuse xy <= n nd y >0, the string y hs to consist of s only. So no mtter wht segment of the string xy covers, pumping y dds to the numer of s nd hence there re more s thn s There is NO WAY to segment w into xyz such tht pumping will not led to string tht is not in the lnguge! CONTRADICTION! L is therefore not regulr Importnt point It is necessry to show there is no segmenttion of the chosen string tht won t led to contrdiction This mens considering every possile mpping of xy onto the first n symols in the chosen string We chose our string to mke this esy, since very possile segmenttion consists of s only Pumping therefore disrupts the equivlence of the numer of s nd s Exmple Consider the set of strings of 's whose length is squre; formlly, L = { i i is squre}. We clim L is not regulr. Suppose L is regulr. Then there is constnt n stisfying the PL conditions. Consider w = n2, which is surely in L. Then w = xyz, where xy <= n nd y ε. 4

5 By PL, xyyz (xy 2 z) is in L. The length of xyyz is greter thn n 2 nd no greter thn n 2 + n. (Why?) However, the next perfect squre fter n 2 is (n+1) 2 = n 2 + 2n + 1. Thus, xyyz is not of squre length nd is not in L. Since we hve derived contrdiction, the only unproved ssumption -- tht L is regulr -- must e t fult, nd we hve "proof y contrdiction" tht L is not regulr. The PL "gme" Gol: win the PL gme ginst our opponent y estlishing contrdiction of the PL, while the opponent tries to foil us. Four steps: 1.The numer of sttes in the utomton is n. Note tht we don't hve to know wht n is, since we use the vrile to define our string. 2. Given n, we pick string w in L of length equl to or greter thn n. We re free to choose ny w, suject to w L nd w n. We usully define the string in terms of n. 3. Our opponent chooses the decomposition xyz, suject to xy <= n, y We try to pick i (the power fctor in xy i z) in such wy tht the pumped string w i is not in L. If we cn do so, we win the gme! Exmple 1 Σ = {,}; L = {ww R w Σ*} Whtever n is, we cn lwys choose w s follows: n n n n x y Becuse of this choice nd the requirement tht xy <= n, the opponent is restricted in step 3 to choosing y tht consists entirely of s. In step 4, we use i=2.the string xy 2 z hs more 's on the left thn on the right, so it cnnot e of form ww R. So L is not regulr. z 5

6 Exmple 2 L = {w w hs n equl numer of 1's nd 0's} Given n, we choose the string (01) n We need to show splitting this string into xyz where xy i z is in L is impossile But it is possile! If x = ε, y = 01, nd z = (01) n-1, xy i z is in L for every vlue of i. Are we out of luck? First lw of PL use: If your string does not succeed, try nother! Let's try 1 n 0 n. Agin, we need to show splitting this string into xyz where xy i z is in L is impossile But it is possile! If x nd z re the empty string nd y is 1 n 0 n, then xy i z lwys hs n equl numer of 0's nd 1's. Are we still in troule? Not this time the PL sys tht our string hs to e divided so tht xy <= n nd y. If xy <= n then y must consist only of 0's, so xyyz L. Contrdiction! We win! Exmple 3 L = {ww w Σ*} We choose the string n n, where n is the numer of sttes in the FA. We now show tht there is no decomposition of this string into xyz where for ny j 0 xy j z is in L. Agin, it is crucil tht the PL insists tht xy <= n, ecuse without it we could could pump the string if we let x nd z e the empty string. With this condition, it's esy to show tht the PL won't pply ecuse y must consist only of 's, so xyyz is not in L. 6

7 In the previous exmple s efore, the choice of string is criticl: hd we chosen n n (which is memer of L) insted of n n, it wouldn't work ecuse it cn e pumped nd still stisfy the PL. MORAL Choose your strings wisely.! Exmple 4 L = {0 i 1 j i > j} Given n, choose s = 0 n+1 1 n. Split into xyz etc. Becuse y the PL xy <= n, y consists only of 0's. Is xyyz in L? The PL sttes tht xy i z is in L even when i = 0 So, consider the string xy 0 z Removing string y decreses the numer of 0's in s s hs only one more 0 thn 1 Therefore, xz cnnot hve more 0's thn 1's, nd is not memer of L. Contrdiction! This strtegy is clled pumping down Exmple 5 L = { i i is prime} Let n e the pumping lemm vlue nd let k e prime greter thn n. If L is regulr, PL implies tht k cn e decomposed into xyz, y > 0, such tht xy i z is in L for ll i 0. Assume such decomposition exists. The length of w = xy k+1 z must e prime if w is in L. But length(xy k+1 z) = length(xyzy k ) = length(xyz) + length(y k ) = k + k(length(y) = k (1 + length(y)) The length of xy k+1 z is therefore not prime, since it is the product of two numers other thn 1. So xy k+1 z is not in L. Contrdiction! 7

8 Exmple 6 L = {w Σ* n (w) > n (w)} Let n e the pumping lemm constnt. Then if L is regulr, PL implies tht s = n n+1 cn e decomposed into xyz, y > 0, xy n, such tht xy i z is in L for ll i 0. Since the length of xy n, y consists of ll s Then xy 2 z = k-j j n-k n+1, where the length of of y = j. We know j > 0 so the length of the pumped string contins t lest s mny s s s, nd is not in L. Contrdiction! Exmple 7 L = { 3 m c m-3 m > 3} Let n e the pumping lemm constnt. Then if L is regulr, PL implies tht s = 3 n c n-3 cn e decomposed into xyz, y > 0, xy n, such tht xy i z is in L for ll i 0. Since the length of xy n, there re three wys to prtition s: 1. y consists of ll s Pumping y will led to string with more thn 3 s -- not in L 2. y consists of ll s Pumping y will led to string with more thn m s, nd leve the numer of c s untouched, such tht there re no longer 3 fewer c s thn s -- not in L 3. y consists of s nd s Pumping y will led to string with s efore s, -- not in L There is no wy to prtition 3 n n-3 so tht pumped strings re still in L. Contrdiction! Rememer You need to find only ONE string for which the PL does not hold to prove lnguge is not regulr But you must show tht for ANY decomposition of tht string into xyz the PL holds This sometimes mens considering severl different cses The Pumping Lemm Poem Any regulr lnguge L hs mgic numer p And ny long-enough word in L hs the following property: Among its first p symols is segment you cn find Whose repetition or omission leves x mong its kind. So if you find lnguge L which fils this cid test, And some long word you pump ecomes distinct from ll the rest, By contrdiction you hve shown tht lnguge L is not A regulr guy, resilient to the dmge you hve wrought. But if, upon the other hnd, x stys within its L, Then either L is regulr, or else you chose not well. For w is xyz, nd y cnnot e null, And y must come efore p symols hve een red in full. As mthemticl postscript, n ddendum to the wise: The sic proof we outlined here does certinly generlize. So there is pumping lemm for ll lnguges context-free, Although we do not hve the sme for those tht re r.e. 8

9 Proving lnguge non-regulr without the pumping lemm The pumping lemm isn't the only wy we cn prove lnguge is non-regulr Other techniques: show tht the desired DFA would require infinite sttes to model the intended lnguge use closure properties to relte to other non-rl lnguges DFA Method Consider the lnguge { i i i >= 0} nd DFA to recognize it For ny i, let i e the stte entered fter processing i, i.e., ˆ δ (q 0, i ) = i. Consider ny i nd j such tht i j. ˆ δ (q 0, i i ) ˆ δ (q 0, j i ), since the former is ccepting, nd the ltter is rejecting. ˆ δ (q 0, i i ) = ˆ δ ( ˆ δ (q 0, i ), i ) = ˆ δ ( i, i ), y definition of ˆ δ nd definition of i, respectively. ˆ (q 0, j i ) = ˆ δ δ ( ˆ δ (q 0, j ), i ) = ˆ δ ( j, i ), y the sme resoning. Since i nd j led to different sttes on the sme input, i j. Since i nd j were ritrry, nd since there re n infinite numer of wys to pick them, there must e n infinite numer of sttes. Thus, there is no DFA to recognize this lnguge, nd the lnguge is non-regulr. 9

10 Closure Properties Certin opertions on regulr lnguges re gurnteed to produce regulr lnguges Closure properties cn lso e used to prove lnguge non-regulr (or regulr) Regulr lnguges re closed under common set opertions Union : L 1 L 2 Intersection : L 1 L 2 Conctention : L 1 L 2 Complementtion : Str-closure : L 1 * L 1 Other closures Difference: If L 1 nd L 2 re regulr, then L 1 - L 2 is lso regulr Proof : Set difference is defined s L 1 - L 2 = L 1 L 2 We know tht if L 2 is regulr, so is L 2. We lso know regulr lnguges re closed under intersection. Therefore, we know tht L 1 L 2 is regulr. Reversl : If L 1 is regulr, then L R is lso regulr. Proof: Suppose L is regulr lnguge. We cn therefore construct n NFA with single finl stte tht ccepts L. We cn then mke the strt stte of this NFA the finl stte, mke the finl stte the strt stte, nd reverse the direction of ll rcs in the NFA. The modified NFA ccepts string w R if nd only if the originl NFA ccepts w. Therefore the modified NFA ccepts L R. Difference sometimes notted s L 1 \ L 2 10

11 Using regulr lnguge closure properties Showing lnguge is regulr show tht y using two or more known regulr lnguges nd one or more of the opertions over which regulr lnguges re closed, you cn produce tht lnguge Lnguges known to e regulr Bsic templte L REG1 [OP] L REG2 = L REG3 Lnguge to prove regulr where OP is one of the opertions over which regulr lnguges re closed L REG3 is the lnguge in question (i.e., the one we need to prove is regulr) L REG1 nd L REG2 re known regulr lnguges If the two lnguges on the left side of the opertor re regulr then so too must e the one on the right side NB: Cnnot ssume tht if the lnguge on the right is regulr, so too must e oth lnguges on the left Exmple If L is regulr lnguge, is L 1 = {uv u L, v = 2} lso regulr? We know L is regulr Every string in L 1 consists of string from L conctented to string of length 2 The set of strings of length 2 (cll it L 2 ) over ny lphet is finite, nd therefore this is regulr lnguge since ll finite lnguges re regulr. Therefore we hve L [conctention] L 2 = L 1 [ L REG1 ] [OP] [ L REG2 ] = [ L REG3 ] Since L 1 is the conctention of two regulr lnguges, L 1 must lso e regulr Exmple Prove the lnguge { n m n,m > 3} is regulr Show tht this lnguge cn e produced using regulr lnguge closure properties on known regulr lnguges L 1 = {**}, L 2 = {,, }, L 3 = {,,} s follows: conctenttion: L 4 = L 2 L 3 complementtion: L 5 = L 4 intersection : L 6 = L 5 L 1 = { n m n,m > 3} 11

12 Using regulr lnguge closure properties Showing lnguge is not regulr Use the sme templte L REG1 [OP] L REG2 = L REG3 However: the lnguge in question is plugged into the templte in the position of L REG1 wnt to use known regulr lnguge for L REG2 If we cn show tht L REG3 is not regulr, then it must e the cse tht L REG1 is not regulr Exmple Show L = {w w in {,}* w hs equl numer of 's nd 's} is non-regulr Use the templte: L ** = { n n n 0} If oth lnguges on the left side of the = re regulr, the lnguge on the right side is regulr (closure of regulr lnguges over intersection) { n n n 0} esily proved non-regulr using the pumping lemm We know ** is regulr Therefore L must e non-regulr Exmple Given L 1 is regulr L 1 L 2 is regulr L 2 is non-regulr Is L 1 L 2 regulr? Use sme strtegy s previous exmple: Mke the unknown lnguge (L 1 L 2 ) one of the lnguges on the left side in templte Mke the other left side lnguge known regulr lnguge Show tht the lnguge on the right side is not regulr The unknown lnguge is it more complicted ecuse it is the union of two other lnguges, ut this doesn t chnge nything Fill the templte: Use one of our known RLs on left side Use known non-rl on right So we hve (L 1 L 2 ) OP [known regulr lnguge] = L 2 Need to put in n opertion nd known regulr lnguge tht we know yields L 2 To do this, get L 2 isolted from L 1 L 2 Given L 1 is regulr L 1 L 2 is regulr L 2 is non-regulr Is L 1 L 2 regulr? L 1 L 2 Σ* 12

13 Cn t extrct L 2 from L 1 L 2 using only L 1 or L 1 L 2, since tking the difference of L 1 L 2 nd L 1 gives us only wht is left of L 2 tht is not in L 1 Hve to remove nything tht is in L 1 L 2 from L 1, then sutrct the result (everything in L 1 tht is not lso in L 2 ) from L 1 L 2 difference nd union re closed for regulr lnguges fter doing this we know we still hve regulr lnguge to sutrct from L 1 L 2 Result: (L 1 L 2 ) (L 1 - (L 1 L 2 )) = L 2 Templte L REG1 is (L 1 L 2 ) [OP] is - (difference) L REG2 is (L 1 - (L 1 L 2 )) L REG3 is L 2 We know L REG2 is regulr produced y pplying the closure opertions on two known regulr lnguges (L 1 nd L 1 L 2 ) if L REG1 is regulr, so is L REG3 But we were given the fct tht L 2 is non-regulr We cn conclude tht L REG1 = L 1 L 2 is non-regulr s well Divide nd Conquer L = {w {,}* w contins n even numer of s nd n odd numer of s nd ll s come in runs of three} Regulr: L = L 1 L 2, where L 1 = {w {,}* w {,}* w contins n even numer of s nd n odd numer of s} nd L 2 = {w {,}* ll s come in runs of three} To prove it, uild n FSA for ech Esier thn FSA for the originl lnguge L 1 : L 2 : Even s Even s Even s Odd s Odd s Even s Odd s Odd s Becuse we cn uild n FSA for ech of these lnguges, they re oth regulr We get L y intersecting these two lnguges RLs re closed under intersection Therefore, L is regulr! 13

14 Wht the Closure Theorem for Union Does Not Sy Closure theorem for union sys : If L 1 nd L 2 re regulr, then L = L 1 L 2 is regulr. Wht hppens if (for exmple) L is regulr? Does tht men tht L 1 nd L 2 re lso? Mye. Exmple We know + is regulr Consider two cses for L 1 nd L = { n n > 0 nd n is prime} { n n > 0 nd n is not prime} + = L 1 L 2 Neither L 1 nor L 2 is regulr! 2. + = { n n > 0 nd n is even} { + = { n n > 0 nd n is odd} + = L 1 L 2 Both L 1 nd L 2 re regulr! Wht the Closure Theorem for Conctention Does Not Sy Closure Theorem for Conctention sys : If L 1 nd L 2 re regulr, then L = L 1 L 2 is regulr. Wht hppens (for exmple) if L 2 is not regulr? Does tht men tht L isn t regulr? Mye. Consider two exmples: 1. { n n n 0} = {} { n n n 0} L = L 1 L 2 L 2 is not regulr! 2. { * } = {*} { n n is prime} L = L 1 L 2 L 2 is not regulr, ut L is! 14

15 True or Flse? If L 1 L 2 nd L 1 is not regulr, then L 2 is not regulr. Flse! {,}* is regulr, nd it hs non-regulr suset { n n n 0} If L 1 L 2 nd L 2 is not regulr, then L 1 is not regulr. Flse! Non-regulr lnguges hve finite susets, nd finite lnguges re regulr Hints When you need known regulr lnguge, rememer tht Σ*,ε, *, **, etc. re regulr When you need known non-regulr lnguge, use n n or ny lnguge with similr dependency 15

Regular Sets and Expressions

Regular Sets and Expressions Regulr Sets nd Expressions Finite utomt re importnt in science, mthemtics, nd engineering. Engineers like them ecuse they re super models for circuits (And, since the dvent of VLSI systems sometimes finite

More information

Homework 3 Solutions

Homework 3 Solutions CS 341: Foundtions of Computer Science II Prof. Mrvin Nkym Homework 3 Solutions 1. Give NFAs with the specified numer of sttes recognizing ech of the following lnguges. In ll cses, the lphet is Σ = {,1}.

More information

One Minute To Learn Programming: Finite Automata

One Minute To Learn Programming: Finite Automata Gret Theoreticl Ides In Computer Science Steven Rudich CS 15-251 Spring 2005 Lecture 9 Fe 8 2005 Crnegie Mellon University One Minute To Lern Progrmming: Finite Automt Let me tech you progrmming lnguge

More information

Polynomial Functions. Polynomial functions in one variable can be written in expanded form as ( )

Polynomial Functions. Polynomial functions in one variable can be written in expanded form as ( ) Polynomil Functions Polynomil functions in one vrible cn be written in expnded form s n n 1 n 2 2 f x = x + x + x + + x + x+ n n 1 n 2 2 1 0 Exmples of polynomils in expnded form re nd 3 8 7 4 = 5 4 +

More information

PROF. BOYAN KOSTADINOV NEW YORK CITY COLLEGE OF TECHNOLOGY, CUNY

PROF. BOYAN KOSTADINOV NEW YORK CITY COLLEGE OF TECHNOLOGY, CUNY MAT 0630 INTERNET RESOURCES, REVIEW OF CONCEPTS AND COMMON MISTAKES PROF. BOYAN KOSTADINOV NEW YORK CITY COLLEGE OF TECHNOLOGY, CUNY Contents 1. ACT Compss Prctice Tests 1 2. Common Mistkes 2 3. Distributive

More information

Appendix D: Completing the Square and the Quadratic Formula. In Appendix A, two special cases of expanding brackets were considered:

Appendix D: Completing the Square and the Quadratic Formula. In Appendix A, two special cases of expanding brackets were considered: Appendi D: Completing the Squre nd the Qudrtic Formul Fctoring qudrtic epressions such s: + 6 + 8 ws one of the topics introduced in Appendi C. Fctoring qudrtic epressions is useful skill tht cn help you

More information

Solution to Problem Set 1

Solution to Problem Set 1 CSE 5: Introduction to the Theory o Computtion, Winter A. Hevi nd J. Mo Solution to Prolem Set Jnury, Solution to Prolem Set.4 ). L = {w w egin with nd end with }. q q q q, d). L = {w w h length t let

More information

Algebra Review. How well do you remember your algebra?

Algebra Review. How well do you remember your algebra? Algebr Review How well do you remember your lgebr? 1 The Order of Opertions Wht do we men when we write + 4? If we multiply we get 6 nd dding 4 gives 10. But, if we dd + 4 = 7 first, then multiply by then

More information

EQUATIONS OF LINES AND PLANES

EQUATIONS OF LINES AND PLANES EQUATIONS OF LINES AND PLANES MATH 195, SECTION 59 (VIPUL NAIK) Corresponding mteril in the ook: Section 12.5. Wht students should definitely get: Prmetric eqution of line given in point-direction nd twopoint

More information

Reasoning to Solve Equations and Inequalities

Reasoning to Solve Equations and Inequalities Lesson4 Resoning to Solve Equtions nd Inequlities In erlier work in this unit, you modeled situtions with severl vriles nd equtions. For exmple, suppose you were given usiness plns for concert showing

More information

MATH 150 HOMEWORK 4 SOLUTIONS

MATH 150 HOMEWORK 4 SOLUTIONS MATH 150 HOMEWORK 4 SOLUTIONS Section 1.8 Show tht the product of two of the numbers 65 1000 8 2001 + 3 177, 79 1212 9 2399 + 2 2001, nd 24 4493 5 8192 + 7 1777 is nonnegtive. Is your proof constructive

More information

Bayesian Updating with Continuous Priors Class 13, 18.05, Spring 2014 Jeremy Orloff and Jonathan Bloom

Bayesian Updating with Continuous Priors Class 13, 18.05, Spring 2014 Jeremy Orloff and Jonathan Bloom Byesin Updting with Continuous Priors Clss 3, 8.05, Spring 04 Jeremy Orloff nd Jonthn Bloom Lerning Gols. Understnd prmeterized fmily of distriutions s representing continuous rnge of hypotheses for the

More information

Section 5-4 Trigonometric Functions

Section 5-4 Trigonometric Functions 5- Trigonometric Functions Section 5- Trigonometric Functions Definition of the Trigonometric Functions Clcultor Evlution of Trigonometric Functions Definition of the Trigonometric Functions Alternte Form

More information

Math 135 Circles and Completing the Square Examples

Math 135 Circles and Completing the Square Examples Mth 135 Circles nd Completing the Squre Exmples A perfect squre is number such tht = b 2 for some rel number b. Some exmples of perfect squres re 4 = 2 2, 16 = 4 2, 169 = 13 2. We wish to hve method for

More information

Example 27.1 Draw a Venn diagram to show the relationship between counting numbers, whole numbers, integers, and rational numbers.

Example 27.1 Draw a Venn diagram to show the relationship between counting numbers, whole numbers, integers, and rational numbers. 2 Rtionl Numbers Integers such s 5 were importnt when solving the eqution x+5 = 0. In similr wy, frctions re importnt for solving equtions like 2x = 1. Wht bout equtions like 2x + 1 = 0? Equtions of this

More information

FORMAL LANGUAGES, AUTOMATA AND THEORY OF COMPUTATION EXERCISES ON REGULAR LANGUAGES

FORMAL LANGUAGES, AUTOMATA AND THEORY OF COMPUTATION EXERCISES ON REGULAR LANGUAGES FORMAL LANGUAGES, AUTOMATA AND THEORY OF COMPUTATION EXERCISES ON REGULAR LANGUAGES Introduction This compendium contins exercises out regulr lnguges for the course Forml Lnguges, Automt nd Theory of Computtion

More information

1.2 The Integers and Rational Numbers

1.2 The Integers and Rational Numbers .2. THE INTEGERS AND RATIONAL NUMBERS.2 The Integers n Rtionl Numers The elements of the set of integers: consist of three types of numers: Z {..., 5, 4, 3, 2,, 0,, 2, 3, 4, 5,...} I. The (positive) nturl

More information

Integration by Substitution

Integration by Substitution Integrtion by Substitution Dr. Philippe B. Lvl Kennesw Stte University August, 8 Abstrct This hndout contins mteril on very importnt integrtion method clled integrtion by substitution. Substitution is

More information

LINEAR TRANSFORMATIONS AND THEIR REPRESENTING MATRICES

LINEAR TRANSFORMATIONS AND THEIR REPRESENTING MATRICES LINEAR TRANSFORMATIONS AND THEIR REPRESENTING MATRICES DAVID WEBB CONTENTS Liner trnsformtions 2 The representing mtrix of liner trnsformtion 3 3 An ppliction: reflections in the plne 6 4 The lgebr of

More information

4.11 Inner Product Spaces

4.11 Inner Product Spaces 314 CHAPTER 4 Vector Spces 9. A mtrix of the form 0 0 b c 0 d 0 0 e 0 f g 0 h 0 cnnot be invertible. 10. A mtrix of the form bc d e f ghi such tht e bd = 0 cnnot be invertible. 4.11 Inner Product Spces

More information

Use Geometry Expressions to create a more complex locus of points. Find evidence for equivalence using Geometry Expressions.

Use Geometry Expressions to create a more complex locus of points. Find evidence for equivalence using Geometry Expressions. Lerning Objectives Loci nd Conics Lesson 3: The Ellipse Level: Preclculus Time required: 120 minutes In this lesson, students will generlize their knowledge of the circle to the ellipse. The prmetric nd

More information

Or more simply put, when adding or subtracting quantities, their uncertainties add.

Or more simply put, when adding or subtracting quantities, their uncertainties add. Propgtion of Uncertint through Mthemticl Opertions Since the untit of interest in n eperiment is rrel otined mesuring tht untit directl, we must understnd how error propgtes when mthemticl opertions re

More information

19. The Fermat-Euler Prime Number Theorem

19. The Fermat-Euler Prime Number Theorem 19. The Fermt-Euler Prime Number Theorem Every prime number of the form 4n 1 cn be written s sum of two squres in only one wy (side from the order of the summnds). This fmous theorem ws discovered bout

More information

Factoring Polynomials

Factoring Polynomials Fctoring Polynomils Some definitions (not necessrily ll for secondry school mthemtics): A polynomil is the sum of one or more terms, in which ech term consists of product of constnt nd one or more vribles

More information

CS99S Laboratory 2 Preparation Copyright W. J. Dally 2001 October 1, 2001

CS99S Laboratory 2 Preparation Copyright W. J. Dally 2001 October 1, 2001 CS99S Lortory 2 Preprtion Copyright W. J. Dlly 2 Octoer, 2 Ojectives:. Understnd the principle of sttic CMOS gte circuits 2. Build simple logic gtes from MOS trnsistors 3. Evlute these gtes to oserve logic

More information

Experiment 6: Friction

Experiment 6: Friction Experiment 6: Friction In previous lbs we studied Newton s lws in n idel setting, tht is, one where friction nd ir resistnce were ignored. However, from our everydy experience with motion, we know tht

More information

Example A rectangular box without lid is to be made from a square cardboard of sides 18 cm by cutting equal squares from each corner and then folding

Example A rectangular box without lid is to be made from a square cardboard of sides 18 cm by cutting equal squares from each corner and then folding 1 Exmple A rectngulr box without lid is to be mde from squre crdbord of sides 18 cm by cutting equl squres from ech corner nd then folding up the sides. 1 Exmple A rectngulr box without lid is to be mde

More information

and thus, they are similar. If k = 3 then the Jordan form of both matrices is

and thus, they are similar. If k = 3 then the Jordan form of both matrices is Homework ssignment 11 Section 7. pp. 249-25 Exercise 1. Let N 1 nd N 2 be nilpotent mtrices over the field F. Prove tht N 1 nd N 2 re similr if nd only if they hve the sme miniml polynomil. Solution: If

More information

Math 314, Homework Assignment 1. 1. Prove that two nonvertical lines are perpendicular if and only if the product of their slopes is 1.

Math 314, Homework Assignment 1. 1. Prove that two nonvertical lines are perpendicular if and only if the product of their slopes is 1. Mth 4, Homework Assignment. Prove tht two nonverticl lines re perpendiculr if nd only if the product of their slopes is. Proof. Let l nd l e nonverticl lines in R of slopes m nd m, respectively. Suppose

More information

Geometry 7-1 Geometric Mean and the Pythagorean Theorem

Geometry 7-1 Geometric Mean and the Pythagorean Theorem Geometry 7-1 Geometric Men nd the Pythgoren Theorem. Geometric Men 1. Def: The geometric men etween two positive numers nd is the positive numer x where: = x. x Ex 1: Find the geometric men etween the

More information

. At first sight a! b seems an unwieldy formula but use of the following mnemonic will possibly help. a 1 a 2 a 3 a 1 a 2

. At first sight a! b seems an unwieldy formula but use of the following mnemonic will possibly help. a 1 a 2 a 3 a 1 a 2 7 CHAPTER THREE. Cross Product Given two vectors = (,, nd = (,, in R, the cross product of nd written! is defined to e: " = (!,!,! Note! clled cross is VECTOR (unlike which is sclr. Exmple (,, " (4,5,6

More information

FAULT TREES AND RELIABILITY BLOCK DIAGRAMS. Harry G. Kwatny. Department of Mechanical Engineering & Mechanics Drexel University

FAULT TREES AND RELIABILITY BLOCK DIAGRAMS. Harry G. Kwatny. Department of Mechanical Engineering & Mechanics Drexel University SYSTEM FAULT AND Hrry G. Kwtny Deprtment of Mechnicl Engineering & Mechnics Drexel University OUTLINE SYSTEM RBD Definition RBDs nd Fult Trees System Structure Structure Functions Pths nd Cutsets Reliility

More information

Lectures 8 and 9 1 Rectangular waveguides

Lectures 8 and 9 1 Rectangular waveguides 1 Lectures 8 nd 9 1 Rectngulr wveguides y b x z Consider rectngulr wveguide with 0 < x b. There re two types of wves in hollow wveguide with only one conductor; Trnsverse electric wves

More information

Lecture 5. Inner Product

Lecture 5. Inner Product Lecture 5 Inner Product Let us strt with the following problem. Given point P R nd line L R, how cn we find the point on the line closest to P? Answer: Drw line segment from P meeting the line in right

More information

2 DIODE CLIPPING and CLAMPING CIRCUITS

2 DIODE CLIPPING and CLAMPING CIRCUITS 2 DIODE CLIPPING nd CLAMPING CIRCUITS 2.1 Ojectives Understnding the operting principle of diode clipping circuit Understnding the operting principle of clmping circuit Understnding the wveform chnge of

More information

A.7.1 Trigonometric interpretation of dot product... 324. A.7.2 Geometric interpretation of dot product... 324

A.7.1 Trigonometric interpretation of dot product... 324. A.7.2 Geometric interpretation of dot product... 324 A P P E N D I X A Vectors CONTENTS A.1 Scling vector................................................ 321 A.2 Unit or Direction vectors...................................... 321 A.3 Vector ddition.................................................

More information

Binary Representation of Numbers Autar Kaw

Binary Representation of Numbers Autar Kaw Binry Representtion of Numbers Autr Kw After reding this chpter, you should be ble to: 1. convert bse- rel number to its binry representtion,. convert binry number to n equivlent bse- number. In everydy

More information

9 CONTINUOUS DISTRIBUTIONS

9 CONTINUOUS DISTRIBUTIONS 9 CONTINUOUS DISTIBUTIONS A rndom vrible whose vlue my fll nywhere in rnge of vlues is continuous rndom vrible nd will be ssocited with some continuous distribution. Continuous distributions re to discrete

More information

Multiplication and Division - Left to Right. Addition and Subtraction - Left to Right.

Multiplication and Division - Left to Right. Addition and Subtraction - Left to Right. Order of Opertions r of Opertions Alger P lese Prenthesis - Do ll grouped opertions first. E cuse Eponents - Second M D er Multipliction nd Division - Left to Right. A unt S hniqu Addition nd Sutrction

More information

Words Symbols Diagram. abcde. a + b + c + d + e

Words Symbols Diagram. abcde. a + b + c + d + e Logi Gtes nd Properties We will e using logil opertions to uild mhines tht n do rithmeti lultions. It s useful to think of these opertions s si omponents tht n e hooked together into omplex networks. To

More information

Vectors 2. 1. Recap of vectors

Vectors 2. 1. Recap of vectors Vectors 2. Recp of vectors Vectors re directed line segments - they cn be represented in component form or by direction nd mgnitude. We cn use trigonometry nd Pythgors theorem to switch between the forms

More information

Operations with Polynomials

Operations with Polynomials 38 Chpter P Prerequisites P.4 Opertions with Polynomils Wht you should lern: Write polynomils in stndrd form nd identify the leding coefficients nd degrees of polynomils Add nd subtrct polynomils Multiply

More information

FUNCTIONS AND EQUATIONS. xεs. The simplest way to represent a set is by listing its members. We use the notation

FUNCTIONS AND EQUATIONS. xεs. The simplest way to represent a set is by listing its members. We use the notation FUNCTIONS AND EQUATIONS. SETS AND SUBSETS.. Definition of set. A set is ny collection of objects which re clled its elements. If x is n element of the set S, we sy tht x belongs to S nd write If y does

More information

0.1 Basic Set Theory and Interval Notation

0.1 Basic Set Theory and Interval Notation 0.1 Bsic Set Theory nd Intervl Nottion 3 0.1 Bsic Set Theory nd Intervl Nottion 0.1.1 Some Bsic Set Theory Notions Like ll good Mth ooks, we egin with definition. Definition 0.1. A set is well-defined

More information

Integration. 148 Chapter 7 Integration

Integration. 148 Chapter 7 Integration 48 Chpter 7 Integrtion 7 Integrtion t ech, by supposing tht during ech tenth of second the object is going t constnt speed Since the object initilly hs speed, we gin suppose it mintins this speed, but

More information

Review guide for the final exam in Math 233

Review guide for the final exam in Math 233 Review guide for the finl exm in Mth 33 1 Bsic mteril. This review includes the reminder of the mteril for mth 33. The finl exm will be cumultive exm with mny of the problems coming from the mteril covered

More information

P.3 Polynomials and Factoring. P.3 an 1. Polynomial STUDY TIP. Example 1 Writing Polynomials in Standard Form. What you should learn

P.3 Polynomials and Factoring. P.3 an 1. Polynomial STUDY TIP. Example 1 Writing Polynomials in Standard Form. What you should learn 33337_0P03.qp 2/27/06 24 9:3 AM Chpter P Pge 24 Prerequisites P.3 Polynomils nd Fctoring Wht you should lern Polynomils An lgeric epression is collection of vriles nd rel numers. The most common type of

More information

6.2 Volumes of Revolution: The Disk Method

6.2 Volumes of Revolution: The Disk Method mth ppliction: volumes of revolution, prt ii Volumes of Revolution: The Disk Method One of the simplest pplictions of integrtion (Theorem ) nd the ccumultion process is to determine so-clled volumes of

More information

Regular Languages and Finite Automata

Regular Languages and Finite Automata N Lecture Notes on Regulr Lnguges nd Finite Automt for Prt IA of the Computer Science Tripos Mrcelo Fiore Cmbridge University Computer Lbortory First Edition 1998. Revised 1999, 2000, 2001, 2002, 2003,

More information

The remaining two sides of the right triangle are called the legs of the right triangle.

The remaining two sides of the right triangle are called the legs of the right triangle. 10 MODULE 6. RADICAL EXPRESSIONS 6 Pythgoren Theorem The Pythgoren Theorem An ngle tht mesures 90 degrees is lled right ngle. If one of the ngles of tringle is right ngle, then the tringle is lled right

More information

Solving BAMO Problems

Solving BAMO Problems Solving BAMO Problems Tom Dvis tomrdvis@erthlink.net http://www.geometer.org/mthcircles Februry 20, 2000 Abstrct Strtegies for solving problems in the BAMO contest (the By Are Mthemticl Olympid). Only

More information

flex Regular Expressions and Lexical Scanning Regular Expressions and flex Examples on Alphabet A = {a,b} (Standard) Regular Expressions on Alphabet A

flex Regular Expressions and Lexical Scanning Regular Expressions and flex Examples on Alphabet A = {a,b} (Standard) Regular Expressions on Alphabet A flex Regulr Expressions nd Lexicl Scnning Using flex to Build Scnner flex genertes lexicl scnners: progrms tht discover tokens. Tokens re the smllest meningful units of progrm (or other string). flex is

More information

Unit 6: Exponents and Radicals

Unit 6: Exponents and Radicals Eponents nd Rdicls -: The Rel Numer Sstem Unit : Eponents nd Rdicls Pure Mth 0 Notes Nturl Numers (N): - counting numers. {,,,,, } Whole Numers (W): - counting numers with 0. {0,,,,,, } Integers (I): -

More information

5.2. LINE INTEGRALS 265. Let us quickly review the kind of integrals we have studied so far before we introduce a new one.

5.2. LINE INTEGRALS 265. Let us quickly review the kind of integrals we have studied so far before we introduce a new one. 5.2. LINE INTEGRALS 265 5.2 Line Integrls 5.2.1 Introduction Let us quickly review the kind of integrls we hve studied so fr before we introduce new one. 1. Definite integrl. Given continuous rel-vlued

More information

Pentominoes. Pentominoes. Bruce Baguley Cascade Math Systems, LLC. The pentominoes are a simple-looking set of objects through which some powerful

Pentominoes. Pentominoes. Bruce Baguley Cascade Math Systems, LLC. The pentominoes are a simple-looking set of objects through which some powerful Pentominoes Bruce Bguley Cscde Mth Systems, LLC Astrct. Pentominoes nd their reltives the polyominoes, polycues, nd polyhypercues will e used to explore nd pply vrious importnt mthemticl concepts. In this

More information

MA 15800 Lesson 16 Notes Summer 2016 Properties of Logarithms. Remember: A logarithm is an exponent! It behaves like an exponent!

MA 15800 Lesson 16 Notes Summer 2016 Properties of Logarithms. Remember: A logarithm is an exponent! It behaves like an exponent! MA 5800 Lesson 6 otes Summer 06 Rememer: A logrithm is n eponent! It ehves like n eponent! In the lst lesson, we discussed four properties of logrithms. ) log 0 ) log ) log log 4) This lesson covers more

More information

Basic Analysis of Autarky and Free Trade Models

Basic Analysis of Autarky and Free Trade Models Bsic Anlysis of Autrky nd Free Trde Models AUTARKY Autrky condition in prticulr commodity mrket refers to sitution in which country does not engge in ny trde in tht commodity with other countries. Consequently

More information

5.6 POSITIVE INTEGRAL EXPONENTS

5.6 POSITIVE INTEGRAL EXPONENTS 54 (5 ) Chpter 5 Polynoils nd Eponents 5.6 POSITIVE INTEGRAL EXPONENTS In this section The product rule for positive integrl eponents ws presented in Section 5., nd the quotient rule ws presented in Section

More information

SPECIAL PRODUCTS AND FACTORIZATION

SPECIAL PRODUCTS AND FACTORIZATION MODULE - Specil Products nd Fctoriztion 4 SPECIAL PRODUCTS AND FACTORIZATION In n erlier lesson you hve lernt multipliction of lgebric epressions, prticulrly polynomils. In the study of lgebr, we come

More information

Repeated multiplication is represented using exponential notation, for example:

Repeated multiplication is represented using exponential notation, for example: Appedix A: The Lws of Expoets Expoets re short-hd ottio used to represet my fctors multiplied together All of the rules for mipultig expoets my be deduced from the lws of multiplictio d divisio tht you

More information

Physics 43 Homework Set 9 Chapter 40 Key

Physics 43 Homework Set 9 Chapter 40 Key Physics 43 Homework Set 9 Chpter 4 Key. The wve function for n electron tht is confined to x nm is. Find the normliztion constnt. b. Wht is the probbility of finding the electron in. nm-wide region t x

More information

Answer, Key Homework 10 David McIntyre 1

Answer, Key Homework 10 David McIntyre 1 Answer, Key Homework 10 Dvid McIntyre 1 This print-out should hve 22 questions, check tht it is complete. Multiple-choice questions my continue on the next column or pge: find ll choices efore mking your

More information

MODULE 3. 0, y = 0 for all y

MODULE 3. 0, y = 0 for all y Topics: Inner products MOULE 3 The inner product of two vectors: The inner product of two vectors x, y V, denoted by x, y is (in generl) complex vlued function which hs the following four properties: i)

More information

DlNBVRGH + Sickness Absence Monitoring Report. Executive of the Council. Purpose of report

DlNBVRGH + Sickness Absence Monitoring Report. Executive of the Council. Purpose of report DlNBVRGH + + THE CITY OF EDINBURGH COUNCIL Sickness Absence Monitoring Report Executive of the Council 8fh My 4 I.I...3 Purpose of report This report quntifies the mount of working time lost s result of

More information

9.3. The Scalar Product. Introduction. Prerequisites. Learning Outcomes

9.3. The Scalar Product. Introduction. Prerequisites. Learning Outcomes The Sclr Product 9.3 Introduction There re two kinds of multipliction involving vectors. The first is known s the sclr product or dot product. This is so-clled becuse when the sclr product of two vectors

More information

Section 7-4 Translation of Axes

Section 7-4 Translation of Axes 62 7 ADDITIONAL TOPICS IN ANALYTIC GEOMETRY Section 7-4 Trnsltion of Aes Trnsltion of Aes Stndrd Equtions of Trnslted Conics Grphing Equtions of the Form A 2 C 2 D E F 0 Finding Equtions of Conics In the

More information

Unambiguous Recognizable Two-dimensional Languages

Unambiguous Recognizable Two-dimensional Languages Unmbiguous Recognizble Two-dimensionl Lnguges Mrcell Anselmo, Dor Gimmrresi, Mri Mdoni, Antonio Restivo (Univ. of Slerno, Univ. Rom Tor Vergt, Univ. of Ctni, Univ. of Plermo) W2DL, My 26 REC fmily I REC

More information

Basic Research in Computer Science BRICS RS-02-13 Brodal et al.: Solving the String Statistics Problem in Time O(n log n)

Basic Research in Computer Science BRICS RS-02-13 Brodal et al.: Solving the String Statistics Problem in Time O(n log n) BRICS Bsic Reserch in Computer Science BRICS RS-02-13 Brodl et l.: Solving the String Sttistics Prolem in Time O(n log n) Solving the String Sttistics Prolem in Time O(n log n) Gerth Stølting Brodl Rune

More information

Mathematics. Vectors. hsn.uk.net. Higher. Contents. Vectors 128 HSN23100

Mathematics. Vectors. hsn.uk.net. Higher. Contents. Vectors 128 HSN23100 hsn.uk.net Higher Mthemtics UNIT 3 OUTCOME 1 Vectors Contents Vectors 18 1 Vectors nd Sclrs 18 Components 18 3 Mgnitude 130 4 Equl Vectors 131 5 Addition nd Subtrction of Vectors 13 6 Multipliction by

More information

Morgan Stanley Ad Hoc Reporting Guide

Morgan Stanley Ad Hoc Reporting Guide spphire user guide Ferury 2015 Morgn Stnley Ad Hoc Reporting Guide An Overview For Spphire Users 1 Introduction The Ad Hoc Reporting tool is ville for your reporting needs outside of the Spphire stndrd

More information

RIGHT TRIANGLES AND THE PYTHAGOREAN TRIPLETS

RIGHT TRIANGLES AND THE PYTHAGOREAN TRIPLETS RIGHT TRIANGLES AND THE PYTHAGOREAN TRIPLETS Known for over 500 yers is the fct tht the sum of the squres of the legs of right tringle equls the squre of the hypotenuse. Tht is +b c. A simple proof is

More information

2005-06 Second Term MAT2060B 1. Supplementary Notes 3 Interchange of Differentiation and Integration

2005-06 Second Term MAT2060B 1. Supplementary Notes 3 Interchange of Differentiation and Integration Source: http://www.mth.cuhk.edu.hk/~mt26/mt26b/notes/notes3.pdf 25-6 Second Term MAT26B 1 Supplementry Notes 3 Interchnge of Differentition nd Integrtion The theme of this course is bout vrious limiting

More information

CHAPTER 11 Numerical Differentiation and Integration

CHAPTER 11 Numerical Differentiation and Integration CHAPTER 11 Numericl Differentition nd Integrtion Differentition nd integrtion re bsic mthemticl opertions with wide rnge of pplictions in mny res of science. It is therefore importnt to hve good methods

More information

Econ 4721 Money and Banking Problem Set 2 Answer Key

Econ 4721 Money and Banking Problem Set 2 Answer Key Econ 472 Money nd Bnking Problem Set 2 Answer Key Problem (35 points) Consider n overlpping genertions model in which consumers live for two periods. The number of people born in ech genertion grows in

More information

5 a LAN 6 a gateway 7 a modem

5 a LAN 6 a gateway 7 a modem STARTER With the help of this digrm, try to descrie the function of these components of typicl network system: 1 file server 2 ridge 3 router 4 ckone 5 LAN 6 gtewy 7 modem Another Novell LAN Router Internet

More information

Treatment Spring Late Summer Fall 0.10 5.56 3.85 0.61 6.97 3.01 1.91 3.01 2.13 2.99 5.33 2.50 1.06 3.53 6.10 Mean = 1.33 Mean = 4.88 Mean = 3.

Treatment Spring Late Summer Fall 0.10 5.56 3.85 0.61 6.97 3.01 1.91 3.01 2.13 2.99 5.33 2.50 1.06 3.53 6.10 Mean = 1.33 Mean = 4.88 Mean = 3. The nlysis of vrince (ANOVA) Although the t-test is one of the most commonly used sttisticl hypothesis tests, it hs limittions. The mjor limittion is tht the t-test cn be used to compre the mens of only

More information

1 Fractions from an advanced point of view

1 Fractions from an advanced point of view 1 Frtions from n vne point of view We re going to stuy frtions from the viewpoint of moern lger, or strt lger. Our gol is to evelop eeper unerstning of wht n men. One onsequene of our eeper unerstning

More information

Chapter. Contents: A Constructing decimal numbers

Chapter. Contents: A Constructing decimal numbers Chpter 9 Deimls Contents: A Construting deiml numers B Representing deiml numers C Deiml urreny D Using numer line E Ordering deimls F Rounding deiml numers G Converting deimls to frtions H Converting

More information

Small Business Networking

Small Business Networking Why network is n essentil productivity tool for ny smll business Effective technology is essentil for smll businesses looking to increse the productivity of their people nd business. Introducing technology

More information

Firm Objectives. The Theory of the Firm II. Cost Minimization Mathematical Approach. First order conditions. Cost Minimization Graphical Approach

Firm Objectives. The Theory of the Firm II. Cost Minimization Mathematical Approach. First order conditions. Cost Minimization Graphical Approach Pro. Jy Bhttchry Spring 200 The Theory o the Firm II st lecture we covered: production unctions Tody: Cost minimiztion Firm s supply under cost minimiztion Short vs. long run cost curves Firm Ojectives

More information

Small Business Networking

Small Business Networking Why network is n essentil productivity tool for ny smll business Effective technology is essentil for smll businesses looking to increse the productivity of their people nd business. Introducing technology

More information

Graphs on Logarithmic and Semilogarithmic Paper

Graphs on Logarithmic and Semilogarithmic Paper 0CH_PHClter_TMSETE_ 3//00 :3 PM Pge Grphs on Logrithmic nd Semilogrithmic Pper OBJECTIVES When ou hve completed this chpter, ou should be ble to: Mke grphs on logrithmic nd semilogrithmic pper. Grph empiricl

More information

All pay auctions with certain and uncertain prizes a comment

All pay auctions with certain and uncertain prizes a comment CENTER FOR RESEARC IN ECONOMICS AND MANAGEMENT CREAM Publiction No. 1-2015 All py uctions with certin nd uncertin prizes comment Christin Riis All py uctions with certin nd uncertin prizes comment Christin

More information

PHY 140A: Solid State Physics. Solution to Homework #2

PHY 140A: Solid State Physics. Solution to Homework #2 PHY 140A: Solid Stte Physics Solution to Homework # TA: Xun Ji 1 October 14, 006 1 Emil: jixun@physics.ucl.edu Problem #1 Prove tht the reciprocl lttice for the reciprocl lttice is the originl lttice.

More information

Small Business Cloud Services

Small Business Cloud Services Smll Business Cloud Services Summry. We re thick in the midst of historic se-chnge in computing. Like the emergence of personl computers, grphicl user interfces, nd mobile devices, the cloud is lredy profoundly

More information

Babylonian Method of Computing the Square Root: Justifications Based on Fuzzy Techniques and on Computational Complexity

Babylonian Method of Computing the Square Root: Justifications Based on Fuzzy Techniques and on Computational Complexity Bbylonin Method of Computing the Squre Root: Justifictions Bsed on Fuzzy Techniques nd on Computtionl Complexity Olg Koshelev Deprtment of Mthemtics Eduction University of Texs t El Pso 500 W. University

More information

Angles 2.1. Exercise 2.1... Find the size of the lettered angles. Give reasons for your answers. a) b) c) Example

Angles 2.1. Exercise 2.1... Find the size of the lettered angles. Give reasons for your answers. a) b) c) Example 2.1 Angles Reognise lternte n orresponing ngles Key wors prllel lternte orresponing vertilly opposite Rememer, prllel lines re stright lines whih never meet or ross. The rrows show tht the lines re prllel

More information

AA1H Calculus Notes Math1115, Honours 1 1998. John Hutchinson

AA1H Calculus Notes Math1115, Honours 1 1998. John Hutchinson AA1H Clculus Notes Mth1115, Honours 1 1998 John Hutchinson Author ddress: Deprtment of Mthemtics, School of Mthemticl Sciences, Austrlin Ntionl University E-mil ddress: John.Hutchinson@nu.edu.u Contents

More information

Regular Repair of Specifications

Regular Repair of Specifications Regulr Repir of Specifictions Michel Benedikt Oxford University michel.enedikt@coml.ox.c.uk Griele Puppis Oxford University griele.puppis@coml.ox.c.uk Cristin Riveros Oxford University cristin.riveros@coml.ox.c.uk

More information

Welch Allyn CardioPerfect Workstation Installation Guide

Welch Allyn CardioPerfect Workstation Installation Guide Welch Allyn CrdioPerfect Worksttion Instlltion Guide INSTALLING CARDIOPERFECT WORKSTATION SOFTWARE & ACCESSORIES ON A SINGLE PC For softwre version 1.6.5 or lter For network instlltion, plese refer to

More information

baby on the way, quit today

baby on the way, quit today for mums-to-be bby on the wy, quit tody WHAT YOU NEED TO KNOW bout smoking nd pregnncy uitting smoking is the best thing you cn do for your bby We know tht it cn be difficult to quit smoking. But we lso

More information

Rotating DC Motors Part II

Rotating DC Motors Part II Rotting Motors rt II II.1 Motor Equivlent Circuit The next step in our consiertion of motors is to evelop n equivlent circuit which cn be use to better unerstn motor opertion. The rmtures in rel motors

More information

Pure C4. Revision Notes

Pure C4. Revision Notes Pure C4 Revision Notes Mrch 0 Contents Core 4 Alger Prtil frctions Coordinte Geometry 5 Prmetric equtions 5 Conversion from prmetric to Crtesin form 6 Are under curve given prmetriclly 7 Sequences nd

More information

COMPONENTS: COMBINED LOADING

COMPONENTS: COMBINED LOADING LECTURE COMPONENTS: COMBINED LOADING Third Edition A. J. Clrk School of Engineering Deprtment of Civil nd Environmentl Engineering 24 Chpter 8.4 by Dr. Ibrhim A. Asskkf SPRING 2003 ENES 220 Mechnics of

More information

DATABASDESIGN FÖR INGENJÖRER - 1056F

DATABASDESIGN FÖR INGENJÖRER - 1056F DATABASDESIGN FÖR INGENJÖRER - 06F Sommr 00 En introuktionskurs i tssystem http://user.it.uu.se/~ul/t-sommr0/ lt. http://www.it.uu.se/eu/course/homepge/esign/st0/ Kjell Orsorn (Rusln Fomkin) Uppsl Dtse

More information

6 Energy Methods And The Energy of Waves MATH 22C

6 Energy Methods And The Energy of Waves MATH 22C 6 Energy Methods And The Energy of Wves MATH 22C. Conservtion of Energy We discuss the principle of conservtion of energy for ODE s, derive the energy ssocited with the hrmonic oscilltor, nd then use this

More information

1.00/1.001 Introduction to Computers and Engineering Problem Solving Fall 2011 - Final Exam

1.00/1.001 Introduction to Computers and Engineering Problem Solving Fall 2011 - Final Exam 1./1.1 Introduction to Computers nd Engineering Problem Solving Fll 211 - Finl Exm Nme: MIT Emil: TA: Section: You hve 3 hours to complete this exm. In ll questions, you should ssume tht ll necessry pckges

More information

Small Business Networking

Small Business Networking Why network is n essentil productivity tool for ny smll business Effective technology is essentil for smll businesses looking to increse the productivity of their people nd processes. Introducing technology

More information

CURVES ANDRÉ NEVES. that is, the curve α has finite length. v = p q p q. a i.e., the curve of smallest length connecting p to q is a straight line.

CURVES ANDRÉ NEVES. that is, the curve α has finite length. v = p q p q. a i.e., the curve of smallest length connecting p to q is a straight line. CURVES ANDRÉ NEVES 1. Problems (1) (Ex 1 of 1.3 of Do Crmo) Show tht the tngent line to the curve α(t) (3t, 3t 2, 2t 3 ) mkes constnt ngle with the line z x, y. (2) (Ex 6 of 1.3 of Do Crmo) Let α(t) (e

More information