> restart; > with(orthopoly); [G, H, L, P, T, U] > N:=14; > Digits:=13; > N := 14 Digits := 13 > R:=1; > Phi:=1; R := 1 Phi := 1 > U:=(r,theta)->sum(u[i]*P(i,cos(theta))*r^i,i=0..N); > V:=(r,theta)->sum(v[i]*P(i,cos(theta))/r^(i+1),i=0..N); N ----- \ i U := (r, theta) -> ) u[i] P(i, cos(theta)) r / ----- i = 0 N ----- \ v[i] P(i, cos(theta)) V := (r, theta) -> ) --------------------- / (i + 1) ----- r i = 0 > w:=(i)->evalf(Pi*i/N); > vzduch:=0..trunc(N/2)-1; > bronz:=rhs(vzduch)+1..N; Pi i w := i -> evalf(----) N vzduch := 0 .. 6 bronz := 7 .. 14 > rovnice:= { > seq( U(R,w(j))=Phi , j=bronz), > seq( V(R,w(j))=Phi , j=bronz), > seq( V(R,w(j))=U(R,w(j)) , j=vzduch), > seq( eval(diff(V(r,w(j))-U(r,w(j)),r),r=R)=0 , j=vzduch) > }: > reseni := solve(rovnice,{u[i]$i=0..N,v[i]$i=0..N} ); reseni := {v[13] = .0002503896106629, u[12] = .04378019261026, v[9] = -.01069640957662, u[6] = -.06776079939038, v[5] = -.04030920157930, u[4] = .08549302049364, v[8] = .05768886009990, u[11] = .003288901175883, u[13] = .0002503896106629, v[3] = .08320689193217, u[5] = -.04030920157930, v[7] = .02133617545862, u[2] = -.1281029234359, u[3] = .08320689193217, v[6] = -.06776079939038, u[14] = -.01706672162353, u[1] = -.2959602921854, u[0] = .8403738139418, v[0] = .8403738139418, v[10] = -.05328898785983, v[2] = -.1281029234359, u[7] = .02133617545862, v[11] = .003288901175883, v[12] = .04378019261026, u[8] = .05768886009990, u[10] = -.05328898785983, v[14] = -.01706672162353, v[4] = .08549302049364, v[1] = -.2959602921854, u[9] = -.01069640957662} > transf :={r=sqrt(x^2+z^2),cos(theta)=z/sqrt(x^2+z^2)}; z 2 2 transf := {cos(theta) = -------------, r = sqrt(x + z )} 2 2 sqrt(x + z ) > uu:=unapply(subs(reseni,transf,U(r,theta)),x,z): > vv:=unapply(subs(reseni,transf,V(r,theta)),x,z): > uv:=proc(x,z) > if not type(evalf(x^2+z^2),numeric) then 'uv(x,z)' else > if x^2+z^2 fi; > end; uv := proc(x, z) if not type(evalf(x^2 + z^2), numeric) then 'uv(x, z)' else if x^2 + z^2 < R^2 then uu(x, z) else vv(x, z) fi fi end > plots[contourplot](uv(x,z),x=1E-10..3,z=-3..3, levels=[(i/20)$i=0..19],scaling=constrained,grid=[150,150],color=black); > > > > > > > > > > > UV:=proc(r,theta) > global R; > > if not type(r,numeric) then 'uv(r,theta)' else > if r fi; > end; > UV := proc(r, theta) global R; if not type(r, numeric) then 'uv(r, theta)' else if r < R then U(r, theta) else V(r, theta) fi fi end > plots[contourplot](subs(r=sqrt(x^2+z^2),cos(theta)=z/sqrt(x^2+z^2),UV(r,theta)), > x=0..3,z=-3..3, levels=[(i/50)$i=0..49],scaling=constrained,grid=[10,10]); Error, (in UV) cannot evaluate boolean: r < 1 > (subs(r=sqrt(x^2+y^2),cos(theta)=y/sqrt(x^2+y^2),UV(r,theta)); Error, (in UV) cannot evaluate boolean: r < 1 > plots[contourplot](, > x=0..3,y=-3..3, levels=[(i/50)$i=0..49],scaling=constrained,grid=[150,150]); > > SR:={}:i:='i':j:='j': > for j from 0 to N do > t:=evalf(Pi*j/N); > if j ee:=diff(U(r,t)-V(r,t),r); > ee:=eval(ee,r=1); > SR:=SR union {U(1,t)=V(1,t),ee}; > else > SR:=SR union {U(1,t)=1,V(1,t)=1}; > fi; > od: > #SR; > vr:=solve(SR,{u[i]$i=0..N,v[i]$i=0..N} ); vr := {v[7] = .02133617545862, v[4] = .08549302049364, u[7] = .02133617545862, u[14] = -.01706672162353, v[2] = -.1281029234359, v[3] = .08320689193217, u[11] = .003288901175883, u[13] = .0002503896106624, u[1] = -.2959602921854, u[10] = -.05328898785983, v[12] = .04378019261026, v[8] = .05768886009990, v[13] = .0002503896106624, u[8] = .05768886009990, u[0] = .8403738139418, v[1] = -.2959602921854, v[14] = -.01706672162353, u[5] = -.04030920157930, u[3] = .08320689193217, u[12] = .04378019261026, v[10] = -.05328898785983, u[9] = -.01069640957662, v[5] = -.04030920157930, v[6] = -.06776079939037, u[6] = -.06776079939037, u[2] = -.1281029234359, u[4] = .08549302049364, v[9] = -.01069640957662, v[11] = .003288901175883, v[0] = .8403738139418} > uu:=unapply(subs(vr,U(r,theta)),r,theta): > vv:=unapply(subs(vr,V(r,theta)),r,theta): > uv:=proc(r,theta) > global uu,vv; > if not type(r,numeric) then 'uv(r,theta)' else > if r<1 then evalf(uu(r,theta)) else evalf(vv(r,theta)) fi; > fi; > end; > plots[contourplot](uv(sqrt(x^2+y^2),arccos(y/sqrt(x^2+y^2+1E-20))), > x=0..3,y=-3..3, levels=[(i/50)$i=0..49],scaling=constrained,grid=[150,150]); uv := proc(r, theta) global uu, vv; if not type(r, numeric) then 'uv(r, theta)' else if r < 1 then evalf(uu(r, theta)) else evalf(vv(r, theta)) fi fi end > > > lsolve:=proc(R,u) > local a,a1,u1,r1,A,i; > r1:=convert(R,list); > u1:=map(q->q=0,u); > for i from 1 to nops(R) do > #print (r1[i]); > if type(r1[i],equation) then r1[i]:=eval('lhs(r1[i])-rhs(r1[i])'); fi; > od: > a1:=subs(u1,r1); > u1:=convert(u,list); > A:=linalg[jacobian](r1,u1); > print(A,a1); > a:=linalg[linsolve](A,-a1); > RETURN({seq(u1[i]=a[i],i=1..nops(u))}); > end; lsolve := proc(R, u) local a, a1, u1, r1, A, i; r1 := convert(R, list); u1 := map(q -> q = 0, u); for i to nops(R) do if type(r1[i], equation) then r1[i] := eval('lhs(r1[i]) - rhs(r1[i])') fi od; a1 := subs(u1, r1); u1 := convert(u, list); A := linalg[jacobian](r1, u1); print(A, a1); a := linalg[linsolve](A, -a1); RETURN({seq(u1[i] = a[i], i = 1 .. nops(u))}) end > #lsolve({u+2*v=1,2*u-v=0},{u,v}); > vr:=lsolve(SR,{u[i]$i=0..N,v[i]$i=0..N} ); [1 , -.974927912181823607018131682993931 , .925726650926814344677076739630583 , -.854242643610702483074577210294009 , .763148756611000876454644020785893 , -.655832928251889946135257139787939 , .536257386538795040022808303381980 , -.408794607963313174710909711868458 , .278047174877666832803388487697422 , -.148659368338849184356972220671654 , .0251286610517394105542102843732387 , .0883747626574049642222023675265760 , -.188172733087794814519403068737770 , .271221084083224948941643788604640 , -.335222972248021379135183576069987 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0] [0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , -1. , -1. , 1 , 1 , -1. , 1 , -1. , 1 , -1. , 1 , 1 , 1 , -1. , 1 , -1.] [1 , 1.94985582436364721403626336598786 , 2.77717995278044303403123021889175 , 3.41697057444280993229830884117604 , 3.81574378305500438227322010392946 , 3.93499756951133967681154283872763 , 3.75380170577156528015965812367386 , 3.27035686370650539768727769494766 , 2.50242457389900149523049638927680 , 1.48659368338849184356972220671654 , .276415271569133516096313128105626 , -1.06049715188885957066642841031891 , -2.44624553014133258875223989359101 , -3.79709517716514928518301304046496 , -5.02834458372032068702775364104980 , .974927912181823607018131682993931 , -3.52587409308192433624136925186032 , -4.69312161147229930789257006497982 , 3.21754431923277024013684982029188 , 2.86156225574319222297636798307921 , 2.22437739902133466242710790157938 , 1.33793431504964265921274998604489 , .251286610517394105542102843732387 , -.972122389231454606444226042792336 , -2.25807279705353777423283682485324 , 0 , 1.85145330185362868935415347926117 , 2.56272793083210744922373163088203 , 3.05259502644400350581857608314357 , 3.27916464125944973067628569893970] [0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , -.222520933956314404288902564496793 , -.0241553519993967016092655345403957 , .210764857821593790172430339685172 , -.0340709996864496304675324620361504 , .292748633421373826521609705550432 , -.0923304365056543627086343939568370 , -.221412925887315544224603765251730 , .176708513866135714805071064299172 , .126216458587193956185270622730763 , -.215813929181129422147500307161447 , 1 , -.425726650926814344677076739630585 , .306235775928090554969789590816350 , .200043214171988922557080071093745 , -.325113465870985652446612125966596] [-1 , -.433883739117558120475768332848360 , .217617351394050147893753663003178 , .446623542944555459207919177053073 , .175906698838213668134557616210512 , -.219917333145693713416175361415067 , -.321522932835539418974633593474959 , -.0705774915950418898129719295159378 , .223915517573356729840018645138954 , .246247340772249713828909326964596 , .00147719641181547602309012251820647 , -.222637622378957892760562556203795 , -.186501881170712459269273896830383 , .0498960099751779976688619537615572 , .214932091024739041837009546485307 , .433883739117558120475768332848360 , -.0498960099751779976688619537615572 , -.214932091024739041837009546485307 , .321522932835539418974633593474959 , .0705774915950418898129719295159378 , -.223915517573356729840018645138954 , -.246247340772249713828909326964596 , -.00147719641181547602309012251820647 , .222637622378957892760562556203795 , .186501881170712459269273896830383 , 1 , -.217617351394050147893753663003178 , -.446623542944555459207919177053073 , -.175906698838213668134557616210512 , .219917333145693713416175361415067] [-1 , -.222520933956314404288902564496796 , .425726650926814344677076739630583 , .306235775928090554969789590816353 , -.200043214171988922557080071093740 , -.325113465870985652446612125966598 , .0340709996864496304675324620361441 , .292748633421373826521609705550432 , .0923304365056543627086343939568438 , -.221412925887315544224603765251726 , -.176708513866135714805071064299178 , .126216458587193956185270622730756 , .215813929181129422147500307161450 , -.0241553519993967016092655345403866 , -.210764857821593790172430339685171 , .222520933956314404288902564496796 , .0241553519993967016092655345403866 , .210764857821593790172430339685171 , -.0340709996864496304675324620361441 , -.292748633421373826521609705550432 , -.0923304365056543627086343939568438 , .221412925887315544224603765251726 , .176708513866135714805071064299178 , -.126216458587193956185270622730756 , -.215813929181129422147500307161450 , 1 , -.425726650926814344677076739630583 , -.306235775928090554969789590816353 , .200043214171988922557080071093740 , .325113465870985652446612125966598] [1 , -1. , 1 , -1. , 1 , -1. , 1 , -1. , 1 , -1. , 1 , -1. , 1 , -1. , 1 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0] [1 , 1.80193773580483825247220463901489 , 2.15285205418215044368126098900954 , 1.90775563674441470007640989050315 , 1.06887213661747394221785218146070 , -.209182443354217241525655391390124 , -1.65012718512014040384904477106757 , -2.91640731116172403163559091876002 , -3.68618419986111944293438871393247 , -3.72983539405329143803656568326487 , -2.96857042655773431544842212480191 , -1.50130819160376040105804162774304 , .407361360806999840071134968574254 , 2.37689383016331023783147636595601 , 3.98859483806916044607069996647704 , .900968867902419126236102319507445 , 2.20711569943735950655779948267344 , 3.72268851553121641633265330204524 , -1.41439473010297748901346694662934 , -2.55185639726650852768114205391501 , -3.27660817765432839371945663460664 , -3.35685185464796229423290911493838 , -2.69870038777975846858947465891083 , -1.37619917563678036763653815876446 , .376025871514153698527201509453158 , 0 , 1.43523470278810029578750732600636 , 1.43081672755831102505730741787736 , .855097709293979153774281745168560 , -.174318702795181034604712826158437] [-1 , -.900968867902419126236102319507445 , -.717617351394050147893753663003180 , -.476938909186103675019102472625788 , -.213774427323494788443570436292140 , .0348637405590362069209425652316874 , .235732455017162914835577824438224 , .364550913895215503954448864845002 , .409576022206791049214932079325830 , .372983539405329143803656568326487 , .269870038777975846858947465891083 , .125109015966980033421503468978587 , -.0313354892928461415439334591210965 , -.169778130725950731273676883282572 , -.265906322537944029738046664431803 , .900968867902419126236102319507445 , .169778130725950731273676883282572 , .265906322537944029738046664431803 , -.235732455017162914835577824438224 , -.364550913895215503954448864845002 , -.409576022206791049214932079325830 , -.372983539405329143803656568326487 , -.269870038777975846858947465891083 , -.125109015966980033421503468978587 , .0313354892928461415439334591210965 , 1 , .717617351394050147893753663003180 , .476938909186103675019102472625788 , .213774427323494788443570436292140 , -.0348637405590362069209425652316874] [0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , -.433883739117558120475768332848357 , .0498960099751779976688619537615672 , -.214932091024739041837009546485310 , .321522932835539418974633593474957 , -.0705774915950418898129719295159303 , -.223915517573356729840018645138959 , .246247340772249713828909326964592 , -.00147719641181547602309012251819740 , -.222637622378957892760562556203799 , .186501881170712459269273896830377 , 1 , -.217617351394050147893753663003182 , .446623542944555459207919177053072 , -.175906698838213668134557616210506 , -.219917333145693713416175361415072] [1 , -.433883739117558120475768332848357 , -.217617351394050147893753663003182 , .446623542944555459207919177053072 , -.175906698838213668134557616210506 , -.219917333145693713416175361415072 , .321522932835539418974633593474957 , -.0705774915950418898129719295159303 , -.223915517573356729840018645138959 , .246247340772249713828909326964592 , -.00147719641181547602309012251819740 , -.222637622378957892760562556203799 , .186501881170712459269273896830377 , .0498960099751779976688619537615672 , -.214932091024739041837009546485310 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0] [1 , 1.24697960371746706105000976800848 , .249327898598292590349969229882213 , -1.31718746696794751980274847276225 , -2.10815070747741855500325253692941 , -1.25850164812830332684598263559054 , .781202307925287817121772005320590 , 2.47207237146728535619153143683653 , 2.37235222020888370731209825954404 , .357615398022989004209471969252406 , -2.14358107509085229740735958248900 , -3.17358239142743162528128910051216 , -1.78633008995451461777863097547542 , 1.11110347571467851348619384952146 , 3.34539694738365084099128243824539 , .623489801858733530525004884004240 , 1.03173894173505861966575143169850 , 3.12237048422474078492519694236236 , .669601978221675271818661718846220 , 2.16306332503387468666759000723196 , 2.10875752907456329538853178626137 , .321853858220690103788524772327165 , -1.94871006826441117946123598408091 , -2.90911719214181232317451500880282 , -1.64892008303493657025719782351578 , 0 , .166218599065528393566646153254809 , -.987890600225960639852061354571689 , -1.68652056598193484400260202954353 , -1.04875137344025277237165219632545] [1 , -.781831482468029808708444526674056 , .416890700467235803216676923372592 , -.0220094689770373529683114894725420 , -.282554557772787208320086404575390 , .415245662988504118730787905297567 , -.359733444374334458997441896856938 , .166398305639955587370244962414034 , .0708378251175648970366301574415374 , -.252522395129972258123237285388544 , .311362878621794815468879838144958 , -.235170488113317256120931764929389 , .0669894363592210271251291719073742 , .116360353761470711251062637237931 , -.237654696105672806566869377444712 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0] [0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , -.623489801858733530525004884004238 , -.0793645339796198938204424178229693 , .223026463158910056066085495883028 , .111600329703612545303110286474376 , -.309009046433410669523941429604567 , .263594691134320411923566473282667 , -.0357615398022989004209471969252335 , -.194871006826441117946123598408096 , .264465199285619302106774091709346 , -.137410006919578047521433151959641 , 1 , .0831092995327641967833230766274005 , .329296866741986879950687118190566 , -.421630141495483711000650507385882 , .209750274688050554474330439265085] [1 , 2 , 3 , 4 , 5 , 6 , 7 , 8 , 9 , 10 , 11 , 12 , 13 , 14 , 15 , 1 , 13 , 14 , 6 , 7 , 8 , 9 , 10 , 11 , 12 , 0 , 2 , 3 , 4 , 5] [0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , -.900968867902419126236102319507444 , -.169778130725950731273676883282581 , .265906322537944029738046664431808 , -.235732455017162914835577824438230 , .364550913895215503954448864845006 , -.409576022206791049214932079325830 , .372983539405329143803656568326484 , -.269870038777975846858947465891076 , .125109015966980033421503468978578 , .0313354892928461415439334591211063 , 1 , .717617351394050147893753663003177 , -.476938909186103675019102472625784 , .213774427323494788443570436292134 , .0348637405590362069209425652316939] [1 , 1.56366296493605961741688905334812 , 1.25067210140170740965003077011780 , .0880378759081494118732459578902052 , -1.41277278886393604160043202287692 , -2.49147397793102471238472743178540 , -2.51813411062034121298209327799861 , -1.33118644511964469896195969931237 , .637540426058084073329671416973713 , 2.52522395129972258123237285388536 , 3.42499166483974297015767821959455 , 2.82204585735980707345118117915279 , .870862672669873352626679234796084 , -1.62904495266058995751487692133081 , -3.56482044158509209850304066167058 , .781831482468029808708444526674059 , -1.51268459889911924626381428409290 , -3.32716574547941929193617128422587 , -2.15840066624600675398465138114166 , -1.16478813947968911159171473689832 , .566702600940519176293041259532190 , 2.27270155616975032310913556849682 , 3.11362878621794815468879838144959 , 2.58687536924648981733024941422339 , .803873236310652325501550062888693 , 0 , .833781400934471606433353846745198 , .0660284069311120589049344684176539 , -1.13021823109114883328034561830153 , -2.07622831494252059365393952648783] [ [0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , -32 .144209858469968755291048747229616 10 , -32 .422912309555972824354511121025915 10 , -.209472656250000000000000000000000 , -.312500000000000000000000000000000 , -32 -.315459065403056652199169134564785 10 , .273437500000000000000000000000000 , -32 .354891448578438733724065276385383 10 , -.246093750000000000000000000000000 , -32 -.390380593436282607096471804023921 10 , .225585937500000000000000000000000 , 1 , -.500000000000000000000000000000000 , -32 -.216314787704953132936573120844424 10 , .375000000000000000000000000000000 , -32] .270393484631191416170716401055530 10 ] [1 , .867767478235116240951536665696720 , -.652852054182150443681260989009534 , -1.78649417177822183683167670821229 , -.879533494191068340672788081052560 , 1.31950399887416228049705216849040 , 2.25066052984877593282243515432471 , .564619932760335118503775436127502 , -2.01523965816021056856016780625059 , -2.46247340772249713828909326964596 , -.0162491605299702362539913477002712 , 2.67165146854749471312675067444554 , 2.42452445521926197050056065879498 , -.698544139652491967364067352661801 , -3.22398136537108562755514319727960 , .433883739117558120475768332848360 , -.648648129677313969695205398900244 , -3.00904927434634658571813365079430 , 1.92913759701323651384780156084975 , .494042441165293228690803506611565 , -1.79132414058685383872014916111163 , -2.21622606695024742446018394268136 , -.0147719641181547602309012251820647 , 2.44901384616853682036618811824174 , 2.23802257404854951123128676196460 , 0 , -.435234702788100295787507326006356 , -1.33987062883366637762375753115922 , -.703626795352854672538230464842048 , 1.09958666572846856708087680707534] [-1 , -1 , -1 , -1 , -1 , -1 , -1 , -1 , -1 , -1 , -1 , -1 , -1 , -1 , -1 , 1 , 1 , 1 , 1 , 1 , 1 , 1 , 1 , 1 , 1 , 1 , 1 , 1 , 1 , 1] [1 , .445041867912628808577805128993592 , -1.27717995278044303403123021889175 , -1.22494310371236221987915836326541 , 1.00021607085994461278540035546870 , 1.95068079522591391467967275579959 , -.238496997805147413272727234253009 , -2.34198906737099061217287764440346 , -.830973928550889264377709545611594 , 2.21412925887315544224603765251726 , 1.94379365252749286285578170729096 , -1.51459750304632747422324747276907 , -2.80558107935468248791750399309885 , .338174927991553822529717483565412 , 3.16147286732390685258645509527756 , .222520933956314404288902564496796 , .314019575992157120920451949025026 , 2.95070800950231306241402475559239 , -.204425998118697782805194772216865 , -2.04924043394961678565126793885302 , -.738643492045234901669075151654750 , 1.99271633298583989802143388726553 , 1.76708513866135714805071064299178 , -1.38838104445913351803797685003832 , -2.58976715017355306577000368593740 , 0 , -.851453301853628689354153479261166 , -.918707327784271664909368772449059 , .800172856687955690228320284374960 , 1.62556732935492826223306062983299] [-1 , -.974927912181823607018131682993931 , -.925726650926814344677076739630583 , -.854242643610702483074577210294009 , -.763148756611000876454644020785893 , -.655832928251889946135257139787939 , -.536257386538795040022808303381980 , -.408794607963313174710909711868458 , -.278047174877666832803388487697422 , -.148659368338849184356972220671654 , -.0251286610517394105542102843732387 , .0883747626574049642222023675265760 , .188172733087794814519403068737770 , .271221084083224948941643788604640 , .335222972248021379135183576069987 , .974927912181823607018131682993931 , -.271221084083224948941643788604640 , -.335222972248021379135183576069987 , .536257386538795040022808303381980 , .408794607963313174710909711868458 , .278047174877666832803388487697422 , .148659368338849184356972220671654 , .0251286610517394105542102843732387 , -.0883747626574049642222023675265760 , -.188172733087794814519403068737770 , 1 , .925726650926814344677076739630583 , .854242643610702483074577210294009 , .763148756611000876454644020785893 , .655832928251889946135257139787939] [ -32 [1 , .144209858469968755291048747229616 10 , -.500000000000000000000000000000000 , -32 -.216314787704953132936573120844424 10 , .375000000000000000000000000000000 , -32 .270393484631191416170716401055530 10 , -.312500000000000000000000000000000 , -32 -.315459065403056652199169134564785 10 , .273437500000000000000000000000000 , -32 .354891448578438733724065276385383 10 , -.246093750000000000000000000000000 , -32 -.390380593436282607096471804023921 10 , .225585937500000000000000000000000 , -32 .422912309555972824354511121025915 10 , -.209472656250000000000000000000000 , 0 , 0 , 0 , 0 , 0 , 0 , ] 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0] [1 , -.623489801858733530525004884004238 , .0831092995327641967833230766274005 , .329296866741986879950687118190566 , -.421630141495483711000650507385882 , .209750274688050554474330439265085 , .111600329703612545303110286474376 , -.309009046433410669523941429604567 , .263594691134320411923566473282667 , -.0357615398022989004209471969252335 , -.194871006826441117946123598408096 , .264465199285619302106774091709346 , -.137410006919578047521433151959641 , -.0793645339796198938204424178229693 , .223026463158910056066085495883028 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0] [-1 , -.623489801858733530525004884004240 , -.0831092995327641967833230766274043 , .329296866741986879950687118190563 , .421630141495483711000650507385882 , .209750274688050554474330439265090 , -.111600329703612545303110286474370 , -.309009046433410669523941429604566 , -.263594691134320411923566473282671 , -.0357615398022989004209471969252406 , .194871006826441117946123598408091 , .264465199285619302106774091709347 , .137410006919578047521433151959648 , -.0793645339796198938204424178229613 , -.223026463158910056066085495883026 , .623489801858733530525004884004240 , .0793645339796198938204424178229613 , .223026463158910056066085495883026 , .111600329703612545303110286474370 , .309009046433410669523941429604566 , .263594691134320411923566473282671 , .0357615398022989004209471969252406 , -.194871006826441117946123598408091 , -.264465199285619302106774091709347 , -.137410006919578047521433151959648 , 1 , .0831092995327641967833230766274043 , -.329296866741986879950687118190563 , -.421630141495483711000650507385882 , -.209750274688050554474330439265090] [1 , -.900968867902419126236102319507444 , .717617351394050147893753663003177 , -.476938909186103675019102472625784 , .213774427323494788443570436292134 , .0348637405590362069209425652316939 , -.235732455017162914835577824438230 , .364550913895215503954448864845006 , -.409576022206791049214932079325830 , .372983539405329143803656568326484 , -.269870038777975846858947465891076 , .125109015966980033421503468978578 , .0313354892928461415439334591211063 , -.169778130725950731273676883282581 , .265906322537944029738046664431808 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0] [-1 , -.781831482468029808708444526674059 , -.416890700467235803216676923372599 , -.0220094689770373529683114894725513 , .282554557772787208320086404575383 , .415245662988504118730787905297566 , .359733444374334458997441896856944 , .166398305639955587370244962414046 , -.0708378251175648970366301574415237 , -.252522395129972258123237285388536 , -.311362878621794815468879838144959 , -.235170488113317256120931764929399 , -.0669894363592210271251291719073911 , .116360353761470711251062637237915 , .237654696105672806566869377444705 , .781831482468029808708444526674059 , -.116360353761470711251062637237915 , -.237654696105672806566869377444705 , -.359733444374334458997441896856944 , -.166398305639955587370244962414046 , .0708378251175648970366301574415237 , .252522395129972258123237285388536 , .311362878621794815468879838144959 , .235170488113317256120931764929399 , .0669894363592210271251291719073911 , 1 , .416890700467235803216676923372599 , .0220094689770373529683114894725513 , -.282554557772787208320086404575383 , -.415245662988504118730787905297566] [1 , -.222520933956314404288902564496793 , -.425726650926814344677076739630585 , .306235775928090554969789590816350 , .200043214171988922557080071093745 , -.325113465870985652446612125966596 , -.0340709996864496304675324620361504 , .292748633421373826521609705550432 , -.0923304365056543627086343939568370 , -.221412925887315544224603765251730 , .176708513866135714805071064299172 , .126216458587193956185270622730763 , -.215813929181129422147500307161447 , -.0241553519993967016092655345403957 , .210764857821593790172430339685172 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0] [0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , -.781831482468029808708444526674056 , .116360353761470711251062637237931 , -.237654696105672806566869377444712 , -.359733444374334458997441896856938 , .166398305639955587370244962414034 , .0708378251175648970366301574415374 , -.252522395129972258123237285388544 , .311362878621794815468879838144958 , -.235170488113317256120931764929389 , .0669894363592210271251291719073742 , 1 , .416890700467235803216676923372592 , -.0220094689770373529683114894725420 , -.282554557772787208320086404575390 , .415245662988504118730787905297567] [0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , 0 , -.974927912181823607018131682993931 , .271221084083224948941643788604640 , -.335222972248021379135183576069987 , .536257386538795040022808303381980 , -.408794607963313174710909711868458 , .278047174877666832803388487697422 , -.148659368338849184356972220671654 , .0251286610517394105542102843732387 , .0883747626574049642222023675265760 , -.188172733087794814519403068737770 , 1 , .925726650926814344677076739630583 , -.854242643610702483074577210294009 , .763148756611000876454644020785893 , -.655832928251889946135257139787939], [-1., -1., 0., -1., 0., 0., -1., 0., 0., -1., -1., 0., -1., -1., 0, -1., 0., -1., 0., 0, 0., 0., -1., -1., 0., -1., 0., -1., -1., -1.] vr := {v[4] = .0854930204935793607383410471800542, v[5] = -.0403092015794234097200871081474098, v[6] = -.0677607993904499989979165250942740, v[7] = .0213361754586976860803965520986972, u[11] = .0032889011758742715107651697061899, u[0] = .840373813941738115285108935468293, u[2] = -.128102923435780282667771473852477, u[3] = .0832068919322870921814126959322407, u[4] = .0854930204935793607383410471800542, u[5] = -.0403092015794234097200871081474094, u[12] = .0437801926105226563249270450831854, v[10] = -.0532889878600746845978509048083115, v[8] = .0576888601000826619199673196755846, v[9] = -.0106964095766408845693966610998596, v[11] = .00328890117587427151076516970619252, v[12] = .0437801926105226563249270450831862, v[13] = .00025038961066522721266613432798045, v[14] = -.0170667216236339932493509575087036, u[1] = -.295960292185476147940302296674474, u[13] = .000250389610665227212666134327981336, u[14] = -.0170667216236339932493509575087025, u[6] = -.0677607993904499989979165250942732, u[7] = .0213361754586976860803965520986972, u[8] = .0576888601000826619199673196755843, u[9] = -.0106964095766408845693966610998712, u[10] = -.0532889878600746845978509048083118, v[0] = .840373813941738115285108935468292, v[1] = -.295960292185476147940302296674475, v[2] = -.128102923435780282667771473852476, v[3] = .083206891932287092181412695932238} > uu:=unapply(subs(vr,U(r,theta)),r,theta): > vv:=unapply(subs(vr,V(r,theta)),r,theta): > > sigma:=-diff(evalf(vv(r,theta)-uu(r,theta)),r): > sigma:=eval(sigma,r=1): > X||N:=plot(sigma,theta=0..Pi,color=green):; > plots[display](X44,X14); > with(plots); Warning, the name changecoords has been redefined [animate, animate3d, animatecurve, changecoords, complexplot, complexplot3d, conformal, contourplot, contourplot3d, coordplot, coordplot3d, cylinderplot, densityplot, display, display3d, fieldplot, fieldplot3d, gradplot, gradplot3d, implicitplot, implicitplot3d, inequal, listcontplot, listcontplot3d, listdensityplot, listplot, listplot3d, loglogplot, logplot, matrixplot, odeplot, pareto, pointplot, pointplot3d, polarplot, polygonplot, polygonplot3d, polyhedra_supported, polyhedraplot, replot, rootlocus, semilogplot, setoptions, setoptions3d, spacecurve, sparsematrixplot, sphereplot, surfdata, textplot, textplot3d, tubeplot] > uv:=proc(r,theta) > global uu,vv; > if not type(r,numeric) then 'uv(r,theta)' else > if r<1 then evalf(uu(r,theta)) else evalf(vv(r,theta)) fi; > fi; > end; uv := proc(r, theta) global uu, vv; if not type(r, numeric) then 'uv(r, theta)' else if r < 1 then evalf(uu(r, theta)) else evalf(vv(r, theta)) fi fi end > contourplot(uv(sqrt(x^2+y^2),arccos(y/sqrt(x^2+y^2+1E-20))), > x=0..3,y=-3..3, levels=[(i/50)$i=0..49],scaling=constrained,grid=[120,120]); > uv(1,0); .5129280410011 > subs(vr,u[0]); .8253470273054 > Eru:=evalf(eval(subs(vr,diff(-U(r,theta),r)),r=1-.03)): > Erv:=evalf(eval(subs(vr,diff(-V(r,theta),r)),r=1+.03)): > Eri:=evalf(eval(subs(vr,diff(-V(r,theta),r)),r=1000+.01)): > > int(Eru*2*Pi*sin(theta),theta=Pi/2..Pi); > int(Erv*2*Pi*sin(theta),theta=Pi/2..Pi); > %-%%; > int(1000^2*2*Pi*Eri*sin(theta),theta=0..Pi); > subs(vr,evalf(u[0]*4*Pi)); -1.262403170173 7.559302619966 8.821705790139 10.56023759479 10.56044880060 > int(Eru*2*Pi*sin(theta),theta=Pi/2..Pi); > int(Erv*2*Pi*sin(theta),theta=Pi/2..Pi); > %-%%; > int(1000^2*2*Pi*Eri*sin(theta),theta=0..Pi); > subs(vr,evalf(u[0]*4*Pi)); > -1.417436312685 7.705906081864 9.123342394549 10.44503589675 10.44524479851 > N; > int(Eru*2*Pi*sin(theta),theta=Pi/2..Pi); > int(Erv*2*Pi*sin(theta),theta=Pi/2..Pi); > %-%%; > int(1000^2*2*Pi*Eri*sin(theta),theta=0..Pi); > subs(vr,evalf(u[0]*4*Pi)); 34 -1.4249339831194042657772 7.1921948771456507025958 8.6171288602650549683730 10.397363643876500210991 10.397571592189114105382 > > > > > plot(uu(1.03,theta),theta=0..Pi); > ?linsolve >