src/HOL/Decision_Procs/ex/Approximation_Ex.thy
changeset 48480 cb03acfae211
parent 47600 e12289b5796b
child 53015 a1119cf551e8
equal deleted inserted replaced
48479:819f7a5f3e7f 48480:cb03acfae211
     1 (* Author:     Johannes Hoelzl <hoelzl@in.tum.de> 2009 *)
     1 (* Author:     Johannes Hoelzl <hoelzl@in.tum.de> 2009 *)
     2 
     2 
     3 theory Approximation_Ex
     3 theory Approximation_Ex
     4 imports Complex_Main "~~/src/HOL/Decision_Procs/Approximation"
     4 imports Complex_Main "../Approximation"
     5 begin
     5 begin
     6 
     6 
     7 text {*
     7 text {*
     8 
     8 
     9 Here are some examples how to use the approximation method.
     9 Here are some examples how to use the approximation method.