diff -r 0bc1db726f81 -r 5e76af0a51f9 Attic/Quot/Examples/FSet_BallBex.thy --- a/Attic/Quot/Examples/FSet_BallBex.thy Mon Aug 30 11:02:13 2010 +0900 +++ b/Attic/Quot/Examples/FSet_BallBex.thy Mon Aug 30 15:55:08 2010 +0900 @@ -11,15 +11,13 @@ apply (metis mem_def) done -(* Should not work and doesn't. thm test[quot_lifted] -*) lemma "\xs \ (\xs. x |\| xs). x |\| finsert y xs" - unfolding Ball_def mem_def - by (lifting test[unfolded Ball_def mem_def]) + unfolding Ball_def + by (lifting test[unfolded Ball_def]) -ML {* Quotient_Tacs.lifted @{context} [@{typ "'a fset"}] @{thms Ball_def Bex_def mem_def} @{thm test}*} +ML {* Quotient_Tacs.lifted @{context} [@{typ "'a fset"}] @{thms Ball_def Bex_def} @{thm test}*} lemma test2: "\xs \ (\xs. xs \ []). xs \ []" @@ -27,14 +25,12 @@ apply (auto simp add: mem_def) done -(* Should not work and doesn't thm test2[quot_lifted] -*) lemma "\xs \ (\xs. xs = {||}). xs = {||}" - unfolding Bex_def mem_def - by (lifting test2[unfolded Bex_def mem_def]) + unfolding Bex_def + by (lifting test2[unfolded Bex_def]) -ML {* Quotient_Tacs.lifted @{context} [@{typ "'a fset"}] @{thms Bex_def mem_def} @{thm test2}*} +ML {* Quotient_Tacs.lifted @{context} [@{typ "'a fset"}] @{thms Bex_def} @{thm test2}*} end