diff -r a394c7337966 -r e576a97e9a3e Quot/QuotMain.thy --- a/Quot/QuotMain.thy Thu Jan 21 07:38:34 2010 +0100 +++ b/Quot/QuotMain.thy Thu Jan 21 09:02:04 2010 +0100 @@ -138,6 +138,7 @@ lemma shows QT_all: "Quot_True (All P) \ Quot_True P" and QT_ex: "Quot_True (Ex P) \ Quot_True P" + and QT_ex1: "Quot_True (Ex1 P) \ Quot_True P" and QT_lam: "Quot_True (\x. P x) \ (\x. Quot_True (P x))" and QT_ext: "(\x. Quot_True (a x) \ f x = g x) \ (Quot_True a \ f = g)" by (simp_all add: Quot_True_def ext)