Maple 17 Questions and Posts

These are Posts and Questions associated with the product, Maple 17

I'm trying to plot the graph of a recursive function in Maple 17 but I keep getting the error Error, (in f) too many levels of recursion.

I need to plot a logarithmic graph in the range of x=1,...40. Here is the code:

with(plots); 
f:=x->(2.25*f(x-1)-0.5*f(x-2));
f(1):=1/3;
f(2):=1/12;
logplot(f(x),1..40);

How can I fix this problem? Maybe I need to write it in an iterative form, but I don't know how. Thank you very much for any help!

As I am trying to solve this integration:

restart; with(linalg); with(stats); with(plots); with(Statistics); with(LinearAlgebra); with(Optimization);
lambda0 := proc (t) options operator, arrow; gamma0+gamma1*t+gamma2*t^2 end proc;
lambda := lambda0(t)*exp(beta*s);
t1 := 145; t3 := 250; t2 := (t1+t3)*(1/2);
s := 1/(273.16+50); s1 := 1/(273.16+t1); s3 := 1/(273.16+t3); s2 := 1/(273.16+t2); gamma0 := 0.1e-3; gamma1 := .5; gamma2 := 0; beta := -3800;
c := 300; n := 200;
Theta := solve(1-exp(-(gamma0*tau1+(1/2)*gamma1*tau1^2+(1/3)*gamma2*tau1^3)*exp(beta*s1)) = 1-exp(-(gamma0*a+(1/2)*gamma1*a^2+(1/3)*gamma2*a^3)*exp(beta*s2)), a);

a := Theta[1];

Delta := solve(1-exp(-(gamma0*(a+tau2-tau1)+(1/2)*gamma1*(a+tau2-tau1)^2+(1/3)*gamma2*(a+tau2-tau1)^3)*exp(beta*s2)) = 1-exp(-(gamma0*b+(1/2)*gamma1*b^2+(1/3)*gamma2*b^3)*exp(beta*s3)), b);

b := Delta[1];

A1 := `assuming`([unapply(int(exp(beta*s1)*exp(-(gamma0*t+(1/2)*gamma1*t^2+(1/3)*gamma2*t^3)*exp(beta*s1))/(gamma0+gamma1*t+gamma2*t^`2`), t = N .. M), N, M)], [N > 0, M > 0]);
A2 := unapply(int(exp(beta*s2)*exp(-(gamma0*(a+t-tau1)+(1/2)*gamma1*(a+t-tau1)^2+(1/3)*gamma2*(a+t-tau1)^3)*exp(beta*s2))/(gamma0+gamma1*(a+t-tau1)+gamma2*(a+t-tau1)^2), t = N .. M), N, M);
A3 := unapply(int(exp(beta*s3)*exp(-(gamma0*(b+t-tau2)+(1/2)*gamma1*(b+t-tau2)^2+(1/3)*gamma2*(b+t-tau2)^3)*exp(beta*s3))/(gamma0+gamma1*(b+t-tau2)+gamma2*(b+t-tau2)^2), t = N .. M), N, M);
B1 := `assuming`([unapply(int(t^2*exp(beta*s1)*exp(-(gamma0*t+(1/2)*gamma1*t^2+(1/3)*gamma2*t^3)*exp(beta*s1))/(gamma2*t^2+gamma1*t+gamma0), t = N .. M), N, M)], [N > 0, M > 0]);
B2 := unapply(int((a+t-tau1)^2*exp(beta*s2)*exp(-(gamma0*(a+t-tau1)+(1/2)*gamma1*(a+t-tau1)^2+(1/3)*gamma2*(a+t-tau1)^3)*exp(beta*s2))/(gamma0+gamma1*(a+t-tau1)+gamma2*(a+t-tau1)^2), t = N .. M), N, M);
B3 := unapply(int((b+t-tau2)^2*exp(beta*s3)*exp(-(gamma0*(b+t-tau2)+(1/2)*gamma1*(b+t-tau2)^2+(1/3)*gamma2*(b+t-tau2)^3)*exp(beta*s3))/(gamma0+gamma1*(b+t-tau2)+gamma2*(b+t-tau2)^2), t = N .. M), N, M);

