src/HOL/Library/Coinductive_List.thy
changeset 32960 69916a850301
parent 32655 dd84779cd191
child 33056 791a4655cae3
equal deleted inserted replaced
32959:23a8c5ac35f8 32960:69916a850301
   458       with h h' MN have ?EqNIL by simp
   458       with h h' MN have ?EqNIL by simp
   459       then show ?thesis ..
   459       then show ?thesis ..
   460     next
   460     next
   461       case (Some p)
   461       case (Some p)
   462       with h h' MN have "M = CONS (fst p) (h (snd p))"
   462       with h h' MN have "M = CONS (fst p) (h (snd p))"
   463 	and "N = CONS (fst p) (h' (snd p))"
   463         and "N = CONS (fst p) (h' (snd p))"
   464         by (simp_all split: prod.split)
   464         by (simp_all split: prod.split)
   465       then have ?EqCONS by (auto iff: Id_on_iff)
   465       then have ?EqCONS by (auto iff: Id_on_iff)
   466       then show ?thesis ..
   466       then show ?thesis ..
   467     qed
   467     qed
   468   qed
   468   qed