| 
37134
 | 
     1  | 
(*  Title:      FOL/ex/Locale_Test/Locale_Test3.thy
  | 
| 
 | 
     2  | 
    Author:     Clemens Ballarin
  | 
| 
 | 
     3  | 
  | 
| 
 | 
     4  | 
Test environment for the locale implementation.
  | 
| 
 | 
     5  | 
*)
  | 
| 
 | 
     6  | 
  | 
| 
 | 
     7  | 
theory Locale_Test3
  | 
| 
 | 
     8  | 
imports Locale_Test1
  | 
| 
 | 
     9  | 
begin
  | 
| 
 | 
    10  | 
  | 
| 
69590
 | 
    11  | 
interpretation le2: mixin_thy_merge \<open>gle\<close> \<open>gle'\<close>
  | 
| 
 | 
    12  | 
  rewrites \<open>reflexive.less(gle', x, y) \<longleftrightarrow> gless'(x, y)\<close>
  | 
| 
37134
 | 
    13  | 
proof -
  | 
| 
69590
 | 
    14  | 
  show \<open>mixin_thy_merge(gle, gle')\<close> by unfold_locales
  | 
| 
37134
 | 
    15  | 
  note reflexive = this[unfolded mixin_thy_merge_def, THEN conjunct2]
  | 
| 
69590
 | 
    16  | 
  show \<open>reflexive.less(gle', x, y) \<longleftrightarrow> gless'(x, y)\<close>
  | 
| 
37134
 | 
    17  | 
    by (simp add: reflexive.less_def[OF reflexive] gless'_def)
  | 
| 
 | 
    18  | 
qed
  | 
| 
 | 
    19  | 
  | 
| 
 | 
    20  | 
end
  |