Timothy Bourke [Mon, 09 Feb 2009 17:25:07 +1100] rev 29848
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.
chaieb [Mon, 09 Feb 2009 17:21:46 +0000] rev 29847
added Determinants to Library
chaieb [Mon, 09 Feb 2009 17:21:19 +0000] rev 29846
Traces, Determinant of square matrices and some properties
chaieb [Mon, 09 Feb 2009 17:09:18 +0000] rev 29845
added Euclidean_Space and Glbs to Library
chaieb [Mon, 09 Feb 2009 17:08:49 +0000] rev 29844
fixed proof -- removed unnecessary sorry
chaieb [Mon, 09 Feb 2009 16:57:10 +0000] rev 29843
Fixed theorem reference
chaieb [Mon, 09 Feb 2009 16:54:03 +0000] rev 29842
(Real) Vectors in Euclidean space, and elementary linear algebra.
chaieb [Mon, 09 Feb 2009 16:43:52 +0000] rev 29841
A generic decision procedure for linear rea arithmetic and normed vector spaces
chaieb [Mon, 09 Feb 2009 16:42:15 +0000] rev 29840
Permutations, both general and specifically on finite sets.
chaieb [Mon, 09 Feb 2009 16:20:24 +0000] rev 29839
Imports Main in order to avoid the typerep problem
chaieb [Mon, 09 Feb 2009 16:19:46 +0000] rev 29838
A theory of greatest lower bounds
chaieb [Mon, 09 Feb 2009 15:38:26 +0000] rev 29837
Now imports Fact as suggested by Florian in order to avoid the typerep problem
chaieb [Mon, 09 Feb 2009 11:15:13 +0000] rev 29836
Added HOL/Library/Finite_Cartesian_Product.thy to Library
chaieb [Mon, 09 Feb 2009 11:07:17 +0000] rev 29835
A formalization of finite cartesian product types
hoelzl [Mon, 09 Feb 2009 11:19:44 +0100] rev 29834
Proof method 'reify' is now reentrant.
nipkow [Sun, 08 Feb 2009 11:59:26 +0100] rev 29833
added noatps
haftmann [Sat, 07 Feb 2009 10:56:44 +0100] rev 29832
check for destination directory, do not allocate it gratuitously
haftmann [Sat, 07 Feb 2009 10:03:09 +0100] rev 29831
Isar proof
haftmann [Sat, 07 Feb 2009 09:58:24 +0100] rev 29830
merged
haftmann [Sat, 07 Feb 2009 09:57:07 +0100] rev 29829
code theorems for nth, list_update
haftmann [Sat, 07 Feb 2009 09:57:03 +0100] rev 29828
added bulkload
haftmann [Sat, 07 Feb 2009 08:37:43 +0100] rev 29827
code theorems for nth, list_update
haftmann [Sat, 07 Feb 2009 08:37:42 +0100] rev 29826
added bulkload
haftmann [Sat, 07 Feb 2009 09:25:59 +0100] rev 29825
added Decision_Procs.thy
haftmann [Fri, 06 Feb 2009 15:15:46 +0100] rev 29824
merged
haftmann [Fri, 06 Feb 2009 15:15:32 +0100] rev 29823
session Reflecion renamed to Decision_Procs, moved Dense_Linear_Order there
haftmann [Fri, 06 Feb 2009 15:15:27 +0100] rev 29822
authentic syntax for List.nth
berghofe [Fri, 06 Feb 2009 14:36:58 +0100] rev 29821
Merged.
blanchet [Fri, 06 Feb 2009 13:43:19 +0100] rev 29820
Rearrange Refute/SAT theory dependencies so as to use even more antiquotations in refute.ML +
find/fix Product_Type.{fst,snd}, which are now called simply fst and snd.
chaieb [Fri, 06 Feb 2009 08:23:15 +0000] rev 29819
Automated merge with ssh://chaieb@atbroy100.informatik.tu-muenchen.de//home/isabelle-repository/repos/isabelle
chaieb [Fri, 06 Feb 2009 08:22:32 +0000] rev 29818
fixed import
haftmann [Fri, 06 Feb 2009 09:06:17 +0100] rev 29817
merged
haftmann [Fri, 06 Feb 2009 09:05:20 +0100] rev 29816
more robust failure in error situations
haftmann [Fri, 06 Feb 2009 09:05:19 +0100] rev 29815
mandatory prefix for index conversion operations
haftmann [Fri, 06 Feb 2009 09:05:19 +0100] rev 29814
added replace operation
chaieb [Fri, 06 Feb 2009 00:13:15 +0000] rev 29813
fixed dependencies : Theory Dense_Linear_Order moved to Library
chaieb@chaieb-laptop [Fri, 06 Feb 2009 00:10:58 +0000] rev 29812
Theory Dense_Linear_Order moved to Library
chaieb@chaieb-laptop [Fri, 06 Feb 2009 00:10:58 +0000] rev 29811
fixed Proofs and dependencies ; Theory Dense_Linear_Order moved to Library
hoelzl [Thu, 05 Feb 2009 15:35:06 +0100] rev 29810
Updated NEWS about approximation
haftmann [Thu, 05 Feb 2009 14:50:43 +0100] rev 29809
merged
haftmann [Thu, 05 Feb 2009 14:14:03 +0100] rev 29808
split of already properly working part of Quickcheck infrastructure
haftmann [Thu, 05 Feb 2009 14:14:03 +0100] rev 29807
code attribute applied before user attributes
haftmann [Thu, 05 Feb 2009 14:14:02 +0100] rev 29806
moved Random.thy to Library
hoelzl [Thu, 05 Feb 2009 11:49:15 +0100] rev 29805
Add approximation method
hoelzl [Thu, 05 Feb 2009 11:45:15 +0100] rev 29804
Added new Float theory and moved old Library/Float.thy to ComputeFloat
hoelzl [Thu, 05 Feb 2009 11:34:42 +0100] rev 29803
Added derivation lemmas for power series and theorems for the pi, arcus tangens and logarithm series
blanchet [Wed, 04 Feb 2009 18:10:07 +0100] rev 29802
Make some Refute functions public so I can use them in Nitpick,
use @{const_name} antiquotation whenever possible (some, like Lfp.lfp
had been renamed since Tjark wrote Refute), and removed some "set"-related
code that is no longer relevant in Isabelle2008. There's still some "set"
code that needs to be ported; see TODO in the file.
chaieb [Wed, 04 Feb 2009 11:32:35 +0000] rev 29801
merged
chaieb [Wed, 04 Feb 2009 11:31:05 +0000] rev 29800
Now catch ERROR exception thrown by find and friends
haftmann [Wed, 04 Feb 2009 10:59:32 +0100] rev 29799
dropped Id
haftmann [Wed, 04 Feb 2009 10:59:31 +0100] rev 29798
proper datatype abstraction example
haftmann [Tue, 03 Feb 2009 21:26:21 +0100] rev 29797
handling type classes without parameters
haftmann [Tue, 03 Feb 2009 19:48:06 +0100] rev 29796
adjusted theory name
haftmann [Tue, 03 Feb 2009 19:37:30 +0100] rev 29795
merged
haftmann [Tue, 03 Feb 2009 19:37:16 +0100] rev 29794
added stub about datatype abstraction
haftmann [Tue, 03 Feb 2009 19:37:00 +0100] rev 29793
changed name space policy for Haskell includes
haftmann [Tue, 03 Feb 2009 18:34:49 +0100] rev 29792
merged Big0
haftmann [Tue, 03 Feb 2009 18:25:31 +0100] rev 29791
added ROOT.ML for Reflection session
haftmann [Tue, 03 Feb 2009 16:54:31 +0100] rev 29790
merged
haftmann [Tue, 03 Feb 2009 16:54:10 +0100] rev 29789
established session HOL-Reflection
haftmann [Tue, 03 Feb 2009 16:50:41 +0100] rev 29788
established session HOL-Reflection
haftmann [Tue, 03 Feb 2009 16:50:40 +0100] rev 29787
regenerated presburger code
haftmann [Tue, 03 Feb 2009 16:50:40 +0100] rev 29786
merged Big0
nipkow [Tue, 03 Feb 2009 16:52:01 +0100] rev 29785
merge
immler@in.tum.de [Tue, 03 Feb 2009 15:29:52 +0100] rev 29784
changed default timeout
haftmann [Tue, 03 Feb 2009 16:40:10 +0100] rev 29783
merged
haftmann [Tue, 03 Feb 2009 16:39:52 +0100] rev 29782
dropped global Nil/Append interpretation
krauss [Tue, 03 Feb 2009 11:16:28 +0100] rev 29781
small fixes; removed Id
krauss [Tue, 03 Feb 2009 11:16:28 +0100] rev 29780
mergesort example: recdef->fun, localized
krauss [Tue, 03 Feb 2009 11:16:28 +0100] rev 29779
declare "nat o abs" as default measure for int
haftmann [Tue, 03 Feb 2009 07:44:10 +0100] rev 29778
repaired accidental commit
wenzelm [Sun, 22 Feb 2009 20:37:18 +0100] rev 29777
result for Swing.now;
wenzelm [Sat, 21 Feb 2009 18:06:17 +0100] rev 29776
replaced \overline by \vec;
wenzelm [Sat, 21 Feb 2009 18:05:34 +0100] rev 29775
updated generated files;
wenzelm [Sat, 21 Feb 2009 18:05:12 +0100] rev 29774
tuned;
wenzelm [Fri, 20 Feb 2009 21:01:52 +0100] rev 29773
updated generated files;
wenzelm [Fri, 20 Feb 2009 21:01:19 +0100] rev 29772
removed junk;
wenzelm [Fri, 20 Feb 2009 21:00:28 +0100] rev 29771
improved section "Rule composition";
tuned;
wenzelm [Fri, 20 Feb 2009 19:07:31 +0100] rev 29770
tuned;
wenzelm [Fri, 20 Feb 2009 18:48:58 +0100] rev 29769
improved section on "Hereditary Harrop Formulae";
wenzelm [Thu, 19 Feb 2009 21:19:49 +0100] rev 29768
more on object-level rules;
tuned;
wenzelm [Wed, 18 Feb 2009 22:44:59 +0100] rev 29767
updated generated files;
wenzelm [Wed, 18 Feb 2009 22:44:52 +0100] rev 29766
tuned;
wenzelm [Wed, 18 Feb 2009 22:37:57 +0100] rev 29765
more on local theories;
tuned;
wenzelm [Tue, 17 Feb 2009 22:47:19 +0100] rev 29764
some text on local theory specifications;
wenzelm [Tue, 17 Feb 2009 22:46:41 +0100] rev 29763
some more Isar macros;
wenzelm [Mon, 16 Feb 2009 21:39:52 +0100] rev 29762
updated genereted files;
wenzelm [Mon, 16 Feb 2009 21:39:19 +0100] rev 29761
minor tuning and typographic fixes;
wenzelm [Mon, 16 Feb 2009 21:23:34 +0100] rev 29760
tuned refs;
wenzelm [Mon, 16 Feb 2009 21:23:34 +0100] rev 29759
removed rudiments of glossary;
tuned outline;
wenzelm [Mon, 16 Feb 2009 21:23:33 +0100] rev 29758
removed rudiments of glossary;
wenzelm [Mon, 16 Feb 2009 21:04:15 +0100] rev 29757
removed unused glossary macros;
wenzelm [Mon, 16 Feb 2009 20:49:39 +0100] rev 29756
updated generated files;
wenzelm [Mon, 16 Feb 2009 20:47:44 +0100] rev 29755
observe usual theory naming conventions;
wenzelm [Mon, 16 Feb 2009 20:25:21 +0100] rev 29754
updated generated files;
wenzelm [Mon, 16 Feb 2009 20:23:43 +0100] rev 29753
tuned;