equal
deleted
inserted
replaced
1 theory BlexerSimp |
1 theory BlexerSimp |
2 imports Blexer |
2 imports Blexer |
3 begin |
3 begin |
|
4 |
|
5 |
|
6 lemma test: |
|
7 assumes "Q \<Longrightarrow> P" |
|
8 shows "~P \<Longrightarrow> ~Q" |
|
9 using assms |
|
10 apply(erule_tac contrapos_nn) |
|
11 apply(simp) |
|
12 done |
4 |
13 |
5 fun distinctWith :: "'a list \<Rightarrow> ('a \<Rightarrow> 'a \<Rightarrow> bool) \<Rightarrow> 'a set \<Rightarrow> 'a list" |
14 fun distinctWith :: "'a list \<Rightarrow> ('a \<Rightarrow> 'a \<Rightarrow> bool) \<Rightarrow> 'a set \<Rightarrow> 'a list" |
6 where |
15 where |
7 "distinctWith [] eq acc = []" |
16 "distinctWith [] eq acc = []" |
8 | "distinctWith (x # xs) eq acc = |
17 | "distinctWith (x # xs) eq acc = |