src/HOL/Decision_Procs/Dense_Linear_Order.thy
changeset 45620 f2a587696afb
parent 44064 5bce8ff0d9ae
child 46497 89ccf66aa73d
equal deleted inserted replaced
45619:76c5f277b234 45620:f2a587696afb
   863          else Ferrante_Rackoff_Data.Nox
   863          else Ferrante_Rackoff_Data.Nox
   864    | _ => Ferrante_Rackoff_Data.Nox
   864    | _ => Ferrante_Rackoff_Data.Nox
   865  in h end;
   865  in h end;
   866 fun class_field_ss phi =
   866 fun class_field_ss phi =
   867    HOL_basic_ss addsimps ([@{thm "linorder_not_less"}, @{thm "linorder_not_le"}])
   867    HOL_basic_ss addsimps ([@{thm "linorder_not_less"}, @{thm "linorder_not_le"}])
   868    addsplits [@{thm "abs_split"},@{thm "split_max"}, @{thm "split_min"}]
   868    |> fold Splitter.add_split [@{thm "abs_split"}, @{thm "split_max"}, @{thm "split_min"}]
   869 
   869 
   870 in
   870 in
   871 Ferrante_Rackoff_Data.funs @{thm "class_dense_linordered_field.ferrack_axiom"}
   871 Ferrante_Rackoff_Data.funs @{thm "class_dense_linordered_field.ferrack_axiom"}
   872   {isolate_conv = field_isolate_conv, whatis = classfield_whatis, simpset = class_field_ss}
   872   {isolate_conv = field_isolate_conv, whatis = classfield_whatis, simpset = class_field_ss}
   873 end
   873 end