src/HOL/Quot/PER0.thy
changeset 3842 b55686a7b22c
parent 3058 9d6526cacc3c
--- a/src/HOL/Quot/PER0.thy	Fri Oct 10 18:37:49 1997 +0200
+++ b/src/HOL/Quot/PER0.thy	Fri Oct 10 19:02:28 1997 +0200
@@ -27,9 +27,9 @@
         D         :: "'a::per set"
 defs
         per_def         "(op ===) == eqv"
-        Dom             "D=={x.x===x}"
+        Dom             "D=={x. x===x}"
 (* define ==== on and function type => *)
-        fun_per_def     "eqv f g == !x y.x:D & y:D & x===y --> f x === g y"
+        fun_per_def     "eqv f g == !x y. x:D & y:D & x===y --> f x === g y"
 
 syntax (symbols)
   "op ==="   :: "['a,'a::per] => bool"        (infixl "\\<sim>" 50)