src/FOL/ex/LocaleTest.thy
changeset 15624 484178635bd8
parent 15598 4ab52355bb53
child 15696 1da4ce092c0b
--- a/src/FOL/ex/LocaleTest.thy	Thu Mar 24 16:36:40 2005 +0100
+++ b/src/FOL/ex/LocaleTest.thy	Thu Mar 24 17:03:37 2005 +0100
@@ -20,7 +20,7 @@
 print_interps L
 print_interps M
 
-interpretation test [simp]: L .
+interpretation test [simp]: L print_interps M .
 
 interpretation L .
 
@@ -52,8 +52,19 @@
 
 print_interps A
 
-(*
-thm asm_A a.asm_A p1.a.asm_A
+(* possible accesses
+thm p1.a.asm_A thm LocaleTest.p1.a.asm_A
+thm LocaleTest.asm_A thm p1.asm_A
+*)
+
+(* without prefix *)
+
+interpretation C ["W::'b" "Z::'b"] by (auto intro: A.intro C_axioms.intro)
+
+print_interps A
+
+(* possible accesses
+thm a.asm_A thm asm_A thm LocaleTest.a.asm_A thm LocaleTest.asm_A
 *)
 
 interpretation p2: D [X Y "Y = X"] by (auto intro: A.intro simp: eq_commute)
@@ -64,7 +75,7 @@
 thm p2.a.asm_A
 *)
 
-interpretation p3: D [X Y] by (auto intro: A.intro)
+interpretation p3: D [X Y] .
 
 (* duplicate: not registered *)
 (*
@@ -87,4 +98,18 @@
 interpretation A [Z] apply - apply (auto intro: A.intro) done
 *)
 
+theorem True
+proof -
+  fix alpha::i and beta::i and gamma::i
+  assume "A(alpha)"
+  then interpret p5: A [alpha] .
+  print_interps A
+  interpret p6: C [alpha beta] by (auto intro: C_axioms.intro)
+  print_interps A   (* p6 not added! *)
+  print_interps C
+qed rule
+
+(* lemma "bla.bla": True by rule *)
+
+
 end