diff -r 93f158d59ead -r 64ac3471005a src/HOL/Codatatype/BNF_FP.thy --- a/src/HOL/Codatatype/BNF_FP.thy Mon Sep 17 21:13:30 2012 +0200 +++ b/src/HOL/Codatatype/BNF_FP.thy Mon Sep 17 21:13:30 2012 +0200 @@ -137,6 +137,18 @@ lemma ex_mem_singleton: "(\y. y \ A \ y \ {x}) = (x \ A)" by simp +lemma prod_set_simps: +"fsts (x, y) = {x}" +"snds (x, y) = {y}" +unfolding fsts_def snds_def by simp+ + +lemma sum_set_simps: +"sum_setl (Inl x) = {x}" +"sum_setl (Inr x) = {}" +"sum_setr (Inl x) = {}" +"sum_setr (Inr x) = {x}" +unfolding sum_setl_def sum_setr_def by simp+ + lemma induct_set_step: "\b \ A; c \ F b\ \ \x. x \ A \ c \ F x" "\B \ A; c \ f B\ \ \C. (\a \ A. C = f a) \c \ C"