src/HOL/Lifting.thy
changeset 67229 4ecf0ef70efb
parent 63343 fb5d8a50c641
child 67399 eab6ce8368fa
--- a/src/HOL/Lifting.thy	Wed Dec 20 12:22:36 2017 +0100
+++ b/src/HOL/Lifting.thy	Wed Dec 20 14:53:34 2017 +0100
@@ -228,7 +228,7 @@
   fixes Abs :: "'a \<Rightarrow> 'b"
   and Rep :: "'b \<Rightarrow> 'a"
   assumes "type_definition Rep Abs (UNIV::'a set)"
-  shows "equivp (op=::'a\<Rightarrow>'a\<Rightarrow>bool)"
+  shows "equivp (op= ::'a\<Rightarrow>'a\<Rightarrow>bool)"
 by (rule identity_equivp)
 
 lemma typedef_to_Quotient: