src/HOL/Ord.thy
changeset 6855 36de02d1a257
parent 6515 18e113be12ee
child 7238 36e58620ffc8
--- a/src/HOL/Ord.thy	Mon Jun 28 23:05:19 1999 +0200
+++ b/src/HOL/Ord.thy	Tue Jun 29 11:58:21 1999 +0200
@@ -66,6 +66,6 @@
  "! x<y.  P"  =>  "! x. x < y  --> P"
  "! x<=y. P"  =>  "! x. x <= y --> P"
  "? x<y.  P"  =>  "? x. x < y  & P"
- "? x<=y. P"  =>  "! x. x <= y & P"
+ "? x<=y. P"  =>  "? x. x <= y & P"
 
 end