src/HOL/Orderings.thy
changeset 22068 00bed5ac9884
parent 21818 4d2ad5445c81
child 22206 8cc04341de38
--- a/src/HOL/Orderings.thy	Tue Jan 16 08:06:55 2007 +0100
+++ b/src/HOL/Orderings.thy	Tue Jan 16 08:06:57 2007 +0100
@@ -122,10 +122,10 @@
 
 subsection {* Partial orderings *}
 
-locale partial_order = preorder + 
+locale order = preorder + 
   assumes antisym: "x \<sqsubseteq> y \<Longrightarrow> y \<sqsubseteq> x \<Longrightarrow> x = y"
 
-context partial_order
+context order
 begin
 
 text {* Asymmetry. *}
@@ -181,7 +181,7 @@
   order_less_le: "(x < y) = (x <= y & x ~= y)"
 
 interpretation order:
-  partial_order ["op \<le> \<Colon> 'a\<Colon>order \<Rightarrow> 'a \<Rightarrow> bool" "op < \<Colon> 'a\<Colon>order \<Rightarrow> 'a \<Rightarrow> bool"]
+  order ["op \<le> \<Colon> 'a\<Colon>order \<Rightarrow> 'a \<Rightarrow> bool" "op < \<Colon> 'a\<Colon>order \<Rightarrow> 'a \<Rightarrow> bool"]
 apply unfold_locales
 apply (rule order_refl)
 apply (erule (1) order_trans)
@@ -192,7 +192,7 @@
 
 subsection {* Linear (total) orders *}
 
-locale linorder = partial_order +
+locale linorder = order +
   assumes linear: "x \<sqsubseteq> y \<or> y \<sqsubseteq> x"
 begin