F0 := A1(0, tau1)+A2(tau1, tau2)+A3(tau2, c);
F1 := B1(0, tau1)+B2(tau1, tau2)+B3(tau2, c);

NLPSolve(1/(n^3*(F0*F1-F1)), tau1 = 115 .. 201, tau2 = 237 .. 273);

I need to have tau1 tau2 as varibles to get there optimal values ..

But this error keeps coming :


Error, (in Optimization:-NLPSolve) integration range or variable must be specified in the second argument, got HFloat(1.0) = HFloat(158.0) .. HFloat(255.0)

Please Help ..

I am a problem with solve differential equation, please help me: THANKS 

g := (y^2-1)^2; I4 := int(g^4, y = -1 .. 1); I5 := 2*(int(g^3*(diff(g, y, y)), y = -1 .. 1)); I6 := int(g^3*(diff(g, y, y, y, y)), y = -1 .. 1); with(Student[Calculus1]); I10 := ApproximateInt(6/(1-f(x)*g)^2, y = -1 .. 1, method = simpson);

dsys3 := {I4*f(x)^2*(diff(f(x), x, x, x, x))+I5*f(x)^2*(diff(f(x), x, x))+I6*f(x)^3 = I10, f(-1) = 0, f(1) = 0, ((D@@1)(f))(-1) = 0, ((D@@1)(f))(1) = 0};

dsol5 := dsolve(dsys3, numeric, output = array([0.]));

              Error, (in dsolve/numeric/bvp) system is singular at left endpoint, use midpoint method instead

****************FORMAT TWO ********************************************************

g := (y^2-1)^2; I4 := int(g^4, y = -1 .. 1); I5 := 2*(int(g^3*(diff(g, y, y)), y = -1 .. 1)); I6 := int(g^3*(diff(g, y, y, y, y)), y = -1 .. 1); with(Student[Calculus1]); I10 := ApproximateInt(6/(1-f(x)*g)^2, y = -1 .. 1, method = simpson);
dsys3 := {I4*f(x)^2*(diff(f(x), x, x, x, x))+I5*f(x)^2*(diff(f(x), x, x))+I6*f(x)^3 = I10, f(-1) = 0, f(1) = 0, ((D@@1)(f))(-1) = 0, ((D@@1)(f))(1) = 0};

dsol5 := dsolve(dsys3, method = bvp[midrich], output = array([0.]));
%;
                                   Error, (in dsolve) too many levels of recursion

I DONT KNOW ABOUT THIS ERROR

PLEASE HELP ME

THANKS A LOT

 

As am trying to solve this integration:


A(c,n,m):=evalf(int(1/(y)*exp(-c*y^(2)),y=n..m))

B(c,n,m):=evalf(int(exp(-c*y^(2)),y=n..m))

C(c,n,m):=evalf(int(y*exp(-c*y^(2)),y=n..m))

d(c,n,m):=evalf(int(y^(2)*exp(-c*y^(2)),y=n..m))

E(c,n,m):=evalf(int(y^(3)*exp(-c*y^(2)),y=n..m))

F0 := exp(beta*s1)*exp(gamma0^2*exp(beta*s1)/(2*gamma1))*A((1/2)*gamma1*exp(beta*s1), gamma0/gamma1,gamma0/gamma1+tau1)/gamma1+exp(beta*s2)*exp(gamma0^2*exp(beta*s2)/(2*gamma1))*A((1/2)*gamma1*exp(beta*s2), gamma0/gamma1+a, gamma0/gamma1+tau2-tau1+a)/gamma1+exp(beta*s3)*exp(gamma0^2*exp(beta*s3)/(2*gamma1))*A((1/2)*gamma1*exp(beta*s3), gamma0/gamma1+b, gamma0/gamma1+c-tau2+b)/gamma1

