equal
deleted
inserted
replaced
1 theory QuotList |
1 theory QuotList |
2 imports QuotScript |
2 imports QuotScript List |
3 begin |
3 begin |
4 |
4 |
5 lemma LIST_map_id: |
5 lemma LIST_map_id: |
6 shows "map (\<lambda>x. x) = (\<lambda>x. x)" |
6 shows "map (\<lambda>x. x) = (\<lambda>x. x)" |
7 by simp |
7 by simp |