Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-3000
-1000
-480
+480
+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.
print_data moved to theory.ML;
1998-06-05, by wenzelm
added THEN: ('a -> 'b seq) * ('b -> 'c seq) -> 'a -> 'c seq;
1998-06-05, by wenzelm
added object.ML;
1998-06-05, by wenzelm
added option_map_o_empty
1998-06-02, by oheimb
added split_etas
1998-06-02, by oheimb
added split_sum_case_asm
1998-06-02, by oheimb
tuned;
1998-05-29, by wenzelm
tuned msgs;
1998-05-29, by wenzelm
auto update
1998-05-28, by paulson
fixed ml_prompts;
1998-05-28, by wenzelm
changed get_single: ('a, 'b) source -> ('a * ('a, 'b) source) option;
1998-05-28, by wenzelm
tuned dist version;
1998-05-28, by wenzelm
tuned header;
1998-05-28, by wenzelm
version under control of Admin/makedist;
1998-05-28, by wenzelm
README, Pure/ROOT.ML: version set automatically;
1998-05-28, by wenzelm
version under control of Admin/makedist;
1998-05-28, by wenzelm
added ml_prompts;
1998-05-28, by wenzelm
added mapfilter: ('a -> 'b option) -> ('a, 'c) source -> ('b, ('a, 'c)
1998-05-28, by wenzelm
tuned error msg;
1998-05-28, by wenzelm
fixed error msgs;
1998-05-28, by wenzelm
Structure Option now declared in MLWorks
1998-05-27, by paulson
mk_all_imp: no longer creates goals that have beta-redexes
1998-05-27, by paulson
more tracing
1998-05-27, by paulson
Changed require to requires for MLWorks
1998-05-27, by paulson
auto update
1998-05-27, by paulson
made SML/NJ happy;
1998-05-26, by wenzelm
foldl_map prep_field;
1998-05-26, by wenzelm
tuned store_theory;
1998-05-25, by wenzelm
tuned local, global;
1998-05-25, by wenzelm
tuned store_theory: theory -> unit;
1998-05-25, by wenzelm
added get_name, put_name, global_path, local_path, begin_theory,
1998-05-25, by wenzelm
global_names moved to pure_thy.ML;
1998-05-25, by wenzelm
certify_term: type_check replaces Term.type_of, providing sensible
1998-05-25, by wenzelm
renamed state_source to source';
1998-05-25, by wenzelm
added recover, source;
1998-05-25, by wenzelm
added catch: ('a -> 'b) -> 'a -> 'b;
1998-05-25, by wenzelm
remove seq2, scan (use seq2, foldl_map from library.ML);
1998-05-25, by wenzelm
added foldl_map: ('a * 'b -> 'a * 'c) -> 'a * 'b list -> 'a * 'c list;
1998-05-25, by wenzelm
Swapped order of params.
1998-05-25, by nipkow
changed get_single: ('a, 'b) source -> 'a option * ('a, 'b) source;
1998-05-20, by wenzelm
source vs. source';
1998-05-20, by wenzelm
tuned keywords;
1998-05-20, by wenzelm
added is_stale;
1998-05-20, by wenzelm
tuned signature;
1998-05-20, by wenzelm
tuned comments;
1998-05-20, by wenzelm
tuned;
1998-05-20, by wenzelm
Small mods.
1998-05-20, by nipkow
prompt made part of source;
1998-05-19, by wenzelm
fixed handle_error: cat_lines;
1998-05-19, by wenzelm
added Thy/position.ML;
1998-05-19, by wenzelm
added source: string -> (string, string list) Source.source;
1998-05-19, by wenzelm
Input positions.
1998-05-19, by wenzelm
added Syntax/source.ML;
1998-05-18, by wenzelm
added Source module;
1998-05-18, by wenzelm
Co-algebraic data sources.
1998-05-18, by wenzelm
Symbol.stopper;
1998-05-18, by wenzelm
improved finite scans: more abstract stopper;
1998-05-18, by wenzelm
snoc_induct/exhaust -> rev_induct_exhaust.
1998-05-18, by nipkow
Cleaned up and simplified etc.
1998-05-18, by nipkow
witnesses: lookup stored thms instead of axioms;
1998-05-15, by wenzelm
added add_axioms_x, add_defs_x;
1998-05-15, by wenzelm
PureThy.add_typedecls;
1998-05-15, by wenzelm
Reordred arguments in AutoChopper.
1998-05-14, by nipkow
extended addsplits and delsplits to handle also split rules for assumptions
1998-05-14, by oheimb
simplifications
1998-05-14, by oheimb
disabled (experimental) geometry option
1998-05-14, by oheimb
keyboard settings now done by loading Tools/8bit/xemacs/isa_xemacs.emacs
1998-05-14, by oheimb
added option_map_o_update
1998-05-14, by oheimb
added welcome;
1998-05-13, by wenzelm
added :-- (dependent pair);
1998-05-13, by wenzelm
added transform_error, exception ERROR_MESSAGE;
1998-05-13, by wenzelm
added thms_closure: theory -> xstring -> tthm list option;
1998-05-13, by wenzelm
adapted to new Scan.fail_with / Scan.!!;
1998-05-13, by wenzelm
pure_nonterms;
1998-05-13, by wenzelm
added fail_with and adapted !!;
1998-05-13, by wenzelm
gen_attr: fixed order of evaluation;
1998-05-13, by wenzelm
tuned msg;
1998-05-13, by wenzelm
get_first: ('a -> 'b option) -> 'a list -> 'b option;
1998-05-13, by wenzelm
HOL/record: now includes concrete syntax for record terms;
1998-05-13, by wenzelm
added Goal, Goalw;
1998-05-12, by wenzelm
branching_level = 250;
1998-05-12, by wenzelm
fixed comment;
1998-05-12, by wenzelm
Removed duplicate list_length_induct
1998-05-12, by nipkow
Reordered a few parameters.
1998-05-11, by nipkow
Lex
1998-05-11, by nipkow
tuned comment;
1998-05-10, by wenzelm
Reshuffeling, renaming and a few simple corollaries.
1998-05-08, by nipkow
fixed translations;
1998-05-08, by wenzelm
proper thy files;
1998-05-08, by wenzelm
fixed update syntax;
1998-05-08, by wenzelm
improved source: state-based;
1998-05-07, by wenzelm
added scan_tvar;
1998-05-07, by wenzelm
added 'space';
1998-05-07, by wenzelm
Got rid of NAe.delta
1998-05-07, by nipkow
HOL/Update
1998-05-06, by paulson
Removed some traces of UNITY
1998-05-06, by paulson
Changed [/] to [:=] and removed actual definition.
1998-05-06, by nipkow
New syntax for function update; moved to main HOL directory
1998-05-05, by paulson
misc tuning;
1998-05-05, by wenzelm
'more' selector;
1998-05-04, by wenzelm
added nth_update: 'a -> int * 'a list -> 'a list;
1998-05-04, by wenzelm
tuned msg;
1998-05-04, by wenzelm
fixed constdefs syntax;
1998-05-04, by wenzelm
concrete syntax for record terms;
1998-05-04, by wenzelm
New behaviour of asm_full_simp_tac.
1998-05-04, by nipkow
added CLASIMPSET(') tacticals;
1998-05-02, by wenzelm
added trfun_names;
1998-05-02, by wenzelm
added accesses: string -> string list;
1998-05-02, by wenzelm
minor corrections
1998-05-01, by oheimb
Auto_tac: now uses enhanced version of asm_full_simp_tac,
1998-05-01, by oheimb
added finite_dom_map_of and ran_update
1998-05-01, by oheimb
added insert_Collect
1998-05-01, by oheimb
corrected and updated description of wrapper mechanism (including addss)
1998-05-01, by oheimb
*** empty log message ***
1998-05-01, by nipkow
"let" is no longer restricted to FOL terms and allows any logical terms
1998-05-01, by paulson
Let.ML and Let.thy had been omitted
1998-05-01, by paulson
fixed simpset(), claset();
1998-04-30, by wenzelm
moved records data to Tools/record_package.ML;
1998-04-29, by wenzelm
nontermials;
1998-04-29, by wenzelm
Theory.require;
1998-04-29, by wenzelm
TypedefPackage.add_typedef;
1998-04-29, by wenzelm
Theory.require;
1998-04-29, by wenzelm
Logic.mk_defpair;
1998-04-29, by wenzelm
Extensible records with structural subtyping in HOL. See
1998-04-29, by wenzelm
new theory section 'setup';
1998-04-29, by wenzelm
nonterminals;
1998-04-29, by wenzelm
package extensible records with structural subtyping in HOL -- still
1998-04-29, by wenzelm
renamed from typedef.ML;
1998-04-29, by wenzelm
reworked and moved to Tools/record_package.ML;
1998-04-29, by wenzelm
removed typedef.ML, record.ML;
1998-04-29, by wenzelm
renamed to Tools/typedef_package.ML;
1998-04-29, by wenzelm
adapted to new PureThy.add_axioms_i;
1998-04-29, by wenzelm
adapted to new PureThy.add_tthmss;
1998-04-29, by wenzelm
Theory.require;
1998-04-29, by wenzelm
adapted to new PureThy.add_axioms;
1998-04-29, by wenzelm
new theory section 'nonterminals';
1998-04-29, by wenzelm
adapted to new PureThy.add_defs;
1998-04-29, by wenzelm
Theory.require;
1998-04-29, by wenzelm
tuned setup;
1998-04-29, by wenzelm
tuned setup;
1998-04-29, by wenzelm
tuned names of (add_)store_XXX functions;
1998-04-29, by wenzelm
replaced thy_setup by 'setup' section;
1998-04-29, by wenzelm
added append;
1998-04-29, by wenzelm
added none: 'a -> 'a * 'b attribute list;
1998-04-29, by wenzelm
tuned error msgs;
1998-04-29, by wenzelm
moved mk_defpair to logic.ML;
1998-04-29, by wenzelm
tuned get_ax (uses ancestry);
1998-04-29, by wenzelm
renamed setup to apply;
1998-04-29, by wenzelm
adapted to new PureThy.add_axioms_i;
1998-04-29, by wenzelm
added defaultS: sg -> sort;
1998-04-29, by wenzelm
added thm, thms;
1998-04-29, by wenzelm
*** empty log message ***
1998-04-29, by wenzelm
new thms, really demos of the final coalgebra theorem
1998-04-28, by paulson
new thms image_0_left, image_Un_left, etc.
1998-04-28, by paulson
new thm mult_lt_mono1
1998-04-28, by paulson
cleanup for split_all_tac as wrapper in claset()
1998-04-27, by oheimb
removed wrong comment
1998-04-27, by oheimb
added option_map_eq_Some via AddIffs
1998-04-27, by oheimb
*** empty log message ***
1998-04-27, by nipkow
delsplits, Addsplits, Delsplits.
1998-04-27, by nipkow
Renamed expand_const -> split_const
1998-04-27, by nipkow
Added conversion of reg.expr. to automata.
1998-04-27, by nipkow
Renamed expand_const -> split_const.
1998-04-27, by nipkow
Added a few lemmas.
1998-04-27, by nipkow
New proof of apply_equality and new thm Pi_image_cons
1998-04-27, by paulson
improved split_all_tac significantly
1998-04-24, by oheimb
improved keyboard modifiers
1998-04-24, by oheimb
added ASCII translation of subseteq
1998-04-24, by oheimb
tidied; div & mod
1998-04-24, by paulson
*** empty log message ***
1998-04-24, by oheimb
added no_syn;
1998-04-22, by wenzelm
added mk_cond_defpair, mk_defpair;
1998-04-22, by wenzelm
Modifications due to improved simplifier.
1998-04-22, by nipkow
Tried to speed up the rewriter by eta-contracting all patterns beforehand and
1998-04-22, by nipkow
improved pair_tac to call prune_params_tac afterwards
1998-04-21, by oheimb
split_all_tac is now added to claset() _before_ other safe tactics
1998-04-21, by oheimb
made proof of zmult_congruent2 more stable
1998-04-21, by oheimb
simplification of explicit theory usage and merges
1998-04-21, by oheimb
removed split_all_tac from claset() globally within IOA
1998-04-21, by oheimb
made modifications of the simpset() local
1998-04-21, by oheimb
layout improvement
1998-04-21, by oheimb
expandshort; new gcd_induct with inbuilt case analysis
1998-04-21, by paulson
Renamed mod_XXX_cancel to mod_XXX_self
1998-04-21, by paulson
New laws for mod
1998-04-20, by paulson
proving fib(gcd(m,n)) = gcd(fib m, fib n)
1998-04-20, by paulson
fixed comment;
1998-04-19, by wenzelm
Fixed bug in inductive sections to allow disjunctive premises;
1998-04-10, by paulson
bug fixes
1998-04-10, by paulson
can prove the empty relation to be WF
1998-04-10, by paulson
Fixed bug in inductive sections to allow disjunctive premises;
1998-04-10, by paulson
Clearer description of recdef, including use of {}
1998-04-09, by paulson
Simplified the syntax description; mentioned FOL vs HOL
1998-04-09, by paulson
*** empty log message ***
1998-04-07, by oheimb
replaced option_map_SomeD by option_map_eq_Some (RS iffD1)
1998-04-07, by oheimb
made split_all_tac as safe wrapper more defensive:
1998-04-07, by oheimb
no open Simplifier;
1998-04-04, by wenzelm
tuned fail;
1998-04-04, by wenzelm
type_error;
1998-04-04, by wenzelm
tuned comments;
1998-04-04, by wenzelm
no open Simplifier;
1998-04-04, by wenzelm
replaced thy_data by thy_setup;
1998-04-04, by wenzelm
type_error;
1998-04-04, by wenzelm
replaced thy_data by setup;
1998-04-04, by wenzelm
removed simple;
1998-04-04, by wenzelm
added triv_goal, rev_triv_goal (for Isar);
1998-04-04, by wenzelm
added Goal_def;
1998-04-04, by wenzelm
replaced thy_data by thy_setup;
1998-04-04, by wenzelm
added local_theory (for Isar);
1998-04-04, by wenzelm
tuned trace msgs;
1998-04-04, by wenzelm
tuned names;
1998-04-03, by wenzelm
added get_tthm(s), store_tthms(s);
1998-04-03, by wenzelm
tuned comments;
1998-04-03, by wenzelm
added attribute.ML;
1998-04-03, by wenzelm
Theorem tags and attributes.
1998-04-03, by wenzelm
UNITY
1998-04-03, by paulson
repaired incompatibility with new SML version by eta-expansion
1998-04-03, by oheimb
New target HOL-UNITY
1998-04-03, by paulson
New UNITY theory
1998-04-03, by paulson
Tidied proofs
1998-04-03, by paulson
Tidied proofs by getting rid of case_tac
1998-04-03, by paulson
improved \tt appearance of many ASCII special symbols like #
1998-04-03, by oheimb
split_all_tac now fails if there is nothing to split
1998-04-02, by oheimb
new theorems
1998-04-02, by paulson
changed if_bool_eq to if_bool_eq_conj
1998-04-02, by paulson
changed if_bool_eq to if_bool_eq_conj and added if_bool_eq_disj
1998-04-02, by paulson
New theorems card_Diff_le and card_insert_le; tidied
1998-04-02, by paulson
introduced functions for updating the wrapper lists
1998-04-02, by oheimb
*** empty log message ***
1998-04-02, by oheimb
merge_cs now also merges safe and unsafe wrappers
1998-03-30, by oheimb
generalized appearance of trancl_into_rtrancl and r_into_trancl
1998-03-30, by oheimb
adapted proof of finite_converse
1998-03-30, by oheimb
added wf_converse_trancl, adapted proof of wfrec
1998-03-30, by oheimb
added caveat
1998-03-30, by oheimb
added introduction and elimination rules for Univalent
1998-03-30, by oheimb
added Univalent_rel_pow
1998-03-30, by oheimb
removed superfluous use_thy
1998-03-30, by oheimb
removed superfluous translations
1998-03-30, by oheimb
added try, single, many;
1998-03-24, by wenzelm
added cproj', and therefore extended prj
1998-03-24, by oheimb
added cproj', and therefore extended prj
1998-03-24, by oheimb
improved checks
1998-03-24, by oheimb
added o2s
1998-03-24, by oheimb
added finite_acyclic_wf_converse: corrected 8bit chars
1998-03-24, by oheimb
added acyclicI
1998-03-24, by oheimb
added finite_acyclic_wf_converse
1998-03-24, by oheimb
more thms
1998-03-23, by paulson
inverse -> converse
1998-03-16, by paulson
inverse -> converse
1998-03-16, by paulson
re-ordered proofs
1998-03-16, by paulson
moved addsplits [expand_if] from HOL_basic_ss to HOL_ss;
1998-03-13, by wenzelm
renamed not1_or to disj_not1, not2_or to disj_not2
1998-03-12, by oheimb
improved coding of delWrapper and delSWrapper
1998-03-12, by oheimb
addloop: added warning in case of overwriting a looper
1998-03-12, by oheimb
Made mutual simplification of prems a special case.
1998-03-12, by nipkow
Used merge_alists for loopers.
1998-03-12, by nipkow
New, stronger rewrites
1998-03-12, by paulson
The theorem nat_neqE, and some tidying
1998-03-12, by paulson
New laws, mostly generalizing old "pred" ones
1998-03-12, by paulson
spy_analz_tac now handles individual conjuncts properly
1998-03-11, by paulson
new theorem
1998-03-11, by paulson
New theorem Image_eq_UN; deleted the silly vimage_inverse_Image
1998-03-11, by paulson
Arith.thy -> thy; proved a few new theorems
1998-03-11, by paulson
New Asm_full_simp_tac shortens proof.
1998-03-11, by nipkow
Simplifier
1998-03-11, by nipkow
More Lex.
1998-03-11, by nipkow
New Asm_full_simp_tac led to a loop.
1998-03-11, by nipkow
Mod because of new simplifier.
1998-03-10, by nipkow
Mod because of not1_or.
1998-03-10, by nipkow
Updated proofs because of new simplifier.
1998-03-10, by nipkow
Updated proofs because of new simplification tactics.
1998-03-10, by nipkow
Adapted proofs because of new simplification tactics.
1998-03-10, by nipkow
The new asm_lr_simp_tac is the old asm_full_simp_tac.
1998-03-10, by nipkow
renamed is_chain to chain, is_tord to tord, replaced chain_finite by chfin
1998-03-10, by oheimb
added not1_or and if_eq_cancel to simpset()
1998-03-10, by oheimb
added not1_or and if_eq_cancel to simpset()
1998-03-10, by oheimb
new rewrite rules not1_or, not2_or, and if_eq_cancel
1998-03-10, by oheimb
renamed smart_tac to force_tac, slight improvement of force_tac
1998-03-10, by oheimb
Asm_full_simp_tac now reorients asm c = t to t = c.
1998-03-10, by nipkow
adhoc fix of is_blank;
1998-03-10, by wenzelm
New scanner in abstract form.
1998-03-10, by nipkow
New simplifier flag for mutual simplification.
1998-03-10, by nipkow
Removed expand_split from simpset.
1998-03-10, by nipkow
removed pred;
1998-03-09, by wenzelm
eliminated pred function;
1998-03-09, by wenzelm
Symbol.explode;
1998-03-09, by wenzelm
replaced $LOGNAME by $USER;
1998-03-09, by wenzelm
tuned;
1998-03-09, by wenzelm
Symbol.is_*;
1998-03-09, by wenzelm
adapted to new scanner, baroque chars;
1998-03-09, by wenzelm
Symbol.input;
1998-03-09, by wenzelm
adapted to symbols, scan;
1998-03-09, by wenzelm
Generic scanners (for potentially infinite input) -- replaces Scanner;
1998-03-09, by wenzelm
adapted to new scanner and abroque chars;
1998-03-09, by wenzelm
read_var;
1998-03-09, by wenzelm
Symbol.output;
1998-03-09, by wenzelm
tuned syntax error msg;
1998-03-09, by wenzelm
Symbol.explode;
1998-03-09, by wenzelm
scan.ML, symbol.ML;
1998-03-09, by wenzelm
adapted to new scanners and baroque chars;
1998-03-09, by wenzelm
tuned some names;
1998-03-09, by wenzelm
adapted to baroque chars;
1998-03-09, by wenzelm
added merge_alists;
1998-03-09, by wenzelm
Syntax.indexname;
1998-03-09, by wenzelm
tuned comment;
1998-03-09, by wenzelm
tuned;
1998-03-09, by wenzelm
replaced Pure/Syntax/symbol_font.ML by Pure/Syntax/symbol.ML;
1998-03-09, by wenzelm
replaced Pure/Syntax/symbol_font.ML by Pure/Syntax/symbol.ML;
1998-03-09, by wenzelm
Removed `addsplits [expand_if]'
1998-03-07, by nipkow
added clasimp.ML;
1998-03-06, by wenzelm
Removed superfluous `op'
1998-03-06, by nipkow
*** empty log message ***
1998-03-06, by nipkow
Added delspilts, Addsplits, Delsplits.
1998-03-06, by nipkow
expand_if is now by default part of the simpset.
1998-03-06, by nipkow
New theorem and simprules
1998-03-05, by paulson
Reorganized simplifier. May now reorient rules.
1998-03-04, by nipkow
Reorganized simplifier. May now reorient rules.
1998-03-04, by nipkow
Reorganized simplifier. May now reorient rules.
1998-03-04, by nipkow
Better simplification allows deletion of parts of proofs
1998-03-03, by paulson
New theorem
1998-03-03, by paulson
New theorems
1998-03-03, by paulson
New theorems; tidied
1998-03-03, by paulson
New theorem diff_Suc_le_Suc_diff; tidied another proof
1998-03-03, by paulson
auto generated
1998-03-03, by paulson
Modified def.
1998-02-28, by nipkow
Splitters via named loopers.
1998-02-28, by nipkow
Little reorganization. Loop tactics have names now.
1998-02-28, by nipkow
Tried to reorganize rewriter a little. More to be done.
1998-02-28, by nipkow
added minimal description of rep_cs: corrections
1998-02-27, by oheimb
added minimal description of rep_cs
1998-02-27, by oheimb
added minimal description of rep_ss
1998-02-27, by oheimb
"choice" moved to Set.ML
1998-02-27, by paulson
New absorbsion laws, etc
1998-02-27, by paulson
Vimage
1998-02-27, by paulson
New vimage laws
1998-02-27, by paulson
added smart_tac
1998-02-26, by oheimb
removed superfluous addss
1998-02-26, by oheimb
New theory, Vimage
1998-02-26, by paulson
Proved choice and bchoice; changed Fun.thy -> thy
1998-02-26, by paulson
*** empty log message ***
1998-02-26, by wenzelm
added clasimp.ML;
1998-02-26, by wenzelm
renamed rep_claset to rep_cs
1998-02-25, by oheimb
factored out common code of HOL/simpdata.ML and FOL/simpdata.ML concerning
1998-02-25, by oheimb
changed wrapper mechanism of classical reasoner
1998-02-25, by oheimb
added split_all_tac to claset()
1998-02-25, by oheimb
changed wrapper mechanism of classical reasoner
1998-02-25, by oheimb
New theory of the inverse image of a function
1998-02-24, by paulson
Added some lemmas.
1998-02-24, by nipkow
Catches bad elim rules, handling exception OPTION
1998-02-23, by paulson
New laws for union
1998-02-23, by paulson
New laws for id
1998-02-23, by paulson
New induction schemas for lists (length and snoc).
1998-02-22, by nipkow
*** empty log message ***
1998-02-20, by nipkow
Congruence rules use == in premises now.
1998-02-20, by nipkow
Congruence rules use == in premises now.
1998-02-20, by nipkow
minor improvements
1998-02-20, by oheimb
re-arranged bindings for many function keys
1998-02-20, by oheimb
extended input syntax to handle names of special keys
1998-02-20, by oheimb
moved Ctrl entry before Alt entry
1998-02-20, by oheimb
New theorem eq_imp_le
1998-02-20, by paulson
Four new Union/Intersection laws
1998-02-19, by paulson
corrected problem with auto_tac: now uses a variant of depth_tac that avoids
1998-02-18, by oheimb
added New Jersey mirror;
1998-02-18, by wenzelm
Improved loop-test for rewrite rules a little.
1998-02-18, by nipkow
tuned comment;
1998-02-18, by wenzelm
added append (curried);
1998-02-13, by wenzelm
*** empty log message ***
1998-02-12, by wenzelm
Sign.merge vs. Sign.nontriv_merge;
1998-02-12, by wenzelm
tuned comments;
1998-02-12, by wenzelm
oops;
1998-02-12, by wenzelm
tuned print_cs;
1998-02-12, by wenzelm
updated;
1998-02-12, by wenzelm
tuned;
1998-02-12, by wenzelm
added explicit signature;
1998-02-12, by wenzelm
improved comments;
1998-02-12, by wenzelm
fixed add_trrules: intern root;
1998-02-12, by wenzelm
export map_trrule;
1998-02-12, by wenzelm
tuned add_trrules;
1998-02-12, by wenzelm
improved is_letter etc.;
1998-02-12, by wenzelm
New Addsimps for Compl rules
1998-02-10, by paulson
New AddIffs le_0_eq and neq0_conv
1998-02-10, by paulson
Replaced ALLNEWSUBGOALS by THEN_ALL_NEW
1998-02-09, by nipkow
Used THEN_ALL_NEW.
1998-02-09, by nipkow
moved freeze_thaw to drule.ML
1998-02-07, by paulson
Tidying; rotate_prems; moved freeze_thaw from tactic.ML
1998-02-07, by paulson
AC and other rewrite rules for Un and Int
1998-02-07, by paulson
auto update
1998-02-07, by paulson
Added reference to rotate_prems
1998-02-07, by paulson
filter_size -> length_filter
1998-02-06, by nipkow
Added `remdups'
1998-02-06, by nipkow
added Vartab: TABLE;
1998-02-06, by wenzelm
added param;
1998-02-05, by wenzelm
added THEN_ALL_NEW;
1998-02-05, by wenzelm
New theorem Image_id
1998-02-05, by paulson
New theorem order_eq_refl
1998-02-05, by paulson
New max, min theorems
1998-02-05, by paulson
Added some more explicit guarantees of key secrecy for agents
1998-02-05, by paulson
Fixed a lot of overfull and underfull lines (hboxes)
1998-02-05, by paulson
Updated the description of how to set up hyp_subst_tac
1998-02-05, by paulson
New example, Pow_Sigma_bij
1998-02-02, by paulson
fixed WWW links
1998-02-02, by paulson
Three new facts about Image
1998-02-02, by paulson
Replaced \\1 by $1 as Perl itself asked me to...
1998-02-02, by paulson
Fixed the description of recdef
1998-01-30, by paulson
tuned msgs;
1998-01-30, by wenzelm
improved tracing of rewrite rule application;
1998-01-30, by wenzelm
removed dead messy code;
1998-01-30, by wenzelm
added read_var;
1998-01-30, by wenzelm
tuned;
1998-01-30, by wenzelm
Updated MOD reference
1998-01-23, by paulson
added symbols syntax;
1998-01-21, by wenzelm
reorganized into individual theories;
1998-01-20, by wenzelm
tuned;
1998-01-19, by wenzelm
make images;
1998-01-19, by wenzelm
tuned URL;
1998-01-15, by wenzelm
polyml-3.1;
1998-01-15, by wenzelm
obsolete;
1998-01-15, by wenzelm
added thms wrt weakening and strengthening in Abstraction;
1998-01-14, by mueller
New Jersey inactive;
Isabelle98
1998-01-14, by wenzelm
HOL/record;
1998-01-14, by wenzelm
error with instantiantion of sub-records removed
1998-01-14, by narasche
added record.ML;
1998-01-14, by wenzelm
tuned;
1998-01-14, by wenzelm
added unit and prod stuff;
1998-01-14, by wenzelm
fixed Id;
1998-01-14, by wenzelm
smlnj-110 factory default;
1998-01-14, by wenzelm
added of_sort;
1998-01-14, by wenzelm
added base_path;
1998-01-13, by wenzelm
added simulations files to IOA;
1998-01-13, by mueller
added forward simulation correectness;
1998-01-13, by mueller
Simplification: sel make and update make
1998-01-13, by narasche
added abstraction files;
1998-01-12, by mueller
added further IOA liles;
1998-01-12, by mueller
updated to Isabelle98;
1998-01-12, by wenzelm
tuned;
1998-01-12, by wenzelm
added files containing temproal logic and abstraction;
1998-01-12, by mueller
Delsimprocs nat_cancel;
1998-01-12, by wenzelm
tuned;
1998-01-12, by wenzelm
Tidying, mostly to do with handling a more specific version of Fake_parts_insert
1998-01-12, by paulson
tuned;
1998-01-12, by wenzelm
tuned;
1998-01-12, by wenzelm
fixed author;
1998-01-12, by wenzelm
Simplified proofs by omitting PA = {|XA, ...|} from RA2
1998-01-10, by paulson
trivial tidy
1998-01-10, by paulson
tuned;
1998-01-09, by wenzelm
automatic index.html patch;
1998-01-09, by wenzelm
tuned;
1998-01-09, by wenzelm
tuned ISABELLE_TMP_PREFIX;
1998-01-09, by wenzelm
thm_ord;
1998-01-09, by wenzelm
eliminated make_ord;
1998-01-09, by wenzelm
ISABELLE_TMP_PREFIX: $LOGNAME
1998-01-09, by wenzelm
several minor updates;
1998-01-09, by wenzelm
tuned;
1998-01-08, by wenzelm
index.html for Isabelle Distribution Area;
1998-01-08, by wenzelm
updated to Isabelle98;
1998-01-08, by wenzelm
tuned;
1998-01-08, by wenzelm
fixed thm_less;
1998-01-08, by wenzelm
Expressed most Oops rules using Notes instead of Says, and other tidying
1998-01-08, by paulson
added split_paired_Ex to the implicit simpset
1998-01-08, by oheimb
added select_equality to the implicit claset
1998-01-08, by oheimb
added select_equality to the implicit claset
1998-01-08, by oheimb
added newline at end of file
1998-01-08, by oheimb
*** empty log message ***
1998-01-08, by oheimb
streamlined specification of included theories
1998-01-08, by oheimb
corrected Title
1998-01-08, by oheimb
removed obsolete comment
1998-01-08, by oheimb
added Univalent
1998-01-08, by oheimb
removed Eps_eq, ex1_Eps_eq, and some unnecessary parentheses
1998-01-08, by oheimb
added update_same, update_other, update_triv, and map_of_SomeD
1998-01-08, by oheimb
replaced fn _ => by K
1998-01-08, by oheimb
*** empty log message ***
1998-01-08, by wenzelm
New rule: image_subset
1998-01-08, by paulson
Restored the ciphertext in OR4 in order to make the spec closer to that in
1998-01-08, by paulson
Tidied by adding more default simprules
1998-01-08, by paulson
adapted to new split order;
1998-01-07, by wenzelm
adapted to new sort function;
1998-01-07, by wenzelm
improved targets;
1998-01-07, by wenzelm
tuned;
1998-01-06, by wenzelm
added -u option (again);
1998-01-05, by wenzelm
Now calls Blast_tac more often
1998-01-05, by paulson
obsolete;
1998-01-02, by wenzelm
less
more
|
(0)
-3000
-1000
-480
+480
+1000
+3000
+10000
+30000
tip