F1 := exp(beta*s1)*exp(gamma0^2*exp(beta*s1)/(2*gamma1))*(gamma0^2*A((1/2)*gamma1*exp(beta*s1), gamma0/gamma1, gamma0/gamma1+tau1)/gamma1^2-2*gamma0*B((1/2)*gamma1*exp(beta*s1), gamma0/gamma1, gamma0/gamma1+tau1)/gamma1+C((1/2)*gamma1*exp(beta*s1), gamma0/gamma1, gamma0/gamma1+tau1))/gamma1+exp(beta*s2)*exp(gamma0^2*exp(beta*s2)/(2*gamma1))*(gamma0^2*A((1/2)*gamma1*exp(beta*s2), gamma0/gamma1+a, gamma0/gamma1+tau2-tau1+a)/gamma1^2-2*gamma0*B((1/2)*gamma1*exp(beta*s2), gamma0/gamma1+a, gamma0/gamma1+tau2-tau1+a)/gamma1+C((1/2)*gamma1*exp(beta*s2), gamma0/gamma1+a, gamma0/gamma1+tau2-tau1+a))/gamma1+exp(beta*s3)*exp(gamma0^2*exp(beta*s3)/(2*gamma1))*(gamma0^2*A((1/2)*gamma1*exp(beta*s3), gamma0/gamma1+b, gamma0/gamma1+c-tau2+b)/gamma1^2-2*gamma0*B((1/2)*gamma1*exp(beta*s3), gamma0/gamma1+b, gamma0/gamma1+c-tau2+b)/gamma1+C((1/2)*gamma1*exp(beta*s3), gamma0/gamma1+b, gamma0/gamma1+c-tau2+b))/gamma1

F01 := exp(beta*s1)*exp(gamma0^2*exp(beta*s1)/(2*gamma1))*(B((1/2)*gamma1*exp(beta*s1), gamma0/gamma1, gamma0/gamma1+tau1)-gamma0*A((1/2)*gamma1*exp(beta*s1), gamma0/gamma1, gamma0/gamma1+tau1)/gamma1)/gamma1+exp(beta*s2)*exp(gamma0^2*exp(beta*s2)/(2*gamma1))*(B((1/2)*gamma1*exp(beta*s2), gamma0/gamma1+a, gamma0/gamma1+tau2-tau1+a)-gamma0*A((1/2)*gamma1*exp(beta*s2), gamma0/gamma1+a, gamma0/gamma1+tau2-tau1+a)/gamma1)/gamma1+exp(beta*s3)*exp(gamma0^2*exp(beta*s3)/(2*gamma1))*(B((1/2)*gamma1*exp(beta*s3), gamma0/gamma1+b, gamma0/gamma1+c-tau2+b)-gamma0*A((1/2)*gamma1*exp(beta*s3), gamma0/gamma1+b, gamma0/gamma1+c-tau2+b)/gamma1)/gamma1

`Fβ` := int((s1^2*(gamma0*t+(1/2)*gamma1*t^2)*exp(beta*s1)*(gamma1*t+gamma0)*exp(beta*s1))*exp(-(gamma0*t+(1/2)*gamma1*t^2)*exp(beta*s1)), t = 0 .. tau1)+int((s2^2*(gamma0*(a+t-tau1)+(1/2)*gamma1*(a+t-tau1)^2)*exp(beta*s2)*(gamma0+gamma1*(a+t-tau1))*exp(beta*s2))*exp(-(gamma0*(a+t-tau1)+(1/2)*gamma1*(a+t-tau1)^2)*exp(beta*s2)), t = tau1 .. tau2)+int((s3^2*(gamma0*(b+t-tau2)+(1/2)*gamma1*(b+t-tau2)^2)*exp(beta*s3)*(gamma0+gamma1*(b+t-tau2))*exp(beta*s3))*exp(-(gamma0*(b+t-tau2)+(1/2)*gamma1*(b+t-tau2)^2)*exp(beta*s3)), t = tau2 .. c)+int((s3^2*(gamma0*(b+t-tau2)+(1/2)*gamma1*(b+t-tau2)^2)*exp(beta*s3)*(gamma0+gamma1*(b+t-tau2))*exp(beta*s3))*exp(-(gamma0*(b+t-tau2)+(1/2)*gamma1*(b+t-tau2)^2)*exp(beta*s3)), t = c .. infinity)

