src/HOL/HOL.thy
changeset 14223 0ee05eef881b
parent 14208 144f45277d5a
child 14248 399a3290936c
--- a/src/HOL/HOL.thy	Wed Oct 08 16:02:54 2003 +0200
+++ b/src/HOL/HOL.thy	Thu Oct 09 18:13:32 2003 +0200
@@ -146,10 +146,11 @@
   Let_def:      "Let s f == f(s)"
   if_def:       "If P x y == THE z::'a. (P=True --> z=x) & (P=False --> z=y)"
 
-  arbitrary_def:  "False ==> arbitrary == (THE x. False)"
-    -- {* @{term arbitrary} is completely unspecified, but is made to appear as a
-    definition syntactically *}
-
+finalconsts
+  "op ="
+  "op -->"
+  The
+  arbitrary
 
 subsubsection {* Generic algebraic operations *}