Slides/Slides6.thy
changeset 2771 66ef2a2c64fb
parent 2764 03de62208942
equal deleted inserted replaced
2766:7a6b87adebc8 2771:66ef2a2c64fb
    10   Cons  ("_::/_" [66,65] 65) 
    10   Cons  ("_::/_" [66,65] 65) 
    11 
    11 
    12 (*>*)
    12 (*>*)
    13 
    13 
    14 text_raw {*
    14 text_raw {*
    15   \renewcommand{\slidecaption}{Shanghai, 12.~April 2011}
    15   \renewcommand{\slidecaption}{Hefei, 15.~April 2011}
    16 
    16 
    17   \newcommand{\abst}[2]{#1.#2}% atom-abstraction
    17   \newcommand{\abst}[2]{#1.#2}% atom-abstraction
    18   \newcommand{\pair}[2]{\langle #1,#2\rangle} % pairing
    18   \newcommand{\pair}[2]{\langle #1,#2\rangle} % pairing
    19   \newcommand{\susp}{{\boldsymbol{\cdot}}}% for suspensions
    19   \newcommand{\susp}{{\boldsymbol{\cdot}}}% for suspensions
    20   \newcommand{\unit}{\langle\rangle}% unit
    20   \newcommand{\unit}{\langle\rangle}% unit
   126   \end{frame}}
   126   \end{frame}}
   127   %%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%     
   127   %%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%     
   128 *}
   128 *}
   129 
   129 
   130 
   130 
       
   131 text_raw {*
       
   132   %%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%
       
   133   \mode<presentation>{
       
   134   \begin{frame}[c]
       
   135   \frametitle{3 Points}
       
   136   \large
       
   137   \begin{itemize}
       
   138   \item It is easy to make mistakes.\bigskip
       
   139   \item Theorem provers can prevent mistakes, {\bf if} the problem
       
   140   is formulated so that it is suitable for theorem provers.\bigskip
       
   141   \item This re-formulation can be done, even in domains where
       
   142   we do not expect it.
       
   143   \end{itemize}
       
   144 
       
   145   \end{frame}}
       
   146   %%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%     
       
   147 *}
   131 
   148 
   132 text_raw {*
   149 text_raw {*
   133 
   150 
   134   %%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%
   151   %%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%
   135   \mode<presentation>{
   152   \mode<presentation>{
   184   \color{gray}{relied on their proof in a safety critical system (proof carrying code)}
   201   \color{gray}{relied on their proof in a safety critical system (proof carrying code)}
   185   \end{tabular}
   202   \end{tabular}
   186 
   203 
   187   \end{tabular}\medskip
   204   \end{tabular}\medskip
   188 
   205 
   189 
   206   \end{frame}}
   190   
   207   %%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%     
   191 
   208 
   192 
   209 *}
   193   \end{frame}}
   210 
   194   %%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%     
       
   195 
       
   196 *}
       
   197 
   211 
   198 text_raw {*
   212 text_raw {*
   199 
   213 
   200   %%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%
   214   %%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%
   201   \mode<presentation>{
   215   \mode<presentation>{
   331 
   345 
   332 text_raw {*
   346 text_raw {*
   333   %%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%
   347   %%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%
   334   \mode<presentation>{
   348   \mode<presentation>{
   335   \begin{frame}<1->[c]
   349   \begin{frame}<1->[c]
   336   \frametitle{Theorem Provers}
   350   \frametitle{Lessons Learned}
   337 
   351 
   338   \begin{itemize}
   352   \begin{itemize}
   339   \item Theorem provers help with keeping large proofs consistent;
   353   \item Theorem provers help with keeping large proofs consistent;
   340   make them modifiable.\medskip
   354   make them modifiable.\medskip
   341   
   355   
   736   \end{flushright}
   750   \end{flushright}
   737   \end{textblock}
   751   \end{textblock}
   738 
   752 
   739   \begin{textblock}{6}(9.5,6.18)
   753   \begin{textblock}{6}(9.5,6.18)
   740   \begin{flushright}
   754   \begin{flushright}
   741   \color{gray}``derivative for a char'' 
   755   \color{gray}``derivative w.r.t.~a char'' 
   742   \end{flushright}
   756   \end{flushright}
   743   \end{textblock}
   757   \end{textblock}
   744 
   758 
   745   \begin{textblock}{6}(9.5,12.1)
   759   \begin{textblock}{6}(9.5,12.1)
   746   \begin{flushright}
   760   \begin{flushright}
   747   \color{gray}``deriv.~for a string'' 
   761   \color{gray}``deriv.~w.r.t.~a string'' 
   748   \end{flushright}
   762   \end{flushright}
   749   \end{textblock}
   763   \end{textblock}
   750 
   764 
   751   \begin{textblock}{6}(9.5,13.98)
   765   \begin{textblock}{6}(9.5,13.98)
   752   \begin{flushright}
   766   \begin{flushright}
   859   \item A \alert{regular language} is one where there is a DFA that 
   873   \item A \alert{regular language} is one where there is a DFA that 
   860   recognises it.\bigskip\pause
   874   recognises it.\bigskip\pause
   861   \end{itemize}
   875   \end{itemize}
   862 
   876 
   863 
   877 
   864   I can think of two reasons why this is a good definition:\medskip
   878   There are many reasons why this is a good definition:\medskip
   865   \begin{itemize}
   879   \begin{itemize}
   866   \item pumping lemma
   880   \item pumping lemma
   867   \item closure properties of regular languages (closed under complement)
   881   \item closure properties of regular languages\\ (e.g.~closure under complement)
   868   \end{itemize}
   882   \end{itemize}
   869 
   883 
   870   \end{frame}}
   884   \end{frame}}
   871   %%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%     
   885   %%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%     
   872 
   886 
   907 
   921 
   908 text_raw {*
   922 text_raw {*
   909   %%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%
   923   %%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%
   910   \mode<presentation>{
   924   \mode<presentation>{
   911   \begin{frame}[c]
   925   \begin{frame}[c]
       
   926   \frametitle{}
       
   927   \large
       
   928   \begin{center}
       
   929   \begin{tabular}{p{9cm}}
       
   930   My point:\bigskip\\
       
   931 
       
   932   The theory about regular languages can be reformulated 
       
   933   to be more suitable for theorem proving.
       
   934   \end{tabular}
       
   935   \end{center}
       
   936   \end{frame}}
       
   937   %%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%     
       
   938 *}
       
   939 
       
   940 text_raw {*
       
   941   %%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%
       
   942   \mode<presentation>{
       
   943   \begin{frame}[c]
   912   \frametitle{\LARGE The Myhill-Nerode Theorem}
   944   \frametitle{\LARGE The Myhill-Nerode Theorem}
   913 
   945 
   914   \begin{itemize}
   946   \begin{itemize}
   915   \item provides necessary and suf\!ficient conditions for a language 
   947   \item provides necessary and suf\!ficient conditions for a language 
   916   being regular (pumping lemma only necessary)\medskip
   948   being regular (pumping lemma only necessary)\medskip
   923   \end{center}
   955   \end{center}
   924   \end{itemize}
   956   \end{itemize}
   925 
   957 
   926   \end{frame}}
   958   \end{frame}}
   927   %%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%     
   959   %%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%     
   928 
       
   929 *}
   960 *}
   930 
   961 
   931 text_raw {*
   962 text_raw {*
   932   %%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%
   963   %%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%
   933   \mode<presentation>{
   964   \mode<presentation>{
  1053   \multicolumn{2}{l}{\smath{U\!N\!IV /\!/\approx_L} produces}\\[4mm]
  1084   \multicolumn{2}{l}{\smath{U\!N\!IV /\!/\approx_L} produces}\\[4mm]
  1054 
  1085 
  1055   \smath{R_1}: & \smath{\{[]\}}\\
  1086   \smath{R_1}: & \smath{\{[]\}}\\
  1056   \smath{R_2}: & \smath{\{[c]\}}\\
  1087   \smath{R_2}: & \smath{\{[c]\}}\\
  1057   \smath{R_3}: & \smath{U\!N\!IV - \{[], [c]\}}\\[6mm]
  1088   \smath{R_3}: & \smath{U\!N\!IV - \{[], [c]\}}\\[6mm]
  1058   \multicolumn{2}{l}{\onslide<2->{\smath{X \stackrel{c}{\longrightarrow} Y \dn X ; [c] \subseteq Y}}}
  1089   \multicolumn{2}{l}{\onslide<2->{\smath{X \stackrel{c}{\longrightarrow} Y \dn X ;; [c] \subseteq Y}}}
  1059   \end{tabular}
  1090   \end{tabular}
  1060 
  1091 
  1061   \end{tabular}
  1092   \end{tabular}
  1062 
  1093 
  1063   \end{frame}}
  1094   \end{frame}}
  1343   \frametitle{\LARGE What Have We Achieved?}
  1374   \frametitle{\LARGE What Have We Achieved?}
  1344 
  1375 
  1345   \begin{itemize}
  1376   \begin{itemize}
  1346   \item \smath{\text{finite}\, (U\!N\!IV /\!/ \approx_L) \;\Leftrightarrow\; L\; \text{is regular}}
  1377   \item \smath{\text{finite}\, (U\!N\!IV /\!/ \approx_L) \;\Leftrightarrow\; L\; \text{is regular}}
  1347   \bigskip\pause
  1378   \bigskip\pause
  1348   \item regular languages are closed under complementation; this is easy
  1379   \item regular languages are closed under complementation; this is now easy\medskip
  1349   \begin{center}
  1380   \begin{center}
  1350   \smath{U\!N\!IV /\!/ \approx_L \;\;=\;\; U\!N\!IV /\!/ \approx_{-L}}
  1381   \smath{U\!N\!IV /\!/ \approx_L \;\;=\;\; U\!N\!IV /\!/ \approx_{-L}}
  1351   \end{center}
  1382   \end{center}
  1352   \end{itemize}
  1383   \end{itemize}
  1353 
  1384 
  1421   \begin{frame}[c]
  1452   \begin{frame}[c]
  1422   \frametitle{\LARGE Conclusion}
  1453   \frametitle{\LARGE Conclusion}
  1423 
  1454 
  1424   \begin{itemize}
  1455   \begin{itemize}
  1425   \item We formalised the Myhill-Nerode theorem based on 
  1456   \item We formalised the Myhill-Nerode theorem based on 
  1426   regular expressions (DFA are difficult to deal with in a theorem prover).\smallskip
  1457   regular expressions only (DFAs are difficult to deal with in a theorem prover).\smallskip
  1427 
  1458 
  1428   \item Seems to be a common theme: algorithms need to be reformulated
  1459   \item Seems to be a common theme: algorithms need to be reformulated
  1429   to better suit formal treatment.\smallskip
  1460   to better suit formal treatment.\smallskip
  1430 
  1461 
  1431   \item The most interesting aspect is that we are able to
  1462   \item The most interesting aspect is that we are able to
  1432   implement the matcher directly inside the theorem prover
  1463   implement the matcher directly inside the theorem prover
  1433   (ongoing work).\smallskip
  1464   (ongoing work).\smallskip
  1434 
  1465 
  1435   \item Parsing is a vast field and seems to offer new results. 
  1466   \item Parsing is a vast field which seem to offer new results. 
  1436   \end{itemize}
  1467   \end{itemize}
  1437 
  1468 
  1438   \end{frame}}
  1469   \end{frame}}
  1439   %%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%     
  1470   %%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%     
  1440 *}
  1471 *}
  1448   \mbox{}\\[13mm]
  1479   \mbox{}\\[13mm]
  1449   \alert{\LARGE Thank you very much!}\\
  1480   \alert{\LARGE Thank you very much!}\\
  1450   \alert{\Large Questions?}
  1481   \alert{\Large Questions?}
  1451   \end{tabular}}
  1482   \end{tabular}}
  1452 
  1483 
  1453   %\begin{center}
  1484   \begin{center}
  1454   %\bf \underline{Short Bio:}
  1485   \bf \underline{Short Bio:}
  1455   %\end{center}
  1486   \end{center}
  1456   %\mbox{}\\[-17mm]\mbox{}\small
  1487   \mbox{}\\[-17mm]\mbox{}\small
  1457   %\begin{itemize}
  1488   \begin{itemize}
  1458   %\item PhD in Cambridge
  1489   \item PhD in Cambridge
  1459   %\item Emmy-Noether Fellowship in Munich
  1490   \item Emmy-Noether Research Fellowship at the TU Munich
  1460   %\item main results in nominal reasoning and nominal unification
  1491   \item talks at: CMU, Yale, Princeton, MIT,$\ldots$
  1461   %\end{itemize}
  1492   \end{itemize}
  1462 
  1493 
  1463   \end{frame}}
  1494   \end{frame}}
  1464   %%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%
  1495   %%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%
  1465 *}
  1496 *}
  1466 
  1497 
  1467 
  1498 text_raw {*
       
  1499   %%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%
       
  1500   \mode<presentation>{
       
  1501   \begin{frame}[c]
       
  1502   \frametitle{Future Research}
       
  1503 
       
  1504   My existing strengths:\bigskip
       
  1505 
       
  1506   \begin{itemize}
       
  1507   \item Isabelle (implementation)\bigskip
       
  1508   \item background in logic, programming languages, formal methods
       
  1509   \end{itemize}
       
  1510 
       
  1511   \end{frame}}
       
  1512   %%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%
       
  1513 *}
       
  1514 
       
  1515 text_raw {*
       
  1516   %%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%
       
  1517   \mode<presentation>{
       
  1518   \begin{frame}[c]
       
  1519   \frametitle{Future Research}
       
  1520 
       
  1521   I want to have a single logic framework in which I can
       
  1522   write programs and prove their correctness.\bigskip
       
  1523 
       
  1524   \begin{itemize}
       
  1525   \item extensions of HOL (IO, modules, advanced types)
       
  1526   \item high-level programming languages
       
  1527   \end{itemize}
       
  1528 
       
  1529   \end{frame}}
       
  1530   %%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%
       
  1531 *}
       
  1532 
       
  1533 text_raw {*
       
  1534   %%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%
       
  1535   \mode<presentation>{
       
  1536   \begin{frame}[c]
       
  1537   \frametitle{Future Research}
       
  1538 
       
  1539   Compilers\bigskip
       
  1540 
       
  1541   \begin{itemize}
       
  1542   \item the high-level language needs to be compiled to correct machine
       
  1543   code
       
  1544   \item compiler verification, machine code verification
       
  1545   \end{itemize}
       
  1546 
       
  1547   \end{frame}}
       
  1548   %%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%
       
  1549 *}
       
  1550 
       
  1551 text_raw {*
       
  1552   %%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%
       
  1553   \mode<presentation>{
       
  1554   \begin{frame}[c]
       
  1555   \frametitle{Future Research}
       
  1556 
       
  1557   Stronger type-systems\bigskip
       
  1558 
       
  1559   \begin{itemize}
       
  1560   \item ``correct by construction''
       
  1561   \item GADTs, dependent types
       
  1562   \end{itemize}
       
  1563 
       
  1564   \end{frame}}
       
  1565   %%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%
       
  1566 *}
       
  1567 
       
  1568 text_raw {*
       
  1569   %%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%
       
  1570   \mode<presentation>{
       
  1571   \begin{frame}[c]
       
  1572   \frametitle{Future Research}
       
  1573 
       
  1574   Proof automation\bigskip
       
  1575 
       
  1576   \begin{itemize}
       
  1577   \item external tools generate ``proof-certificates''
       
  1578   \item certificates are imported into Isabelle
       
  1579   \item GPU based external provers
       
  1580   \end{itemize}
       
  1581 
       
  1582   \end{frame}}
       
  1583   %%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%
       
  1584 *}
       
  1585 
       
  1586 text_raw {*
       
  1587   %%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%
       
  1588   \mode<presentation>{
       
  1589   \begin{frame}[c]
       
  1590   \frametitle{Future Research}
       
  1591 
       
  1592   Large-scale applications\bigskip
       
  1593 
       
  1594   \begin{itemize}
       
  1595   \item verification of Java-Script, Scala,$\ldots$
       
  1596   \item interesting code (INTEL in Shanghai)
       
  1597   \end{itemize}
       
  1598 
       
  1599   \end{frame}}
       
  1600   %%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%
       
  1601 *}
  1468 
  1602 
  1469 
  1603 
  1470 (*<*)
  1604 (*<*)
  1471 end
  1605 end
  1472 (*>*)
  1606 (*>*)