aboutsummaryrefslogtreecommitdiff
path: root/scratch.thy
blob: 331b60718c7ead592e00fb6d0d42ea92f82faeba (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
22
23
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