I need to have tau2 as varibles to get there optimal values ..

Minimize(1/((F0*F1-F01^2)*n^3*`Fβ`), tau2 = 237..273})

But this error keeps coming :

Error, (in Optimization:-NLPSolve) integration range or variable must be specified in the second argument, got HFloat(1.0) = 121.0828419 .. HFloat(193.0828419)

Please Help ..

Dear all, 

I'm trying to extract the coefficients from the equation below, the fat expressions in the equation. I don't have any trouble seperating the sine or cosine functions. But the constants are a problem. Since t is the only variable in the function i tried, coeff(R, t, 0). This does not work apparantly. Any suggestions? 

 

R:=(1/12)*C2^3*cos(2*t) - (1/48)*C2^3*cos(4*t) - C2^3*sin(t) + C2^3*sin(3*t)-C2^2*C4*cos(t) + C2^2*C4*cos(3*t) - (1/8)*C2^2*C4*sin(2*t) + (1/16)*C2^2*C4*sin(4*t) + (1/16)*C2*C4^2*cos(4*t) - C2*C4^2*sin(t) - C2*C4^2*sin(3*t) - C4^3*cos(t) - C4^3*cos(3*t) - (1/24)*C4^3*sin(2*t) - (1/48)*C4^3*sin(4*t) - (1/16)*C2^3 - (1/16)*C2*C4^2 - (1/2)*C2*cos(2*t) + C2*sin(t) + C4*cos(t) + (1/2)*C4*sin(2*t) + (1/2)*C2

Hello everyone,

i'm trying to simulate a diffusion problem. It contains two connected regions in which a species is diffusing at different speeds. In one region (zeta) one boundary is set to be constant whereas in the other region (c) there is some oscillation at the boundary.The code i try to use is as follows:

sys1 := [diff(c(x, t), t) = gDiffusion*10^5*diff(c(x, t), x$2), diff(zeta(x, t), t) = KDiffusion*10^6*diff(zeta(x, t), x$2)]

pds := pdsolve(sys1, IBC, numeric, time = t, range = 0 .. 3000, spacestep = 3)

However the main problem are my boundary conditions:

IBC := {c(0, t) = 0, c(x > 0, 0) = 0, zeta(0, t) = .4, zeta(x > 0, 0) = .4, (D[1](c))(3000, t) = sin((1/100)*t), (D[1](zeta))(0, t) = 0}

Like this it principally works (however it is apparently ill-posed).

Now what i do like is that the two equations are coupled at x=2000 with the condition that c(2000,t)=zeta(2000,t). This however i dont seem to be able to implement.

I appreciate your comments

Goon

Hi,

Hello Maple-Primers!

I am trying to evaluate a system at many different points.  I would like to include an interpolation function in this system, but have thusfar been unsuccessful.

Usually, I solve a system symbolically by using eliminate and unapply:

eq[1] := A = M^3;
eq[2] := C = A*2;
eq[3] := D = N+3;
eq[4] := B = piecewise(A = 0, 0,C);
eq[5] := E = B*D;
elimsol:=eliminate(convert(eq,list),[A,B,C,D,E])[1];

unappsol:=unapply(elimsol,[N,M]);

unappsol(1,2);
{A = 8, B = 16, C = 16, D = 4, E = 64} <--- great!

Now, I want to include an interpolation function in the system of equations.  They look like this (see worksheet for actual interpolation function):

B_interp := (W,T) -> CurveFitting:-ArrayInterpolation([FC_Map_W,FC_Map_T],FC_Map,Array(1 .. 1, 1 .. 1, 1 .. 2, [[[W, T]]]),method=linear);

eq[5] := E = B_interp(N,M);

Error, (in CurveFitting:-ArrayInterpolation) invalid input: coordinates of xvalues must be of type numeric <-- bad!

