QuotList.thy
changeset 535 a19a5179fbca
parent 533 4318ab0df27b
child 537 57073b0b8fac
equal deleted inserted replaced
534:051bd9e90e92 535:a19a5179fbca
     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