.hgtags
author Timothy Bourke
Mon, 09 Feb 2009 17:25:07 +1100
changeset 29848 a7c164e228e1
parent 28933 6c9d81544b26
child 30877 27cf197214c8
permissions -rw-r--r--
Nicer names in FindTheorems. * Patch NameSpace.get_accesses, contributed by Timothy Bourke: NameSpace.get_accesses has been patched to fix the following bug: theory OverHOL imports Main begin lemma conjI: "a & b --> b" by blast ML {* val ns = PureThy.facts_of @{theory} |> Facts.space_of; val x1 = NameSpace.get_accesses ns "HOL.conjI"; val x2 = NameSpace.get_accesses ns "OverHOL.conjI"; *} end where x1 = ["conjI", "HOL.conjI"] and x2 = ["conjI", "OverHOL.conjI"], but x1 should be just ["HOL.conjI"]. NameSpace.get_accesses is only used within the NameSpace structure itself. The two uses have been modified to retain their original behaviour. Note that NameSpace.valid_accesses gives different results: get_accesses ns "HOL.eq_class.eq" gives ["eq", "eq_class.eq", "HOL.eq_class.eq"] but, valid_accesses ns "HOL.eq_class.eq" gives ["HOL.eq_class.eq", "eq_class.eq", "HOL.eq", "eq"] * Patch FindTheorems: Prefer names that are shorter to type in the current context. * Re-export space_of.
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
28119
bdf7d5f4d5b0 update tags
convert-repo
parents:
diff changeset
     1
0140ff702b232f48cb4c7414dca663e41acad213 Isabelle94-3
bdf7d5f4d5b0 update tags
convert-repo
parents:
diff changeset
     2
0a604b2fc2b1df524a3cf81f5a7b2255b19fda92 Isabelle99
bdf7d5f4d5b0 update tags
convert-repo
parents:
diff changeset
     3
0b268cff9344268b18ab5241b5c45e3374f107cd Isabelle94-8
bdf7d5f4d5b0 update tags
convert-repo
parents:
diff changeset
     4
213dcc39358faefae737f8e7d2eea67658e9eedf Isabelle2003
bdf7d5f4d5b0 update tags
convert-repo
parents:
diff changeset
     5
23ceb1dc9755a8ad6f0230697d0cc52f54102bf4 Isabelle94-5
bdf7d5f4d5b0 update tags
convert-repo
parents:
diff changeset
     6
2cf13a72e1704d0094d21e7dc68e7271a282ed31 Isabelle2008
bdf7d5f4d5b0 update tags
convert-repo
parents:
diff changeset
     7
33b9b5da3e6faee6ca6969d17e79634d49e5b46a Isabelle94-1
bdf7d5f4d5b0 update tags
convert-repo
parents:
diff changeset
     8
35fba71ec6ef550178e5f5e44d95d96c6f36eae6 nominal_01
bdf7d5f4d5b0 update tags
convert-repo
parents:
diff changeset
     9
3e47692e3a3e4c695f6345b3534ed0c36817fd40 Isabelle99-2
bdf7d5f4d5b0 update tags
convert-repo
parents:
diff changeset
    10
50be659d4222b68f95e9c966097e59091f26acf3 Isabelle99-1
bdf7d5f4d5b0 update tags
convert-repo
parents:
diff changeset
    11
67692db44c7099ad8789f088003213aeb095e914 Isabelle94-2
bdf7d5f4d5b0 update tags
convert-repo
parents:
diff changeset
    12
6a422b22ba02f6275fa3ac5f9df1428705552d50 Isabelle98-1
bdf7d5f4d5b0 update tags
convert-repo
parents:
diff changeset
    13
6f79698f294df13edfba9c790df18a545570c81e Isabelle2007
bdf7d5f4d5b0 update tags
convert-repo
parents:
diff changeset
    14
7d6b0241afabbf87d4d94a412a1c1ebbba71c088 Isabelle94-4
bdf7d5f4d5b0 update tags
convert-repo
parents:
diff changeset
    15
805fa01ac2337790fd555991f1231d3ef6b2e3fb Isabelle2004_0
bdf7d5f4d5b0 update tags
convert-repo
parents:
diff changeset
    16
831a9a7ab9f352c65b0f449630b428304c89362b Isabelle93
bdf7d5f4d5b0 update tags
convert-repo
parents:
diff changeset
    17
836950047d8508e3c200edc1e07a46c2c5e09cd7 Isabelle94-6
bdf7d5f4d5b0 update tags
convert-repo
parents:
diff changeset
    18
8d42a7bccf0b0880dff8e46c71c4811be8b2e7ec Isabelle94-7
bdf7d5f4d5b0 update tags
convert-repo
parents:
diff changeset
    19
a23af144eb47f12354dff090813c796f278e2eb8 nominal_03
bdf7d5f4d5b0 update tags
convert-repo
parents:
diff changeset
    20
be6b5edbca9ffeb3bace5f4bac5c6478bf8cbdb2 Isabelle98
bdf7d5f4d5b0 update tags
convert-repo
parents:
diff changeset
    21
cd41a57221d07441647284e239b8d8d77d498ef5 isa94
bdf7d5f4d5b0 update tags
convert-repo
parents:
diff changeset
    22
ce180e5b7fa056003791fff19cc5cefba193b135 Isabelle2002
bdf7d5f4d5b0 update tags
convert-repo
parents:
diff changeset
    23
dde117622dace696123b023d1f06cf8d8ef9eb46 nominal_02
bdf7d5f4d5b0 update tags
convert-repo
parents:
diff changeset
    24
f9eb0f819642b2ad77119dbf8935bf13248f205d Isabelle94
bdf7d5f4d5b0 update tags
convert-repo
parents:
diff changeset
    25
fc385ce6187d5ad2cef90f1e6240cc691e02d827 Isabelle2005