Anyone have any ideas?  I've tried to use polynomials, but I can't seem to get a fit close enough for my purposes.

Maple_2D_Interpolate_FC.mw

Hello,

       How long can I expect Maple17 to take to algebraically solve a system of 14 nonlinear equations that has approximately 40% nonlinearity in its terms? I am running it on the machine right now, but have no idea what to expect. As mentioned before, I'm new to Maple...

Here is my code:

restart; eq1 := A*z-B*a*z-V*a*q-W*(b+d)*a = 0; eq2 := W*(b+d)*a-V*b*q-(F*G+B+D)*b*z = 0; eq3 := V*a*q-W*c*(b+d)-(B+C+E)*c*z = 0; eq4 := V*b*q+W*(b+d)*c-(B+C+D+F)*d*z = 0; eq5 := G*F*b*z-V*q*e-(B+H)*e*z = 0; eq6 := H*e*z-V*q*f-(B+S)*f*z = 0; eq7 := S*f*z-V*q*g-B*g*z = 0; eq8 := V*q*g+S*s*z-(B+C+E)*h*z = 0; eq9 := F*d*z+V*q*e-(B+C+H+T)*t*z = 0; eq10 := H*t*z+V*q*f-(U+B+C+2*S)*s*z = 0; eq11 := T*t*z-(B+H+Y)*u*z = 0; eq12 := U*s*z-(B+S)*v*z+H*u*z-Y*H*v*z/(H+S) = 0; eq13 := g-c-d-t-s-h = 0; eq14 := z-a-b-c-d-e-f-g-h-s-t-u-v = 0; soln := solve({eq1, eq10, eq11, eq12, eq13, eq14, eq2, eq3, eq4, eq5, eq6, eq7, eq8, eq9}, {a, b, c, d, e, f, g, h, q, s, t, u, v, z});

Thanks.

 

 

Greetings,

       I am new to Maple and this forum. I would like to obtain a Jacobian of a system of 12 ODEs. What have I done wrongly with my code?

eq_1 := -B*a+A-V*(c+d+t+s+h)*a/(a+b+c+d+e+f+g+h+s+t+u+v)-W*(b+d)*a/(a+b+c+d+e+f+g+h+s+t+u+v);
eq_2 := W*(b+d)*a/(a+b+c+d+e+f+g+h+s+t+u+v)-V*(c+d+t+s+h)*b/(a+b+c+d+e+f+g+h+s+t+u+v)-(F*G+B+D)*b;
eq_3 := V*(c+d+t+s+h)*a/(a+b+c+d+e+f+g+h+s+t+u+v)-W*(b+d)*c/(a+b+c+d+e+f+g+h+s+t+u+v)-(B+E+C)*c;
eq_4 := V*(c+d+t+s+h)*b/(a+b+c+d+e+f+g+h+s+t+u+v)+W*(b+d)*c/(a+b+c+d+e+f+g+h+s+t+u+v)-(B+C+D+F)*d;
eq_5 := G*F*b-V*(c+d+t+s+h)*e/(a+b+c+d+e+f+g+h+s+t+u+v)-(B+H)*e;
eq_6 := H*e-V*(c+d+t+s+h)*f/(a+b+c+d+e+f+g+h+s+t+u+v)-(B+S)*f;
eq_7 := S*f-V*(c+d+t+s+h)*g/(a+b+c+d+e+f+g+h+s+t+u+v)-B*g;
eq_8 := V*(c+d+t+s+h)*g/(a+b+c+d+e+f+g+h+s+t+u+v)+S*s-(B+E+C)*h;
eq_9 := F*d+V*(c+d+t+s+h)*e/(a+b+c+d+e+f+g+h+s+t+u+v)-(B+C+H+T)*t;
eq_10 := H*t+V*(c+d+t+s+h)*f/(a+b+c+d+e+f+g+h+s+t+u+v)-(U+B+C+S+S)*s;
eq_11 := T*t+W*(b+d)*x/(a+b+c+d+e+f+g+h+s+t+u+v)-(B+H+Y)*u;
eq_12 := U*s-(B+S)*v+H*u-Y*H*v/(H+S);
with(linalg);
J := Jacobian([eq_1, eq_2, eq_3, eq_4, eq_5, eq_6, eq_7, eq_8, eq_9, eq_10, eq_11, eq_12], [a, b, c, d, e, f, g, h, s, t, u, v]);

