src/HOL/Codatatype/BNF_FP.thy
changeset 49451 7a28d22c33c6
parent 49430 6df729c6a1a6
child 49457 1d2825673cec
--- a/src/HOL/Codatatype/BNF_FP.thy	Thu Sep 20 02:42:48 2012 +0200
+++ b/src/HOL/Codatatype/BNF_FP.thy	Thu Sep 20 02:42:48 2012 +0200
@@ -113,11 +113,11 @@
 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+
+"setl (Inl x) = {x}"
+"setl (Inr x) = {}"
+"setr (Inl x) = {}"
+"setr (Inr x) = {x}"
+unfolding sum_set_defs by simp+
 
 ML_file "Tools/bnf_fp_util.ML"
 ML_file "Tools/bnf_fp_sugar_tactics.ML"