Quot/QuotMain.thy
changeset 833 129caba33c03
parent 825 970e86082cd7
child 834 fb7fe6aca6f0
equal deleted inserted replaced
832:b3bb2bad952f 833:129caba33c03
   105 
   105 
   106 (* Lemmas about simplifying id's. *)
   106 (* Lemmas about simplifying id's. *)
   107 lemmas [id_simps] =
   107 lemmas [id_simps] =
   108   fun_map_id[THEN eq_reflection]
   108   fun_map_id[THEN eq_reflection]
   109   id_apply[THEN eq_reflection]
   109   id_apply[THEN eq_reflection]
   110   id_def[THEN eq_reflection, symmetric]
   110   (*id_def[THEN eq_reflection, symmetric]*)
   111   id_o[THEN eq_reflection]
   111   id_o[THEN eq_reflection]
   112   o_id[THEN eq_reflection]
   112   o_id[THEN eq_reflection]
   113   eq_comp_r
   113   eq_comp_r
   114 
   114 
   115 (* The translation functions for the lifting process. *)
   115 (* The translation functions for the lifting process. *)