I am getting the message: 

 Vector(4, {(1) = ` 12 x 12 `*Matrix, (2) = `Data Type: `*anything, (3) = `Storage: `*rectangular, (4) = `Order: `*Fortran_order})

Thanks!!

Hello,

       I am new to this forum. I have typed the follwing code in Maple17:

restart; eq1 := A-B*a-V*a*q/z-W*(b+d)*a/z = 0; eq2 := W*(b+d)*a/z-V*b*q/z-(F*G+B+D)*b = 0; eq3 := V*a*q/z-W*c(b+d)/z-(B+C+E)*c = 0; eq4 := V*b*q/z+W*(b+d)*c/z-(B+C+D+F)*d = 0; eq5 := G*F*b-V*q*e/z-(B+H)*e = 0; eq6 := H*e-V*q*f/z-(B+S)*f = 0; eq7 := S*f-V*q*g/z-B*g = 0; eq8 := V*q*g/z+S*s-(B+C+E)*h = 0; eq9 := F*d+V*q*e/z-(B+C+H+T)*t = 0; eq10 := H*t+V*q*f/z-(U+B+C+2*S)*s = 0; eq11 := T*t+W*(b+d)*x/z-(B+H+Y)*u = 0; eq12 := U*s-(B+S)*v+H*u-Y*H*v/(H+S) = 0; eq13 := g-c-d-t-s-h = 0; eq14 := z-a-b-c-d-e-f-g-h-s-t-u-v = 0; soln := solve({eq1, eq10, eq11, eq12, eq13, eq14, eq2, eq3, eq4, eq5, eq6, eq7, eq8, eq9}, {a, b, c, d, e, f, g, h, q, s, t, u, v, z});

 

This is to symbolically solve a nonlinear system of (14) equations. But when I press Enter, it just returns the message "Ready". Shouldn't it say "Evaluating"?

I don't see anything syntactically wrong with my code...

Hello there!

There seems to be an issue with indexed variables and the instruction "DGsetup" of the differential geometry package when used with Maple 17. An error is returned to the effect that DGsetup is expecting independent variables to be unassigned names. This phenomenon does not occur with Maple 16!

Here is what I get:

> restart;
> with(DifferentialGeometry); with(Tools); with(Tensor); with(LinearAlgebra);

Executing the following command, I get an error with Maple 17 which does not occur with Maple 16!

> DGsetup([seq(x[i], i = 1 .. 4)], M, verbose);
Error, (in DifferentialGeometry:-DGsetup) expected 1st independent variable to be an unassigned name, received: x[1]

Is there any fix for this problem?

Kind regards
Freddy Baudine

 

solve Differential equation "a-y=y' bc" use maple 17

the result is y(x)=a+_C1e^-(1/bc)

but the correct result  isn't y(x)=a-_C1e^-(1/bc) ?

Thank you in advance for your help

 

 

hi.i encountered this erroe  [Error, (in dsolve/numeric/bvp/convertsys) unable to convert to an explicit first-order system] with solving set of differential equation.please help me.thanks a lot  

