Fri, 06 Feb 2009 15:57:47 +0100 Added "nitpick_const_simps" and "nitpick_ind_intros" attributes for theorems;
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.
Wed, 11 Feb 2009 23:07:50 +1100 fixed typo
kleing [Wed, 11 Feb 2009 23:07:50 +1100] rev 29862
fixed typo
Wed, 11 Feb 2009 23:05:58 +1100 updated NEWS etc with "solves" criterion and auto_solves
kleing [Wed, 11 Feb 2009 23:05:58 +1100] rev 29861
updated NEWS etc with "solves" criterion and auto_solves
Wed, 11 Feb 2009 10:51:31 +0100 merged
nipkow [Wed, 11 Feb 2009 10:51:31 +0100] rev 29860
merged
Wed, 11 Feb 2009 10:51:07 +0100 Moved Order_Relation into Library and moved some of it into Relation.
nipkow [Wed, 11 Feb 2009 10:51:07 +0100] rev 29859
Moved Order_Relation into Library and moved some of it into Relation.
Wed, 11 Feb 2009 16:03:10 +1100 Autosolve feature for detecting duplicate theorems; patch by Timothy Bourke
kleing [Wed, 11 Feb 2009 16:03:10 +1100] rev 29858
Autosolve feature for detecting duplicate theorems; patch by Timothy Bourke
Wed, 11 Feb 2009 14:48:14 +1100 FindTheorems: add solves feature; tidy up const name subsettin; 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
Tue, 10 Feb 2009 17:53:51 -0800 const_name antiquotations
huffman [Tue, 10 Feb 2009 17:53:51 -0800] rev 29856
const_name antiquotations
Tue, 10 Feb 2009 10:25:09 +0000 Repaired a proof that did, after all, refer to the theorem nat_induct2.
paulson [Tue, 10 Feb 2009 10:25:09 +0000] rev 29855
Repaired a proof that did, after all, refer to the theorem nat_induct2.
Tue, 10 Feb 2009 09:58:58 +0000 merged
paulson [Tue, 10 Feb 2009 09:58:58 +0000] rev 29854
merged
Tue, 10 Feb 2009 09:51:23 +0000 Strengthened the induction rule nat_induct2.
paulson [Tue, 10 Feb 2009 09:51:23 +0000] rev 29853
Strengthened the induction rule nat_induct2.
Tue, 10 Feb 2009 09:46:11 +0000 Deleted the induction rule nat_induct2, which was too weak and not used even once.
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.
Mon, 09 Feb 2009 22:15:37 +0100 merged
nipkow [Mon, 09 Feb 2009 22:15:37 +0100] rev 29851
merged
Mon, 09 Feb 2009 22:14:33 +0100 fix to [arith]
nipkow [Mon, 09 Feb 2009 22:14:33 +0100] rev 29850
fix to [arith]
Mon, 09 Feb 2009 18:50:10 +0100 new attribute "arith" for facts supplied to arith.
nipkow [Mon, 09 Feb 2009 18:50:10 +0100] rev 29849
new attribute "arith" for facts supplied to arith.
Mon, 09 Feb 2009 17:25:07 +1100 Nicer names in FindTheorems.
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.
Mon, 09 Feb 2009 17:21:46 +0000 added Determinants to Library
chaieb [Mon, 09 Feb 2009 17:21:46 +0000] rev 29847
added Determinants to Library
Mon, 09 Feb 2009 17:21:19 +0000 Traces, Determinant of square matrices and some properties
chaieb [Mon, 09 Feb 2009 17:21:19 +0000] rev 29846
Traces, Determinant of square matrices and some properties
Mon, 09 Feb 2009 17:09:18 +0000 added Euclidean_Space and Glbs to Library
chaieb [Mon, 09 Feb 2009 17:09:18 +0000] rev 29845
added Euclidean_Space and Glbs to Library
Mon, 09 Feb 2009 17:08:49 +0000 fixed proof -- removed unnecessary sorry
chaieb [Mon, 09 Feb 2009 17:08:49 +0000] rev 29844
fixed proof -- removed unnecessary sorry
Mon, 09 Feb 2009 16:57:10 +0000 Fixed theorem reference
chaieb [Mon, 09 Feb 2009 16:57:10 +0000] rev 29843
Fixed theorem reference
Mon, 09 Feb 2009 16:54:03 +0000 (Real) Vectors in Euclidean space, and elementary linear algebra.
chaieb [Mon, 09 Feb 2009 16:54:03 +0000] rev 29842
(Real) Vectors in Euclidean space, and elementary linear algebra.
Mon, 09 Feb 2009 16:43:52 +0000 A generic decision procedure for linear rea arithmetic and normed vector spaces
chaieb [Mon, 09 Feb 2009 16:43:52 +0000] rev 29841
A generic decision procedure for linear rea arithmetic and normed vector spaces
Mon, 09 Feb 2009 16:42:15 +0000 Permutations, both general and specifically on finite sets.
chaieb [Mon, 09 Feb 2009 16:42:15 +0000] rev 29840
Permutations, both general and specifically on finite sets.
Mon, 09 Feb 2009 16:20:24 +0000 Imports Main in order to avoid the typerep problem
chaieb [Mon, 09 Feb 2009 16:20:24 +0000] rev 29839
Imports Main in order to avoid the typerep problem
Mon, 09 Feb 2009 16:19:46 +0000 A theory of greatest lower bounds
chaieb [Mon, 09 Feb 2009 16:19:46 +0000] rev 29838
A theory of greatest lower bounds
Mon, 09 Feb 2009 15:38:26 +0000 Now imports Fact as suggested by Florian in order to avoid the typerep problem
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
Mon, 09 Feb 2009 11:15:13 +0000 Added HOL/Library/Finite_Cartesian_Product.thy to Library
chaieb [Mon, 09 Feb 2009 11:15:13 +0000] rev 29836
Added HOL/Library/Finite_Cartesian_Product.thy to Library
(0) -10000 -3000 -1000 -300 -100 -50 -28 +28 +50 +100 +300 +1000 +3000 +10000 +30000 tip