aboutsummaryrefslogtreecommitdiff
path: root/scratch.thy
diff options
context:
space:
mode:
Diffstat (limited to 'scratch.thy')
-rw-r--r--scratch.thy20
1 files changed, 2 insertions, 18 deletions
diff --git a/scratch.thy b/scratch.thy
index 331b607..b90fd59 100644
--- a/scratch.thy
+++ b/scratch.thy
@@ -1,24 +1,8 @@
theory scratch
- imports IFOL
+ imports HoTT
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
+schematic_goal "\<lbrakk>a : A; b : B\<rbrakk> \<Longrightarrow> ?x : A \<times> B" by simple
end \ No newline at end of file