src/FOL/ex/LocaleTest.thy
author huffman
Wed, 24 Dec 2008 13:16:26 -0800
changeset 29170 dad3933c88dd
parent 28611 983c1855a7af
permissions -rw-r--r--
clean up lemmas about exp
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
15596
8665d08085df First version of global registration command.
ballarin
parents:
diff changeset
     1
(*  Title:      FOL/ex/LocaleTest.thy
8665d08085df First version of global registration command.
ballarin
parents:
diff changeset
     2
    ID:         $Id$
8665d08085df First version of global registration command.
ballarin
parents:
diff changeset
     3
    Author:     Clemens Ballarin
8665d08085df First version of global registration command.
ballarin
parents:
diff changeset
     4
    Copyright (c) 2005 by Clemens Ballarin
8665d08085df First version of global registration command.
ballarin
parents:
diff changeset
     5
8665d08085df First version of global registration command.
ballarin
parents:
diff changeset
     6
Collection of regression tests for locales.
8665d08085df First version of global registration command.
ballarin
parents:
diff changeset
     7
*)
8665d08085df First version of global registration command.
ballarin
parents:
diff changeset
     8
16102
c5f6726d9bb1 Locale expressions: rename with optional mixfix syntax.
ballarin
parents: 15837
diff changeset
     9
header {* Test of Locale Interpretation *}
15596
8665d08085df First version of global registration command.
ballarin
parents:
diff changeset
    10
16102
c5f6726d9bb1 Locale expressions: rename with optional mixfix syntax.
ballarin
parents: 15837
diff changeset
    11
theory LocaleTest
c5f6726d9bb1 Locale expressions: rename with optional mixfix syntax.
ballarin
parents: 15837
diff changeset
    12
imports FOL
c5f6726d9bb1 Locale expressions: rename with optional mixfix syntax.
ballarin
parents: 15837
diff changeset
    13
begin
15596
8665d08085df First version of global registration command.
ballarin
parents:
diff changeset
    14
16168
adb83939177f Locales: new element constrains, parameter renaming with syntax,
ballarin
parents: 16102
diff changeset
    15
ML {* set Toplevel.debug *}
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
    16
ML {* set show_hyps *}
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
    17
ML {* set show_sorts *}
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
    18
17139
165c97f9bb63 Printing of interpretations: option to show witness theorems;
ballarin
parents: 17096
diff changeset
    19
ML {*
165c97f9bb63 Printing of interpretations: option to show witness theorems;
ballarin
parents: 17096
diff changeset
    20
  fun check_thm name = let
165c97f9bb63 Printing of interpretations: option to show witness theorems;
ballarin
parents: 17096
diff changeset
    21
    val thy = the_context ();
26343
0dd2eab7b296 simplified get_thm(s): back to plain name argument;
wenzelm
parents: 26336
diff changeset
    22
    val thm = PureThy.get_thm thy name;
17139
165c97f9bb63 Printing of interpretations: option to show witness theorems;
ballarin
parents: 17096
diff changeset
    23
    val {prop, hyps, ...} = rep_thm thm;
165c97f9bb63 Printing of interpretations: option to show witness theorems;
ballarin
parents: 17096
diff changeset
    24
    val prems = Logic.strip_imp_prems prop;
165c97f9bb63 Printing of interpretations: option to show witness theorems;
ballarin
parents: 17096
diff changeset
    25
    val _ = if null hyps then ()
165c97f9bb63 Printing of interpretations: option to show witness theorems;
ballarin
parents: 17096
diff changeset
    26
        else error ("Theorem " ^ quote name ^ " has meta hyps.\n" ^
165c97f9bb63 Printing of interpretations: option to show witness theorems;
ballarin
parents: 17096
diff changeset
    27
          "Consistency check of locales package failed.");
165c97f9bb63 Printing of interpretations: option to show witness theorems;
ballarin
parents: 17096
diff changeset
    28
    val _ = if null prems then ()
165c97f9bb63 Printing of interpretations: option to show witness theorems;
ballarin
parents: 17096
diff changeset
    29
        else error ("Theorem " ^ quote name ^ " has premises.\n" ^
165c97f9bb63 Printing of interpretations: option to show witness theorems;
ballarin
parents: 17096
diff changeset
    30
          "Consistency check of locales package failed.");
165c97f9bb63 Printing of interpretations: option to show witness theorems;
ballarin
parents: 17096
diff changeset
    31
  in () end;
165c97f9bb63 Printing of interpretations: option to show witness theorems;
ballarin
parents: 17096
diff changeset
    32
*}
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
    33
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
    34
section {* Context Elements and Locale Expressions *}
16102
c5f6726d9bb1 Locale expressions: rename with optional mixfix syntax.
ballarin
parents: 15837
diff changeset
    35
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
    36
text {* Naming convention for global objects: prefixes L and l *}
16168
adb83939177f Locales: new element constrains, parameter renaming with syntax,
ballarin
parents: 16102
diff changeset
    37
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
    38
subsection {* Renaming with Syntax *}
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
    39
27681
8cedebf55539 dropped locale (open)
haftmann
parents: 27618
diff changeset
    40
locale LS = var mult +
16102
c5f6726d9bb1 Locale expressions: rename with optional mixfix syntax.
ballarin
parents: 15837
diff changeset
    41
  assumes "mult(x, y) = mult(y, x)"
c5f6726d9bb1 Locale expressions: rename with optional mixfix syntax.
ballarin
parents: 15837
diff changeset
    42
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
    43
print_locale LS
16168
adb83939177f Locales: new element constrains, parameter renaming with syntax,
ballarin
parents: 16102
diff changeset
    44
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
    45
locale LS' = LS mult (infixl "**" 60)
16102
c5f6726d9bb1 Locale expressions: rename with optional mixfix syntax.
ballarin
parents: 15837
diff changeset
    46
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
    47
print_locale LS'
16102
c5f6726d9bb1 Locale expressions: rename with optional mixfix syntax.
ballarin
parents: 15837
diff changeset
    48
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
    49
locale LT = var mult (infixl "**" 60) +
16102
c5f6726d9bb1 Locale expressions: rename with optional mixfix syntax.
ballarin
parents: 15837
diff changeset
    50
  assumes "x ** y = y ** x"
c5f6726d9bb1 Locale expressions: rename with optional mixfix syntax.
ballarin
parents: 15837
diff changeset
    51
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
    52
locale LU = LT mult (infixl "**" 60) + LT add (infixl "++" 55) + var h +
16102
c5f6726d9bb1 Locale expressions: rename with optional mixfix syntax.
ballarin
parents: 15837
diff changeset
    53
  assumes hom: "h(x ** y) = h(x) ++ h(y)"
c5f6726d9bb1 Locale expressions: rename with optional mixfix syntax.
ballarin
parents: 15837
diff changeset
    54
25282
1cc04c8e1253 Tests enforce proper export behaviour.
ballarin
parents: 24788
diff changeset
    55
1cc04c8e1253 Tests enforce proper export behaviour.
ballarin
parents: 24788
diff changeset
    56
(* FIXME: graceful handling of type errors?
19783
82f365a14960 Improved parameter management of locales.
ballarin
parents: 17436
diff changeset
    57
locale LY = LT mult (infixl "**" 60) + LT add (binder "++" 55) + var h +
82f365a14960 Improved parameter management of locales.
ballarin
parents: 17436
diff changeset
    58
  assumes "mult(x) == add"
82f365a14960 Improved parameter management of locales.
ballarin
parents: 17436
diff changeset
    59
*)
82f365a14960 Improved parameter management of locales.
ballarin
parents: 17436
diff changeset
    60
25282
1cc04c8e1253 Tests enforce proper export behaviour.
ballarin
parents: 24788
diff changeset
    61
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
    62
