src/Doc/ProgProve/Isar.thy
changeset 52059 2f970c7f722b
parent 51445 1c9538a04e63
child 52361 7d5ad23b8245
equal deleted inserted replaced
52058:387dc978422b 52059:2f970c7f722b
     1 (*<*)
     1 (*<*)
     2 theory Isar
     2 theory Isar
     3 imports LaTeXsugar
     3 imports LaTeXsugar
     4 begin
     4 begin
     5 ML{* quick_and_dirty := true *}
     5 declare [[quick_and_dirty]]
     6 (*>*)
     6 (*>*)
     7 text{*
     7 text{*
     8 Apply-scripts are unreadable and hard to maintain. The language of choice
     8 Apply-scripts are unreadable and hard to maintain. The language of choice
     9 for larger proofs is \concept{Isar}. The two key features of Isar are:
     9 for larger proofs is \concept{Isar}. The two key features of Isar are:
    10 \begin{itemize}
    10 \begin{itemize}