src/HOL/Decision_Procs/Dense_Linear_Order.thy
changeset 35043 07dbdf60d5ad
parent 35028 108662d50512
child 35084 e25eedfc15ce
--- a/src/HOL/Decision_Procs/Dense_Linear_Order.thy	Mon Feb 08 14:22:22 2010 +0100
+++ b/src/HOL/Decision_Procs/Dense_Linear_Order.thy	Mon Feb 08 14:22:22 2010 +0100
@@ -637,7 +637,7 @@
   using eq_diff_eq[where a= x and b=t and c=0] by simp
 
 
-interpretation class_dense_linlinordered_field: constr_dense_linorder
+interpretation class_dense_linordered_field: constr_dense_linorder
  "op <=" "op <"
    "\<lambda> x y. 1/2 * ((x::'a::{linordered_field,number_ring}) + y)"
 proof (unfold_locales, dlo, dlo, auto)
@@ -871,7 +871,7 @@
    addsplits [@{thm "abs_split"},@{thm "split_max"}, @{thm "split_min"}]
 
 in
-Ferrante_Rackoff_Data.funs @{thm "class_dense_linlinordered_field.ferrack_axiom"}
+Ferrante_Rackoff_Data.funs @{thm "class_dense_linordered_field.ferrack_axiom"}
   {isolate_conv = field_isolate_conv, whatis = classfield_whatis, simpset = class_field_ss}
 end
 *}