locale LV = LU _ add
16102
c5f6726d9bb1 Locale expressions: rename with optional mixfix syntax.
ballarin
parents: 15837
diff changeset
    63
19783
82f365a14960 Improved parameter management of locales.
ballarin
parents: 17436
diff changeset
    64
locale LW = LU _ mult (infixl "**" 60)
82f365a14960 Improved parameter management of locales.
ballarin
parents: 17436
diff changeset
    65
16168
adb83939177f Locales: new element constrains, parameter renaming with syntax,
ballarin
parents: 16102
diff changeset
    66
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
    67
subsection {* Constrains *}
16102
c5f6726d9bb1 Locale expressions: rename with optional mixfix syntax.
ballarin
parents: 15837
diff changeset
    68
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
    69
locale LZ = fixes a (structure)
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
    70
locale LZ' = LZ +
16168
adb83939177f Locales: new element constrains, parameter renaming with syntax,
ballarin
parents: 16102
diff changeset
    71
  constrains a :: "'a => 'b"
adb83939177f Locales: new element constrains, parameter renaming with syntax,
ballarin
parents: 16102
diff changeset
    72
  assumes "a (x :: 'a) = a (y)"
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
    73
print_locale LZ'
16102
c5f6726d9bb1 Locale expressions: rename with optional mixfix syntax.
ballarin
parents: 15837
diff changeset
    74
c5f6726d9bb1 Locale expressions: rename with optional mixfix syntax.
ballarin
parents: 15837
diff changeset
    75
c5f6726d9bb1 Locale expressions: rename with optional mixfix syntax.
ballarin
parents: 15837
diff changeset
    76
section {* Interpretation *}
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
    77
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
    78
text {* Naming convention for global objects: prefixes I and i *}
15596
8665d08085df First version of global registration command.
ballarin
parents:
diff changeset
    79
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
    80
text {* interpretation input syntax *}
15596
8665d08085df First version of global registration command.
ballarin
parents:
diff changeset
    81
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
    82
locale IL
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
    83
locale IM = fixes a and b and c
15596
8665d08085df First version of global registration command.
ballarin
parents:
diff changeset
    84
28085
914183e229e9 Interpretation commands no longer accept interpretation attributes.
ballarin
parents: 27761
diff changeset
    85
interpretation test: IL + IM a b c [x y z] .
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
    86
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
    87
print_interps IL    (* output: test *)
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
    88
print_interps IM    (* output: test *)
15596
8665d08085df First version of global registration command.
ballarin
parents:
diff changeset
    89
28085
914183e229e9 Interpretation commands no longer accept interpretation attributes.
ballarin
parents: 27761
diff changeset
    90
interpretation test: IL print_interps IM .
15596
8665d08085df First version of global registration command.
ballarin
parents:
diff changeset
    91
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
    92
interpretation IL .
15596
8665d08085df First version of global registration command.
ballarin
parents:
diff changeset
    93
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
    94
text {* Processing of locale expression *}
15596
8665d08085df First version of global registration command.
ballarin
parents:
diff changeset
    95
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
    96
locale IA = fixes a assumes asm_A: "a = a"
15596
8665d08085df First version of global registration command.
ballarin
parents:
diff changeset
    97
27681
8cedebf55539 dropped locale (open)
haftmann
parents: 27618
diff changeset
    98
locale IB = fixes b assumes asm_B [simp]: "b = b"
15596
8665d08085df First version of global registration command.
ballarin
parents:
diff changeset
    99
28235
89e4d2232ed2 No interpretation of locale with dangling type frees.
ballarin
parents: 28085
diff changeset
   100
locale IC = IA + IB + assumes asm_C: "b = b"
89e4d2232ed2 No interpretation of locale with dangling type frees.
ballarin
parents: 28085
diff changeset
   101
89e4d2232ed2 No interpretation of locale with dangling type frees.
ballarin
parents: 28085
diff changeset
   102
locale IC' = IA + IB + assumes asm_C: "c = c"
89e4d2232ed2 No interpretation of locale with dangling type frees.
ballarin
parents: 28085
diff changeset
   103
  (* independent type var in c *)
15596
8665d08085df First version of global registration command.
ballarin
parents:
diff changeset
   104
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   105
locale ID = IA + IB + fixes d defines def_D: "d == (a = b)"
15596
8665d08085df First version of global registration command.
ballarin
parents:
diff changeset
   106
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   107
theorem (in ID) True ..
15596
8665d08085df First version of global registration command.
ballarin
parents:
diff changeset
   108
8665d08085df First version of global registration command.
ballarin
parents:
diff changeset
   109
typedecl i
8665d08085df First version of global registration command.
ballarin
parents:
diff changeset
   110
arities i :: "term"
8665d08085df First version of global registration command.
ballarin
parents:
diff changeset
   111
15598
4ab52355bb53 Registrations of global locale interpretations: improved, better naming.
ballarin
parents: 15596
diff changeset
   112
19984
29bb4659f80a Method intro_locales replaced by intro_locales and unfold_locales.
ballarin
parents: 19931
diff changeset
   113
interpretation i1: IC ["X::i" "Y::i"] by unfold_locales auto
15596
8665d08085df First version of global registration command.
ballarin
parents:
diff changeset
   114
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   115
print_interps IA  (* output: i1 *)
15596
8665d08085df First version of global registration command.
ballarin
parents:
diff changeset
   116
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   117
(* possible accesses *)
26645
e114be97befe Changed naming scheme for theorems generated by interpretations.
ballarin
parents: 26343
diff changeset
   118
thm i1.a.asm_A thm LocaleTest.IA_locale.i1.a.asm_A thm IA_locale.i1.a.asm_A
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   119
thm i1.asm_A thm LocaleTest.i1.asm_A
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   120
17139
165c97f9bb63 Printing of interpretations: option to show witness theorems;
ballarin
parents: 17096
diff changeset
   121
ML {* check_thm "i1.a.asm_A" *}
15624
484178635bd8 Further work on interpretation commands. New command `interpret' for
ballarin
parents: 15598
diff changeset
   122
484178635bd8 Further work on interpretation commands. New command `interpret' for
ballarin
parents: 15598
diff changeset
   123
