| 62858 |      1 | (*  Title:      HOL/Corec_Examples/Tests/Merge_B.thy
 | 
| 62696 |      2 |     Author:     Aymeric Bouzy, Ecole polytechnique
 | 
|  |      3 |     Author:     Jasmin Blanchette, Inria, LORIA, MPII
 | 
|  |      4 |     Copyright   2015, 2016
 | 
|  |      5 | 
 | 
|  |      6 | Tests theory merges.
 | 
|  |      7 | *)
 | 
|  |      8 | 
 | 
| 62726 |      9 | section \<open>Tests Theory Merges\<close>
 | 
| 62696 |     10 | 
 | 
|  |     11 | theory Merge_B
 | 
|  |     12 | imports Merge_A
 | 
|  |     13 | begin
 | 
|  |     14 | 
 | 
|  |     15 | consts fb :: "'a ta \<Rightarrow> 'a ta"
 | 
|  |     16 | consts gb :: "'a ta \<Rightarrow> 'a ta"
 | 
|  |     17 | 
 | 
|  |     18 | friend_of_corec fb :: "'a ta \<Rightarrow> 'a ta" where
 | 
|  |     19 |   "fb t = Ca (sa1 t) (sa2 t)"
 | 
|  |     20 |   sorry
 | 
|  |     21 | 
 | 
|  |     22 | friend_of_corec gb :: "'a ta \<Rightarrow> 'a ta" where
 | 
|  |     23 |   "gb t = Ca (sa1 t) (sa2 t)"
 | 
|  |     24 |   sorry
 | 
|  |     25 | 
 | 
|  |     26 | end
 |