Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-240
+240
+1000
+3000
+10000
+30000
tip
Find changesets by keywords (author, files, the commit message), revision number or hash, or
revset expression
.
The revision graph only works with JavaScript-enabled browsers.
moved type bstring from name_space.ML to binding.ML -- it is the primitive concept behind bindings;
2009-03-03, by wenzelm
added markup for binding;
2009-03-03, by wenzelm
Binding.str_of;
2009-03-03, by wenzelm
Binding.str_of;
2009-03-03, by wenzelm
Binding.str_of;
2009-03-03, by wenzelm
renamed Binding.display to Binding.str_of, which is slightly more canonical;
2009-03-03, by wenzelm
nicer_shortest: use NameSpace.extern_flags with disabled "features" instead of internal NameSpace.get_accesses;
2009-03-03, by wenzelm
moved name space externalization flags back to name_space.ML;
2009-03-03, by wenzelm
moved name space externalization flags back to name_space.ML;
2009-03-03, by wenzelm
reverted change introduced in a7c164e228e1 -- there cannot be a "bug" in a perfectly normal operation on the internal data representation that merely escaped into public by accident (cf. 0a981c596372);
2009-03-03, by wenzelm
merged
2009-03-03, by wenzelm
Thm.binding;
2009-03-03, by wenzelm
added type binding and val empty_binding;
2009-03-03, by wenzelm
updated generated files;
2009-03-03, by wenzelm
ignore "source" option in antiquotations @{ML}, @{ML_type}, @{ML_struct} -- did not really make sense, without it users can enable source mode globally with less surprises;
2009-03-03, by wenzelm
Implement Makarius's suggestion for improved type pattern parsing.
2009-03-03, by Timothy Bourke
find_consts: fold in preference to foldl; hide internal constants; remove redundant exception catch
2009-03-02, by Timothy Bourke
adapted to lates experimental version;
2009-03-02, by wenzelm
removed Ids;
2009-03-02, by wenzelm
merged
2009-03-02, by haftmann
reduced confusion code_funcgr vs. code_wellsorted
2009-03-02, by haftmann
better markup
2009-03-02, by haftmann
name fix
2009-03-02, by nipkow
merged
2009-03-02, by nipkow
name changes
2009-03-02, by nipkow
Automated merge with ssh://chaieb@atbroy100.informatik.tu-muenchen.de//home/isabelle-repository/repos/isabelle
2009-03-02, by chaieb
Moved a few theorems about monotonic sequences from Fundamental_Theorem_Algebra to SEQ.thy
2009-03-02, by chaieb
fixed broken @{file} refs;
2009-03-02, by wenzelm
merged
2009-03-02, by wenzelm
using plain ISABELLE_PROCESS
2009-03-02, by haftmann
merged
2009-03-02, by haftmann
ignore ISABELLE_LINE_EDITOR for code generation
2009-03-02, by haftmann
use long names for old-style fold combinators;
2009-03-01, by wenzelm
discontinued experimental support for Alice -- too hard to maintain its many language incompatibilities, never really worked anyway;
2009-03-01, by wenzelm
avoid fragile parsing of end_timing result -- would have produced GC time on MosML, for example;
2009-03-01, by wenzelm
end_timing: generalized result -- message plus with explicit time values;
2009-03-01, by wenzelm
replaced archaic Display.pretty_fact by FindTheorems.pretty_thm, which observes the context properly (as did the former prt_fact already);
2009-03-01, by wenzelm
updated contributors;
2009-03-01, by wenzelm
removed parts of the manual that are clearly obsolete, or covered by
2009-03-01, by wenzelm
merged
2009-03-01, by wenzelm
minor update of Mercurial HOWTO;
2009-03-01, by wenzelm
removed redundant lemmas
2009-03-01, by nipkow
added lemmas by Jeremy Avigad
2009-03-01, by nipkow
A Serbian theory, by Filip Maric.
2009-02-28, by wenzelm
more accurate deps;
2009-02-28, by wenzelm
merged
2009-02-28, by wenzelm
add news for HOLCF; fixed some typos and inaccuracies
2009-02-28, by huffman
fixed headers;
2009-02-28, by wenzelm
moved isabelle_system.scala to src/Pure/System/;
2009-02-28, by wenzelm
moved isabelle_process.ML, isabelle_process.scala, isar.ML, session.ML to Pure/System/ (together with associated Isar commands);
2009-02-28, by wenzelm
updated generated files;
2009-02-28, by wenzelm
added method "coherent";
2009-02-28, by wenzelm
more refs;
2009-02-28, by wenzelm
moved method "iprover" to HOL specific part;
2009-02-28, by wenzelm
removed Ids;
2009-02-28, by wenzelm
simultaneous use_thys;
2009-02-28, by wenzelm
replaced low-level 'no_syntax' by 'no_notation';
2009-02-28, by wenzelm
moved generic intuitionistic prover to src/Tools/intuitionistic.ML;
2009-02-28, by wenzelm
tuned message;
2009-02-28, by wenzelm
* New prover for coherent logic (see src/Tools/coherent.ML).
2009-02-28, by wenzelm
more CONTRIBUTORS;
2009-02-28, by wenzelm
removed Ids;
2009-02-28, by wenzelm
moved some generic tools to src/Tools/ -- src/Provers is essentially obsolete;
2009-02-28, by wenzelm
some updates on ancient README;
2009-02-28, by wenzelm
fixrec package uses new-style syntax and local-theory interface
2009-02-27, by huffman
add function taken_names
2009-02-27, by huffman
merged
2009-02-27, by huffman
make list-style polynomial syntax work when show_sorts is on
2009-02-27, by huffman
more CONTRIBUTORS;
2009-02-27, by wenzelm
turned "read-only refs" typ_level and minimize_applies into constant values;
2009-02-27, by wenzelm
merged
2009-02-27, by wenzelm
removed global ref dfg_format
2009-02-26, by immler
removed local ref const_needs_hBOOL;
2009-02-25, by immler
removed local ref const_min_arity
2009-02-24, by immler
eliminated private clones of List.partition;
2009-02-27, by wenzelm
observe some Isabelle/ML coding conventions;
2009-02-27, by wenzelm
eliminated NJ's List.nth;
2009-02-27, by wenzelm
tuned CHANGED_GOAL: use Thm.cprem_of instead of selecting from Thm.prems_of;
2009-02-27, by wenzelm
tuned/unified size_of_term and size_of_typ, eliminated obsolete foldl;
2009-02-27, by wenzelm
observe basic Isabelle/ML coding conventions;
2009-02-27, by wenzelm
moved find_theorems.ML and find_consts.ML to Pure/Tools, collecting main implementation in one place each;
2009-02-27, by wenzelm
added ML-Systems/polyml-experimental.ML;
2009-02-27, by wenzelm
tuned;
2009-02-27, by wenzelm
even less default memory for sunbroy2;
2009-02-27, by wenzelm
merged
2009-02-27, by boehmes
merged
2009-02-27, by boehmes
Made then_conv and else_conv available as infix operations.
2009-02-26, by boehmes
merged
2009-02-27, by haftmann
fixed typo
2009-02-27, by haftmann
merged
2009-02-26, by huffman
avoid using legacy type inference
2009-02-26, by huffman
use TheoryData to keep track of pattern match combinators
2009-02-26, by huffman
merged
2009-02-26, by huffman
remove unnecessary simp rules
2009-02-26, by huffman
revert some Suc 0 lemmas back to their original forms; added some simp rules for (1::nat)
2009-02-26, by huffman
merged
2009-02-26, by wenzelm
back to canonical ROOT, to see if memory problems still persist;
2009-02-26, by wenzelm
trying less default memory for sunbroy2 test
2009-02-27, by kleing
basic setup for chapter "Syntax and type-checking";
2009-02-26, by wenzelm
merged
2009-02-26, by wenzelm
standard headers;
2009-02-26, by wenzelm
updated generated files;
2009-02-26, by wenzelm
uniform treatment of ML indexing, using general \indexdef macro for formal Isabelle/Isar entities;
2009-02-26, by wenzelm
fixed import of ~~/src/HOL/Decision_Procs/Ferrack;
2009-02-26, by wenzelm
more explicit indication of old manuals;
2009-02-26, by wenzelm
merged
2009-02-26, by wenzelm
\bibliographystyle{abbrv} for newer ref manuals;
2009-02-26, by wenzelm
added Haftmann-Wenzel:2009;
2009-02-26, by wenzelm
updated generated files;
2009-02-26, by wenzelm
isabelle document: adapted (postulated) defaults for tags to actual isabelle.sty;
2009-02-26, by wenzelm
merged
2009-02-26, by wenzelm
include HOL-Decision_Procs in stats;
2009-02-26, by wenzelm
back to plain http;
2009-02-26, by wenzelm
merged
2009-02-26, by berghofe
Added postprocessing rules for fresh_star.
2009-02-26, by berghofe
Fixed nonexhaustive match problem in decomp, to make it fail more gracefully
2009-02-26, by berghofe
tuned NEWS;
2009-02-26, by wenzelm
merged
2009-02-26, by wenzelm
merged
2009-02-26, by huffman
add type annotation
2009-02-26, by huffman
disable floor_minus and ceiling_minus [simp]
2009-02-26, by huffman
merged
2009-02-26, by wenzelm
merged
2009-02-26, by paulson
Updated the theory syntax. Corrected an error in a command.
2009-02-26, by paulson
merged
2009-02-25, by huffman
generalize floor/ceiling to work with real and rat; rename floor_mono2 to floor_mono
2009-02-25, by huffman
new theory of Archimedean fields
2009-02-25, by huffman
add lemmas about comparisons of Fract a b with 0 and 1
2009-02-25, by huffman
merged
2009-02-25, by huffman
add lemma diff_Suc_1
2009-02-25, by huffman
Added lemmas for normalizing freshness results involving fresh_star.
2009-02-25, by berghofe
Added typing and evaluation relations, together with proofs of preservation
2009-02-25, by berghofe
merged
2009-02-25, by berghofe
Use LocalTheory.full_name instead of Sign.full_name, because the latter does
2009-02-25, by berghofe
Replaced Logic.unvarify by Variable.import_terms to make declaration of
2009-02-25, by berghofe
nominal_inductive and equivariance now work on local_theory.
2009-02-25, by berghofe
Added equivariance lemmas for fresh_star.
2009-02-25, by berghofe
NEWS
2009-02-25, by nipkow
merged
2009-02-25, by haftmann
robustified
2009-02-25, by haftmann
make more proofs work whether or not One_nat_def is a simp rule
2009-02-24, by huffman
add simp rules for numerals with 1::nat
2009-02-24, by huffman
fix lemma hypreal_hnorm_def
2009-02-24, by huffman
make proofs work whether or not One_nat_def is a simp rule; replace 1 with Suc 0 in the rhs of some simp rules
2009-02-23, by huffman
move lemma dvd_mod_imp_dvd into class semiring_div
2009-02-23, by huffman
merged
2009-02-23, by haftmann
improved treatment of case certificates
2009-02-23, by haftmann
repaired order of variable node allocation
2009-02-23, by haftmann
explicitly import Fact
2009-02-23, by huffman
change imports to move Fact.thy outside Plain
2009-02-23, by huffman
add lemmas poly_{div,mod}_minus_{left,right}
2009-02-23, by huffman
merged
2009-02-23, by huffman
declare scaleR distrib rules [algebra_simps]; cleaned up
2009-02-22, by huffman
clean up instantiations
2009-02-22, by huffman
merged
2009-02-22, by huffman
simplify some proofs
2009-02-22, by huffman
remove duplicate instance declaration
2009-02-22, by huffman
stripped classrels_of, instances_of
2009-02-23, by haftmann
use canonical subalgebra projection
2009-02-23, by haftmann
experimental switch to new well-sorting algorithm
2009-02-22, by haftmann
handle NONE case in arity function properly
2009-02-22, by haftmann
clarified status of variables in evaluation terms; tuned header
2009-02-22, by haftmann
subalgebra: drop arities if desired
2009-02-22, by haftmann
merged
2009-02-22, by haftmann
more liberality needed
2009-02-22, by haftmann
merged
2009-02-22, by nipkow
added lemmas
2009-02-22, by nipkow
merged
2009-02-22, by haftmann
simplified evaluation
2009-02-22, by haftmann
merged
2009-02-22, by nipkow
added dvd_div_mult
2009-02-22, by nipkow
merged
2009-02-22, by haftmann
first attempt to solve evaluation bootstrap problem
2009-02-22, by haftmann
formal dependency on newly emerging algorithm
2009-02-22, by haftmann
merged
2009-02-22, by nipkow
name fix
2009-02-22, by nipkow
fix spelling
2009-02-21, by huffman
real_inner class instance for vectors
2009-02-21, by huffman
NEWS
2009-02-21, by nipkow
merged
2009-02-21, by nipkow
Removed subsumed lemmas
2009-02-21, by nipkow
remove duplicated lemmas about norm
2009-02-21, by huffman
real_normed_vector instance
2009-02-21, by huffman
fix real_vector, real_algebra instances
2009-02-21, by huffman
merged
2009-02-21, by huffman
generalize lemmas from nat to 'a::wellorder
2009-02-20, by huffman
generalize some lemmas
2009-02-20, by huffman
merged
2009-02-21, by nipkow
removed redundant thms
2009-02-21, by nipkow
merged
2009-02-20, by huffman
class instances for num1
2009-02-20, by huffman
Removed redundant lemmas
2009-02-20, by nipkow
merged
2009-02-20, by haftmann
also consider superclasses properly
2009-02-20, by haftmann
merged
2009-02-20, by nipkow
removed subsumed lemmas
2009-02-20, by nipkow
merged
2009-02-20, by haftmann
datatype antiquotation: always bracket types with spaces in between
2009-02-20, by haftmann
consequent use of term `code equation`
2009-02-20, by haftmann
permissive check for pattern discipline in case schemes
2009-02-20, by haftmann
maintain order of constructors in datatypes; clarified conventions for type schemes
2009-02-20, by haftmann
stripped Id
2009-02-20, by haftmann
merged
2009-02-20, by huffman
add theory of products as real vector spaces to Library
2009-02-20, by huffman
add new theory Product_plus.thy to Library
2009-02-20, by huffman
merged
2009-02-20, by immler
changed message
2009-02-20, by immler
detailed information on atp-failure via Output.debug
2009-02-20, by immler
merged
2009-02-20, by haftmann
reverted to old wellsorting algorithm
2009-02-20, by haftmann
fixed spurious proof failure
2009-02-20, by haftmann
consider changes variable names in theorem le_imp_power_dvd
2009-02-20, by haftmann
tuned and incremental version of wellsorting algorithm
2009-02-20, by haftmann
ignore sorts in bare types
2009-02-20, by haftmann
defensive implementation of pretty serialisation of lists and characters
2009-02-20, by haftmann
dropped Id
2009-02-20, by haftmann
experimental inclusion of new wellsorting algorithm for code equations
2009-02-20, by haftmann
merged
2009-02-20, by chaieb
merged
2009-02-17, by chaieb
merged
2009-02-17, by chaieb
fixed selection of premises
2009-02-17, by chaieb
cleaned up
2009-02-19, by huffman
declare of_int_number_of_eq [simp]
2009-02-19, by huffman
fix case_names
2009-02-19, by huffman
nicer induction/cases rules for numeral types
2009-02-19, by huffman
number_ring instances for numeral types
2009-02-19, by huffman
declare xor_compl_{left,right} [simp]
2009-02-19, by huffman
add rule for minus 1 at type bit
2009-02-19, by huffman
add formalization of a type of integers mod 2 to Library
2009-02-19, by huffman
new theory of real inner product spaces
2009-02-19, by huffman
add Powerdomain_ex.thy
2009-02-19, by huffman
add more ordering lemmas
2009-02-19, by huffman
avoid using ab_semigroup_idem_mult locale for powerdomains
2009-02-19, by huffman
merged
2009-02-19, by huffman
add header
2009-02-18, by huffman
move Polynomial.thy to Library
2009-02-18, by huffman
move FrechetDeriv.thy to Library
2009-02-18, by huffman
split polynomial-related stuff from Deriv.thy into Library/Poly_Deriv.thy
2009-02-18, by huffman
half auto_solve default time out; increase manually in PG for large projects
2009-02-19, by kleing
merged
2009-02-18, by huffman
less
more
|
(0)
-30000
-10000
-3000
-1000
-240
+240
+1000
+3000
+10000
+30000
tip