ProgTutorial/Appendix.thy
author Norbert Schirmer <norbert.schirmer@web.de>
Fri, 17 May 2019 07:29:51 +0200
changeset 568 be23597e81db
parent 565 cecd7a941885
child 569 f875a25aa72d
permissions -rw-r--r--
adding to "how to understand code"
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
13
2b07da8b310d polished and added a subdirectory for the recipes
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
     1
2b07da8b310d polished and added a subdirectory for the recipes
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
     2
theory Appendix
346
0fea8b7a14a1 tuned the ML-output mechanism; tuned slightly the text
Christian Urban <urbanc@in.tum.de>
parents: 189
diff changeset
     3
imports Base
13
2b07da8b310d polished and added a subdirectory for the recipes
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
     4
begin
2b07da8b310d polished and added a subdirectory for the recipes
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
     5
565
cecd7a941885 isabelle update_cartouches -t
Norbert Schirmer <norbert.schirmer@web.de>
parents: 517
diff changeset
     6
text \<open>\appendix\<close>
13
2b07da8b310d polished and added a subdirectory for the recipes
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
     7
129
e0d368a45537 started a section about simprocs
Christian Urban <urbanc@in.tum.de>
parents: 73
diff changeset
     8
565
cecd7a941885 isabelle update_cartouches -t
Norbert Schirmer <norbert.schirmer@web.de>
parents: 517
diff changeset
     9
chapter \<open>Recipes\<close>
13
2b07da8b310d polished and added a subdirectory for the recipes
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    10
565
cecd7a941885 isabelle update_cartouches -t
Norbert Schirmer <norbert.schirmer@web.de>
parents: 517
diff changeset
    11
text \<open>
184
c7f04a008c9c some polishing
Christian Urban <urbanc@in.tum.de>
parents: 182
diff changeset
    12
  Possible topics: 
162
3fb9f820a294 some additions to the simplifier section and general tuning
Christian Urban <urbanc@in.tum.de>
parents: 131
diff changeset
    13
168
009ca4807baa polished somewhat the recipes and solutions
Christian Urban <urbanc@in.tum.de>
parents: 164
diff changeset
    14
  \begin{itemize}
009ca4807baa polished somewhat the recipes and solutions
Christian Urban <urbanc@in.tum.de>
parents: 164
diff changeset
    15
  \item translations/print translations; 
475
25371f74c768 updated to post-2011-1 Isabelle
Christian Urban <urbanc@in.tum.de>
parents: 407
diff changeset
    16
  @{ML "Proof_Context.print_syntax"}
131
8db9195bb3e9 polished
Christian Urban <urbanc@in.tum.de>
parents: 129
diff changeset
    17
  
168
009ca4807baa polished somewhat the recipes and solutions
Christian Urban <urbanc@in.tum.de>
parents: 164
diff changeset
    18
  \item user space type systems (in the form that already exists)
164
3f617d7a2691 more work on simple_inductive
Christian Urban <urbanc@in.tum.de>
parents: 162
diff changeset
    19
407
Christian Urban <urbanc@in.tum.de>
parents: 356
diff changeset
    20
  \item useful datastructures: discrimination nets, graphs, association lists
356
43df2d59fb98 updated to new Isabelle
Christian Urban <urbanc@in.tum.de>
parents: 346
diff changeset
    21
43df2d59fb98 updated to new Isabelle
Christian Urban <urbanc@in.tum.de>
parents: 346
diff changeset
    22
  \item Brief history of Isabelle
168
009ca4807baa polished somewhat the recipes and solutions
Christian Urban <urbanc@in.tum.de>
parents: 164
diff changeset
    23
  \end{itemize}
565
cecd7a941885 isabelle update_cartouches -t
Norbert Schirmer <norbert.schirmer@web.de>
parents: 517
diff changeset
    24
\<close>
131
8db9195bb3e9 polished
Christian Urban <urbanc@in.tum.de>
parents: 129
diff changeset
    25
517
d8c376662bb4 removed special ML-setup and replaced it by explicit markups (i.e., %grayML)
Christian Urban <urbanc@in.tum.de>
parents: 475
diff changeset
    26
end