Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-3000
-1000
-112
+112
+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.
renamed 'with' to 'using';
1999-07-19, by wenzelm
*** empty log message ***
1999-07-19, by wenzelm
NatBin: binary arithmetic for the naturals
1999-07-19, by paulson
examples of arithmetic on the naturals
1999-07-19, by paulson
deleted a reference to "nat", now erroneous because "nat" is a function
1999-07-19, by paulson
many new laws about div and mod
1999-07-19, by paulson
new theorem zless_zero_nat
1999-07-19, by paulson
removal of rewrites for Suc(Suc(Suc...)))
1999-07-19, by paulson
NatBin: binary arithmetic for the naturals
1999-07-19, by paulson
getting rid of qed_goal
1999-07-19, by paulson
getting rid of qed_goal
1999-07-19, by paulson
new division laws taking advantage of (m div 0) = 0 and (m mod 0) = m
1999-07-19, by paulson
Modifid length_tl
1999-07-18, by nipkow
adapted to dest_keywords, dest_parsers;
1999-07-16, by wenzelm
separate command tokens;
1999-07-16, by wenzelm
tuned dest_lexicon;
1999-07-16, by wenzelm
tuned;
1999-07-16, by wenzelm
removed break;
1999-07-16, by wenzelm
removed BREAK, ROLLBACK;
1999-07-16, by wenzelm
structure LocalDefs = LocalDefs;
1999-07-16, by wenzelm
Exported function unify_consts (workaround to avoid inconsistently
1999-07-16, by berghofe
Added new example (infinitely branching trees).
1999-07-16, by berghofe
Infinitely branching trees.
1999-07-16, by berghofe
Replaced datatype_info by datatype_info_err.
1999-07-16, by berghofe
- Now also supports arbitrarily branching datatypes.
1999-07-16, by berghofe
- Datatype package now also supports arbitrarily branching datatypes
1999-07-16, by berghofe
Added some definitions and theorems needed for the
1999-07-16, by berghofe
Some rather large datatype examples (from John Harrison).
1999-07-16, by berghofe
improved print_thms;
1999-07-15, by wenzelm
export init_state;
1999-07-15, by wenzelm
more renaming of theorems from _nat to _int (corresponding to a function that
1999-07-15, by paulson
more renaming of theorems from _nat to _int (corresponding to a function that
1999-07-15, by paulson
qed_goal -> Goal; new theorems nat_le_0, nat_le_eq_zle and zdiff_int
1999-07-15, by paulson
qed_goal -> Goal
1999-07-15, by paulson
tuned;
1999-07-14, by wenzelm
tuned comments;
1999-07-14, by wenzelm
tuned contradiction method;
1999-07-14, by wenzelm
improved comment;
1999-07-14, by wenzelm
more marg_comments;
1999-07-14, by wenzelm
Deriving rules in Isabelle;
1999-07-14, by wenzelm
rewrite add1_zle_eq is no longer in the default simpset
1999-07-14, by paulson
optimization for division by powers of 2
1999-07-14, by paulson
new montonicity theorems
1999-07-14, by paulson
new constant folding rewrites
1999-07-14, by paulson
handle cgoal;
1999-07-13, by wenzelm
added mk_cgoal, assume_goal;
1999-07-13, by wenzelm
same_tac;
1999-07-13, by wenzelm
change to force (m div 0 = 0)
1999-07-13, by paulson
many new theorems
1999-07-13, by paulson
renamed inj_nat to inj_int
1999-07-13, by paulson
new monotonicity theorems
1999-07-13, by paulson
new theorem zmult_eq_0_iff
1999-07-13, by paulson
renamed sort "numeral" to "number"
1999-07-13, by paulson
simplified the <= monotonicity proof
1999-07-13, by paulson
local qeds: print rule;
1999-07-12, by wenzelm
added show_hyps flag;
1999-07-12, by wenzelm
local qed; print rule;
1999-07-12, by wenzelm
term/prop: include number;
1999-07-12, by wenzelm
added show_hyps flag;
1999-07-12, by wenzelm
export assumption_tac;
1999-07-12, by wenzelm
removed merge_theories;
1999-07-12, by wenzelm
removed metacuts_tac;
1999-07-12, by wenzelm
tmp_path: *add* path;
1999-07-12, by wenzelm
thms_containing: undeclared consts error;
1999-07-12, by wenzelm
removed pretty_thm_no_hyps (again);
1999-07-12, by wenzelm
removed merge_theories;
1999-07-12, by wenzelm
may get BASH_PATH etc. from env;
1999-07-12, by wenzelm
new theorems for the "at most" relation
1999-07-12, by paulson
def: ==;
1999-07-12, by wenzelm
tuned Interrupt msgs;
1999-07-10, by wenzelm
pass exn;
1999-07-10, by wenzelm
handle THM exn;
1999-07-10, by wenzelm
handle THM/TERM exn;
1999-07-10, by wenzelm
dup_elim: use try to handle general exn;
1999-07-10, by wenzelm
handle THM exn;
1999-07-10, by wenzelm
fixed interrupts (eliminated races);
1999-07-10, by wenzelm
defer_tac: use try for general exn handling;
1999-07-10, by wenzelm
Symtab.lookup_multi;
1999-07-10, by wenzelm
more specific exn;
1999-07-10, by wenzelm
err_method: pass exn;
1999-07-10, by wenzelm
prove_goalw_cterm_general: pass exeption;
1999-07-10, by wenzelm
try/can: pass Interrupt and ERROR;
1999-07-10, by wenzelm
rmdir pdf;
1999-07-09, by wenzelm
mono: extra I/E;
1999-07-09, by wenzelm
mono: AddXI/Es;
1999-07-09, by wenzelm
type claset: added extra I/E rules;
1999-07-09, by wenzelm
added Isar/local_defs.ML;
1999-07-09, by wenzelm
added 'def';
1999-07-09, by wenzelm
added local_def(_i);
1999-07-09, by wenzelm
global_qed: removed alt_name, alt_att;
1999-07-09, by wenzelm
global_qed: removed alt_name, alt_att;
1999-07-09, by wenzelm
added termp;
1999-07-09, by wenzelm
COMP: optional position;
1999-07-09, by wenzelm
write_keywords: default file name;
1999-07-09, by wenzelm
added compose_single;
1999-07-09, by wenzelm
added HOL.trans;
1999-07-09, by wenzelm
removed qed_with;
1999-07-09, by wenzelm
faster division algorithm; monotonicity of div in 2nd arg
1999-07-09, by paulson
more monotonicity laws for times
1999-07-09, by paulson
products of signs as equivalences
1999-07-09, by paulson
-B option;
1999-07-08, by wenzelm
removed old version;
1999-07-08, by wenzelm
tuned indentation;
1999-07-08, by wenzelm
added export_chain;
1999-07-08, by wenzelm
propp: 'concl' patterns;
1999-07-08, by wenzelm
propp: 'concl' patterns;
1999-07-08, by wenzelm
terminal_proof: 2nd method;
1999-07-08, by wenzelm
'export';
1999-07-08, by wenzelm
propp: 'concl' patterns;
1999-07-08, by wenzelm
propp: 'concl' patterns;
1999-07-08, by wenzelm
improved error msgs of cterm_instantiate;
1999-07-08, by wenzelm
aprop: ??id, ...;
1999-07-08, by wenzelm
less
more
|
(0)
-3000
-1000
-112
+112
+1000
+3000
+10000
+30000
tip