src/HOL/ex/LSC_Examples.thy
changeset 41912 1848775589e5
parent 41910 709c04e7b703
child 41913 34360908cb78
equal deleted inserted replaced
41911:c6e66b32ce16 41912:1848775589e5
   121 function series_tree
   121 function series_tree
   122 where
   122 where
   123   "series_tree d = sum (cons ET) (apply (apply (apply (apply (cons MKT) series) series_tree) series_tree) series) d"
   123   "series_tree d = sum (cons ET) (apply (apply (apply (apply (cons MKT) series) series_tree) series_tree) series) d"
   124 by pat_completeness auto
   124 by pat_completeness auto
   125 
   125 
   126 termination sorry
   126 termination proof (relation "measure nat_of")
       
   127 qed (auto simp add: of_int_inverse nat_of_def)
   127 
   128 
   128 instance ..
   129 instance ..
   129 
   130 
   130 end
   131 end
   131 
   132