doc-src/IsarImplementation/Thy/Prelim.thy
changeset 35408 b48ab741683b
parent 34928 c4cd36411983
child 36611 b0c047d03208
equal deleted inserted replaced
35407:980d4194a212 35408:b48ab741683b
   434   (
   434   (
   435     type T = term OrdList.T;
   435     type T = term OrdList.T;
   436     val empty = [];
   436     val empty = [];
   437     val extend = I;
   437     val extend = I;
   438     fun merge (ts1, ts2) =
   438     fun merge (ts1, ts2) =
   439       OrdList.union TermOrd.fast_term_ord ts1 ts2;
   439       OrdList.union Term_Ord.fast_term_ord ts1 ts2;
   440   )
   440   )
   441 
   441 
   442   val get = Terms.get;
   442   val get = Terms.get;
   443 
   443 
   444   fun add raw_t thy =
   444   fun add raw_t thy =
   445     let val t = Sign.cert_term thy raw_t
   445     let val t = Sign.cert_term thy raw_t
   446     in Terms.map (OrdList.insert TermOrd.fast_term_ord t) thy end;
   446     in Terms.map (OrdList.insert Term_Ord.fast_term_ord t) thy end;
   447 
   447 
   448   end;
   448   end;
   449 *}
   449 *}
   450 
   450 
   451 text {* We use @{ML_type "term OrdList.T"} for reasonably efficient
   451 text {* We use @{ML_type "term OrdList.T"} for reasonably efficient