QuotList.thy
changeset 57 13be92f5b638
parent 0 ebe0ea8fe247
child 511 28bb34eeedc5
equal deleted inserted replaced
56:ec5fbe7ab427 57:13be92f5b638
     1 theory QuotList
     1 theory QuotList
     2 imports QuotScript
     2 imports QuotScript
     3 begin
     3 begin
     4 
       
     5 
     4 
     6 lemma LIST_map_I:
     5 lemma LIST_map_I:
     7   shows "map (\<lambda>x. x) = (\<lambda>x. x)"
     6   shows "map (\<lambda>x. x) = (\<lambda>x. x)"
     8   by simp
     7   by simp
     9 
     8