src/HOL/Product_Type.thy
changeset 63566 e5abbdee461a
parent 63400 249fa34faba2
child 63575 b9bd9e61fd63
equal deleted inserted replaced
63560:3e3097ac37d1 63566:e5abbdee461a
   262 lemmas simps = prod.inject prod.case prod.rec
   262 lemmas simps = prod.inject prod.case prod.rec
   263 
   263 
   264 setup \<open>Sign.parent_path\<close>
   264 setup \<open>Sign.parent_path\<close>
   265 
   265 
   266 declare prod.case [nitpick_simp del]
   266 declare prod.case [nitpick_simp del]
   267 declare prod.case_cong_weak [cong del]
   267 declare old.prod.case_cong_weak [cong del]
   268 declare prod.case_eq_if [mono]
   268 declare prod.case_eq_if [mono]
   269 declare prod.split [no_atp]
   269 declare prod.split [no_atp]
   270 declare prod.split_asm [no_atp]
   270 declare prod.split_asm [no_atp]
   271 
   271 
   272 text \<open>
   272 text \<open>