linorder_neqE_ordered_idom: proper proof, avoid illegal schematic type vars;
authorwenzelm
Sat, 01 Sep 2007 18:17:38 +0200
changeset 24515 d4dc5dc2db98
parent 24514 540eaf87e42d
child 24516 c121834a8808
linorder_neqE_ordered_idom: proper proof, avoid illegal schematic type vars;
src/HOL/Ring_and_Field.thy
--- a/src/HOL/Ring_and_Field.thy	Sat Sep 01 18:17:36 2007 +0200
+++ b/src/HOL/Ring_and_Field.thy	Sat Sep 01 18:17:38 2007 +0200
@@ -347,8 +347,10 @@
 
 class ordered_field = field + ordered_idom
 
-lemmas linorder_neqE_ordered_idom =
- linorder_neqE[where 'a = "?'b::ordered_idom"]
+lemma linorder_neqE_ordered_idom:
+  fixes x y :: "'a :: ordered_idom"
+  assumes "x \<noteq> y" obtains "x < y" | "y < x"
+  using assms by (rule linorder_neqE)
 
 lemma eq_add_iff1:
   "(a*e + c = b*e + d) = ((a-b)*e + c = (d::'a::ring))"