dsys3 := {`1`*h1(theta)+`1`*(diff(h1(theta), theta, theta))+`1`*(diff(h2(theta), theta))+`1`*(diff(h2(theta), theta, theta, theta))+`1`*h3(theta)+`1`*(diff(h3(theta), theta, theta))+`1`*(diff(h1(theta), theta, theta, theta, theta)) = 0, `1`*h2(theta)+`1`*(diff(h2(theta), theta, theta, theta, theta))+`1`*(diff(h2(theta), theta, theta))+`1`*(diff(h1(theta), theta))+`1`*(diff(h1(theta), theta, theta, theta))+`1`*(diff(h3(theta), theta))+`1`*(diff(h3(theta), theta, theta, theta)) = 0, h3(theta)^5*(`1`+ln(h3(theta))^2*`1`+2*ln(h3(theta))*`1`)+(diff(h3(theta), theta, theta))*h3(theta)^4*(`1`+ln(h3(theta))^2*`1`+2*ln(h3(theta))*`1`)+(diff(h3(theta), theta, theta, theta, theta))*h3(theta)^4*(`1`+ln(h3(theta))^2*`1`+2*ln(h3(theta))*`1`)+h1(theta)*h3(theta)^4*(`1`+ln(h3(theta))^2*`1`+2*ln(h3(theta))*`1`)+(diff(h1(theta), theta, theta))*h3(theta)^4*(`1`+ln(h3(theta))^2*`1`+2*ln(h3(theta))*`1`)+(diff(h2(theta), theta))*h3(theta)^4*(`1`+ln(h3(theta))^2*`1`+2*ln(h3(theta))*`1`)+(diff(h2(theta), theta, theta, theta))*h3(theta)^4*(`1`+ln(h3(theta))^2*`1`+2*ln(h3(theta))*`1`)+h3(theta)^4*(`1`+ln(h3(theta))^2*`1`+2*ln(h3(theta))*`1`)+h3(theta)^4*(diff(h2(theta), theta, theta, theta, theta, theta, theta))*(`1`+ln(h3(theta))^2*`1`+2*ln(h3(theta))*`1`)-beta*h3(theta)^3*`1`-chi*ln(h3(theta))^2*`1`/kappa-chi*`1`/kappa-2*chi*ln(h3(theta))*`1`/kappa = 0, h1(0) = 0, h1(1) = 0, h2(0) = 0, h2(1) = 0, h3(0) = 1, h3(1) = 1, ((D@@1)(h1))(0) = 0, ((D@@1)(h1))(1) = 0, ((D@@1)(h2))(0) = 0, ((D@@1)(h2))(1) = 0, ((D@@1)(h3))(0) = 0, ((D@@1)(h3))(1) = 0, ((D@@2)(h3))(0) = 0, ((D@@2)(h3))(1) = 0}; dsol5 := dsolve(dsys3, 'maxmesh' = 600, numeric, output = listprocedure);
%;
Error, (in dsolve/numeric/bvp/convertsys) unable to convert to an explicit first-order system

 

What´s the error here??????

Solução do Sistema de EDO's por Transformada de Laplace

 

restart

with(inttrans):

eq1 := diff(x(t), t)+(2.2*x(t)*y(t)+0.5e-1*x(t)/(5+0.5e-1*t)) = 0;

diff(x(t), t)+2.2*x(t)*y(t)+0.5e-1*x(t)/(5+0.5e-1*t) = 0

(1)

eq2 := diff(y(t), t)+(2.2*x(t)*y(t)-(0.5e-1*(0.25e-1-y(t)))/(5+0.5e-1*t)) = 0;

diff(y(t), t)+2.2*x(t)*y(t)-0.5e-1*(0.25e-1-y(t))/(5+0.5e-1*t) = 0

(2)

eq3 := diff(z(t), t)-2.2*x(t)*y(t)+0.5e-1*z(t)/(5+0.5e-1*t) = 0;

diff(z(t), t)-2.2*x(t)*y(t)+0.5e-1*z(t)/(5+0.5e-1*t) = 0

(3)

EQ := [eq1, eq2, eq3]:

for i to 3 do La[i] := laplace(EQ[i], t, s) end do;

s*laplace(x(t), t, s)-1.*x(0.)+2.200000000*laplace(x(t)*y(t), t, s)+laplace(x(t)/(100.+t)^1., t, s) = 0.

 

-1.*y(0.)-0.2500000000e-1*(exp(100.*s))^1.*Ei(1., 100.*s)^1.+1.*s^1.*laplace(y(t), t, s)^1.+2.200000000*laplace(x(t)^1.*y(t)^1., t, s)+1.*laplace(y(t)^1./(100.+1.*t)^1., t, s) = 0.

 

