Plans. Memoryless plans Definition. Memoryless plans Example. Images Formal definition. Images. Preimages. Preimages. Definition

Size: px
Start display at page:

Download "Plans. Memoryless plans Definition. Memoryless plans Example. Images Formal definition. Images. Preimages. Preimages. Definition"

Transcription

1 Noetermnstc plannng (May 25, 2005) Plans AND-OR search Dynamc programmng (Albert-Ludwgs-Unverstät Freburg) 1 / 56 Plans Plans 1. map a state/an observaton to an operator. We use ths defnton of plans for fully observable problems only. 2. Cotonal plans generalze memoryless plans. They are needed for problems wthout full observablty. The state of the executon of a cotonal plan depes on observatons on earler executon steps. The state of the executon = a prmtve form of memory. The operator to be executed depes on the state of the executon. (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 Let S be the set of all states. A memoryless plan s a partal functon π : S O. Executon of a memoryless plan 1. Determne the current state s (full observablty!!!). 2. If π(s) s not defned then termnate executon. If the objectve s to reach a goal state, then π(s) s not defned f s s a goal state so that the executon termnates. 3. Execute acton π(s). 4. Goto step 1. (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 Formal defnton Image The mage of a set T of states wth respect to an operator o s the set of those states that can be reached by executng o n a state n T. T mg o (T ) (Image of a state) mg o (s) = {s S sos } (Image of a set of states) mg o (T ) = s T mg o(s) (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 Weak premage The premage of a set T of states wth respect to an operator o s the set of those states from whch a state n T can be reached by executng o. premg o (T ) T Formal defnton (Weak premage of a state) premg o (s ) = {s S sos } (Weak premage of a set of states) premg o (T ) = s T premg o(s). (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56

2 Strong premage The strong premage of a set T of states wth respect to an operator o s the set of those states from whch a state n T s always reached when executng o. Formal defnton spremg o (T ) T (Strong premage of a set of states) spremg o (T ) = {s S s T, sos, mg o (s) T } (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 AND-OR search for fully observable problems AND-OR search 1. Heurstc search (forward) Noetermnstc plannng can be vewed as AND-OR search. OR nodes: Choce between operators AND nodes: Noetermnstcally reached state Heurstc AND-OR search algorthms: AO*, Dynamc programmng (backward) Idea Compute operator/dstance/value for a state based on the operators/dstances/values of ts all successor states actons needed for goal states. 2.2 If states wth actons to goals are known, states wth + 1 actons to goals can be easly dentfed. Automatc reuse of already fou plan suffxes. OR s 1 s 2 s 3 s 4 OR OR OR OR s 5 s 6 s 7 s 8 s 9 s 10 s 11 s 12 s 13 s 14 s 15 s 16 s 17 s 18 s 19 s 20 (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 Dynamc programmng Dynamc programmng Dynamc programmng Plannng by dynamc programmng If for all successors of state s wth respect to operator o a plan exsts, assgn operator o to s. Base case = 0: In goal states there s nothng to do. Iuctve case 1: If there s o O such that for all s mg o (s) s s a goal state or π(s ) was assgned on teraton 1, then assgn π(s) = o. dstance to G G Connecton to dstances If s s assgned a value on teraton 1, then the backward dstance of s s. The dynamc programmng algorthm essentally computes the backward dstances of states. (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 of dstance sets Let G be a set of states a O a set of operators. Defne the backward dstance sets D bwd for G, O that consst of those states for whch there s a guarantee of reachng a state n G wth at most operator applcatons. D bwd D bwd 0 = G = D 1 bwd spremg o(d 1 bwd ) for all 1 Let G be as set of states a O a set of operators, a let D0 bwd, D1 bwd,... be the backward dstance sets for G a O. Then the backward dstance from a state s to G s If s D bwd δ bwd G { 0 f s G (s) = f s D bwd for all 0 then δg bwd (s) =. \D 1 bwd (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56

3 Constructon of a plan based on dstances Makng the algorthm a logc-based algorthm Extracton of a plan from dstance sets 1. Let S S be those states havng a fnte backward dstance. 2. Let s be a state wth dstance = δg bwd (s) Assgn to π(s) any operator o O such that mg o (s) D 1 bwd. Hence o decreases the backward dstance by at least one. The plan π solves the plannng problem for S, I, O, G, P ff I S. An algorthm that represents the states explctly s feasble for transton systems wth at most 10 6 or 10 7 states. For plannng wth bgger transton systems structural propertes of the transton system have to be taken advantage of. Representng state sets as propostonal formulae often allow takng advantage of the structural propertes: a formula that represents a set of states or a transton relaton that has certan regulartes may be very small n comparson to the set or relaton. (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 Makng the algorthm a logc-based algorthm for noetermnstc operators We use a formula φ as a data structure for representng the set {s S s = φ}. We show that regresson regr o (φ) for noetermnstc operators s one way of computng strong premages. We present general technques for computng mages, premages a strong premages of sets of states represented as formulae. Many of the algorthms presented later n the lecture can be lfted to use a logc-based representaton, thereby expang ther range of applcablty to much bgger transton systems. We can easly generalze our regresson operaton for determnstc operators to regresson for noetermnstc operators of a restrcted syntactc form. ( for noetermnstc operators) Let φ be a propostonal formula a o = c, e 1 e n an operator where e 1,..., e n are determnstc. Defne regr o (φ) = regr c,e1 (φ) regr c,en (φ). (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 for noetermnstc operators Illustraton for noetermnstc operators Correctness regr c,(e1 e 2) (φ) = regr c,e1 (φ) regr c,e2 (φ) regr c,e2 (φ) regr c,e1 (φ) φ Let φ be a formula over A, o an operator over A, a S the set of all states over A. Then {s S s = regr o (φ)} = spremg o ({s S s = φ}). Let o = c, (e 1 e n ). {s S s = regr o (φ)} = {s S s = regr c,e1 (φ) regr c,en (φ)} = {s S s = regr c,e1 (φ),..., s = regr c,en (φ)} = {s S app c,e1 (s) = φ,..., app c,en (s) = φ} = {s S s = φ for all s mg o (s), there s s = φ wth sos } = spremg o ({s S s = φ}) 3rd = s by propertes of determnstc regresson. 4th = s by mg o (s) = {app c,e1 (s),..., app c,en (s)}. (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 for noetermnstc operators wth formulas Let o = d, (b c). Then regr o (b c) = regr d,b (b c) regr d, c (b c) = (d ( c)) (d (b )) d c b. By usng regresson we can compute formulas that represent backward dstance sets. Let G be a formula a O a set of operators. The backward dstance sets D bwd for G, O are represented by the followng formulae. D bwd D bwd 0 = G = D bwd 1 regr o (D 1 bwd ) for all 1 (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56

4 wth formulas General mages a premages wth formulas Let G be a formula a O a set of operators, a let D0 bwd, D1 bwd,... be the formulae representng the backward dstance sets for G a O. Then the backward dstance from a state s to G s If s = D bwd δ bwd G { 0 f s = G (s) = f s = D bwd for all 0 then δg bwd (s) =. D bwd 1 The defnton of regresson covers only a subclass of noetermnstc operators. How to defne strong premages for all operators, a mages a premages? Now we apply a general dea: 1. Vew operators/actons as bnary relatons. 2. Represent these bnary relatons as formulae. 3. Defne relatonal operatons for relatons represented as formulae. (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 General mages a premages wth formulas General mages a premages wth formulas Defne the set of state varables possbly changed by e as changes(a) = {a} changes( a) = {a} changes(c e) = changes(e) changes(e 1 e n ) = changes(e 1 ) changes(e n ) changes(e 1 e n ) = changes(e 1 ) changes(e n ) Assumpton Let e 1 e n occur n the effect of an operator. If e 1,..., e n are not all determnstc then a a a may occur as an atomc effect n at most one of e 1,..., e n. Ths assumpton rules out effects lke (a b) ( a c) that may make a smultaneously true a false. In noetermnstc choces e 1 e n the formula for each e has to express the changes for exactly the same set B of state varables. τ B (e) = τ B(e) when e s determnstc τ B (e 1 e n ) = τ B (e 1) τ B (e n) τ B (e 1 e n ) = τ B\(B2 Bn) (e 1) τ (e B2 2) τ (e Bn n) where B = changes(e ) for {2,..., n} (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 General mages a premages wth formulas General mages a premages wth formulas We translate the effect e = (a (d a)) (c d) nto a propostonal formula. The set of state varables s A = {a, b, c, d}. τ{a,b,c,d} (e) = τ {a,b}(a (d a)) τ (a) τ = (τ {a,b} {a,b} {c,d} (c d) (d a)) (τ {c,d} (c) τ {c,d} (d)) = ((a (b b )) (((a d) a ) (b b ))) ((c (d d )) ((c c ) d )) Let A be a set of state varables. Let o = c, e be an operator over A n normal form. Defne τa (o) = c τ A (e). Lemma Let o be an operator. Then {v v s a valuaton of A A, v = τ } = {s s [A /A] s, s S, s mg o (s)}. (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 Exstental a unversal abstracton The most mportant operatons performed on transton relatons represented as propostonal formulae are based on exstental abstracton a unversal abstracton. Exstental abstracton of a formula φ wth respect to a A: a.φ = φ[ /a] φ[ /a]. Unversal abstracton s defned analogously by usng conjuncton nstead of dsjuncton. Unversal abstracton of a formula φ wth respect to a A: a.φ = φ[ /a] φ[ /a]. -abstracton s b.((a b) (b c)) = ((a ) ( c)) ((a ) ( c)) c a a c ab.(a b) = b.( b) ( b) = (( ) ( )) (( ) ( )) = ( ) ( ) = -abstracton s also known as forgettng: mon tue((mon tue) (mon work) (tue work)) tue((work (tue work)) (tue (tue work))) work (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56

5 a -abstracton n terms of truth-tables Propertes of abstracton operatons a a a correspo to combnng pars of lnes wth the same valuaton for varables other than a. a b c a (b c) c.(a (b c)) a b a b c.(a (b c)) c.(a (b c)) a a b c.(a (b c)) (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 Exstental a unversal abstracton of φ wth respect to a set of atomc propostons B = {b 1,..., b n } are B.φ = b 1.( b 2.(... b n.φ...)) B.φ = b 1.( b 2.(... b n.φ...)). (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 Propertes of abstracted formulas Propertes of a abstracton 1. Let φ be a formula over A. Then A.φ a A.φ are formulae that consst of the constants a a the logcal connectves only. 2. The truth-values of these formulae are epeent of the valuaton of A, that s, ther values are the same for all valuatons. 3. A.φ f a only f φ s satsfable. 4. A.φ f a only f φ s vald. Lemma If φ s a formula over A A a v a valuaton of A then 1. v = A.φ ff v v = φ for some valuaton v of A. 2. v = A.φ ff v v = φ for all valuatons v of A. (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 Sze of abstracted formulae Abstractng one varable takes polynomal tme n the sze of the formula. Abstractng one varable may double the formula sze. Abstractng n varables may ncrease sze by factor 2 n. For makng abstracton practcal the formulae must be smplfed, for example wth equvalences lke φ φ, φ, φ, φ φ,, a. by -abstracton Let A = {a 1,..., a n }, A = {a 1,..., a n}, φ 1 be a formula on A representng a row vector V 1 2 n (equvalently, a set of valuatons of A), a φ 2 a formula on A A representng a matrx M 2 n 2 n (equvalently, a bnary relaton on valuatons of A). The product matrx V M of sze 1 2 n s represented by A.(φ 1 φ 2 ) whch s a formula on A. To obtan a formula over A we have to rename the varables. ( A.(φ 1 φ 2 ))[A/A ] (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 by -abstracton Matrx multplcaton by -abstracton Let A = {a, b} be the state varables ( ) = ( ) represents the mage of {00, 10} wth respect to a relaton. a. b.( b (b b )) b.( b (b b )) ( ( b )) ( ( b )) b The formula b represents {01, 11}. (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 Let A = {a 1,..., a n }, A = {a 1,..., a n}, A = {a 1,..., a n}, φ 1 be a formula on A A representng matrx M 1 a φ 2 a formula on A A representng matrx M 2. The matrces M 1 a M 2 have sze 2 n 2 n. The product matrx M 1 M 2 s represented by whch s a formula on A A. A.(φ 1 φ 2 ) (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56

6 Matrx multplcaton by -abstracton Matrx multplcaton Let φ 1 = a a a φ 2 = a a represent two actons, reversng the truth-value of a a dong nothng. The sequental composton of these actons s a.φ 1 φ 2 = ((a ) ( a )) ((a ) ( a )) ((a ) ( a )) ((a ) ( a )) ( a a ) (a a ) a a. Multply ( a a ) ( b b ) a (a b ) (b a ): Ths s = a. b.( a a ) ( b b ) (a b ) (b a ) ( a b ) ( b a ). (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 a premages by formula manpulaton by formula manpulaton Defne s[a /A] = { a, s(a) a A}. Lemma Let φ be a formula on A a v a valuaton of A. Then v = φ ff v[a /A] = φ[a /A]. Let o be an operator a φ a formula. Defne mg o (φ) = ( A.(φ τa (o)))[a/a ] premg o (φ) = A.(τA (o) φ[a /A]) spremg o (φ) = A.(τA (o) φ[a /A]) A.τA (o). Let T = {s S s = φ}. Then {s S s = mg o (φ)} = {s S s = ( A.(φ τ ))[A/A ]} = mg o (T ). s = ( A.(φ τ ))[A/A ] ff s [A /A] = A.(φ τ ) ff there s valuaton s of A s.t. (s s [A /A]) = φ τ ff there s valuaton s of A s.t. s = φ a (s s [A /A]) = τ ff there s s T s.t. (s s [A /A]) = τ ff there s s T s.t. s mg o (s) ff s mg o (T ). (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 by formula manpulaton by formula manpulaton Let T = {s S s = φ}. Then {s S s = premg o (φ)} = {s S s = A.(τ φ[a /A])} = premg o (T ). s = A.(τ φ[a /A]) ff there s s 0 : A {0, 1} s.t. (s s 0 ) = τ φ[a /A] ff there s s 0 : A {0, 1} s.t. s 0 = φ[a /A] a (s s 0 ) = τ ff there s s : A {0, 1} s.t. s = φ a (s s 0 ) = τ ff there s s T s.t. (s s [A /A]) = τ ff there s s T s.t. s mg o (s) ff there s s T s.t. s premg o (s ) ff s premg o (T ). Above we defne s = s 0 [A/A ] (a hence s 0 = s [A /A].) Let T = {s S s = φ}. Then {s S s = spremg o (φ)} = {s S s = A.(τA (o) φ[a /A]) A.τA (o)} = spremg o(t ). See the lecture notes. (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 vs. regresson Summary Summary of matrx/logc/relatonal operatons Corollary Let o = c, (e 1 e n ) be an operator such that all e are determnstc. The formula spremg o (φ) s logcally equvalent to regr o (φ). {s S s = regr o (φ)} = spremg o ({s S s = φ}) = {s S s = spremg o (φ)}. matrces formulas state sets vector V 1 n formula on A set matrx M n n formula on A A relaton V 1 n + V 1 n φ 1 φ 2 unon φ 1 φ 2 ntersecton V 1 n M n n ( A.(φ τa (o)))[a/a ] mg o (T ) M n n V n 1 A.(τA (o) /A]) premg o (T ) A.(τA (o) φ[a /A]) A.τA (o) o(t ) (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56

7 vs. SAT a premages of sets of operators vs. SAT Image computaton vs. plannng by satsfablty We tested plan exstence by testng satsfablty of The unon of mages of φ wth respect to all operators o O s mg o (φ). Ths can be computed more drectly by usng the dsjuncton τ A(o) of the transton formulae: A.(φ ( τ ))[A/A ]. Same works for premages. ι 0 R 1 (A 0, A 1 ) R 1 (A t 1, A t ) G t where R 1 (A, A ) = τ A(o). -abstractng A 0 A t 1 yelds A t 1.( A 0.(ι 0 R 1 (A 0, A 1 )) R 1 (A t 1, A t ) G t ). Ths s equvalent to conjonng the t-fold mage of ι mg o ( mg o (ι) ) wth G to test goal reachablty n t steps. We can do the same wth premages startng from G. (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 Shannon expanson Bnary decson dagrams 3-place connectve f-then-else s defned by where a s a proposton. te(a, φ 1, φ 2 ) = (a φ 1 ) ( a φ 2 ) Shannon expanson of a formula φ wth respect to a A s φ (a φ[ /a]) ( a φ[ /a]) = te(a, φ[ /a], φ[ /a]) By repeated applcaton of Shannon expanson any propostonal formula can be transformed to an equvalent formula contanng no other connectves than te a propostonal varables only n the frst poston of te. (a b) (b c) te(a, ( b) (b c), ( b) (b c)) te(a, b c, b) te(a, te(b, c, c), te(b,, )) te(a, te(b,, c), te(b,, )) te(a, te(b,, te(c,, )), te(b,, )) (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 Bnary decson dagrams Canoncty Bnary decson dagrams: example a Transformaton to ordered BDDs 1. Fx an orderng a 1,..., a n on all propostonal varables. 2. Apply Shannon expanson to all varables n ths order. 3. Represent the resultng formulae as drected acyclc graphs (DAG) so that shared subformulae occur only once. b c b Let φ 1 a φ 2 be two ordered BDDs obtaned by usng the same varable orderng. Then φ 1 φ 2 f a only f φ 1 a φ 2 are somorphc (the same DAG.) 1 0 (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 Satsfablty algorthms vs. BDDs Propertes of CPC normal forms Comparson: formula sze, runtme technque sze of R 1 (P, P ) runtme for plan length n satsfablty not a problem exponental n n BDDs major problem less depeent on n Comparson: resource consumpton technque crtcal resource satsfablty runtme BDDs memory Comparson: applcaton doman technque types of problems satsfablty lots of state varables, short plans BDDs few state varables, long plans Trade-offs between dfferent CPC normal forms Normal forms that allow faster reasonng are more expensve to construct from an arbtrary propostonal formula a may be much bgger. Propertes of dfferent normal forms φ TAUT? φ SAT? φ φ? crcuts poly poly poly co-np-hard NP-hard co-np-hard formulae poly poly poly co-np-hard NP-hard co-np-hard DNF poly exp exp co-np-hard n P co-np-hard CNF exp poly exp n P NP-hard co-np-hard BDD exp exp poly n P n P n P For BDDs one / s polynomal tme/sze (sze s doubled) but repeated / lead to exponental sze. (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56 (Albert-Ludwgs-Unverstät Freburg) AI Plannng May 30, / 56

Inner Product. Euclidean Space. Orthonormal Basis. Orthogonal

Inner Product. Euclidean Space. Orthonormal Basis. Orthogonal Inner Product Defnton 1 () A Eucldean space s a fnte-dmensonal vector space over the reals R, wth an nner product,. Defnton 2 (Inner Product) An nner product, on a real vector space X s a symmetrc, blnear,

More information

NP-Completeness : Proofs

NP-Completeness : Proofs NP-Completeness : Proofs Proof Methods A method to show a decson problem Π NP-complete s as follows. (1) Show Π NP. (2) Choose an NP-complete problem Π. (3) Show Π Π. A method to show an optmzaton problem

More information

Week 2. This week, we covered operations on sets and cardinality.

Week 2. This week, we covered operations on sets and cardinality. Week 2 Ths week, we covered operatons on sets and cardnalty. Defnton 0.1 (Correspondence). A correspondence between two sets A and B s a set S contaned n A B = {(a, b) a A, b B}. A correspondence from

More information

Calculation of time complexity (3%)

Calculation of time complexity (3%) Problem 1. (30%) Calculaton of tme complexty (3%) Gven n ctes, usng exhaust search to see every result takes O(n!). Calculaton of tme needed to solve the problem (2%) 40 ctes:40! dfferent tours 40 add

More information

Singular Value Decomposition: Theory and Applications

Singular Value Decomposition: Theory and Applications Sngular Value Decomposton: Theory and Applcatons Danel Khashab Sprng 2015 Last Update: March 2, 2015 1 Introducton A = UDV where columns of U and V are orthonormal and matrx D s dagonal wth postve real

More information

Problem Set 9 Solutions

Problem Set 9 Solutions Desgn and Analyss of Algorthms May 4, 2015 Massachusetts Insttute of Technology 6.046J/18.410J Profs. Erk Demane, Srn Devadas, and Nancy Lynch Problem Set 9 Solutons Problem Set 9 Solutons Ths problem

More information

Basic Regular Expressions. Introduction. Introduction to Computability. Theory. Motivation. Lecture4: Regular Expressions

Basic Regular Expressions. Introduction. Introduction to Computability. Theory. Motivation. Lecture4: Regular Expressions Introducton to Computablty Theory Lecture: egular Expressons Prof Amos Israel Motvaton If one wants to descrbe a regular language, La, she can use the a DFA, Dor an NFA N, such L ( D = La that that Ths

More information

8.4 COMPLEX VECTOR SPACES AND INNER PRODUCTS

8.4 COMPLEX VECTOR SPACES AND INNER PRODUCTS SECTION 8.4 COMPLEX VECTOR SPACES AND INNER PRODUCTS 493 8.4 COMPLEX VECTOR SPACES AND INNER PRODUCTS All the vector spaces you have studed thus far n the text are real vector spaces because the scalars

More information

A CLASS OF RECURSIVE SETS. Florentin Smarandache University of New Mexico 200 College Road Gallup, NM 87301, USA

A CLASS OF RECURSIVE SETS. Florentin Smarandache University of New Mexico 200 College Road Gallup, NM 87301, USA A CLASS OF RECURSIVE SETS Florentn Smarandache Unversty of New Mexco 200 College Road Gallup, NM 87301, USA E-mal: smarand@unmedu In ths artcle one bulds a class of recursve sets, one establshes propertes

More information

9 Characteristic classes

9 Characteristic classes THEODORE VORONOV DIFFERENTIAL GEOMETRY. Sprng 2009 [under constructon] 9 Characterstc classes 9.1 The frst Chern class of a lne bundle Consder a complex vector bundle E B of rank p. We shall construct

More information

= z 20 z n. (k 20) + 4 z k = 4

= z 20 z n. (k 20) + 4 z k = 4 Problem Set #7 solutons 7.2.. (a Fnd the coeffcent of z k n (z + z 5 + z 6 + z 7 + 5, k 20. We use the known seres expanson ( n+l ( z l l z n below: (z + z 5 + z 6 + z 7 + 5 (z 5 ( + z + z 2 + z + 5 5

More information

Some Consequences. Example of Extended Euclidean Algorithm. The Fundamental Theorem of Arithmetic, II. Characterizing the GCD and LCM

Some Consequences. Example of Extended Euclidean Algorithm. The Fundamental Theorem of Arithmetic, II. Characterizing the GCD and LCM Example of Extended Eucldean Algorthm Recall that gcd(84, 33) = gcd(33, 18) = gcd(18, 15) = gcd(15, 3) = gcd(3, 0) = 3 We work backwards to wrte 3 as a lnear combnaton of 84 and 33: 3 = 18 15 [Now 3 s

More information

Computing Correlated Equilibria in Multi-Player Games

Computing Correlated Equilibria in Multi-Player Games Computng Correlated Equlbra n Mult-Player Games Chrstos H. Papadmtrou Presented by Zhanxang Huang December 7th, 2005 1 The Author Dr. Chrstos H. Papadmtrou CS professor at UC Berkley (taught at Harvard,

More information

Real-Time Systems. Multiprocessor scheduling. Multiprocessor scheduling. Multiprocessor scheduling

Real-Time Systems. Multiprocessor scheduling. Multiprocessor scheduling. Multiprocessor scheduling Real-Tme Systems Multprocessor schedulng Specfcaton Implementaton Verfcaton Multprocessor schedulng -- -- Global schedulng How are tasks assgned to processors? Statc assgnment The processor(s) used for

More information

For now, let us focus on a specific model of neurons. These are simplified from reality but can achieve remarkable results.

For now, let us focus on a specific model of neurons. These are simplified from reality but can achieve remarkable results. Neural Networks : Dervaton compled by Alvn Wan from Professor Jtendra Malk s lecture Ths type of computaton s called deep learnng and s the most popular method for many problems, such as computer vson

More information

Lecture 3. Ax x i a i. i i

Lecture 3. Ax x i a i. i i 18.409 The Behavor of Algorthms n Practce 2/14/2 Lecturer: Dan Spelman Lecture 3 Scrbe: Arvnd Sankar 1 Largest sngular value In order to bound the condton number, we need an upper bound on the largest

More information

Module 9. Lecture 6. Duality in Assignment Problems

Module 9. Lecture 6. Duality in Assignment Problems Module 9 1 Lecture 6 Dualty n Assgnment Problems In ths lecture we attempt to answer few other mportant questons posed n earler lecture for (AP) and see how some of them can be explaned through the concept

More information

Feature Selection: Part 1

Feature Selection: Part 1 CSE 546: Machne Learnng Lecture 5 Feature Selecton: Part 1 Instructor: Sham Kakade 1 Regresson n the hgh dmensonal settng How do we learn when the number of features d s greater than the sample sze n?

More information

Notes on Frequency Estimation in Data Streams

Notes on Frequency Estimation in Data Streams Notes on Frequency Estmaton n Data Streams In (one of) the data streamng model(s), the data s a sequence of arrvals a 1, a 2,..., a m of the form a j = (, v) where s the dentty of the tem and belongs to

More information

Differential Polynomials

Differential Polynomials JASS 07 - Polynomals: Ther Power and How to Use Them Dfferental Polynomals Stephan Rtscher March 18, 2007 Abstract Ths artcle gves an bref ntroducton nto dfferental polynomals, deals and manfolds and ther

More information

Decision Diagrams Derivatives

Decision Diagrams Derivatives Decson Dagrams Dervatves Logc Crcuts Desgn Semnars WS2010/2011, Lecture 3 Ing. Petr Fšer, Ph.D. Department of Dgtal Desgn Faculty of Informaton Technology Czech Techncal Unversty n Prague Evropský socální

More information

Errors for Linear Systems

Errors for Linear Systems Errors for Lnear Systems When we solve a lnear system Ax b we often do not know A and b exactly, but have only approxmatons  and ˆb avalable. Then the best thng we can do s to solve ˆx ˆb exactly whch

More information

Solutions of Boolean equations by orthonormal expansion

Solutions of Boolean equations by orthonormal expansion Solutons of Boolean equatons by orthonormal expanson Vrendra Sule Department of Electrcal Engneerng Indan Insttute of Technology Bombay, Powa Mumba 400076, Inda (vrs@ee.tb.ac.n) December 29, 2012 1 Introducton

More information

The Minimum Universal Cost Flow in an Infeasible Flow Network

The Minimum Universal Cost Flow in an Infeasible Flow Network Journal of Scences, Islamc Republc of Iran 17(2): 175-180 (2006) Unversty of Tehran, ISSN 1016-1104 http://jscencesutacr The Mnmum Unversal Cost Flow n an Infeasble Flow Network H Saleh Fathabad * M Bagheran

More information

5 The Rational Canonical Form

5 The Rational Canonical Form 5 The Ratonal Canoncal Form Here p s a monc rreducble factor of the mnmum polynomal m T and s not necessarly of degree one Let F p denote the feld constructed earler n the course, consstng of all matrces

More information

Outline and Reading. Dynamic Programming. Dynamic Programming revealed. Computing Fibonacci. The General Dynamic Programming Technique

Outline and Reading. Dynamic Programming. Dynamic Programming revealed. Computing Fibonacci. The General Dynamic Programming Technique Outlne and Readng Dynamc Programmng The General Technque ( 5.3.2) -1 Knapsac Problem ( 5.3.3) Matrx Chan-Product ( 5.3.1) Dynamc Programmng verson 1.4 1 Dynamc Programmng verson 1.4 2 Dynamc Programmng

More information

DATA STRUCTURES FOR LOGIC OPTIMIZATION

DATA STRUCTURES FOR LOGIC OPTIMIZATION DATA STRUCTURES FOR LOGIC OPTIMIZATION Outlne Revew of Boolean algera. c Govann De Mchel Stanford Unversty Representatons of logc functons. Matrx representatons of covers. Operatons on logc covers. Background

More information

Week 5: Neural Networks

Week 5: Neural Networks Week 5: Neural Networks Instructor: Sergey Levne Neural Networks Summary In the prevous lecture, we saw how we can construct neural networks by extendng logstc regresson. Neural networks consst of multple

More information

2 More examples with details

2 More examples with details Physcs 129b Lecture 3 Caltech, 01/15/19 2 More examples wth detals 2.3 The permutaton group n = 4 S 4 contans 4! = 24 elements. One s the dentty e. Sx of them are exchange of two objects (, j) ( to j and

More information

The Order Relation and Trace Inequalities for. Hermitian Operators

The Order Relation and Trace Inequalities for. Hermitian Operators Internatonal Mathematcal Forum, Vol 3, 08, no, 507-57 HIKARI Ltd, wwwm-hkarcom https://doorg/0988/mf088055 The Order Relaton and Trace Inequaltes for Hermtan Operators Y Huang School of Informaton Scence

More information

Transfer Functions. Convenient representation of a linear, dynamic model. A transfer function (TF) relates one input and one output: ( ) system

Transfer Functions. Convenient representation of a linear, dynamic model. A transfer function (TF) relates one input and one output: ( ) system Transfer Functons Convenent representaton of a lnear, dynamc model. A transfer functon (TF) relates one nput and one output: x t X s y t system Y s The followng termnology s used: x y nput output forcng

More information

20. Mon, Oct. 13 What we have done so far corresponds roughly to Chapters 2 & 3 of Lee. Now we turn to Chapter 4. The first idea is connectedness.

20. Mon, Oct. 13 What we have done so far corresponds roughly to Chapters 2 & 3 of Lee. Now we turn to Chapter 4. The first idea is connectedness. 20. Mon, Oct. 13 What we have done so far corresponds roughly to Chapters 2 & 3 of Lee. Now we turn to Chapter 4. The frst dea s connectedness. Essentally, we want to say that a space cannot be decomposed

More information

Generalized Linear Methods

Generalized Linear Methods Generalzed Lnear Methods 1 Introducton In the Ensemble Methods the general dea s that usng a combnaton of several weak learner one could make a better learner. More formally, assume that we have a set

More information

APPENDIX A Some Linear Algebra

APPENDIX A Some Linear Algebra APPENDIX A Some Lnear Algebra The collecton of m, n matrces A.1 Matrces a 1,1,..., a 1,n A = a m,1,..., a m,n wth real elements a,j s denoted by R m,n. If n = 1 then A s called a column vector. Smlarly,

More information

VQ widely used in coding speech, image, and video

VQ widely used in coding speech, image, and video at Scalar quantzers are specal cases of vector quantzers (VQ): they are constraned to look at one sample at a tme (memoryless) VQ does not have such constrant better RD perfomance expected Source codng

More information

LINEAR TRANSFORMATION OF BINARY DECISION DIAGRAMS TROUGH SPECTRAL DOMAIN

LINEAR TRANSFORMATION OF BINARY DECISION DIAGRAMS TROUGH SPECTRAL DOMAIN LINEAR TRANSFORMATION OF BINARY DECISION DIAGRAMS TROUGH SPECTRAL DOMAIN Mlena Stankovc, Suzana Stokovc 2 Faculty of Electronc Engneerng, Unversty of Ns, A Medvedeva 4, 8 Ns, SERBIA, mstankovc@elfaknacyu,

More information

C/CS/Phy191 Problem Set 3 Solutions Out: Oct 1, 2008., where ( 00. ), so the overall state of the system is ) ( ( ( ( 00 ± 11 ), Φ ± = 1

C/CS/Phy191 Problem Set 3 Solutions Out: Oct 1, 2008., where ( 00. ), so the overall state of the system is ) ( ( ( ( 00 ± 11 ), Φ ± = 1 C/CS/Phy9 Problem Set 3 Solutons Out: Oct, 8 Suppose you have two qubts n some arbtrary entangled state ψ You apply the teleportaton protocol to each of the qubts separately What s the resultng state obtaned

More information

MATH 241B FUNCTIONAL ANALYSIS - NOTES EXAMPLES OF C ALGEBRAS

MATH 241B FUNCTIONAL ANALYSIS - NOTES EXAMPLES OF C ALGEBRAS MATH 241B FUNCTIONAL ANALYSIS - NOTES EXAMPLES OF C ALGEBRAS These are nformal notes whch cover some of the materal whch s not n the course book. The man purpose s to gve a number of nontrval examples

More information

An efficient algorithm for multivariate Maclaurin Newton transformation

An efficient algorithm for multivariate Maclaurin Newton transformation Annales UMCS Informatca AI VIII, 2 2008) 5 14 DOI: 10.2478/v10065-008-0020-6 An effcent algorthm for multvarate Maclaurn Newton transformaton Joanna Kapusta Insttute of Mathematcs and Computer Scence,

More information

Lectures - Week 4 Matrix norms, Conditioning, Vector Spaces, Linear Independence, Spanning sets and Basis, Null space and Range of a Matrix

Lectures - Week 4 Matrix norms, Conditioning, Vector Spaces, Linear Independence, Spanning sets and Basis, Null space and Range of a Matrix Lectures - Week 4 Matrx norms, Condtonng, Vector Spaces, Lnear Independence, Spannng sets and Bass, Null space and Range of a Matrx Matrx Norms Now we turn to assocatng a number to each matrx. We could

More information

CS 331 DESIGN AND ANALYSIS OF ALGORITHMS DYNAMIC PROGRAMMING. Dr. Daisy Tang

CS 331 DESIGN AND ANALYSIS OF ALGORITHMS DYNAMIC PROGRAMMING. Dr. Daisy Tang CS DESIGN ND NLYSIS OF LGORITHMS DYNMIC PROGRMMING Dr. Dasy Tang Dynamc Programmng Idea: Problems can be dvded nto stages Soluton s a sequence o decsons and the decson at the current stage s based on the

More information

Lecture 5 Decoding Binary BCH Codes

Lecture 5 Decoding Binary BCH Codes Lecture 5 Decodng Bnary BCH Codes In ths class, we wll ntroduce dfferent methods for decodng BCH codes 51 Decodng the [15, 7, 5] 2 -BCH Code Consder the [15, 7, 5] 2 -code C we ntroduced n the last lecture

More information

The Problem: Mapping programs to architectures

The Problem: Mapping programs to architectures Complng for Parallelsm & Localty!Last tme! SSA and ts uses!today! Parallelsm and localty! Data dependences and loops CS553 Lecture Complng for Parallelsm & Localty 1 The Problem: Mappng programs to archtectures

More information

Report on Image warping

Report on Image warping Report on Image warpng Xuan Ne, Dec. 20, 2004 Ths document summarzed the algorthms of our mage warpng soluton for further study, and there s a detaled descrpton about the mplementaton of these algorthms.

More information

A New Refinement of Jacobi Method for Solution of Linear System Equations AX=b

A New Refinement of Jacobi Method for Solution of Linear System Equations AX=b Int J Contemp Math Scences, Vol 3, 28, no 17, 819-827 A New Refnement of Jacob Method for Soluton of Lnear System Equatons AX=b F Naem Dafchah Department of Mathematcs, Faculty of Scences Unversty of Gulan,

More information

CHAPTER-5 INFORMATION MEASURE OF FUZZY MATRIX AND FUZZY BINARY RELATION

CHAPTER-5 INFORMATION MEASURE OF FUZZY MATRIX AND FUZZY BINARY RELATION CAPTER- INFORMATION MEASURE OF FUZZY MATRI AN FUZZY BINARY RELATION Introducton The basc concept of the fuzz matr theor s ver smple and can be appled to socal and natural stuatons A branch of fuzz matr

More information

Lecture 13 APPROXIMATION OF SECOMD ORDER DERIVATIVES

Lecture 13 APPROXIMATION OF SECOMD ORDER DERIVATIVES COMPUTATIONAL FLUID DYNAMICS: FDM: Appromaton of Second Order Dervatves Lecture APPROXIMATION OF SECOMD ORDER DERIVATIVES. APPROXIMATION OF SECOND ORDER DERIVATIVES Second order dervatves appear n dffusve

More information

On the Complexity of Partial Order Trace Model Checking

On the Complexity of Partial Order Trace Model Checking On the Complexty of Partal Order Trace Model Checkng Therry Massart Cédrc Meuter Laurent Van Begn Unversté Lbre de Bruxelles (U.L.B.), Boulevard du Tromphe, CP-212, 1050 Bruxelles, Belgum {tmassart,cmeuter,lvbegn}@ulb.ac.be

More information

Maximum Likelihood Estimation of Binary Dependent Variables Models: Probit and Logit. 1. General Formulation of Binary Dependent Variables Models

Maximum Likelihood Estimation of Binary Dependent Variables Models: Probit and Logit. 1. General Formulation of Binary Dependent Variables Models ECO 452 -- OE 4: Probt and Logt Models ECO 452 -- OE 4 Maxmum Lkelhood Estmaton of Bnary Dependent Varables Models: Probt and Logt hs note demonstrates how to formulate bnary dependent varables models

More information

Numerical Heat and Mass Transfer

Numerical Heat and Mass Transfer Master degree n Mechancal Engneerng Numercal Heat and Mass Transfer 06-Fnte-Dfference Method (One-dmensonal, steady state heat conducton) Fausto Arpno f.arpno@uncas.t Introducton Why we use models and

More information

Linear, affine, and convex sets and hulls In the sequel, unless otherwise specified, X will denote a real vector space.

Linear, affine, and convex sets and hulls In the sequel, unless otherwise specified, X will denote a real vector space. Lnear, affne, and convex sets and hulls In the sequel, unless otherwse specfed, X wll denote a real vector space. Lnes and segments. Gven two ponts x, y X, we defne xy = {x + t(y x) : t R} = {(1 t)x +

More information

The Geometry of Logit and Probit

The Geometry of Logit and Probit The Geometry of Logt and Probt Ths short note s meant as a supplement to Chapters and 3 of Spatal Models of Parlamentary Votng and the notaton and reference to fgures n the text below s to those two chapters.

More information

Fixed points of IA-endomorphisms of a free metabelian Lie algebra

Fixed points of IA-endomorphisms of a free metabelian Lie algebra Proc. Indan Acad. Sc. (Math. Sc.) Vol. 121, No. 4, November 2011, pp. 405 416. c Indan Academy of Scences Fxed ponts of IA-endomorphsms of a free metabelan Le algebra NAIME EKICI 1 and DEMET PARLAK SÖNMEZ

More information

CSci 6974 and ECSE 6966 Math. Tech. for Vision, Graphics and Robotics Lecture 21, April 17, 2006 Estimating A Plane Homography

CSci 6974 and ECSE 6966 Math. Tech. for Vision, Graphics and Robotics Lecture 21, April 17, 2006 Estimating A Plane Homography CSc 6974 and ECSE 6966 Math. Tech. for Vson, Graphcs and Robotcs Lecture 21, Aprl 17, 2006 Estmatng A Plane Homography Overvew We contnue wth a dscusson of the major ssues, usng estmaton of plane projectve

More information

Common loop optimizations. Example to improve locality. Why Dependence Analysis. Data Dependence in Loops. Goal is to find best schedule:

Common loop optimizations. Example to improve locality. Why Dependence Analysis. Data Dependence in Loops. Goal is to find best schedule: 15-745 Lecture 6 Data Dependence n Loops Copyrght Seth Goldsten, 2008 Based on sldes from Allen&Kennedy Lecture 6 15-745 2005-8 1 Common loop optmzatons Hostng of loop-nvarant computatons pre-compute before

More information

The Second Anti-Mathima on Game Theory

The Second Anti-Mathima on Game Theory The Second Ant-Mathma on Game Theory Ath. Kehagas December 1 2006 1 Introducton In ths note we wll examne the noton of game equlbrum for three types of games 1. 2-player 2-acton zero-sum games 2. 2-player

More information

Hidden Markov Models & The Multivariate Gaussian (10/26/04)

Hidden Markov Models & The Multivariate Gaussian (10/26/04) CS281A/Stat241A: Statstcal Learnng Theory Hdden Markov Models & The Multvarate Gaussan (10/26/04) Lecturer: Mchael I. Jordan Scrbes: Jonathan W. Hu 1 Hdden Markov Models As a bref revew, hdden Markov models

More information

find (x): given element x, return the canonical element of the set containing x;

find (x): given element x, return the canonical element of the set containing x; COS 43 Sprng, 009 Dsjont Set Unon Problem: Mantan a collecton of dsjont sets. Two operatons: fnd the set contanng a gven element; unte two sets nto one (destructvely). Approach: Canoncal element method:

More information

Ensemble Methods: Boosting

Ensemble Methods: Boosting Ensemble Methods: Boostng Ncholas Ruozz Unversty of Texas at Dallas Based on the sldes of Vbhav Gogate and Rob Schapre Last Tme Varance reducton va baggng Generate new tranng data sets by samplng wth replacement

More information

Boolean games revisited

Boolean games revisited Boolean games revsted Else Bonzon and Mare-Chrstne Lagasque-Schex and Jérôme Lang and Bruno Zanuttn 2 Abstract. Game theory s a wdely used formal model for studyng strategcal nteractons between agents.

More information

Chapter 8 Indicator Variables

Chapter 8 Indicator Variables Chapter 8 Indcator Varables In general, e explanatory varables n any regresson analyss are assumed to be quanttatve n nature. For example, e varables lke temperature, dstance, age etc. are quanttatve n

More information

Lecture Notes on Linear Regression

Lecture Notes on Linear Regression Lecture Notes on Lnear Regresson Feng L fl@sdueducn Shandong Unversty, Chna Lnear Regresson Problem In regresson problem, we am at predct a contnuous target value gven an nput feature vector We assume

More information

Dynamic Programming. Preview. Dynamic Programming. Dynamic Programming. Dynamic Programming (Example: Fibonacci Sequence)

Dynamic Programming. Preview. Dynamic Programming. Dynamic Programming. Dynamic Programming (Example: Fibonacci Sequence) /24/27 Prevew Fbonacc Sequence Longest Common Subsequence Dynamc programmng s a method for solvng complex problems by breakng them down nto smpler sub-problems. It s applcable to problems exhbtng the propertes

More information

Formulas for the Determinant

Formulas for the Determinant page 224 224 CHAPTER 3 Determnants e t te t e 2t 38 A = e t 2te t e 2t e t te t 2e 2t 39 If 123 A = 345, 456 compute the matrx product A adj(a) What can you conclude about det(a)? For Problems 40 43, use

More information

Salmon: Lectures on partial differential equations. Consider the general linear, second-order PDE in the form. ,x 2

Salmon: Lectures on partial differential equations. Consider the general linear, second-order PDE in the form. ,x 2 Salmon: Lectures on partal dfferental equatons 5. Classfcaton of second-order equatons There are general methods for classfyng hgher-order partal dfferental equatons. One s very general (applyng even to

More information

Finding Primitive Roots Pseudo-Deterministically

Finding Primitive Roots Pseudo-Deterministically Electronc Colloquum on Computatonal Complexty, Report No 207 (205) Fndng Prmtve Roots Pseudo-Determnstcally Ofer Grossman December 22, 205 Abstract Pseudo-determnstc algorthms are randomzed search algorthms

More information

Lecture Space-Bounded Derandomization

Lecture Space-Bounded Derandomization Notes on Complexty Theory Last updated: October, 2008 Jonathan Katz Lecture Space-Bounded Derandomzaton 1 Space-Bounded Derandomzaton We now dscuss derandomzaton of space-bounded algorthms. Here non-trval

More information

College of Computer & Information Science Fall 2009 Northeastern University 20 October 2009

College of Computer & Information Science Fall 2009 Northeastern University 20 October 2009 College of Computer & Informaton Scence Fall 2009 Northeastern Unversty 20 October 2009 CS7880: Algorthmc Power Tools Scrbe: Jan Wen and Laura Poplawsk Lecture Outlne: Prmal-dual schema Network Desgn:

More information

Introductory Cardinality Theory Alan Kaylor Cline

Introductory Cardinality Theory Alan Kaylor Cline Introductory Cardnalty Theory lan Kaylor Clne lthough by name the theory of set cardnalty may seem to be an offshoot of combnatorcs, the central nterest s actually nfnte sets. Combnatorcs deals wth fnte

More information

Chapter - 2. Distribution System Power Flow Analysis

Chapter - 2. Distribution System Power Flow Analysis Chapter - 2 Dstrbuton System Power Flow Analyss CHAPTER - 2 Radal Dstrbuton System Load Flow 2.1 Introducton Load flow s an mportant tool [66] for analyzng electrcal power system network performance. Load

More information

MEM 255 Introduction to Control Systems Review: Basics of Linear Algebra

MEM 255 Introduction to Control Systems Review: Basics of Linear Algebra MEM 255 Introducton to Control Systems Revew: Bascs of Lnear Algebra Harry G. Kwatny Department of Mechancal Engneerng & Mechancs Drexel Unversty Outlne Vectors Matrces MATLAB Advanced Topcs Vectors A

More information

where a is any ideal of R. Lemma 5.4. Let R be a ring. Then X = Spec R is a topological space Moreover the open sets

where a is any ideal of R. Lemma 5.4. Let R be a ring. Then X = Spec R is a topological space Moreover the open sets 5. Schemes To defne schemes, just as wth algebrac varetes, the dea s to frst defne what an affne scheme s, and then realse an arbtrary scheme, as somethng whch s locally an affne scheme. The defnton of

More information

Canonical transformations

Canonical transformations Canoncal transformatons November 23, 2014 Recall that we have defned a symplectc transformaton to be any lnear transformaton M A B leavng the symplectc form nvarant, Ω AB M A CM B DΩ CD Coordnate transformatons,

More information

Lecture 14 (03/27/18). Channels. Decoding. Preview of the Capacity Theorem.

Lecture 14 (03/27/18). Channels. Decoding. Preview of the Capacity Theorem. Lecture 14 (03/27/18). Channels. Decodng. Prevew of the Capacty Theorem. A. Barg The concept of a communcaton channel n nformaton theory s an abstracton for transmttng dgtal (and analog) nformaton from

More information

CALCULUS CLASSROOM CAPSULES

CALCULUS CLASSROOM CAPSULES CALCULUS CLASSROOM CAPSULES SESSION S86 Dr. Sham Alfred Rartan Valley Communty College salfred@rartanval.edu 38th AMATYC Annual Conference Jacksonvlle, Florda November 8-, 202 2 Calculus Classroom Capsules

More information

Subset Topological Spaces and Kakutani s Theorem

Subset Topological Spaces and Kakutani s Theorem MOD Natural Neutrosophc Subset Topologcal Spaces and Kakutan s Theorem W. B. Vasantha Kandasamy lanthenral K Florentn Smarandache 1 Copyrght 1 by EuropaNova ASBL and the Authors Ths book can be ordered

More information

A new construction of 3-separable matrices via an improved decoding of Macula s construction

A new construction of 3-separable matrices via an improved decoding of Macula s construction Dscrete Optmzaton 5 008 700 704 Contents lsts avalable at ScenceDrect Dscrete Optmzaton journal homepage: wwwelsevercom/locate/dsopt A new constructon of 3-separable matrces va an mproved decodng of Macula

More information

Hidden Markov Models

Hidden Markov Models Hdden Markov Models Namrata Vaswan, Iowa State Unversty Aprl 24, 204 Hdden Markov Model Defntons and Examples Defntons:. A hdden Markov model (HMM) refers to a set of hdden states X 0, X,..., X t,...,

More information

Equivalence Checking of Dissimilar Circuits II

Equivalence Checking of Dissimilar Circuits II Equvalence Checkng of Dssmlar Crcuts II Cadence Berkeley Labs 1995 Unversty Ave.,Sute 460, Berkeley, Calforna,94704 phone: (510)-647-2825, fax: (510)-486-0205 CDNL-TR-2004-0830 August 2004 Eugene Goldberg

More information

The Feynman path integral

The Feynman path integral The Feynman path ntegral Aprl 3, 205 Hesenberg and Schrödnger pctures The Schrödnger wave functon places the tme dependence of a physcal system n the state, ψ, t, where the state s a vector n Hlbert space

More information

Laboratory 1c: Method of Least Squares

Laboratory 1c: Method of Least Squares Lab 1c, Least Squares Laboratory 1c: Method of Least Squares Introducton Consder the graph of expermental data n Fgure 1. In ths experment x s the ndependent varable and y the dependent varable. Clearly

More information

Composite Hypotheses testing

Composite Hypotheses testing Composte ypotheses testng In many hypothess testng problems there are many possble dstrbutons that can occur under each of the hypotheses. The output of the source s a set of parameters (ponts n a parameter

More information

CHAPTER 17 Amortized Analysis

CHAPTER 17 Amortized Analysis CHAPTER 7 Amortzed Analyss In an amortzed analyss, the tme requred to perform a sequence of data structure operatons s averaged over all the operatons performed. It can be used to show that the average

More information

Stanford University CS254: Computational Complexity Notes 7 Luca Trevisan January 29, Notes for Lecture 7

Stanford University CS254: Computational Complexity Notes 7 Luca Trevisan January 29, Notes for Lecture 7 Stanford Unversty CS54: Computatonal Complexty Notes 7 Luca Trevsan January 9, 014 Notes for Lecture 7 1 Approxmate Countng wt an N oracle We complete te proof of te followng result: Teorem 1 For every

More information

Introduction to Algorithms

Introduction to Algorithms Introducton to Algorthms 6.046J/8.40J Lecture 7 Prof. Potr Indyk Data Structures Role of data structures: Encapsulate data Support certan operatons (e.g., INSERT, DELETE, SEARCH) Our focus: effcency of

More information

Lecture 10 Support Vector Machines II

Lecture 10 Support Vector Machines II Lecture 10 Support Vector Machnes II 22 February 2016 Taylor B. Arnold Yale Statstcs STAT 365/665 1/28 Notes: Problem 3 s posted and due ths upcomng Frday There was an early bug n the fake-test data; fxed

More information

Finite Difference Method

Finite Difference Method 7/0/07 Instructor r. Ramond Rump (9) 747 698 rcrump@utep.edu EE 337 Computatonal Electromagnetcs (CEM) Lecture #0 Fnte erence Method Lecture 0 These notes ma contan coprghted materal obtaned under ar use

More information

12 MATH 101A: ALGEBRA I, PART C: MULTILINEAR ALGEBRA. 4. Tensor product

12 MATH 101A: ALGEBRA I, PART C: MULTILINEAR ALGEBRA. 4. Tensor product 12 MATH 101A: ALGEBRA I, PART C: MULTILINEAR ALGEBRA Here s an outlne of what I dd: (1) categorcal defnton (2) constructon (3) lst of basc propertes (4) dstrbutve property (5) rght exactness (6) localzaton

More information

Lecture 4: November 17, Part 1 Single Buffer Management

Lecture 4: November 17, Part 1 Single Buffer Management Lecturer: Ad Rosén Algorthms for the anagement of Networs Fall 2003-2004 Lecture 4: November 7, 2003 Scrbe: Guy Grebla Part Sngle Buffer anagement In the prevous lecture we taled about the Combned Input

More information

A 2D Bounded Linear Program (H,c) 2D Linear Programming

A 2D Bounded Linear Program (H,c) 2D Linear Programming A 2D Bounded Lnear Program (H,c) h 3 v h 8 h 5 c h 4 h h 6 h 7 h 2 2D Lnear Programmng C s a polygonal regon, the ntersecton of n halfplanes. (H, c) s nfeasble, as C s empty. Feasble regon C s unbounded

More information

R n α. . The funny symbol indicates DISJOINT union. Define an equivalence relation on this disjoint union by declaring v α R n α, and v β R n β

R n α. . The funny symbol indicates DISJOINT union. Define an equivalence relation on this disjoint union by declaring v α R n α, and v β R n β Readng. Ch. 3 of Lee. Warner. M s an abstract manfold. We have defned the tangent space to M va curves. We are gong to gve two other defntons. All three are used n the subject and one freely swtches back

More information

FACTORIZATION IN KRULL MONOIDS WITH INFINITE CLASS GROUP

FACTORIZATION IN KRULL MONOIDS WITH INFINITE CLASS GROUP C O L L O Q U I U M M A T H E M A T I C U M VOL. 80 1999 NO. 1 FACTORIZATION IN KRULL MONOIDS WITH INFINITE CLASS GROUP BY FLORIAN K A I N R A T H (GRAZ) Abstract. Let H be a Krull monod wth nfnte class

More information

Yong Joon Ryang. 1. Introduction Consider the multicommodity transportation problem with convex quadratic cost function. 1 2 (x x0 ) T Q(x x 0 )

Yong Joon Ryang. 1. Introduction Consider the multicommodity transportation problem with convex quadratic cost function. 1 2 (x x0 ) T Q(x x 0 ) Kangweon-Kyungk Math. Jour. 4 1996), No. 1, pp. 7 16 AN ITERATIVE ROW-ACTION METHOD FOR MULTICOMMODITY TRANSPORTATION PROBLEMS Yong Joon Ryang Abstract. The optmzaton problems wth quadratc constrants often

More information

SUPER PRINCIPAL FIBER BUNDLE WITH SUPER ACTION

SUPER PRINCIPAL FIBER BUNDLE WITH SUPER ACTION talan journal of pure appled mathematcs n. 33 2014 (63 70) 63 SUPER PRINCIPAL FIBER BUNDLE WITH SUPER ACTION M.R. Farhangdoost Department of Mathematcs College of Scences Shraz Unversty Shraz, 71457-44776

More information

Bayesian Networks. Course: CS40022 Instructor: Dr. Pallab Dasgupta

Bayesian Networks. Course: CS40022 Instructor: Dr. Pallab Dasgupta Bayesan Networks Course: CS40022 Instructor: Dr. Pallab Dasgupta Department of Computer Scence & Engneerng Indan Insttute of Technology Kharagpur Example Burglar alarm at home Farly relable at detectng

More information

Bézier curves. Michael S. Floater. September 10, These notes provide an introduction to Bézier curves. i=0

Bézier curves. Michael S. Floater. September 10, These notes provide an introduction to Bézier curves. i=0 Bézer curves Mchael S. Floater September 1, 215 These notes provde an ntroducton to Bézer curves. 1 Bernsten polynomals Recall that a real polynomal of a real varable x R, wth degree n, s a functon of

More information

Assortment Optimization under MNL

Assortment Optimization under MNL Assortment Optmzaton under MNL Haotan Song Aprl 30, 2017 1 Introducton The assortment optmzaton problem ams to fnd the revenue-maxmzng assortment of products to offer when the prces of products are fxed.

More information

International Journal of Mathematical Archive-3(3), 2012, Page: Available online through ISSN

International Journal of Mathematical Archive-3(3), 2012, Page: Available online through   ISSN Internatonal Journal of Mathematcal Archve-3(3), 2012, Page: 1136-1140 Avalable onlne through www.ma.nfo ISSN 2229 5046 ARITHMETIC OPERATIONS OF FOCAL ELEMENTS AND THEIR CORRESPONDING BASIC PROBABILITY

More information

p-adic Galois representations of G E with Char(E) = p > 0 and the ring R

p-adic Galois representations of G E with Char(E) = p > 0 and the ring R p-adc Galos representatons of G E wth Char(E) = p > 0 and the rng R Gebhard Böckle December 11, 2008 1 A short revew Let E be a feld of characterstc p > 0 and denote by σ : E E the absolute Frobenus endomorphsm

More information

Embedded Systems. 4. Aperiodic and Periodic Tasks

Embedded Systems. 4. Aperiodic and Periodic Tasks Embedded Systems 4. Aperodc and Perodc Tasks Lothar Thele 4-1 Contents of Course 1. Embedded Systems Introducton 2. Software Introducton 7. System Components 10. Models 3. Real-Tme Models 4. Perodc/Aperodc

More information