aboutsummaryrefslogtreecommitdiff
path: root/scratch.thy
diff options
context:
space:
mode:
authorJosh Chen2018-06-17 00:48:01 +0200
committerJosh Chen2018-06-17 00:48:01 +0200
commit5161a0356d8752f3b1b4f4385e799bca92718814 (patch)
treec7cf1dfd80311af85dd81229ec8f1302395c1c9f /scratch.thy
parent602ad9fe0e2ed1ad4ab6f16e720de878aadc0fba (diff)
Decided on a new proper scheme for type rules using the idea of implicit well-formed contexts and guaranteed conclusion well-formedness. Product type rules now follow this scheme.
Diffstat (limited to 'scratch.thy')
-rw-r--r--scratch.thy24
1 files changed, 24 insertions, 0 deletions
diff --git a/scratch.thy b/scratch.thy
new file mode 100644
index 0000000..331b607
--- /dev/null
+++ b/scratch.thy
@@ -0,0 +1,24 @@
+theory scratch
+ imports IFOL
+
+begin
+
+lemma disj_swap: "P \<or> Q \<Longrightarrow> Q \<or> P"
+apply (erule disjE) (* Compare with the less useful \<open>rule disjE\<close> *)
+ apply (rule disjI2)
+ apply assumption
+apply (rule disjI1)
+apply assumption
+done
+
+lemma imp_uncurry: "P \<longrightarrow> (Q \<longrightarrow> R) \<Longrightarrow> P \<and> Q \<longrightarrow> R"
+apply (rule impI)
+apply (erule conjE)
+apply (drule mp)
+apply assumption
+apply (drule mp)
+apply assumption
+apply assumption
+done
+
+end \ No newline at end of file