haftmann [Wed, 11 Feb 2009 15:05:40 +0100] rev 29876
merged
haftmann [Wed, 11 Feb 2009 15:05:26 +0100] rev 29875
liberal inst_meet
haftmann [Wed, 11 Feb 2009 15:05:25 +0100] rev 29874
display code theorems with HOL equality
blanchet [Wed, 11 Feb 2009 13:47:28 +0100] rev 29873
merged
blanchet [Tue, 10 Feb 2009 18:57:02 +0100] rev 29872
Added serial_string to SAT solver input and output files, to prevent multithreading chaos.
Bug reported by Tobias.
blanchet [Tue, 10 Feb 2009 14:58:15 +0100] rev 29871
Added nitpick_const_simp attribute to recdef and record packages.
blanchet [Tue, 10 Feb 2009 14:20:47 +0100] rev 29870
Added nitpick_const_simp attribute to 'simps' produced by the old primrec package.
blanchet [Tue, 10 Feb 2009 14:02:45 +0100] rev 29869
Renamed descriptions of Nitpick (and ATP) attributes, so that they fit well with the rest of the sentence in ProofGeneral.
blanchet [Mon, 09 Feb 2009 12:31:36 +0100] rev 29868
Reintroduced nitpick_ind_intro attribute.
It looks like I need it nonetheless.
blanchet [Mon, 09 Feb 2009 10:39:57 +0100] rev 29867
merged
blanchet [Mon, 09 Feb 2009 10:37:59 +0100] rev 29866
Added Nitpick_Const_Psimp attribute, dropped the 's' in Nitpick_Const_Simps, and killed the Nitpick_Ind_Intros attribute.
This should now be all.
blanchet [Fri, 06 Feb 2009 16:00:05 +0100] rev 29865
merged
blanchet [Fri, 06 Feb 2009 15:59:49 +0100] rev 29864
Merged.
blanchet [Fri, 06 Feb 2009 15:57:47 +0100] rev 29863
Added "nitpick_const_simps" and "nitpick_ind_intros" attributes for theorems;
these will be used by Nitpick, which will be released independently of Isabelle
2009, but they need to be in.
kleing [Wed, 11 Feb 2009 23:07:50 +1100] rev 29862
fixed typo
kleing [Wed, 11 Feb 2009 23:05:58 +1100] rev 29861
updated NEWS etc with "solves" criterion and auto_solves
nipkow [Wed, 11 Feb 2009 10:51:31 +0100] rev 29860
merged
nipkow [Wed, 11 Feb 2009 10:51:07 +0100] rev 29859
Moved Order_Relation into Library and moved some of it into Relation.
kleing [Wed, 11 Feb 2009 16:03:10 +1100] rev 29858
Autosolve feature for detecting duplicate theorems; patch by Timothy Bourke
kleing [Wed, 11 Feb 2009 14:48:14 +1100] rev 29857
FindTheorems: add solves feature; tidy up const name subsettin; patch by Timothy Bourke
huffman [Tue, 10 Feb 2009 17:53:51 -0800] rev 29856
const_name antiquotations
paulson [Tue, 10 Feb 2009 10:25:09 +0000] rev 29855
Repaired a proof that did, after all, refer to the theorem nat_induct2.
paulson [Tue, 10 Feb 2009 09:58:58 +0000] rev 29854
merged
paulson [Tue, 10 Feb 2009 09:51:23 +0000] rev 29853
Strengthened the induction rule nat_induct2.
paulson [Tue, 10 Feb 2009 09:46:11 +0000] rev 29852
Deleted the induction rule nat_induct2, which was too weak and not used even once.
nipkow [Mon, 09 Feb 2009 22:15:37 +0100] rev 29851
merged
nipkow [Mon, 09 Feb 2009 22:14:33 +0100] rev 29850
fix to [arith]
nipkow [Mon, 09 Feb 2009 18:50:10 +0100] rev 29849
new attribute "arith" for facts supplied to arith.
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