author | wenzelm |
Fri, 19 Feb 2010 22:29:30 +0100 | |
changeset 35243 | 024fef37a65d |
parent 35242 | 1c80c29086d7 |
child 35244 | 5cb9cdc75a4a |
--- a/src/HOL/Library/Quotient_Sum.thy Fri Feb 19 22:25:26 2010 +0100 +++ b/src/HOL/Library/Quotient_Sum.thy Fri Feb 19 22:29:30 2010 +0100 @@ -24,7 +24,7 @@ declare [[map "+" = (sum_map, sum_rel)]] -text {* should probably be in Sum_Type.thy *} +text {* should probably be in @{theory Sum_Type} *} lemma split_sum_all: shows "(\<forall>x. P x) \<longleftrightarrow> (\<forall>x. P (Inl x)) \<and> (\<forall>x. P (Inr x))" apply(auto)