diff options
Diffstat (limited to 'isar/Example.thy')
| -rw-r--r-- | isar/Example.thy | 2 |
1 files changed, 1 insertions, 1 deletions
diff --git a/isar/Example.thy b/isar/Example.thy index f9807888..f1657227 100644 --- a/isar/Example.thy +++ b/isar/Example.thy @@ -4,7 +4,7 @@ theory Example = Main:; text {* Just a few tiny examples to get an idea of how Isabelle/Isar proof documents may look like. - *} + *}; lemma I: "A --> A"; proof; |