(* without prefix *)
484178635bd8 Further work on interpretation commands. New command `interpret' for
ballarin
parents: 15598
diff changeset
   124
27761
b95e9ba0ca1d Interpretation command (theory/proof context) no longer simplifies goal.
ballarin
parents: 27718
diff changeset
   125
interpretation IC ["W::i" "Z::i"] by intro_locales  (* subsumed by i1: IC *)
19984
29bb4659f80a Method intro_locales replaced by intro_locales and unfold_locales.
ballarin
parents: 19931
diff changeset
   126
interpretation IC ["W::'a" "Z::i"] by unfold_locales auto
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   127
  (* subsumes i1: IA and i1: IC *)
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   128
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   129
print_interps IA  (* output: <no prefix>, i1 *)
15596
8665d08085df First version of global registration command.
ballarin
parents:
diff changeset
   130
15837
7a567dcd4cda Subsumption of locale interpretations.
ballarin
parents: 15763
diff changeset
   131
(* possible accesses *)
26645
e114be97befe Changed naming scheme for theorems generated by interpretations.
ballarin
parents: 26343
diff changeset
   132
thm asm_C thm a_b.asm_C thm LocaleTest.IC_locale.a_b.asm_C thm IC_locale.a_b.asm_C
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   133
17139
165c97f9bb63 Printing of interpretations: option to show witness theorems;
ballarin
parents: 17096
diff changeset
   134
ML {* check_thm "asm_C" *}
15596
8665d08085df First version of global registration command.
ballarin
parents:
diff changeset
   135
19931
fb32b43e7f80 Restructured locales with predicates: import is now an interpretation.
ballarin
parents: 19783
diff changeset
   136
interpretation i2: ID [X "Y::i" "Y = X"]
19984
29bb4659f80a Method intro_locales replaced by intro_locales and unfold_locales.
ballarin
parents: 19931
diff changeset
   137
  by (simp add: eq_commute) unfold_locales
15837
7a567dcd4cda Subsumption of locale interpretations.
ballarin
parents: 15763
diff changeset
   138
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   139
print_interps IA  (* output: <no prefix>, i1 *)
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   140
print_interps ID  (* output: i2 *)
15837
7a567dcd4cda Subsumption of locale interpretations.
ballarin
parents: 15763
diff changeset
   141
7a567dcd4cda Subsumption of locale interpretations.
ballarin
parents: 15763
diff changeset
   142
19984
29bb4659f80a Method intro_locales replaced by intro_locales and unfold_locales.
ballarin
parents: 19931
diff changeset
   143
interpretation i3: ID [X "Y::i"] by simp unfold_locales
15598
4ab52355bb53 Registrations of global locale interpretations: improved, better naming.
ballarin
parents: 15596
diff changeset
   144
17436
ballarin
parents: 17228
diff changeset
   145
(* duplicate: thm not added *)
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   146
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   147
(* thm i3.a.asm_A *)
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   148
15596
8665d08085df First version of global registration command.
ballarin
parents:
diff changeset
   149
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   150
print_interps IA  (* output: <no prefix>, i1 *)
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   151
print_interps IB  (* output: i1 *)
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   152
print_interps IC  (* output: <no prefix, i1 *)
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   153
print_interps ID  (* output: i2, i3 *)
15596
8665d08085df First version of global registration command.
ballarin
parents:
diff changeset
   154
8665d08085df First version of global registration command.
ballarin
parents:
diff changeset
   155
27761
b95e9ba0ca1d Interpretation command (theory/proof context) no longer simplifies goal.
ballarin
parents: 27718
diff changeset
   156
interpretation i10: ID + ID a' b' d' [X "Y::i" _ u "v::i" _] by intro_locales
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   157
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   158
corollary (in ID) th_x: True ..
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   159
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   160
(* possible accesses: for each registration *)
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   161
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   162
thm i2.th_x thm i3.th_x
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   163
17139
165c97f9bb63 Printing of interpretations: option to show witness theorems;
ballarin
parents: 17096
diff changeset
   164
ML {* check_thm "i2.th_x"; check_thm "i3.th_x" *}
165c97f9bb63 Printing of interpretations: option to show witness theorems;
ballarin
parents: 17096
diff changeset
   165
26199
04817a8802f2 explicit referencing of background facts;
wenzelm
parents: 25282
diff changeset
   166
lemma (in ID) th_y: "d == (a = b)" by (rule d_def)
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   167
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   168
thm i2.th_y thm i3.th_y
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   169
17139
165c97f9bb63 Printing of interpretations: option to show witness theorems;
ballarin
parents: 17096
diff changeset
   170
ML {* check_thm "i2.th_y"; check_thm "i3.th_y" *}
165c97f9bb63 Printing of interpretations: option to show witness theorems;
ballarin
parents: 17096
diff changeset
   171
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   172
lemmas (in ID) th_z = th_y
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   173
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   174
thm i2.th_z
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   175
17139
165c97f9bb63 Printing of interpretations: option to show witness theorems;
ballarin
parents: 17096
diff changeset
   176
ML {* check_thm "i2.th_z" *}
165c97f9bb63 Printing of interpretations: option to show witness theorems;
ballarin
parents: 17096
diff changeset
   177
15596
8665d08085df First version of global registration command.
ballarin
parents:
diff changeset
   178
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   179
subsection {* Interpretation in Proof Contexts *}
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   180
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   181
locale IF = fixes f assumes asm_F: "f & f --> f"
16102
c5f6726d9bb1 Locale expressions: rename with optional mixfix syntax.
ballarin
parents: 15837
diff changeset
   182
25282
1cc04c8e1253 Tests enforce proper export behaviour.
ballarin
parents: 24788
diff changeset
   183
consts default :: "'a"
1cc04c8e1253 Tests enforce proper export behaviour.
ballarin
parents: 24788
diff changeset
   184
15624
484178635bd8 Further work on interpretation commands. New command `interpret' for
ballarin
parents: 15598
diff changeset
   185
theorem True
484178635bd8 Further work on interpretation commands. New command `interpret' for
ballarin
parents: 15598
diff changeset
   186
proof -
25282
1cc04c8e1253 Tests enforce proper export behaviour.
ballarin
parents: 24788
diff changeset
   187
  fix alpha::i and beta
1cc04c8e1253 Tests enforce proper export behaviour.
ballarin
parents: 24788
diff changeset
   188
  have alpha_A: "IA(alpha)" by unfold_locales
27761
b95e9ba0ca1d Interpretation command (theory/proof context) no longer simplifies goal.
ballarin
parents: 27718
diff changeset
   189
  interpret i5: IA [alpha] by intro_locales  (* subsumed *)
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   190
  print_interps IA  (* output: <no prefix>, i1 *)
19984
29bb4659f80a Method intro_locales replaced by intro_locales and unfold_locales.
ballarin
parents: 19931
diff changeset
   191
  interpret i6: IC [alpha beta] by unfold_locales auto
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   192
  print_interps IA   (* output: <no prefix>, i1 *)
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   193
  print_interps IC   (* output: <no prefix>, i1, i6 *)
25282
1cc04c8e1253 Tests enforce proper export behaviour.
ballarin
parents: 24788
diff changeset
   194
  interpret i11: IF ["default = default"] by (fast intro: IF.intro)
1cc04c8e1253 Tests enforce proper export behaviour.
ballarin
parents: 24788
diff changeset
   195
  thm i11.asm_F [where 'a = i]     (* default has schematic type *)
15624
484178635bd8 Further work on interpretation commands. New command `interpret' for
ballarin
parents: 15598
diff changeset
   196
qed rule
484178635bd8 Further work on interpretation commands. New command `interpret' for
ballarin
parents: 15598
diff changeset
   197
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   198
theorem (in IA) True
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   199
proof -
19931
fb32b43e7f80 Restructured locales with predicates: import is now an interpretation.
ballarin
parents: 19783
diff changeset
   200
  print_interps! IA
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   201
  fix beta and gamma
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   202
  interpret i9: ID [a beta _]
19931
fb32b43e7f80 Restructured locales with predicates: import is now an interpretation.
ballarin
parents: 19783
diff changeset
   203
    apply - apply assumption
19984
29bb4659f80a Method intro_locales replaced by intro_locales and unfold_locales.
ballarin
parents: 19931
diff changeset
   204
    apply unfold_locales
19931
fb32b43e7f80 Restructured locales with predicates: import is now an interpretation.
ballarin
parents: 19783
diff changeset
   205
    apply (rule refl) done
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   206
qed rule
15624
484178635bd8 Further work on interpretation commands. New command `interpret' for
ballarin
parents: 15598
diff changeset
   207
