Journal/Paper.thy
changeset 170 b1258b7d2789
parent 167 61d0a412a3ae
child 172 21ee3a852a02
equal deleted inserted replaced
169:b794db0b79db 170:b1258b7d2789
    91   Science, with many beautiful theorems and many useful algorithms. There is a
    91   Science, with many beautiful theorems and many useful algorithms. There is a
    92   wide range of textbooks on this subject, many of which are aimed at students
    92   wide range of textbooks on this subject, many of which are aimed at students
    93   and contain very detailed `pencil-and-paper' proofs
    93   and contain very detailed `pencil-and-paper' proofs
    94   (e.g.~\cite{Kozen97}). It seems natural to exercise theorem provers by
    94   (e.g.~\cite{Kozen97}). It seems natural to exercise theorem provers by
    95   formalising the theorems and by verifying formally the algorithms.
    95   formalising the theorems and by verifying formally the algorithms.
       
    96   Some of the popular theorem provers are based on Higher-Order Logic (HOL).
    96 
    97 
    97   There is however a problem: the typical approach to regular languages is to
    98   There is however a problem: the typical approach to regular languages is to
    98   introduce finite automata and then define everything in terms of them.  For
    99   introduce finite automata and then define everything in terms of them.  For
    99   example, a regular language is normally defined as one whose strings are
   100   example, a regular language is normally defined as one whose strings are
   100   recognised by a finite deterministic automaton. This approach has many
   101   recognised by a finite deterministic automaton. This approach has many