Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-10000
-3000
-1000
-120
+120
+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.
fixed title
2007-09-15, by haftmann
replaced Symbol.is_hex_letter to Symbol.is_ascii_hex;
2007-09-15, by wenzelm
ML_Lex.keywords;
2007-09-15, by wenzelm
tuned comments;
2007-09-15, by wenzelm
replaced Symbol.is_hex_letter to Symbol.is_ascii_hex;
2007-09-15, by wenzelm
Lexical syntax for SML.
2007-09-15, by wenzelm
added ML/ml_lex.ML;
2007-09-15, by wenzelm
removed redundant OuterLex.make_lexicon;
2007-09-15, by wenzelm
lexicographic_order method uses "<*mlex*>" instead of "measures" => no longer depends on List.thy
2007-09-14, by krauss
added "<*mlex*>" which lexicographically combines a measure function with a relation
2007-09-14, by krauss
moved ML_XXX.ML files to Pure/ML;
2007-09-14, by wenzelm
tidied
2007-09-14, by paulson
reverted back to the old version of the equivariance lemma for ALL
2007-09-14, by urbanc
some cleaning up to do with contexts
2007-09-13, by urbanc
Generalized equivariance and nominal_inductive commands to
2007-09-13, by berghofe
Added equivariance lemmas for induct_forall.
2007-09-13, by berghofe
Added equivariance lemma for induct_implies.
2007-09-13, by berghofe
typo fixed, dead link removed
2007-09-11, by webertj
added lemma
2007-09-10, by nipkow
Auto quickcheck now displays counterexample using Proof.goal_message
2007-09-10, by berghofe
added String.isSubstring;
2007-09-08, by wenzelm
export is_finished;
2007-09-08, by wenzelm
Present.session_name;
2007-09-08, by wenzelm
tuned signature;
2007-09-08, by wenzelm
thy_deps: ThyInfo.thy_ord, improved dir/unfold entry;
2007-09-08, by wenzelm
removed thy_ord (erratic due to multi-threading);
2007-09-08, by wenzelm
some cleaning up
2007-09-08, by urbanc
theorem: apply hook last;
2007-09-07, by wenzelm
reset goal messages after goal update;
2007-09-07, by wenzelm
added hilite markup;
2007-09-07, by wenzelm
fixed type alias in signature;
2007-09-07, by wenzelm
added lemma
2007-09-07, by nipkow
allow TVars during type inference
2007-09-07, by paulson
tidied the proofs
2007-09-07, by paulson
made smlnj happy;
2007-09-07, by wenzelm
new fun declaration
2007-09-06, by paulson
Auto-config of E_HOME, SPASS_HOME, VAMPIRE_HOME
2007-09-06, by paulson
Vampire structured proofs. Better parsing; some bug fixes.
2007-09-06, by paulson
chained facts are now included
2007-09-06, by paulson
new proofs found
2007-09-06, by paulson
trivial cleaning up
2007-09-06, by urbanc
added goal_message;
2007-09-06, by wenzelm
theorem hooks: apply in declaration order;
2007-09-06, by wenzelm
Generalized code generator for numerals.
2007-09-06, by berghofe
- New theories Lambda/NormalForm and Lambda/Standardization
2007-09-06, by berghofe
Added lecture notes by Matthes and Loader.
2007-09-06, by berghofe
New proof of standardization theorem (inspired by Ralph Matthes).
2007-09-06, by berghofe
Definition of normal forms (taken from theory WeakNorm).
2007-09-06, by berghofe
Moved definition of normal forms to new NormalForm theory.
2007-09-06, by berghofe
Added Standardization theory.
2007-09-06, by berghofe
New code generator setup (taken from Library/Executable_Real.thy,
2007-09-06, by berghofe
Added code generator setup (taken from Library/Executable_Rat.thy,
2007-09-06, by berghofe
Integrated code generator setup into RealDef theory.
2007-09-06, by berghofe
Integrated code generator setup into Rational theory.
2007-09-06, by berghofe
Integrated Executable_Rat and Executable_Real theories into
2007-09-06, by berghofe
use preferences.ML: do setmp *here*, to capture intended default values;
2007-09-05, by wenzelm
tuned;
2007-09-05, by wenzelm
modified proofs so that they are not using claset()
2007-09-05, by urbanc
tuned lemma; replaced !! by arbitrary
2007-09-04, by nipkow
Improved comment.
2007-09-04, by ballarin
Documented function package in IsarRef-manual.
2007-09-03, by krauss
added variations on infinite descent
2007-09-03, by nipkow
fixed Rat.inv
2007-09-03, by haftmann
fixed Rat.inv
2007-09-03, by haftmann
fix sgn_div_norm class
2007-09-02, by huffman
made theorem-references safe
2007-09-02, by urbanc
removed unused join_mode;
2007-09-01, by wenzelm
read_def_terms: replaced full Syntax.check_typs by certify_typ, to workaround problems with illegal schematic type vars;
2007-09-01, by wenzelm
removed obsolete ML bindings;
2007-09-01, by wenzelm
linorder_neqE_ordered_idom: proper proof, avoid illegal schematic type vars;
2007-09-01, by wenzelm
mono_Int/Un: proper proof, avoid illegal schematic type vars;
2007-09-01, by wenzelm
removed spurious Toplevel.debug, which actually makes Poly/ML crash in certain situations;
2007-09-01, by wenzelm
added singleton check_typ/term/prop;
2007-09-01, by wenzelm
removed obsolete read/cert variations (cf. Syntax.read/check);
2007-09-01, by wenzelm
replaced ProofContext.cert_term/prop by general Syntax.check_term/prop (which also includes type-inference);
2007-09-01, by wenzelm
replaced ProofContext.read_term/prop by general Syntax.read_term/prop;
2007-09-01, by wenzelm
replaced ProofContext.read_term/prop by general Syntax.read_term/prop;
2007-09-01, by wenzelm
*** empty log message ***
2007-09-01, by nipkow
final(?) iteration of sgn saga.
2007-09-01, by nipkow
reject_vars: accept type-inference params;
2007-08-31, by wenzelm
exported is_param;
2007-08-31, by wenzelm
legacy_infer_term: ProofContext.mode_schematic;
2007-08-31, by wenzelm
prove: setmp quick_and_dirty (avoids race condition);
2007-08-31, by wenzelm
export various inner syntax modes;
2007-08-31, by wenzelm
type_infer: mode_pattern;
2007-08-31, by wenzelm
do not touch quick_and_dirty;
2007-08-31, by wenzelm
tuned multithreading entry -- no longer experimental;
2007-08-31, by wenzelm
explained \isatstyle(minor)
2007-08-31, by nipkow
added short_names explanation
2007-08-31, by nipkow
added join_mode;
2007-08-30, by wenzelm
replaced ProofContext.infer_types by general Syntax.check_terms;
2007-08-30, by wenzelm
replaced ProofContext.infer_types by general Syntax.check_terms;
2007-08-30, by wenzelm
*** empty log message ***
2007-08-30, by nipkow
added constant sgn
2007-08-30, by nipkow
added lemma
2007-08-30, by nipkow
added some more entries;
2007-08-30, by wenzelm
turned type_check into separate typ/term_check;
2007-08-30, by wenzelm
tuned;
2007-08-30, by wenzelm
moved type_mode to type.ML;
2007-08-30, by wenzelm
infer_types: general check_typs instead of Type.cert_typ_mode;
2007-08-30, by wenzelm
maintain mode in context (get/set/restore_mode);
2007-08-30, by wenzelm
added burrow_types;
2007-08-30, by wenzelm
- tuned section about inductive predicates
2007-08-30, by berghofe
ported div/mod simprocs from HOL/ex/Binary.thy
2007-08-30, by huffman
renamed POLYML_LINK_OPTIONS to POLY_LINK_OPTIONS;
2007-08-29, by wenzelm
added POLYML_LINK_OPTIONS, which is required for unusual platforms (notably cygwin);
2007-08-29, by wenzelm
some simultaneous use_thys;
2007-08-29, by wenzelm
Updated section about inductive definitions.
2007-08-29, by berghofe
turned list comprehension translations into ML to optimize base case
2007-08-29, by nipkow
added Hoare/hoare_tac.ML (code from Hoare/Hoare.thy, also required in Isar_examples/Hoare.thy);
2007-08-29, by wenzelm
added x86-solaris;
2007-08-29, by wenzelm
fixed Proofs
2007-08-29, by chaieb
added Hoare/hoare_tac.ML (code from Hoare/Hoare.thy, also required in Isar_examples/Hoare.thy);
2007-08-29, by wenzelm
removed unused theorems ; added lifting properties for foldr and foldl
2007-08-29, by chaieb
removed Hoare/hoare.ML, Hoare/hoareAbort.ML, ex/svc_oracle.ML (which can be mistaken as attached ML script on case-insensitive file-system);
2007-08-29, by wenzelm
Deleted unused fillin_mixfix function.
2007-08-29, by berghofe
mark all parallel sessions as experimental
2007-08-29, by kleing
atbroy99 is 64bit
2007-08-29, by kleing
fixed pattern comnpletion; untabified
2007-08-28, by krauss
revert to Word library version from 2007/08/20
2007-08-28, by huffman
less
more
|
(0)
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip