A brief introduction to finite element methods

Size: px
Start display at page:

Download "A brief introduction to finite element methods"

Transcription

1 CHAPTER A brief introduction to finite element methods 1. Two-point boundary value problem and the variational formulation 1.1. The model problem. Consider the two-point boundary value problem: Given a constant a and a function f(x, find u(x such that { u +au = f(x, < x < 1, u( =, u (.1 (1 = The variational formulation. If u is the solution to (.1 and v(x is any (sufficiently regular function such that v( =, then integration by parts yields u vdx+ auvdx = u (1v(1+u (v(+ = fvdx. Let us introduce the bilinear form and define A(u,v = u (xv (xdx+ (u v +auvdx, V = { v L 2 ([,1] : A(v,v < and v( = }. Then we can see that the solution u to (.1 is characterized by u V such that A(u,v = which is called the variational or weak formulation of (.1. auvdx f(xv(xdx v V. (.2 Theorem 1.1. Suppose f C ([,1] and u C 2 ([,1] satisfies (.2. Then u solves (.1. Proof. Let v V C 1 ([,1]. Then integration by parts gives fvdx = A(u,v = u vdx+ auvdx+u (1v(1. (.3 Thus, (f +u auvdx = for all v V C 1 ([,1] such that v(1 =. Let w = f +u au C ([,1]. If w, then w(x is of one sign in some interval [b,c] [,1], with b < c. Choose v(x = (x b 2 (x c 2 in [b,c] and v outside 1

2 2. A BRIEF INTRODUCTION TO FINITE ELEMENT METHODS [b,c]. But then wvdx which is a contradiction. Thus u +au = f. Now apply (.3 with v(x = x to find u (1 =. So u solves (.1. Weremarkthattheboundaryconditionu( = iscalledessential asitappears in the variational formulation explicitly, i.e., in the definition of V. This type of boundary condition is also called Dirichlet boundary condition. The boundary condition u ( = is called natural as it is incorporated implicitly. This type of boundary condition is often referred to by the name Neumann. 2. The finite element method 2.1. Meshes. Let M h be a partition of [,1]: = x < x 1 < x 2 < < x n 1 < x n = 1. The points {x i } are called nodes. Let h i = x i be the length of the i-th subinterval [,x i ]. Define h = max 1 i n h i Finite element spaces. We shall approximate the solution u(x by using the continuous piecewise linear functions over M h. Introduce the linear space of functions V h = { v C ([,1] : v( =, It is clear that V h V. v [xi 1,x i] is a linear polynomial, i = 1,,n }. ( The finite element method. The finite element discretization of (.2 reads as: Find u h V h such that A(u h,v h = f(xv h (xdx v h V h. ( A nodal basis. For i = 1,,n, define φ i V h by the requirement that φ i (x j = δ ij = the Kronecker delta, as shown in Fig. 1: φ i (x φ n (x x 1 x i x i+1 1 x 1 x i x n 1 1 Figure 1. piecewise linear basis function φ i.

3 φ i = φ n = x 2. THE FINITE ELEMENT METHOD 3 h i, x x i, x i+1 x h i+1, x i < x x i+1,, x < or x > x i+1, { x xn 1 h n, x n 1 x 1,, x < x n 1. For any v h V h, let v i be the value of v h at the node x i, i.e., then v i = v h (x i, i = 1,2,,n, v h = v 1 φ 1 (x+v 2 φ 2 (x+ +v n φ n (x The finite element equations. Let 1 i n 1. u h = u 1 φ 1 +u 2 φ 2 + +u n φ n, u 1,,u n R, where u i = u h (x i. Let v h = φ i, i = 1,,n in (.5, then we obtain an algebraic linear system in unknowns u 1,u 2,,u n : Denote by A(φ 1,φ i u 1 +A(φ 2,φ i u 2 + +A(φ n,φ i u n = k ij = A(φ j,φ i = φ j φ i +aφ jφ i dx, f i = i = 1,,n. f(xφ i dx, f(xφ i dx, (.6 and K = ( k ij n n, F = ( f i n 1, U = ( u i n 1, then (.6 can be rewritten as: KU = F (.7 Here K is called the stiffness matrix. It is clear that k ij = if x i and x j are not adjacent to each other. Therefore K is sparse. Next we compute k ij = A(φ j,φ i. Note that xl k ij = A(φ j,φ i = φ jφ i +aφ j φ i dx. On the interval [,x l ], the following integrals are involved. k l 11 := xl k l 12 := xl l=1 φ l 1 φ l 1 +aφ l 1φ l 1 dx, k l 21 := xl φ l φ l 1 +aφ lφ l 1 dx, k l 22 := φ l 1 φ l +aφ l 1φ l dx, xl x l φ l φ l +aφ lφ l dx, Some simple calculations yield k l 11 = kl 22 = 1 h l + a 3 h l, k l 12 = kl 21 = 1 h l + a 6 h l.

4 4. A BRIEF INTRODUCTION TO FINITE ELEMENT METHODS The matrix K l := (k ij 2 2 is called the element stiffness matrix on [,x l ]. The stiffness matrix K can be assembled by using the element stiffness matrices as follows. k22 i +ki+1 11 = a k ii = h i h i+1 3 (h i +h i+1, i = 1,,n 1, k22 n = 1 + a h n 3 h n, i = n, k i 1,i = k i,i 1 = k i 12 = 1 h i + a 6 h i, i = 2,,n. Combining the above equations and (.6 yields [ a(h1+h 2 ] h h u1 2 + ( ah h u2 2 = f 1, ( ahi 6 1 h ui 1 i + [ a(h i+h i+1 ] h i + 1 h ui i+1 + ( ah i h ui+1 i+1 = f i i = 2,,n 1, ( ahn 6 1 h un 1 n + [ ah n ] h un n = f n The interpolant. Given u C ([,1], the interpolant u I V h of u is determined by u I = u(x i φ i. It is clear that u I (x i = u(x i, i =,1,,n, and u I (x = x i x u( + x u(x i for x [,x i ]. h i h i Denote by τ i = [,x i ] and by g L2 (τ i = ( x i g 2 dx 1/2. Theorem 2.1. u u I L2 (τ i 1 π h i u L2 (τ i, (.8 u u I L2 (τ i 1 π 2h2 i u L2 (τ i, (.9 u u I L 2 (τ i 1 π h i u L 2 (τ i. (.1 Proof. We only prove (.8 and leave the others as an exercise. We first change (.8 to the reference interval [,1]. Let ˆx = (x /h i and let ê(ˆx = u(x u I (x. Note that ê( = ê(1 = and k = u I is a constant. The inequality (.8 is equivalent to that is ê 2 L 2 ([,1] = 1 h i u u I 2 L 2 (τ i h i π 2 u 2 L 2 (τ i = 1 π 2 ê +kh i 2 L 2 ([,1], ê 2 L 2 ([,1] 1 π 2 ê 2 L 2 ([,1] + 1 π 2 kh i 2 L 2 ([,1]. (.11 Sinceê( = ê(1 =, it followsfromthe Fourierexpansionê(ˆx = n=1 a nsinnπˆx and the Parseval s identity that ê 2 L 2 ([,1] 1 π ê 2 2 L 2 ([,1], which implies (.11. This completes the proof of (.8.

5 2. THE FINITE ELEMENT METHOD A priori error estimate. Introduce the energy norm From the Cauchy inequality, v = A(v,v 1/2. A(u,v u v. By taking v = v h V h in (.2 and subtracting it from (.5, we have the following fundamental orthogonality Therefore A(u u h,v h = v h V h. (.12 u u h 2 = A(u u h,u u h = A(u u h,u u I u u h u u I, It follows from Theorem 2.1 that [ n ] 1/2 u u h u u I = ( u u I 2 L 2 (τ +a u u i I 2 L 2 (τ i [ n (( h 2 u ( 2 h 4 u ] 1/2 L π 2 (τ +a i 2 L π 2 (τ i = h [ ( ( h 2 1+a π π 1/2 (u dx] 2. We have proved the following error estimate. Theorem 2.2. u u h h ( ( h 2 1/2 u 1+a π π L2([,1]. Since the above estimate depends on the unknown solution u, it is called the a priori error estimate A posteriori error estimates. We will derive error estimates independent of the unknown solution u. Let e = u u h. Then A(e,e = A(u u h,e e I = = f (e e I dx (f au h (e e I dx u h (e e I dx u h (e e I dx Since u h is constant on each interval (,x i, A(e,e = (f au h (e e I dx f au h L 2 (τ e e i I L 2 (τ i h i π f au h L2 (τ i e L2 (τ i. au h (e e I dx

6 6. A BRIEF INTRODUCTION TO FINITE ELEMENT METHODS Here we have used Theorem 2.1 to derive the last inequality. Define the local error estimator on the element τ i = [,x i ] as follows Then η i = 1 π h i f au h L2 (τ i. (.13 ( n 1/2 ( n 1/2 e 2 ηi 2 e ηi 2 e. That is, we have the following a posteriori error estimate. Theorem 2.3 (Upper bound. ( n 1/2 u u h ηi 2. (.14 Now a question is if the above upper bound overestimates the true error. To answer this question we introduce the following theorem that gives a lower bound of the true error. Theorem 2.4 (Lower bound. Define φ τi = ( x i ((φ 2 +aφ 2 dx 1/2. Let (f au h i = 1 xi h i (f au h dx and osc i = 1 π h i f au h (f au h i L2 (τ. i Then As a consequence ( n 5π 2 u u h 6+6ah 2 i η i 5+ 3 ( 6+6ah 2 1 osc i i 2 5 5π 2 u u h τi. (.15 ( ( max η i /2 osc i,. (.16 Proof. For simplicity, denote by R = f au h and R i = (f au h i. For any ψ V, it is clear that A(e,ψ = Rψdx u h ψ dx (.17 Define ψ i (x = φ i 1 (xφ i (x if x τ i and ψ i (x = otherwise. Choose ψ = ψ i R i. By simple calculations, we obtain R i ψdx = 1 6 R i 2 L 2 (τ i, 3 ψ L 2 (τ i = 3h i ψ L 2 (τ i = R i L 2 (τ i. From (.17, We have, which implies A(e,ψ = Rψdx = (R R i ψdx+ 1 6 R i 2 L 2 (τ i. R i 2 L 2 (τ 6 e i τi ψ τi +6πosc i ψ L 2 (τ i (( = 12+ 6ah2 1 2 i e τi + π 3 osc i h 1 i R i 5 5 L2 (τ, i ( h i R i L 2 (τ i 12+ 6ah2 1 i 2 5 e τi + π 3 osc i 5

7 3. EXERCISES 7 Now the proof is completed by using η i 1 π h i R i L 2 (τ i +osc i. We remark that the term osc i is of high order compared to η i if f and a are smooth enough on τ i. Example 2.5. We solve the following problem by the linear finite element method. The true solution (see Fig. 2 is u +1u = 1, < x < 1, u( = u(1 =. u = 1 1 (1 e1x +e 1(1 x 1+e 1 If we use the uniform mesh obtained by dividing the interval [,1] into 18 subintervals of equal length, then the error u u h On the other hand, if we use a non-uniform mesh as shown in Fig. 2 which also contains 18 subintervals, then the error u u h is smaller than that obtained by using the uniform mesh.. x Figure 2. Example 2.5. The finite element solution and the mesh. 3. Exercises Exercise.1. Prove (.9 and (.1. Exercise.2. Use Example 2.5 to verify numerically the a posteriori error estimates in Theorem 2.3 and (.16 in Theorem 2.4.

1 Discretizing BVP with Finite Element Methods.

1 Discretizing BVP with Finite Element Methods. 1 Discretizing BVP with Finite Element Methods In this section, we will discuss a process for solving boundary value problems numerically, the Finite Element Method (FEM) We note that such method is a

More information

1. Let a(x) > 0, and assume that u and u h are the solutions of the Dirichlet problem:

1. Let a(x) > 0, and assume that u and u h are the solutions of the Dirichlet problem: Mathematics Chalmers & GU TMA37/MMG800: Partial Differential Equations, 011 08 4; kl 8.30-13.30. Telephone: Ida Säfström: 0703-088304 Calculators, formula notes and other subject related material are not

More information

Chapter 1: The Finite Element Method

Chapter 1: The Finite Element Method Chapter 1: The Finite Element Method Michael Hanke Read: Strang, p 428 436 A Model Problem Mathematical Models, Analysis and Simulation, Part Applications: u = fx), < x < 1 u) = u1) = D) axial deformation

More information

Numerical Methods for Partial Differential Equations

Numerical Methods for Partial Differential Equations Numerical Methods for Partial Differential Equations Eric de Sturler University of Illinois at Urbana-Champaign Read section 8. to see where equations of type (au x ) x = f show up and their (exact) solution

More information

Scientific Computing I

Scientific Computing I Scientific Computing I Module 8: An Introduction to Finite Element Methods Tobias Neckel Winter 2013/2014 Module 8: An Introduction to Finite Element Methods, Winter 2013/2014 1 Part I: Introduction to

More information

Lehrstuhl Informatik V. Lehrstuhl Informatik V. 1. solve weak form of PDE to reduce regularity properties. Lehrstuhl Informatik V

Lehrstuhl Informatik V. Lehrstuhl Informatik V. 1. solve weak form of PDE to reduce regularity properties. Lehrstuhl Informatik V Part I: Introduction to Finite Element Methods Scientific Computing I Module 8: An Introduction to Finite Element Methods Tobias Necel Winter 4/5 The Model Problem FEM Main Ingredients Wea Forms and Wea

More information

Finite Element Method for Ordinary Differential Equations

Finite Element Method for Ordinary Differential Equations 52 Chapter 4 Finite Element Method for Ordinary Differential Equations In this chapter we consider some simple examples of the finite element method for the approximate solution of ordinary differential

More information

One-dimensional and nonlinear problems

One-dimensional and nonlinear problems Solving PDE s with FEniCS One-dimensional and nonlinear problems L. Ridgway Scott The Institute for Biophysical Dynamics, The Computation Institute, and the Departments of Computer Science and Mathematics,

More information

AMS 529: Finite Element Methods: Fundamentals, Applications, and New Trends

AMS 529: Finite Element Methods: Fundamentals, Applications, and New Trends AMS 529: Finite Element Methods: Fundamentals, Applications, and New Trends Lecture 3: Finite Elements in 2-D Xiangmin Jiao SUNY Stony Brook Xiangmin Jiao Finite Element Methods 1 / 18 Outline 1 Boundary

More information

Scientific Computing WS 2018/2019. Lecture 15. Jürgen Fuhrmann Lecture 15 Slide 1

Scientific Computing WS 2018/2019. Lecture 15. Jürgen Fuhrmann Lecture 15 Slide 1 Scientific Computing WS 2018/2019 Lecture 15 Jürgen Fuhrmann juergen.fuhrmann@wias-berlin.de Lecture 15 Slide 1 Lecture 15 Slide 2 Problems with strong formulation Writing the PDE with divergence and gradient

More information

Numerical Solutions to Partial Differential Equations

Numerical Solutions to Partial Differential Equations Numerical Solutions to Partial Differential Equations Zhiping Li LMAM and School of Mathematical Sciences Peking University Variational Problems of the Dirichlet BVP of the Poisson Equation 1 For the homogeneous

More information

The Finite Element Method for the Wave Equation

The Finite Element Method for the Wave Equation The Finite Element Method for the Wave Equation 1 The Wave Equation We consider the scalar wave equation modelling acoustic wave propagation in a bounded domain 3, with boundary Γ : 1 2 u c(x) 2 u 0, in

More information

Simple Examples on Rectangular Domains

Simple Examples on Rectangular Domains 84 Chapter 5 Simple Examples on Rectangular Domains In this chapter we consider simple elliptic boundary value problems in rectangular domains in R 2 or R 3 ; our prototype example is the Poisson equation

More information

DISCRETE MAXIMUM PRINCIPLES in THE FINITE ELEMENT SIMULATIONS

DISCRETE MAXIMUM PRINCIPLES in THE FINITE ELEMENT SIMULATIONS DISCRETE MAXIMUM PRINCIPLES in THE FINITE ELEMENT SIMULATIONS Sergey Korotov BCAM Basque Center for Applied Mathematics http://www.bcamath.org 1 The presentation is based on my collaboration with several

More information

Chapter Two: Numerical Methods for Elliptic PDEs. 1 Finite Difference Methods for Elliptic PDEs

Chapter Two: Numerical Methods for Elliptic PDEs. 1 Finite Difference Methods for Elliptic PDEs Chapter Two: Numerical Methods for Elliptic PDEs Finite Difference Methods for Elliptic PDEs.. Finite difference scheme. We consider a simple example u := subject to Dirichlet boundary conditions ( ) u

More information

Exercises - Chapter 1 - Chapter 2 (Correction)

Exercises - Chapter 1 - Chapter 2 (Correction) Université de Nice Sophia-Antipolis Master MathMods - Finite Elements - 28/29 Exercises - Chapter 1 - Chapter 2 Correction) Exercise 1. a) Let I =], l[, l R. Show that Cl) >, u C Ī) Cl) u H 1 I), u DĪ).

More information

Numerical Methods for Two Point Boundary Value Problems

Numerical Methods for Two Point Boundary Value Problems Numerical Methods for Two Point Boundary Value Problems Graeme Fairweather and Ian Gladwell 1 Finite Difference Methods 1.1 Introduction Consider the second order linear two point boundary value problem

More information

INTRODUCTION TO FINITE ELEMENT METHODS

INTRODUCTION TO FINITE ELEMENT METHODS INTRODUCTION TO FINITE ELEMENT METHODS LONG CHEN Finite element methods are based on the variational formulation of partial differential equations which only need to compute the gradient of a function.

More information

Algorithms for Scientific Computing

Algorithms for Scientific Computing Algorithms for Scientific Computing Finite Element Methods Michael Bader Technical University of Munich Summer 2016 Part I Looking Back: Discrete Models for Heat Transfer and the Poisson Equation Modelling

More information

Lecture Notes: African Institute of Mathematics Senegal, January Topic Title: A short introduction to numerical methods for elliptic PDEs

Lecture Notes: African Institute of Mathematics Senegal, January Topic Title: A short introduction to numerical methods for elliptic PDEs Lecture Notes: African Institute of Mathematics Senegal, January 26 opic itle: A short introduction to numerical methods for elliptic PDEs Authors and Lecturers: Gerard Awanou (University of Illinois-Chicago)

More information

Finite Element Methods

Finite Element Methods Solving Operator Equations Via Minimization We start with several definitions. Definition. Let V be an inner product space. A linear operator L: D V V is said to be positive definite if v, Lv > for every

More information

Boundary Value Problems and Iterative Methods for Linear Systems

Boundary Value Problems and Iterative Methods for Linear Systems Boundary Value Problems and Iterative Methods for Linear Systems 1. Equilibrium Problems 1.1. Abstract setting We want to find a displacement u V. Here V is a complete vector space with a norm v V. In

More information

Applied/Numerical Analysis Qualifying Exam

Applied/Numerical Analysis Qualifying Exam Applied/Numerical Analysis Qualifying Exam August 9, 212 Cover Sheet Applied Analysis Part Policy on misprints: The qualifying exam committee tries to proofread exams as carefully as possible. Nevertheless,

More information

(f P Ω hf) vdx = 0 for all v V h, if and only if Ω (f P hf) φ i dx = 0, for i = 0, 1,..., n, where {φ i } V h is set of hat functions.

(f P Ω hf) vdx = 0 for all v V h, if and only if Ω (f P hf) φ i dx = 0, for i = 0, 1,..., n, where {φ i } V h is set of hat functions. Answer ALL FOUR Questions Question 1 Let I = [, 2] and f(x) = (x 1) 3 for x I. (a) Let V h be the continous space of linear piecewise function P 1 (I) on I. Write a MATLAB code to compute the L 2 -projection

More information

Numerical Solution I

Numerical Solution I Numerical Solution I Stationary Flow R. Kornhuber (FU Berlin) Summerschool Modelling of mass and energy transport in porous media with practical applications October 8-12, 2018 Schedule Classical Solutions

More information

Basic Concepts of Adaptive Finite Element Methods for Elliptic Boundary Value Problems

Basic Concepts of Adaptive Finite Element Methods for Elliptic Boundary Value Problems Basic Concepts of Adaptive Finite lement Methods for lliptic Boundary Value Problems Ronald H.W. Hoppe 1,2 1 Department of Mathematics, University of Houston 2 Institute of Mathematics, University of Augsburg

More information

Finite difference method for elliptic problems: I

Finite difference method for elliptic problems: I Finite difference method for elliptic problems: I Praveen. C praveen@math.tifrbng.res.in Tata Institute of Fundamental Research Center for Applicable Mathematics Bangalore 560065 http://math.tifrbng.res.in/~praveen

More information

A very short introduction to the Finite Element Method

A very short introduction to the Finite Element Method A very short introduction to the Finite Element Method Till Mathis Wagner Technical University of Munich JASS 2004, St Petersburg May 4, 2004 1 Introduction This is a short introduction to the finite element

More information

FINITE ELEMENT METHODS

FINITE ELEMENT METHODS FINITE ELEMENT METHODS Lecture notes arxiv:1709.08618v1 [math.na] 25 Sep 2017 Christian Clason September 25, 2017 christian.clason@uni-due.de https://udue.de/clason CONTENTS I BACKGROUND 1 overview of

More information

CIV-E1060 Engineering Computation and Simulation Examination, December 12, 2017 / Niiranen

CIV-E1060 Engineering Computation and Simulation Examination, December 12, 2017 / Niiranen CIV-E16 Engineering Computation and Simulation Examination, December 12, 217 / Niiranen This examination consists of 3 problems rated by the standard scale 1...6. Problem 1 Let us consider a long and tall

More information

APPENDIX B GRAM-SCHMIDT PROCEDURE OF ORTHOGONALIZATION. Let V be a finite dimensional inner product space spanned by basis vector functions

APPENDIX B GRAM-SCHMIDT PROCEDURE OF ORTHOGONALIZATION. Let V be a finite dimensional inner product space spanned by basis vector functions 301 APPENDIX B GRAM-SCHMIDT PROCEDURE OF ORTHOGONALIZATION Let V be a finite dimensional inner product space spanned by basis vector functions {w 1, w 2,, w n }. According to the Gram-Schmidt Process an

More information

TMA4220 Numerical Solution of Partial Differential Equations Using Element Methods Høst 2014

TMA4220 Numerical Solution of Partial Differential Equations Using Element Methods Høst 2014 Norwegian University of Science and Technology Department of Mathematical Sciences TMA422 Numerical Solution of Partial Differential Equations Using Element Methods Høst 214 Exercise set 2 1 Consider the

More information

PDE & FEM TERMINOLOGY. BASIC PRINCIPLES OF FEM.

PDE & FEM TERMINOLOGY. BASIC PRINCIPLES OF FEM. PDE & FEM TERMINOLOGY. BASIC PRINCIPLES OF FEM. Sergey Korotov Basque Center for Applied Mathematics / IKERBASQUE http://www.bcamath.org & http://www.ikerbasque.net 1 Introduction The analytical solution

More information

Chapter 1 Foundations of Elliptic Boundary Value Problems 1.1 Euler equations of variational problems

Chapter 1 Foundations of Elliptic Boundary Value Problems 1.1 Euler equations of variational problems Chapter 1 Foundations of Elliptic Boundary Value Problems 1.1 Euler equations of variational problems Elliptic boundary value problems often occur as the Euler equations of variational problems the latter

More information

arxiv: v1 [math.na] 1 May 2013

arxiv: v1 [math.na] 1 May 2013 arxiv:3050089v [mathna] May 03 Approximation Properties of a Gradient Recovery Operator Using a Biorthogonal System Bishnu P Lamichhane and Adam McNeilly May, 03 Abstract A gradient recovery operator based

More information

A simple FEM solver and its data parallelism

A simple FEM solver and its data parallelism A simple FEM solver and its data parallelism Gundolf Haase Institute for Mathematics and Scientific Computing University of Graz, Austria Chile, Jan. 2015 Partial differential equation Considered Problem

More information

Numerical methods for PDEs FEM convergence, error estimates, piecewise polynomials

Numerical methods for PDEs FEM convergence, error estimates, piecewise polynomials Platzhalter für Bild, Bild auf Titelfolie hinter das Logo einsetzen Numerical methods for PDEs FEM convergence, error estimates, piecewise polynomials Dr. Noemi Friedman Contents of the course Fundamentals

More information

Solutions of Selected Problems

Solutions of Selected Problems 1 Solutions of Selected Problems October 16, 2015 Chapter I 1.9 Consider the potential equation in the disk := {(x, y) R 2 ; x 2 +y 2 < 1}, with the boundary condition u(x) = g(x) r for x on the derivative

More information

Lecture 9 Approximations of Laplace s Equation, Finite Element Method. Mathématiques appliquées (MATH0504-1) B. Dewals, C.

Lecture 9 Approximations of Laplace s Equation, Finite Element Method. Mathématiques appliquées (MATH0504-1) B. Dewals, C. Lecture 9 Approximations of Laplace s Equation, Finite Element Method Mathématiques appliquées (MATH54-1) B. Dewals, C. Geuzaine V1.2 23/11/218 1 Learning objectives of this lecture Apply the finite difference

More information

Finite Elements. Colin Cotter. January 15, Colin Cotter FEM

Finite Elements. Colin Cotter. January 15, Colin Cotter FEM Finite Elements January 15, 2018 Why Can solve PDEs on complicated domains. Have flexibility to increase order of accuracy and match the numerics to the physics. has an elegant mathematical formulation

More information

[2] (a) Develop and describe the piecewise linear Galerkin finite element approximation of,

[2] (a) Develop and describe the piecewise linear Galerkin finite element approximation of, 269 C, Vese Practice problems [1] Write the differential equation u + u = f(x, y), (x, y) Ω u = 1 (x, y) Ω 1 n + u = x (x, y) Ω 2, Ω = {(x, y) x 2 + y 2 < 1}, Ω 1 = {(x, y) x 2 + y 2 = 1, x 0}, Ω 2 = {(x,

More information

Chapter 4: Interpolation and Approximation. October 28, 2005

Chapter 4: Interpolation and Approximation. October 28, 2005 Chapter 4: Interpolation and Approximation October 28, 2005 Outline 1 2.4 Linear Interpolation 2 4.1 Lagrange Interpolation 3 4.2 Newton Interpolation and Divided Differences 4 4.3 Interpolation Error

More information

Finite Element Methods

Finite Element Methods Finite Element Methods Max D. Gunzburger Janet S. Peterson August 26, 214 2 Chapter 1 Introduction Many mathematical models of phenomena occurring in the universe involve differential equations for which

More information

Chapter 12. Partial di erential equations Di erential operators in R n. The gradient and Jacobian. Divergence and rotation

Chapter 12. Partial di erential equations Di erential operators in R n. The gradient and Jacobian. Divergence and rotation Chapter 12 Partial di erential equations 12.1 Di erential operators in R n The gradient and Jacobian We recall the definition of the gradient of a scalar function f : R n! R, as @f grad f = rf =,..., @f

More information

6 Non-homogeneous Heat Problems

6 Non-homogeneous Heat Problems 6 Non-homogeneous Heat Problems Up to this point all the problems we have considered for the heat or wave equation we what we call homogeneous problems. This means that for an interval < x < l the problems

More information

Introduction to Finite Element Method

Introduction to Finite Element Method Introduction to Finite Element Method Dr. Rakesh K Kapania Aerospace and Ocean Engineering Department Virginia Polytechnic Institute and State University, Blacksburg, VA AOE 524, Vehicle Structures Summer,

More information

Hamburger Beiträge zur Angewandten Mathematik

Hamburger Beiträge zur Angewandten Mathematik Hamburger Beiträge zur Angewandten Mathematik Numerical analysis of a control and state constrained elliptic control problem with piecewise constant control approximations Klaus Deckelnick and Michael

More information

Numerical Solutions to Partial Differential Equations

Numerical Solutions to Partial Differential Equations Numerical Solutions to Partial Differential Equations Zhiping Li LMAM and School of Mathematical Sciences Peking University Nonconformity and the Consistency Error First Strang Lemma Abstract Error Estimate

More information

Question 9: PDEs Given the function f(x, y), consider the problem: = f(x, y) 2 y2 for 0 < x < 1 and 0 < x < 1. x 2 u. u(x, 0) = u(x, 1) = 0 for 0 x 1

Question 9: PDEs Given the function f(x, y), consider the problem: = f(x, y) 2 y2 for 0 < x < 1 and 0 < x < 1. x 2 u. u(x, 0) = u(x, 1) = 0 for 0 x 1 Question 9: PDEs Given the function f(x, y), consider the problem: 2 u x 2 u = f(x, y) 2 y2 for 0 < x < 1 and 0 < x < 1 u(x, 0) = u(x, 1) = 0 for 0 x 1 u(0, y) = u(1, y) = 0 for 0 y 1. a. Discuss how you

More information

Math 5520 Homework 2 Solutions

Math 5520 Homework 2 Solutions Math 552 Homework 2 Solutions March, 26. Consider the function fx) = 2x ) 3 if x, 3x ) 2 if < x 2. Determine for which k there holds f H k, 2). Find D α f for α k. Solution. We show that k = 2. The formulas

More information

The Closed Form Reproducing Polynomial Particle Shape Functions for Meshfree Particle Methods

The Closed Form Reproducing Polynomial Particle Shape Functions for Meshfree Particle Methods The Closed Form Reproducing Polynomial Particle Shape Functions for Meshfree Particle Methods by Hae-Soo Oh Department of Mathematics, University of North Carolina at Charlotte, Charlotte, NC 28223 June

More information

Chapter 6: Rational Expr., Eq., and Functions Lecture notes Math 1010

Chapter 6: Rational Expr., Eq., and Functions Lecture notes Math 1010 Section 6.1: Rational Expressions and Functions Definition of a rational expression Let u and v be polynomials. The algebraic expression u v is a rational expression. The domain of this rational expression

More information

WRT in 2D: Poisson Example

WRT in 2D: Poisson Example WRT in 2D: Poisson Example Consider 2 u f on [, L x [, L y with u. WRT: For all v X N, find u X N a(v, u) such that v u dv v f dv. Follows from strong form plus integration by parts: ( ) 2 u v + 2 u dx

More information

LECTURE 1: SOURCES OF ERRORS MATHEMATICAL TOOLS A PRIORI ERROR ESTIMATES. Sergey Korotov,

LECTURE 1: SOURCES OF ERRORS MATHEMATICAL TOOLS A PRIORI ERROR ESTIMATES. Sergey Korotov, LECTURE 1: SOURCES OF ERRORS MATHEMATICAL TOOLS A PRIORI ERROR ESTIMATES Sergey Korotov, Institute of Mathematics Helsinki University of Technology, Finland Academy of Finland 1 Main Problem in Mathematical

More information

LECTURE # 0 BASIC NOTATIONS AND CONCEPTS IN THE THEORY OF PARTIAL DIFFERENTIAL EQUATIONS (PDES)

LECTURE # 0 BASIC NOTATIONS AND CONCEPTS IN THE THEORY OF PARTIAL DIFFERENTIAL EQUATIONS (PDES) LECTURE # 0 BASIC NOTATIONS AND CONCEPTS IN THE THEORY OF PARTIAL DIFFERENTIAL EQUATIONS (PDES) RAYTCHO LAZAROV 1 Notations and Basic Functional Spaces Scalar function in R d, d 1 will be denoted by u,

More information

Chapter 1 Piecewise Polynomial Approximation in 1D

Chapter 1 Piecewise Polynomial Approximation in 1D Chapter 1 Piecewise Polynomial Approximation in 1D Abstract n this chapter we introduce a type of functions called piecewise polynomials that can be used to approximate other more general functions, and

More information

Finite Difference Methods for Boundary Value Problems

Finite Difference Methods for Boundary Value Problems Finite Difference Methods for Boundary Value Problems October 2, 2013 () Finite Differences October 2, 2013 1 / 52 Goals Learn steps to approximate BVPs using the Finite Difference Method Start with two-point

More information

2 Two-Point Boundary Value Problems

2 Two-Point Boundary Value Problems 2 Two-Point Boundary Value Problems Another fundamental equation, in addition to the heat eq. and the wave eq., is Poisson s equation: n j=1 2 u x 2 j The unknown is the function u = u(x 1, x 2,..., x

More information

Scientific Computing WS 2017/2018. Lecture 18. Jürgen Fuhrmann Lecture 18 Slide 1

Scientific Computing WS 2017/2018. Lecture 18. Jürgen Fuhrmann Lecture 18 Slide 1 Scientific Computing WS 2017/2018 Lecture 18 Jürgen Fuhrmann juergen.fuhrmann@wias-berlin.de Lecture 18 Slide 1 Lecture 18 Slide 2 Weak formulation of homogeneous Dirichlet problem Search u H0 1 (Ω) (here,

More information

A posteriori error estimation for elliptic problems

A posteriori error estimation for elliptic problems A posteriori error estimation for elliptic problems Praveen. C praveen@math.tifrbng.res.in Tata Institute of Fundamental Research Center for Applicable Mathematics Bangalore 560065 http://math.tifrbng.res.in

More information

Technische Universität Graz

Technische Universität Graz Technische Universität Graz A note on the stable coupling of finite and boundary elements O. Steinbach Berichte aus dem Institut für Numerische Mathematik Bericht 2009/4 Technische Universität Graz A

More information

New class of finite element methods: weak Galerkin methods

New class of finite element methods: weak Galerkin methods New class of finite element methods: weak Galerkin methods Xiu Ye University of Arkansas at Little Rock Second order elliptic equation Consider second order elliptic problem: a u = f, in Ω (1) u = 0, on

More information

Numerical Analysis Comprehensive Exam Questions

Numerical Analysis Comprehensive Exam Questions Numerical Analysis Comprehensive Exam Questions 1. Let f(x) = (x α) m g(x) where m is an integer and g(x) C (R), g(α). Write down the Newton s method for finding the root α of f(x), and study the order

More information

NUMERICAL PARTIAL DIFFERENTIAL EQUATIONS

NUMERICAL PARTIAL DIFFERENTIAL EQUATIONS NUMERICAL PARTIAL DIFFERENTIAL EQUATIONS Lecture Notes, Winter 2011/12 Christian Clason January 31, 2012 Institute for Mathematics and Scientific Computing Karl-Franzens-Universität Graz CONTENTS I BACKGROUND

More information

Schwarz Preconditioner for the Stochastic Finite Element Method

Schwarz Preconditioner for the Stochastic Finite Element Method Schwarz Preconditioner for the Stochastic Finite Element Method Waad Subber 1 and Sébastien Loisel 2 Preprint submitted to DD22 conference 1 Introduction The intrusive polynomial chaos approach for uncertainty

More information

Finite Elements. Colin Cotter. February 22, Colin Cotter FEM

Finite Elements. Colin Cotter. February 22, Colin Cotter FEM Finite Elements February 22, 2019 In the previous sections, we introduced the concept of finite element spaces, which contain certain functions defined on a domain. Finite element spaces are examples of

More information

Time-dependent variational forms

Time-dependent variational forms Time-dependent variational forms Hans Petter Langtangen 1,2 1 Center for Biomedical Computing, Simula Research Laboratory 2 Department of Informatics, University of Oslo Oct 30, 2015 PRELIMINARY VERSION

More information

Applications of the Maximum Principle

Applications of the Maximum Principle Jim Lambers MAT 606 Spring Semester 2015-16 Lecture 26 Notes These notes correspond to Sections 7.4-7.6 in the text. Applications of the Maximum Principle The maximum principle for Laplace s equation is

More information

Nodal O(h 4 )-superconvergence of piecewise trilinear FE approximations

Nodal O(h 4 )-superconvergence of piecewise trilinear FE approximations Preprint, Institute of Mathematics, AS CR, Prague. 2007-12-12 INSTITTE of MATHEMATICS Academy of Sciences Czech Republic Nodal O(h 4 )-superconvergence of piecewise trilinear FE approximations Antti Hannukainen

More information

ASYMPTOTICALLY EXACT A POSTERIORI ESTIMATORS FOR THE POINTWISE GRADIENT ERROR ON EACH ELEMENT IN IRREGULAR MESHES. PART II: THE PIECEWISE LINEAR CASE

ASYMPTOTICALLY EXACT A POSTERIORI ESTIMATORS FOR THE POINTWISE GRADIENT ERROR ON EACH ELEMENT IN IRREGULAR MESHES. PART II: THE PIECEWISE LINEAR CASE MATEMATICS OF COMPUTATION Volume 73, Number 246, Pages 517 523 S 0025-5718(0301570-9 Article electronically published on June 17, 2003 ASYMPTOTICALLY EXACT A POSTERIORI ESTIMATORS FOR TE POINTWISE GRADIENT

More information

10 The Finite Element Method for a Parabolic Problem

10 The Finite Element Method for a Parabolic Problem 1 The Finite Element Method for a Parabolic Problem In this chapter we consider the approximation of solutions of the model heat equation in two space dimensions by means of Galerkin s method, using piecewise

More information

Solving PDE s with FEniCS. L. Ridgway Scott. Laplace and Poisson

Solving PDE s with FEniCS. L. Ridgway Scott. Laplace and Poisson Solving PDE s with FEniCS Laplace and Poisson L. Ridgway Scott The Institute for Biophysical Dynamics, The Computation Institute, and the Departments of Computer Science and Mathematics, The University

More information

Chapter 10. Function approximation Function approximation. The Lebesgue space L 2 (I)

Chapter 10. Function approximation Function approximation. The Lebesgue space L 2 (I) Capter 1 Function approximation We ave studied metods for computing solutions to algebraic equations in te form of real numbers or finite dimensional vectors of real numbers. In contrast, solutions to

More information

Weighted Residual Methods

Weighted Residual Methods Weighted Residual Methods Introductory Course on Multiphysics Modelling TOMASZ G. ZIELIŃSKI bluebox.ippt.pan.pl/ tzielins/ Table of Contents Problem definition. oundary-value Problem..................

More information

DIFFERENTIAL EQUATIONS

DIFFERENTIAL EQUATIONS NUMERICAL PARTIAL DIFFERENTIAL EQUATIONS Lecture Notes, Winter 2013/14 Christian Clason July 15, 2014 Institute for Mathematics and Scientific Computing Karl-Franzens-Universität Graz CONTENTS I BACKGROUND

More information

Adaptive Finite Element Methods Lecture 1: A Posteriori Error Estimation

Adaptive Finite Element Methods Lecture 1: A Posteriori Error Estimation Adaptive Finite Element Methods Lecture 1: A Posteriori Error Estimation Department of Mathematics and Institute for Physical Science and Technology University of Maryland, USA www.math.umd.edu/ rhn 7th

More information

Weighted Residual Methods

Weighted Residual Methods Weighted Residual Methods Introductory Course on Multiphysics Modelling TOMASZ G. ZIELIŃSKI bluebox.ippt.pan.pl/ tzielins/ Institute of Fundamental Technological Research of the Polish Academy of Sciences

More information

Preliminary Examination, Numerical Analysis, August 2016

Preliminary Examination, Numerical Analysis, August 2016 Preliminary Examination, Numerical Analysis, August 2016 Instructions: This exam is closed books and notes. The time allowed is three hours and you need to work on any three out of questions 1-4 and any

More information

Numerical Functional Analysis

Numerical Functional Analysis Numerical Functional Analysis T. Betcke December 17, 28 These notes are in development and only for internal use at the University of Mancheser. For questions, comments or typos please e-mail timo.betcke@manchester.ac.uk.

More information

Traces, extensions and co-normal derivatives for elliptic systems on Lipschitz domains

Traces, extensions and co-normal derivatives for elliptic systems on Lipschitz domains Traces, extensions and co-normal derivatives for elliptic systems on Lipschitz domains Sergey E. Mikhailov Brunel University West London, Department of Mathematics, Uxbridge, UB8 3PH, UK J. Math. Analysis

More information

PIECEWISE LINEAR FINITE ELEMENT METHODS ARE NOT LOCALIZED

PIECEWISE LINEAR FINITE ELEMENT METHODS ARE NOT LOCALIZED PIECEWISE LINEAR FINITE ELEMENT METHODS ARE NOT LOCALIZED ALAN DEMLOW Abstract. Recent results of Schatz show that standard Galerkin finite element methods employing piecewise polynomial elements of degree

More information

Remarks on the analysis of finite element methods on a Shishkin mesh: are Scott-Zhang interpolants applicable?

Remarks on the analysis of finite element methods on a Shishkin mesh: are Scott-Zhang interpolants applicable? Remarks on the analysis of finite element methods on a Shishkin mesh: are Scott-Zhang interpolants applicable? Thomas Apel, Hans-G. Roos 22.7.2008 Abstract In the first part of the paper we discuss minimal

More information

ELEMENTARY MATRIX ALGEBRA

ELEMENTARY MATRIX ALGEBRA ELEMENTARY MATRIX ALGEBRA Third Edition FRANZ E. HOHN DOVER PUBLICATIONS, INC. Mineola, New York CONTENTS CHAPTER \ Introduction to Matrix Algebra 1.1 Matrices 1 1.2 Equality of Matrices 2 13 Addition

More information

Matrix square root and interpolation spaces

Matrix square root and interpolation spaces Matrix square root and interpolation spaces Mario Arioli and Daniel Loghin m.arioli@rl.ac.uk STFC-Rutherford Appleton Laboratory, and University of Birmingham Sparse Days,CERFACS, Toulouse, 2008 p.1/30

More information

On the relationship of local projection stabilization to other stabilized methods for one-dimensional advection-diffusion equations

On the relationship of local projection stabilization to other stabilized methods for one-dimensional advection-diffusion equations On the relationship of local projection stabilization to other stabilized methods for one-dimensional advection-diffusion equations Lutz Tobiska Institut für Analysis und Numerik Otto-von-Guericke-Universität

More information

Formulation of the displacement-based Finite Element Method and General Convergence Results

Formulation of the displacement-based Finite Element Method and General Convergence Results Formulation of the displacement-based Finite Element Method and General Convergence Results z Basics of Elasticity Theory strain e: measure of relative distortions u r r' y for small displacements : x

More information

Partially Penalized Immersed Finite Element Methods for Parabolic Interface Problems

Partially Penalized Immersed Finite Element Methods for Parabolic Interface Problems Partially Penalized Immersed Finite Element Methods for Parabolic Interface Problems Tao Lin, Qing Yang and Xu Zhang Abstract We present partially penalized immersed finite element methods for solving

More information

Iterative Methods for Linear Systems

Iterative Methods for Linear Systems Iterative Methods for Linear Systems 1. Introduction: Direct solvers versus iterative solvers In many applications we have to solve a linear system Ax = b with A R n n and b R n given. If n is large the

More information

TD M1 EDP 2018 no 2 Elliptic equations: regularity, maximum principle

TD M1 EDP 2018 no 2 Elliptic equations: regularity, maximum principle TD M EDP 08 no Elliptic equations: regularity, maximum principle Estimates in the sup-norm I Let be an open bounded subset of R d of class C. Let A = (a ij ) be a symmetric matrix of functions of class

More information

Numerical Solutions to Partial Differential Equations

Numerical Solutions to Partial Differential Equations Numerical Solutions to Partial Differential Equations Zhiping Li LMAM and School of Mathematical Sciences Peking University Numerical Methods for Partial Differential Equations Finite Difference Methods

More information

FEniCS Course. Lecture 0: Introduction to FEM. Contributors Anders Logg, Kent-Andre Mardal

FEniCS Course. Lecture 0: Introduction to FEM. Contributors Anders Logg, Kent-Andre Mardal FEniCS Course Lecture 0: Introduction to FEM Contributors Anders Logg, Kent-Andre Mardal 1 / 46 What is FEM? The finite element method is a framework and a recipe for discretization of mathematical problems

More information

A Gradient Recovery Operator Based on an Oblique Projection

A Gradient Recovery Operator Based on an Oblique Projection A Gradient Recovery Operator Based on an Bishnu P. Lamichhane, bishnu.lamichhane@newcastle.edu.au School of Mathematical and Physical Sciences, University of Newcastle, Australia CARMA Retreat July 18,

More information

Introduction to Finite Element computations

Introduction to Finite Element computations Non Linear Computational Mechanics Athens MP06/2012 Introduction to Finite Element computations Vincent Chiaruttini, Georges Cailletaud vincent.chiaruttini@onera.fr Outline Continuous to discrete problem

More information

TMA4220: Programming project - part 1

TMA4220: Programming project - part 1 TMA4220: Programming project - part 1 TMA4220 - Numerical solution of partial differential equations using the finite element method The programming project will be split into two parts. This is the first

More information

Finite Element Superconvergence Approximation for One-Dimensional Singularly Perturbed Problems

Finite Element Superconvergence Approximation for One-Dimensional Singularly Perturbed Problems Finite Element Superconvergence Approximation for One-Dimensional Singularly Perturbed Problems Zhimin Zhang Department of Mathematics Wayne State University Detroit, MI 48202 Received 19 July 2000; accepted

More information

Numerical Analysis of Differential Equations Numerical Solution of Elliptic Boundary Value

Numerical Analysis of Differential Equations Numerical Solution of Elliptic Boundary Value Numerical Analysis of Differential Equations 188 5 Numerical Solution of Elliptic Boundary Value Problems 5 Numerical Solution of Elliptic Boundary Value Problems TU Bergakademie Freiberg, SS 2012 Numerical

More information

Numerical Solutions to Partial Differential Equations

Numerical Solutions to Partial Differential Equations Numerical Solutions to Partial Differential Equations Zhiping Li LMAM and School of Mathematical Sciences Peking University The Residual and Error of Finite Element Solutions Mixed BVP of Poisson Equation

More information

How to solve the stochastic partial differential equation that gives a Matérn random field using the finite element method

How to solve the stochastic partial differential equation that gives a Matérn random field using the finite element method arxiv:1803.03765v1 [stat.co] 10 Mar 2018 How to solve the stochastic partial differential equation that gives a Matérn random field using the finite element method Haakon Bakka bakka@r-inla.org March 13,

More information

arxiv: v1 [math.ap] 6 Dec 2011

arxiv: v1 [math.ap] 6 Dec 2011 LECTURE NOTES: THE GALERKIN METHOD arxiv:1112.1176v1 [math.ap] 6 Dec 211 Raghavendra Venkatraman 1 In these notes, we consider the analysis of Galerkin Method and its application to computing approximate

More information

Projected Surface Finite Elements for Elliptic Equations

Projected Surface Finite Elements for Elliptic Equations Available at http://pvamu.edu/aam Appl. Appl. Math. IN: 1932-9466 Vol. 8, Issue 1 (June 2013), pp. 16 33 Applications and Applied Mathematics: An International Journal (AAM) Projected urface Finite Elements

More information