484178635bd8 Further work on interpretation commands. New command `interpret' for
ballarin
parents: 15598
diff changeset
   208
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   209
(* Definition involving free variable *)
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   210
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   211
ML {* reset show_sorts *}
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   212
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   213
locale IE = fixes e defines e_def: "e(x) == x & x"
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   214
  notes e_def2 = e_def
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   215
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   216
lemma (in IE) True thm e_def by fast
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   217
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   218
interpretation i7: IE ["%x. x"] by simp
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   219
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   220
thm i7.e_def2 (* has no premise *)
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   221
17139
165c97f9bb63 Printing of interpretations: option to show witness theorems;
ballarin
parents: 17096
diff changeset
   222
ML {* check_thm "i7.e_def2" *}
165c97f9bb63 Printing of interpretations: option to show witness theorems;
ballarin
parents: 17096
diff changeset
   223
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   224
locale IE' = fixes e defines e_def: "e == (%x. x & x)"
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   225
  notes e_def2 = e_def
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   226
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   227
interpretation i7': IE' ["(%x. x)"] by simp
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   228
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   229
thm i7'.e_def2
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   230
17139
165c97f9bb63 Printing of interpretations: option to show witness theorems;
ballarin
parents: 17096
diff changeset
   231
ML {* check_thm "i7'.e_def2" *}
165c97f9bb63 Printing of interpretations: option to show witness theorems;
ballarin
parents: 17096
diff changeset
   232
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   233
(* Definition involving free variable in assm *)
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   234
27681
8cedebf55539 dropped locale (open)
haftmann
parents: 27618
diff changeset
   235
locale IG = fixes g assumes asm_G: "g --> x"
16102
c5f6726d9bb1 Locale expressions: rename with optional mixfix syntax.
ballarin
parents: 15837
diff changeset
   236
  notes asm_G2 = asm_G
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   237
27718
3a85bc6bfd73 Updated locale tests.
ballarin
parents: 27681
diff changeset
   238
interpretation i8: IG ["False"] by unfold_locales fast
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   239
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   240
thm i8.asm_G2
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   241
17139
165c97f9bb63 Printing of interpretations: option to show witness theorems;
ballarin
parents: 17096
diff changeset
   242
ML {* check_thm "i8.asm_G2" *}
165c97f9bb63 Printing of interpretations: option to show witness theorems;
ballarin
parents: 17096
diff changeset
   243
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   244
text {* Locale without assumptions *}
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   245
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   246
locale IL1 = notes rev_conjI [intro] = conjI [THEN iffD1 [OF conj_commute]]
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   247
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   248
lemma "[| P; Q |] ==> P & Q"
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   249
proof -
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   250
  interpret my: IL1 .          txt {* No chained fact required. *}
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   251
  assume Q and P               txt {* order reversed *}
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   252
  then show "P & Q" ..         txt {* Applies @{thm my.rev_conjI}. *}
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   253
qed
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   254
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   255
locale IL11 = notes rev_conjI = conjI [THEN iffD1 [OF conj_commute]]
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   256
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   257
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   258
subsection {* Simple locale with assumptions *}
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   259
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   260
consts ibin :: "[i, i] => i" (infixl "#" 60)
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   261
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   262
axioms i_assoc: "(x # y) # z = x # (y # z)"
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   263
  i_comm: "x # y = y # x"
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   264
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   265
locale IL2 =
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   266
  fixes OP (infixl "+" 60)
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   267
  assumes assoc: "(x + y) + z = x + (y + z)"
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   268
    and comm: "x + y = y + x"
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   269
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   270
lemma (in IL2) lcomm: "x + (y + z) = y + (x + z)"
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   271
proof -
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   272
  have "x + (y + z) = (x + y) + z" by (simp add: assoc)
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   273
  also have "... = (y + x) + z" by (simp add: comm)
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   274
  also have "... = y + (x + z)" by (simp add: assoc)
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   275
  finally show ?thesis .
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   276
qed
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   277
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   278
lemmas (in IL2) AC = comm assoc lcomm
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   279
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   280
lemma "(x::i) # y # z # w = y # x # w # z"
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   281
proof -
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   282
  interpret my: IL2 ["op #"] by (rule IL2.intro [of "op #", OF i_assoc i_comm])
17033
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   283
  show ?thesis by (simp only: my.OP.AC)  (* or my.AC *)
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   284
qed
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   285
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   286
subsection {* Nested locale with assumptions *}
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   287
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   288
locale IL3 =
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   289
  fixes OP (infixl "+" 60)
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   290
  assumes assoc: "(x + y) + z = x + (y + z)"
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   291
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   292
locale IL4 = IL3 +
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   293
  assumes comm: "x + y = y + x"
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   294
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   295
lemma (in IL4) lcomm: "x + (y + z) = y + (x + z)"
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   296
proof -
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   297
  have "x + (y + z) = (x + y) + z" by (simp add: assoc)
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   298
  also have "... = (y + x) + z" by (simp add: comm)
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   299
  also have "... = y + (x + z)" by (simp add: assoc)
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   300
  finally show ?thesis .
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   301
qed
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   302
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   303
lemmas (in IL4) AC = comm assoc lcomm
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   304
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   305
lemma "(x::i) # y # z # w = y # x # w # z"
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   306
proof -
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   307
  interpret my: IL4 ["op #"]
19931
fb32b43e7f80 Restructured locales with predicates: import is now an interpretation.
ballarin
parents: 19783
diff changeset
   308
    by (auto intro: IL4.intro IL3.intro IL4_axioms.intro i_assoc i_comm)
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   309
  show ?thesis by (simp only: my.OP.AC)  (* or simply AC *)
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   310
qed
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   311
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   312
text {* Locale with definition *}
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   313
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   314
text {* This example is admittedly not very creative :-) *}
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   315
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   316
locale IL5 = IL4 + var A +
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   317
  defines A_def: "A == True"
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   318
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   319
lemma (in IL5) lem: A
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   320
  by (unfold A_def) rule
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   321
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   322
lemma "IL5(op #) ==> True"
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   323
proof -
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   324
  assume "IL5(op #)"
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   325
  then interpret IL5 ["op #"] by (auto intro: IL5.axioms)
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   326
  show ?thesis by (rule lem)  (* lem instantiated to True *)
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   327
qed
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   328
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   329
text {* Interpretation in a context with target *}
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   330
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   331
lemma (in IL4)
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   332
  fixes A (infixl "$" 60)
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   333
  assumes A: "IL4(A)"
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   334
  shows "(x::i) $ y $ z $ w = y $ x $ w $ z"
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   335
proof -
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   336
  from A interpret A: IL4 ["A"] by (auto intro: IL4.axioms)
15696
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   337
  show ?thesis by (simp only: A.OP.AC)
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   338
qed
1da4ce092c0b First release of interpretation commands.
ballarin
parents: 15624
diff changeset
   339
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   340
16736
1e792b32abef Preparations for interpretation of locales in locales.
ballarin
parents: 16620
diff changeset
   341
section {* Interpretation in Locales *}
1e792b32abef Preparations for interpretation of locales in locales.
ballarin
parents: 16620
diff changeset
   342
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   343
text {* Naming convention for global objects: prefixes R and r *}
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   344
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   345
(* locale with many parameters ---
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   346
   interpretations generate alternating group A5 *)
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   347
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   348
locale RA5 = var A + var B + var C + var D + var E +
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   349
  assumes eq: "A <-> B <-> C <-> D <-> E"
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   350
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   351
interpretation RA5 < RA5 _ _ D E C
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   352
print_facts
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   353
print_interps RA5
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   354
  using A_B_C_D_E.eq apply (blast intro: RA5.intro) done
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   355
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   356
interpretation RA5 < RA5 C _ E _ A
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   357
print_facts
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   358
print_interps RA5
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   359
  using A_B_C_D_E.eq apply (blast intro: RA5.intro) done
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   360
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   361
interpretation RA5 < RA5 B C A _ _
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   362
print_facts
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   363
print_interps RA5
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   364
  using A_B_C_D_E.eq apply (blast intro: RA5.intro) done
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   365
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   366
interpretation RA5 < RA5 _ C D B _ .
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   367
  (* Any even permutation of parameters is subsumed by the above. *)
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   368
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   369
(* circle of three locales, forward direction *)
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   370
27681
8cedebf55539 dropped locale (open)
haftmann
parents: 27618
diff changeset
   371
locale RA1 = var A + var B + assumes p: "A <-> B"
8cedebf55539 dropped locale (open)
haftmann
parents: 27618
diff changeset
   372
locale RA2 = var A + var B + assumes q: "A & B | ~ A & ~ B"
8cedebf55539 dropped locale (open)
haftmann
parents: 27618
diff changeset
   373
locale RA3 = var A + var B + assumes r: "(A --> B) & (B --> A)"
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   374
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   375
interpretation RA1 < RA2
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   376
  print_facts
27681
8cedebf55539 dropped locale (open)
haftmann
parents: 27618
diff changeset
   377
  using p apply unfold_locales apply fast done
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   378
interpretation RA2 < RA3
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   379
  print_facts
27681
8cedebf55539 dropped locale (open)
haftmann
parents: 27618
diff changeset
   380
  using q apply unfold_locales apply fast done
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   381
interpretation RA3 < RA1
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   382
  print_facts
27681
8cedebf55539 dropped locale (open)
haftmann
parents: 27618
diff changeset
   383
  using r apply unfold_locales apply fast done
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   384
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   385
(* circle of three locales, backward direction *)
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   386
27681
8cedebf55539 dropped locale (open)
haftmann
parents: 27618
diff changeset
   387
locale RB1 = var A + var B + assumes p: "A <-> B"
8cedebf55539 dropped locale (open)
haftmann
parents: 27618
diff changeset
   388
locale RB2 = var A + var B + assumes q: "A & B | ~ A & ~ B"
8cedebf55539 dropped locale (open)
haftmann
parents: 27618
diff changeset
   389
locale RB3 = var A + var B + assumes r: "(A --> B) & (B --> A)"
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   390
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   391
interpretation RB1 < RB2
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   392
  print_facts
27681
8cedebf55539 dropped locale (open)
haftmann
parents: 27618
diff changeset
   393
  using p apply unfold_locales apply fast done
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   394
interpretation RB3 < RB1
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   395
  print_facts
27681
8cedebf55539 dropped locale (open)
haftmann
parents: 27618
diff changeset
   396
  using r apply unfold_locales apply fast done
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   397
interpretation RB2 < RB3
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   398
  print_facts
27681
8cedebf55539 dropped locale (open)
haftmann
parents: 27618
diff changeset
   399
  using q apply unfold_locales apply fast done
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   400
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   401
lemma (in RB1) True
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   402
  print_facts
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   403
  ..
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   404
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   405
27718
3a85bc6bfd73 Updated locale tests.
ballarin
parents: 27681
diff changeset
   406
(* Group example *)
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   407
27718
3a85bc6bfd73 Updated locale tests.
ballarin
parents: 27681
diff changeset
   408
locale Rsemi = var prod (infixl "**" 65) +
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   409
  assumes assoc: "(x ** y) ** z = x ** (y ** z)"
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   410
27718
3a85bc6bfd73 Updated locale tests.
ballarin
parents: 27681
diff changeset
   411
locale Rlgrp = Rsemi + var one + var inv +
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   412
  assumes lone: "one ** x = x"
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   413
    and linv: "inv(x) ** x = one"
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   414
27718
3a85bc6bfd73 Updated locale tests.
ballarin
parents: 27681
diff changeset
   415
lemma (in Rlgrp) lcancel:
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   416
  "x ** y = x ** z <-> y = z"
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   417
proof
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   418
  assume "x ** y = x ** z"
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   419
  then have "inv(x) ** x ** y = inv(x) ** x ** z" by (simp add: assoc)
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   420
  then show "y = z" by (simp add: lone linv)
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   421
qed simp
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   422
27718
3a85bc6bfd73 Updated locale tests.
ballarin
parents: 27681
diff changeset
   423
locale Rrgrp = Rsemi + var one + var inv +
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   424
  assumes rone: "x ** one = x"
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   425
    and rinv: "x ** inv(x) = one"
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   426
27718
3a85bc6bfd73 Updated locale tests.
ballarin
parents: 27681
diff changeset
   427
lemma (in Rrgrp) rcancel:
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   428
  "y ** x = z ** x <-> y = z"
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   429
proof
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   430
  assume "y ** x = z ** x"
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   431
  then have "y ** (x ** inv(x)) = z ** (x ** inv(x))"
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   432
    by (simp add: assoc [symmetric])
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   433
  then show "y = z" by (simp add: rone rinv)
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   434
qed simp
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   435
27718
3a85bc6bfd73 Updated locale tests.
ballarin
parents: 27681
diff changeset
   436
interpretation Rlgrp < Rrgrp
19984
29bb4659f80a Method intro_locales replaced by intro_locales and unfold_locales.
ballarin
parents: 19931
diff changeset
   437
  proof unfold_locales
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   438
    {
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   439
      fix x
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   440
      have "inv(x) ** x ** one = inv(x) ** x" by (simp add: linv lone)
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   441
      then show "x ** one = x" by (simp add: assoc lcancel)
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   442
    }
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   443
    note rone = this
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   444
    {
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   445
      fix x
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   446
      have "inv(x) ** x ** inv(x) = inv(x) ** one"
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   447
	by (simp add: linv lone rone)
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   448
      then show "x ** inv(x) = one" by (simp add: assoc lcancel)
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   449
    }
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   450
  qed
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   451
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   452
(* effect on printed locale *)
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   453
27718
3a85bc6bfd73 Updated locale tests.
ballarin
parents: 27681
diff changeset
   454
print_locale! Rlgrp
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   455
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   456
(* use of derived theorem *)
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   457
27718
3a85bc6bfd73 Updated locale tests.
ballarin
parents: 27681
diff changeset
   458
lemma (in Rlgrp)
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   459
  "y ** x = z ** x <-> y = z"
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   460
  apply (rule rcancel)
27718
3a85bc6bfd73 Updated locale tests.
ballarin
parents: 27681
diff changeset
   461
  print_interps Rrgrp thm lcancel rcancel
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   462
  done
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   463
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   464
(* circular interpretation *)
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   465
27718
3a85bc6bfd73 Updated locale tests.
ballarin
parents: 27681
diff changeset
   466
interpretation Rrgrp < Rlgrp
19984
29bb4659f80a Method intro_locales replaced by intro_locales and unfold_locales.
ballarin
parents: 19931
diff changeset
   467
  proof unfold_locales
17000
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   468
    {
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   469
      fix x
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   470
      have "one ** (x ** inv(x)) = x ** inv(x)" by (simp add: rinv rone)
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   471
      then show "one ** x = x" by (simp add: assoc [symmetric] rcancel)
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   472
    }
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   473
    note lone = this
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   474
    {
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   475
      fix x
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   476
      have "inv(x) ** (x ** inv(x)) = one ** inv(x)"
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   477
	by (simp add: rinv lone rone)
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   478
      then show "inv(x) ** x = one" by (simp add: assoc [symmetric] rcancel)
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   479
    }
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   480
  qed
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   481
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   482
(* effect on printed locale *)
552df70f52c2 First version of interpretation in locales. Not yet fully functional.
ballarin
parents: 16736
diff changeset
   483
27718
3a85bc6bfd73 Updated locale tests.
ballarin
parents: 27681
diff changeset
   484
print_locale! Rrgrp
3a85bc6bfd73 Updated locale tests.
ballarin
parents: 27681
diff changeset
   485
print_locale! Rlgrp
16736
1e792b32abef Preparations for interpretation of locales in locales.
ballarin
parents: 16620
diff changeset
   486
17033
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   487
subsection {* Interaction of Interpretation in Theories and Locales:
17096
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   488
  in Locale, then in Theory *}
17033
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   489
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   490
consts
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   491
  rone :: i
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   492
  rinv :: "i => i"
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   493
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   494
axioms
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   495
  r_one : "rone # x = x"
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   496
  r_inv : "rinv(x) # x = rone"
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   497
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   498
interpretation Rbool: Rlgrp ["op #" "rone" "rinv"]
27681
8cedebf55539 dropped locale (open)
haftmann
parents: 27618
diff changeset
   499
proof
17033
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   500
  fix x y z
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   501
  {
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   502
    show "(x # y) # z = x # (y # z)" by (rule i_assoc)
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   503
  next
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   504
    show "rone # x = x" by (rule r_one)
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   505
  next
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   506
    show "rinv(x) # x = rone" by (rule r_inv)
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   507
  }
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   508
qed
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   509
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   510
(* derived elements *)
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   511
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   512
print_interps Rrgrp
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   513
print_interps Rlgrp
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   514
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   515
lemma "y # x = z # x <-> y = z" by (rule Rbool.rcancel)
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   516
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   517
(* adding lemma to derived element *)
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   518
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   519
lemma (in Rrgrp) new_cancel:
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   520
  "b ** a = c ** a <-> b = c"
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   521
  by (rule rcancel)
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   522
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   523
thm Rbool.new_cancel (* additional prems discharged!! *)
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   524
17139
165c97f9bb63 Printing of interpretations: option to show witness theorems;
ballarin
parents: 17096
diff changeset
   525
ML {* check_thm "Rbool.new_cancel" *}
165c97f9bb63 Printing of interpretations: option to show witness theorems;
ballarin
parents: 17096
diff changeset
   526
17033
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   527
lemma "b # a = c # a <-> b = c" by (rule Rbool.new_cancel)
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   528
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   529
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   530
subsection {* Interaction of Interpretation in Theories and Locales:
17096
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   531
  in Theory, then in Locale *}
17033
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   532
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   533
(* Another copy of the group example *)
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   534
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   535
locale Rqsemi = var prod (infixl "**" 65) +
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   536
  assumes assoc: "(x ** y) ** z = x ** (y ** z)"
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   537
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   538
locale Rqlgrp = Rqsemi + var one + var inv +
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   539
  assumes lone: "one ** x = x"
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   540
    and linv: "inv(x) ** x = one"
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   541
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   542
lemma (in Rqlgrp) lcancel:
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   543
  "x ** y = x ** z <-> y = z"
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   544
proof
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   545
  assume "x ** y = x ** z"
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   546
  then have "inv(x) ** x ** y = inv(x) ** x ** z" by (simp add: assoc)
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   547
  then show "y = z" by (simp add: lone linv)
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   548
qed simp
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   549
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   550
locale Rqrgrp = Rqsemi + var one + var inv +
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   551
  assumes rone: "x ** one = x"
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   552
    and rinv: "x ** inv(x) = one"
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   553
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   554
lemma (in Rqrgrp) rcancel:
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   555
  "y ** x = z ** x <-> y = z"
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   556
proof
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   557
  assume "y ** x = z ** x"
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   558
  then have "y ** (x ** inv(x)) = z ** (x ** inv(x))"
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   559
    by (simp add: assoc [symmetric])
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   560
  then show "y = z" by (simp add: rone rinv)
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   561
qed simp
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   562
27718
3a85bc6bfd73 Updated locale tests.
ballarin
parents: 27681
diff changeset
   563
interpretation Rqrgrp < Rrgrp
19984
29bb4659f80a Method intro_locales replaced by intro_locales and unfold_locales.
ballarin
parents: 19931
diff changeset
   564
  apply unfold_locales
19931
fb32b43e7f80 Restructured locales with predicates: import is now an interpretation.
ballarin
parents: 19783
diff changeset
   565
  apply (rule assoc)
fb32b43e7f80 Restructured locales with predicates: import is now an interpretation.
ballarin
parents: 19783
diff changeset
   566
  apply (rule rone)
fb32b43e7f80 Restructured locales with predicates: import is now an interpretation.
ballarin
parents: 19783
diff changeset
   567
  apply (rule rinv)
fb32b43e7f80 Restructured locales with predicates: import is now an interpretation.
ballarin
parents: 19783
diff changeset
   568
  done
17139
165c97f9bb63 Printing of interpretations: option to show witness theorems;
ballarin
parents: 17096
diff changeset
   569
17033
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   570
interpretation R2: Rqlgrp ["op #" "rone" "rinv"] 
19984
29bb4659f80a Method intro_locales replaced by intro_locales and unfold_locales.
ballarin
parents: 19931
diff changeset
   571
  apply unfold_locales  (* FIXME: unfold_locales is too eager and shouldn't
19931
fb32b43e7f80 Restructured locales with predicates: import is now an interpretation.
ballarin
parents: 19783
diff changeset
   572
                          solve this. *)
27681
8cedebf55539 dropped locale (open)
haftmann
parents: 27618
diff changeset
   573
  apply (rule i_assoc)
8cedebf55539 dropped locale (open)
haftmann
parents: 27618
diff changeset
   574
  apply (rule r_one)
8cedebf55539 dropped locale (open)
haftmann
parents: 27618
diff changeset
   575
  apply (rule r_inv)
19931
fb32b43e7f80 Restructured locales with predicates: import is now an interpretation.
ballarin
parents: 19783
diff changeset
   576
  done
17033
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   577
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   578
print_interps Rqsemi
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   579
print_interps Rqlgrp
27718
3a85bc6bfd73 Updated locale tests.
ballarin
parents: 27681
diff changeset
   580
print_interps Rlgrp  (* no interpretations yet *)
17139
165c97f9bb63 Printing of interpretations: option to show witness theorems;
ballarin
parents: 17096
diff changeset
   581
17033
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   582
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   583
interpretation Rqlgrp < Rqrgrp
19984
29bb4659f80a Method intro_locales replaced by intro_locales and unfold_locales.
ballarin
parents: 19931
diff changeset
   584
  proof unfold_locales
17033
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   585
    {
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   586
      fix x
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   587
      have "inv(x) ** x ** one = inv(x) ** x" by (simp add: linv lone)
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   588
      then show "x ** one = x" by (simp add: assoc lcancel)
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   589
    }
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   590
    note rone = this
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   591
    {
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   592
      fix x
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   593
      have "inv(x) ** x ** inv(x) = inv(x) ** one"
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   594
	by (simp add: linv lone rone)
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   595
      then show "x ** inv(x) = one" by (simp add: assoc lcancel)
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   596
    }
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   597
  qed
f4c1ce91aa3c Release of interpretation in locale.
ballarin
parents: 17000
diff changeset
   598
17139
165c97f9bb63 Printing of interpretations: option to show witness theorems;
ballarin
parents: 17096
diff changeset
   599
print_interps! Rqrgrp
27718
3a85bc6bfd73 Updated locale tests.
ballarin
parents: 27681
diff changeset
   600
print_interps! Rsemi  (* witness must not have meta hyps *)
3a85bc6bfd73 Updated locale tests.
ballarin
parents: 27681
diff changeset
   601
print_interps! Rrgrp  (* witness must not have meta hyps *)
3a85bc6bfd73 Updated locale tests.
ballarin
parents: 27681
diff changeset
   602
print_interps! Rlgrp  (* witness must not have meta hyps *)
17139
165c97f9bb63 Printing of interpretations: option to show witness theorems;
ballarin
parents: 17096
diff changeset
   603
thm R2.rcancel
165c97f9bb63 Printing of interpretations: option to show witness theorems;
ballarin
parents: 17096
diff changeset
   604
thm R2.lcancel
165c97f9bb63 Printing of interpretations: option to show witness theorems;
ballarin
parents: 17096
diff changeset
   605
165c97f9bb63 Printing of interpretations: option to show witness theorems;
ballarin
parents: 17096
diff changeset
   606
ML {* check_thm "R2.rcancel"; check_thm "R2.lcancel" *}
165c97f9bb63 Printing of interpretations: option to show witness theorems;
ballarin
parents: 17096
diff changeset
   607
17096
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   608
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   609
subsection {* Generation of Witness Theorems for Transitive Interpretations *}
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   610
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   611
locale Rtriv = var x +
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   612
  assumes x: "x = x"
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   613
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   614
locale Rtriv2 = var x + var y +
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   615
  assumes x: "x = x" and y: "y = y"
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   616
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   617
interpretation Rtriv2 < Rtriv x
19984
29bb4659f80a Method intro_locales replaced by intro_locales and unfold_locales.
ballarin
parents: 19931
diff changeset
   618
  apply unfold_locales
17096
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   619
  apply (rule x)
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   620
  done
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   621
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   622
interpretation Rtriv2 < Rtriv y
19984
29bb4659f80a Method intro_locales replaced by intro_locales and unfold_locales.
ballarin
parents: 19931
diff changeset
   623
  apply unfold_locales
17096
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   624
  apply (rule y)
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   625
  done
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   626
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   627
print_locale Rtriv2
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   628
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   629
locale Rtriv3 = var x + var y + var z +
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   630
  assumes x: "x = x" and y: "y = y" and z: "z = z"
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   631
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   632
interpretation Rtriv3 < Rtriv2 x y
19984
29bb4659f80a Method intro_locales replaced by intro_locales and unfold_locales.
ballarin
parents: 19931
diff changeset
   633
  apply unfold_locales
17096
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   634
  apply (rule x)
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   635
  apply (rule y)
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   636
  done
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   637
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   638
print_locale Rtriv3
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   639
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   640
interpretation Rtriv3 < Rtriv2 x z
19984
29bb4659f80a Method intro_locales replaced by intro_locales and unfold_locales.
ballarin
parents: 19931
diff changeset
   641
  apply unfold_locales
17096
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   642
  apply (rule x_y_z.x)
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   643
  apply (rule z)
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   644
  done
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   645
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   646
ML {* set show_types *}
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   647
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   648
print_locale Rtriv3
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   649
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   650
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   651
subsection {* Normalisation Replaces Assumed Element by Derived Element *}
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   652
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   653
typedecl ('a, 'b) pair
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   654
arities pair :: ("term", "term") "term"
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   655
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   656
consts
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   657
  pair :: "['a, 'b] => ('a, 'b) pair"
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   658
  fst :: "('a, 'b) pair => 'a"
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   659
  snd :: "('a, 'b) pair => 'b"
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   660
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   661
axioms
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   662
  fst [simp]: "fst(pair(x, y)) = x"
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   663
  snd [simp]: "snd(pair(x, y)) = y"
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   664
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   665
locale Rpair = var prod (infixl "**" 65) + var prodP (infixl "***" 65) +
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   666
  defines P_def: "x *** y == pair(fst(x) ** fst(y), snd(x) ** snd(y))"
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   667
27718
3a85bc6bfd73 Updated locale tests.
ballarin
parents: 27681
diff changeset
   668
locale Rpair_semi = Rpair + Rsemi
17096
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   669
27718
3a85bc6bfd73 Updated locale tests.
ballarin
parents: 27681
diff changeset
   670
interpretation Rpair_semi < Rsemi prodP (infixl "***" 65)
3a85bc6bfd73 Updated locale tests.
ballarin
parents: 27681
diff changeset
   671
proof unfold_locales
17096
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   672
  fix x y z
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   673
  show "(x *** y) *** z = x *** (y *** z)"
19931
fb32b43e7f80 Restructured locales with predicates: import is now an interpretation.
ballarin
parents: 19783
diff changeset
   674
    apply (simp only: P_def) apply (simp add: assoc) (* FIXME: unfold P_def fails *)
fb32b43e7f80 Restructured locales with predicates: import is now an interpretation.
ballarin
parents: 19783
diff changeset
   675
    done
17096
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   676
qed
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   677
27718
3a85bc6bfd73 Updated locale tests.
ballarin
parents: 27681
diff changeset
   678
locale Rsemi_rev = Rsemi + var rprod (infixl "++" 65) +
17096
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   679
  defines r_def: "x ++ y == y ** x"
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   680
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   681
lemma (in Rsemi_rev) r_assoc:
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   682
  "(x ++ y) ++ z = x ++ (y ++ z)"
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   683
  by (simp add: r_def assoc)
8327b71282ce Improved generation of witnesses in interpretation.
ballarin
parents: 17033
diff changeset
   684
20469
bb75c1cdf913 More locale test code.
ballarin
parents: 20034
diff changeset
   685
bb75c1cdf913 More locale test code.
ballarin
parents: 20034
diff changeset
   686
subsection {* Import of Locales with Predicates as Interpretation *}
bb75c1cdf913 More locale test code.
ballarin
parents: 20034
diff changeset
   687
bb75c1cdf913 More locale test code.
ballarin
parents: 20034
diff changeset
   688
locale Ra =
bb75c1cdf913 More locale test code.
ballarin
parents: 20034
diff changeset
   689
  assumes Ra: "True"
bb75c1cdf913 More locale test code.
ballarin
parents: 20034
diff changeset
   690
bb75c1cdf913 More locale test code.
ballarin
parents: 20034
diff changeset
   691
locale Rb = Ra +
bb75c1cdf913 More locale test code.
ballarin
parents: 20034
diff changeset
   692
  assumes Rb: "True"
bb75c1cdf913 More locale test code.
ballarin
parents: 20034
diff changeset
   693
bb75c1cdf913 More locale test code.
ballarin
parents: 20034
diff changeset
   694
locale Rc = Rb +
bb75c1cdf913 More locale test code.
ballarin
parents: 20034
diff changeset
   695
  assumes Rc: "True"
bb75c1cdf913 More locale test code.
ballarin
parents: 20034
diff changeset
   696
bb75c1cdf913 More locale test code.
ballarin
parents: 20034
diff changeset
   697
print_locale! Rc
bb75c1cdf913 More locale test code.
ballarin
parents: 20034
diff changeset
   698
22659
f792579b6e59 Experimental code for the interpretation of definitions.
ballarin
parents: 20469
diff changeset
   699
f792579b6e59 Experimental code for the interpretation of definitions.
ballarin
parents: 20469
diff changeset
   700
section {* Interpretation of Defined Concepts *}
f792579b6e59 Experimental code for the interpretation of definitions.
ballarin
parents: 20469
diff changeset
   701
f792579b6e59 Experimental code for the interpretation of definitions.
ballarin
parents: 20469
diff changeset
   702
text {* Naming convention for global objects: prefixes D and d *}
f792579b6e59 Experimental code for the interpretation of definitions.
ballarin
parents: 20469
diff changeset
   703
23919
af871d13e320 interpretation: equations are propositions not pairs of terms;
ballarin
parents: 22931
diff changeset
   704
af871d13e320 interpretation: equations are propositions not pairs of terms;
ballarin
parents: 22931
diff changeset
   705
subsection {* Simple examples *}
af871d13e320 interpretation: equations are propositions not pairs of terms;
ballarin
parents: 22931
diff changeset
   706
22659
f792579b6e59 Experimental code for the interpretation of definitions.
ballarin
parents: 20469
diff changeset
   707
locale Da = fixes a :: o
f792579b6e59 Experimental code for the interpretation of definitions.
ballarin
parents: 20469
diff changeset
   708
  assumes true: a
f792579b6e59 Experimental code for the interpretation of definitions.
ballarin
parents: 20469
diff changeset
   709
22757
d3298d63b7b6 Interpretation equations applied to attributes
ballarin
parents: 22659
diff changeset
   710
text {* In the following examples, @{term "~ a"} is the defined concept. *}
d3298d63b7b6 Interpretation equations applied to attributes
ballarin
parents: 22659
diff changeset
   711
22659
f792579b6e59 Experimental code for the interpretation of definitions.
ballarin
parents: 20469
diff changeset
   712
lemma (in Da) not_false: "~ a <-> False"
f792579b6e59 Experimental code for the interpretation of definitions.
ballarin
parents: 20469
diff changeset
   713
  apply simp apply (rule true) done
f792579b6e59 Experimental code for the interpretation of definitions.
ballarin
parents: 20469
diff changeset
   714
f792579b6e59 Experimental code for the interpretation of definitions.
ballarin
parents: 20469
diff changeset
   715
interpretation D1: Da ["True"]
23919
af871d13e320 interpretation: equations are propositions not pairs of terms;
ballarin
parents: 22931
diff changeset
   716
  where "~ True == False"
22659
f792579b6e59 Experimental code for the interpretation of definitions.
ballarin
parents: 20469
diff changeset
   717
  apply -
f792579b6e59 Experimental code for the interpretation of definitions.
ballarin
parents: 20469
diff changeset
   718
  apply unfold_locales [1] apply rule
f792579b6e59 Experimental code for the interpretation of definitions.
ballarin
parents: 20469
diff changeset
   719
  by simp
f792579b6e59 Experimental code for the interpretation of definitions.
ballarin
parents: 20469
diff changeset
   720
f792579b6e59 Experimental code for the interpretation of definitions.
ballarin
parents: 20469
diff changeset
   721
thm D1.not_false
f792579b6e59 Experimental code for the interpretation of definitions.
ballarin
parents: 20469
diff changeset
   722
lemma "False <-> False" apply (rule D1.not_false) done
f792579b6e59 Experimental code for the interpretation of definitions.
ballarin
parents: 20469
diff changeset
   723
f792579b6e59 Experimental code for the interpretation of definitions.
ballarin
parents: 20469
diff changeset
   724
interpretation D2: Da ["x | ~ x"]
23919
af871d13e320 interpretation: equations are propositions not pairs of terms;
ballarin
parents: 22931
diff changeset
   725
  where "~ (x | ~ x) <-> ~ x & x"
22659
f792579b6e59 Experimental code for the interpretation of definitions.
ballarin
parents: 20469
diff changeset
   726
  apply -
f792579b6e59 Experimental code for the interpretation of definitions.
ballarin
parents: 20469
diff changeset
   727
  apply unfold_locales [1] apply fast
f792579b6e59 Experimental code for the interpretation of definitions.
ballarin
parents: 20469
diff changeset
   728
  by simp
f792579b6e59 Experimental code for the interpretation of definitions.
ballarin
parents: 20469
diff changeset
   729
f792579b6e59 Experimental code for the interpretation of definitions.
ballarin
parents: 20469
diff changeset
   730
thm D2.not_false
f792579b6e59 Experimental code for the interpretation of definitions.
ballarin
parents: 20469
diff changeset
   731
lemma "~ x & x <-> False" apply (rule D2.not_false) done
f792579b6e59 Experimental code for the interpretation of definitions.
ballarin
parents: 20469
diff changeset
   732
f792579b6e59 Experimental code for the interpretation of definitions.
ballarin
parents: 20469
diff changeset
   733
print_interps! Da
f792579b6e59 Experimental code for the interpretation of definitions.
ballarin
parents: 20469
diff changeset
   734
f792579b6e59 Experimental code for the interpretation of definitions.
ballarin
parents: 20469
diff changeset
   735
(* Subscriptions of interpretations *)
f792579b6e59 Experimental code for the interpretation of definitions.
ballarin
parents: 20469
diff changeset
   736
f792579b6e59 Experimental code for the interpretation of definitions.
ballarin
parents: 20469
diff changeset
   737
lemma (in Da) not_false2: "~a <-> False"
f792579b6e59 Experimental code for the interpretation of definitions.
ballarin
parents: 20469
diff changeset
   738
  apply simp apply (rule true) done
f792579b6e59 Experimental code for the interpretation of definitions.
ballarin
parents: 20469
diff changeset
   739
f792579b6e59 Experimental code for the interpretation of definitions.
ballarin
parents: 20469
diff changeset
   740
thm D1.not_false2 D2.not_false2
f792579b6e59 Experimental code for the interpretation of definitions.
ballarin
parents: 20469
diff changeset
   741
lemma "False <-> False" apply (rule D1.not_false2) done
f792579b6e59 Experimental code for the interpretation of definitions.
ballarin
parents: 20469
diff changeset
   742
lemma "~x & x <-> False" apply (rule D2.not_false2) done
f792579b6e59 Experimental code for the interpretation of definitions.
ballarin
parents: 20469
diff changeset
   743
22757
d3298d63b7b6 Interpretation equations applied to attributes
ballarin
parents: 22659
diff changeset
   744
(* Unfolding in attributes *)
d3298d63b7b6 Interpretation equations applied to attributes
ballarin
parents: 22659
diff changeset
   745
d3298d63b7b6 Interpretation equations applied to attributes
ballarin
parents: 22659
diff changeset
   746
locale Db = Da +
d3298d63b7b6 Interpretation equations applied to attributes
ballarin
parents: 22659
diff changeset
   747
  fixes b :: o
d3298d63b7b6 Interpretation equations applied to attributes
ballarin
parents: 22659
diff changeset
   748
  assumes a_iff_b: "~a <-> b"
d3298d63b7b6 Interpretation equations applied to attributes
ballarin
parents: 22659
diff changeset
   749
d3298d63b7b6 Interpretation equations applied to attributes
ballarin
parents: 22659
diff changeset
   750
lemmas (in Db) not_false_b = not_false [unfolded a_iff_b]
d3298d63b7b6 Interpretation equations applied to attributes
ballarin
parents: 22659
diff changeset
   751
d3298d63b7b6 Interpretation equations applied to attributes
ballarin
parents: 22659
diff changeset
   752
interpretation D2: Db ["x | ~ x" "~ (x <-> x)"]
d3298d63b7b6 Interpretation equations applied to attributes
ballarin
parents: 22659
diff changeset
   753
  apply unfold_locales apply fast done
d3298d63b7b6 Interpretation equations applied to attributes
ballarin
parents: 22659
diff changeset
   754
d3298d63b7b6 Interpretation equations applied to attributes
ballarin
parents: 22659
diff changeset
   755
thm D2.not_false_b
d3298d63b7b6 Interpretation equations applied to attributes
ballarin
parents: 22659
diff changeset
   756
lemma "~(x <-> x) <-> False" apply (rule D2.not_false_b) done
d3298d63b7b6 Interpretation equations applied to attributes
ballarin
parents: 22659
diff changeset
   757
d3298d63b7b6 Interpretation equations applied to attributes
ballarin
parents: 22659
diff changeset
   758
(* Subscription and attributes *)
d3298d63b7b6 Interpretation equations applied to attributes
ballarin
parents: 22659
diff changeset
   759
d3298d63b7b6 Interpretation equations applied to attributes
ballarin
parents: 22659
diff changeset
   760
lemmas (in Db) not_false_b2 = not_false [unfolded a_iff_b]
d3298d63b7b6 Interpretation equations applied to attributes
ballarin
parents: 22659
diff changeset
   761
d3298d63b7b6 Interpretation equations applied to attributes
ballarin
parents: 22659
diff changeset
   762
thm D2.not_false_b2
d3298d63b7b6 Interpretation equations applied to attributes
ballarin
parents: 22659
diff changeset
   763
lemma "~(x <-> x) <-> False" apply (rule D2.not_false_b2) done
d3298d63b7b6 Interpretation equations applied to attributes
ballarin
parents: 22659
diff changeset
   764
15596
8665d08085df First version of global registration command.
ballarin
parents:
diff changeset
   765
end