src/FOL/ex/Locale_Test/Locale_Test.thy
author blanchet
Tue, 07 Dec 2010 11:56:01 +0100
changeset 41051 2ed1b971fc20
parent 37134 29bd6c2ffba8
child 60770 240563fbf41d
permissions -rw-r--r--
give the inner timeout mechanism a chance, since it gives more precise information to the user
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
37134
29bd6c2ffba8 Revise locale test theory layout.
ballarin
parents:
diff changeset
     1
(*  Title:      FOL/ex/Locale_Test/Locale_Test.thy
29bd6c2ffba8 Revise locale test theory layout.
ballarin
parents:
diff changeset
     2
    Author:     Clemens Ballarin
29bd6c2ffba8 Revise locale test theory layout.
ballarin
parents:
diff changeset
     3
29bd6c2ffba8 Revise locale test theory layout.
ballarin
parents:
diff changeset
     4
Test environment for the locale implementation.
29bd6c2ffba8 Revise locale test theory layout.
ballarin
parents:
diff changeset
     5
*)
29bd6c2ffba8 Revise locale test theory layout.
ballarin
parents:
diff changeset
     6
29bd6c2ffba8 Revise locale test theory layout.
ballarin
parents:
diff changeset
     7
theory Locale_Test
29bd6c2ffba8 Revise locale test theory layout.
ballarin
parents:
diff changeset
     8
imports Locale_Test1 Locale_Test2 Locale_Test3
29bd6c2ffba8 Revise locale test theory layout.
ballarin
parents:
diff changeset
     9
begin
29bd6c2ffba8 Revise locale test theory layout.
ballarin
parents:
diff changeset
    10
29bd6c2ffba8 Revise locale test theory layout.
ballarin
parents:
diff changeset
    11
text {* Result of theory merge with distinct but identical interpretations *}
29bd6c2ffba8 Revise locale test theory layout.
ballarin
parents:
diff changeset
    12
29bd6c2ffba8 Revise locale test theory layout.
ballarin
parents:
diff changeset
    13
context mixin_thy_merge
29bd6c2ffba8 Revise locale test theory layout.
ballarin
parents:
diff changeset
    14
begin
29bd6c2ffba8 Revise locale test theory layout.
ballarin
parents:
diff changeset
    15
lemmas less_mixin_thy_merge1 = le.less_def
29bd6c2ffba8 Revise locale test theory layout.
ballarin
parents:
diff changeset
    16
lemmas less_mixin_thy_merge2 = le'.less_def
29bd6c2ffba8 Revise locale test theory layout.
ballarin
parents:
diff changeset
    17
end
29bd6c2ffba8 Revise locale test theory layout.
ballarin
parents:
diff changeset
    18
29bd6c2ffba8 Revise locale test theory layout.
ballarin
parents:
diff changeset
    19
lemma "gless(x, y) <-> gle(x, y) & x ~= y" (* mixin from first interpretation applied *)
29bd6c2ffba8 Revise locale test theory layout.
ballarin
parents:
diff changeset
    20
  by (rule le1.less_mixin_thy_merge1)
29bd6c2ffba8 Revise locale test theory layout.
ballarin
parents:
diff changeset
    21
lemma "gless'(x, y) <-> gle'(x, y) & x ~= y" (* mixin from second interpretation applied *)
29bd6c2ffba8 Revise locale test theory layout.
ballarin
parents:
diff changeset
    22
  by (rule le1.less_mixin_thy_merge2)
29bd6c2ffba8 Revise locale test theory layout.
ballarin
parents:
diff changeset
    23
29bd6c2ffba8 Revise locale test theory layout.
ballarin
parents:
diff changeset
    24
end