src/HOL/Quotient.thy
changeset 63343 fb5d8a50c641
parent 61799 4cf66f21b764
child 67091 1393c2340eec
--- a/src/HOL/Quotient.thy	Tue Jun 21 17:35:45 2016 +0200
+++ b/src/HOL/Quotient.thy	Wed Jun 22 10:09:20 2016 +0200
@@ -28,9 +28,8 @@
   shows "((op =) OOO R) = R"
   by (auto simp add: fun_eq_iff)
 
-context
+context includes lifting_syntax
 begin
-interpretation lifting_syntax .
 
 subsection \<open>Quotient Predicate\<close>
 
@@ -805,9 +804,8 @@
 lemma QT_imp: "Quot_True a \<equiv> Quot_True b"
   by (simp add: Quot_True_def)
 
-context 
+context includes lifting_syntax
 begin
-interpretation lifting_syntax .
 
 text \<open>Tactics for proving the lifted theorems\<close>
 ML_file "Tools/Quotient/quotient_tacs.ML"