# HG changeset patch # User Christian Urban # Date 1283581569 -28800 # Node ID cda25f9aa67884b29e318fd4f48a0c656da9d7d2 # Parent 894599a50af3c42dfb27970d76a2473ef80d4ec5# Parent 1b31d514a087921de5bf6f6d6dcbdb79dcf7fa86 merged diff -r 894599a50af3 -r cda25f9aa678 Attic/Quot/Examples/FSet_BallBex.thy --- a/Attic/Quot/Examples/FSet_BallBex.thy Sat Sep 04 07:39:38 2010 +0800 +++ b/Attic/Quot/Examples/FSet_BallBex.thy Sat Sep 04 14:26:09 2010 +0800 @@ -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 diff -r 894599a50af3 -r cda25f9aa678 Quotient-Paper/Paper.thy --- a/Quotient-Paper/Paper.thy Sat Sep 04 07:39:38 2010 +0800 +++ b/Quotient-Paper/Paper.thy Sat Sep 04 14:26:09 2010 +0800 @@ -23,7 +23,7 @@ notation (latex output) rel_conj ("_ \\\ _" [53, 53] 52) and pred_comp ("_ \\ _" [1, 1] 30) and - "op -->" (infix "\" 100) and + implies (infix "\" 100) and "==>" (infix "\" 100) and fun_map ("_ \ _" 51) and fun_rel ("_ \ _" 51) and