s*laplace(z(t), t, s)-1.*z(0.)-2.200000000*laplace(x(t)*y(t), t, s)+laplace(z(t)/(100.+t)^1., t, s) = 0.

(4)

LL := subs({laplace(x(t), t, s) = X, laplace(y(t), t, s) = Y, laplace(z(t), t, s) = Z}, [La[1], La[2], La[3]]);

[s*X-1.*x(0.)+2.200000000*laplace(x(t)*y(t), t, s)+laplace(x(t)/(100.+t)^1., t, s) = 0., -1.*y(0.)-0.2500000000e-1*(exp(100.*s))^1.*Ei(1., 100.*s)^1.+1.*s^1.*Y^1.+2.200000000*laplace(x(t)*y(t), t, s)+1.*laplace(y(t)/(100.+t)^1., t, s) = 0., s*Z-1.*z(0.)-2.200000000*laplace(x(t)*y(t), t, s)+laplace(z(t)/(100.+t)^1., t, s) = 0.]

(5)

sol := solve(LL, [X, Y, Z]):

assign(sol):

SOLS[X, Y, Z]:

SOLT := map(invlaplace, [X, Y, Z], s, t);

[-2.200000000*(int(x(_U1)*y(_U1), _U1 = 0. .. t))-1.*(int(x(_U1)/(100.+_U1), _U1 = 0. .. t))+x(0), -1.*(int(y(_U1)/(100.+_U1), _U1 = 0. .. t))-2.200000000*(int(x(_U1)*y(_U1), _U1 = 0. .. t))+y(0)+0.2500000000e-1*ln(1.+0.1000000000e-1*t), 2.200000000*(int(x(_U1)*y(_U1), _U1 = 0. .. t))-1.*(int(z(_U1)/(100.+_U1), _U1 = 0. .. t))+z(0)]

(6)

SOLTT := evalf(subs({x(0) = 0.5e-1, y(0) = 0, z(0) = 0}, SOLT));

[-2.200000000*(int(x(_U1)*y(_U1), _U1 = 0. .. t))-1.*(int(x(_U1)/(100.+_U1), _U1 = 0. .. t))+0.5e-1, -1.*(int(y(_U1)/(100.+_U1), _U1 = 0. .. t))-2.200000000*(int(x(_U1)*y(_U1), _U1 = 0. .. t))+0.2500000000e-1*ln(1.+0.1000000000e-1*t), 2.200000000*(int(x(_U1)*y(_U1), _U1 = 0. .. t))-1.*(int(z(_U1)/(100.+_U1), _U1 = 0. .. t))]

(7)

xx := evalc(Re(SOLTT[1]));

-2.200000000*(int(x(_U1)*y(_U1), _U1 = 0. .. t))-1.*(int(x(_U1)/(100.+_U1), _U1 = 0. .. t))+0.5e-1

(8)

yy := evalc(Re(SOLTT[2]));

0.2500000000e-1*ln(abs(1.+0.1000000000e-1*t))-1.*(int(y(_U1)/(100.+_U1), _U1 = 0. .. t))-2.200000000*(int(x(_U1)*y(_U1), _U1 = 0. .. t))

(9)

zz := evalc(Re(SOLTT[3]));

2.200000000*(int(x(_U1)*y(_U1), _U1 = 0. .. t))-1.*(int(z(_U1)/(100.+_U1), _U1 = 0. .. t))

(10)

plot([xx, yy, zz], t = 0 .. 500, legend = [x, y, z]);

Warning, expecting only range variable t in expression -2.200000000*int(x(_U1)*y(_U1),_U1 = 0. .. t)-1.*int(x(_U1)/(100.+_U1),_U1 = 0. .. t)+.5e-1 to be plotted but found names [_U1, x, y]

 

 

NULL

NULL


Download laplace.mw

First 32 33 34 35 36 37 38 Last Page 34 of 61