diff -r c7069b09730b -r 9f6c606d5b59 Quot/QuotMain.thy --- a/Quot/QuotMain.thy Wed Feb 10 10:55:14 2010 +0100 +++ b/Quot/QuotMain.thy Wed Feb 10 11:09:30 2010 +0100 @@ -140,7 +140,7 @@ 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_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) @@ -169,7 +169,7 @@ {* Sets up the three goals for the lifting procedure. *} method_setup regularize = - {* Scan.succeed (mk_method2 Quotient_Tacs.regularize_tac) *} + {* Scan.succeed (mk_method2 Quotient_Tacs.regularize_tac) *} {* Proves automatically the regularization goals from the lifting procedure. *} method_setup injection =