aboutsummaryrefslogtreecommitdiffhomepage
path: root/isar/Example.thy
diff options
context:
space:
mode:
authorGravatar Makarius Wenzel <makarius@sketis.net>1999-05-25 12:19:10 +0000
committerGravatar Makarius Wenzel <makarius@sketis.net>1999-05-25 12:19:10 +0000
commitf582f005a4b337deef93995db1a918ea34a6c6d5 (patch)
tree01f40415679ba9ca3c83139e673f69d873d71669 /isar/Example.thy
parent5133be01ed715bcd877e41153145b12fd31b9066 (diff)
more examples;
Diffstat (limited to 'isar/Example.thy')
-rw-r--r--isar/Example.thy29
1 files changed, 28 insertions, 1 deletions
diff --git a/isar/Example.thy b/isar/Example.thy
index b8b7328b..8dc4b04a 100644
--- a/isar/Example.thy
+++ b/isar/Example.thy
@@ -1,12 +1,39 @@
theory Example = Main:;
-lemma "A --> B --> A";
+
+lemma I: "A --> A";
+proof;
+ assume A;
+ show A; .;
+qed;
+
+lemma K: "A --> B --> A";
proof;
assume A;
show "B --> A";
proof;
+ show A; .;
qed;
qed;
+lemma S: "(A --> B --> C) --> (A --> B) --> A --> C";
+proof;
+ assume "A --> B --> C";
+ show "(A --> B) --> A --> C";
+ proof;
+ assume "A --> B";
+ show "A --> C";
+ proof;
+ assume A;
+ show C;
+ proof (rule mp);
+ show "B --> C"; by (rule mp);
+ show B; by (rule mp);
+ qed;
+ qed;
+ qed;
+qed;
+
+
end;