Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-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.
adapted tuple syntax;
2000-07-16, by wenzelm
tuned;
2000-07-16, by wenzelm
use pair_tac;
2000-07-16, by wenzelm
use split syntax;
2000-07-16, by wenzelm
fixed tuple translations;
2000-07-16, by wenzelm
defs (overloaded);
2000-07-16, by wenzelm
added is_unitT;
2000-07-16, by wenzelm
instance unit :: finite;
2000-07-16, by wenzelm
more robust tuple syntax (still improper, though!);
2000-07-16, by wenzelm
improved unit theory: unit_all_eq1, unit_all_eq2, split_all_tac;
2000-07-16, by wenzelm
added syntax for proper / improper selector functions;
2000-07-16, by wenzelm
tuned;
2000-07-16, by wenzelm
tuned;
2000-07-16, by wenzelm
avoid 'split';
2000-07-16, by wenzelm
added Tuple.thy;
2000-07-16, by wenzelm
added ex/Tuple.thy;
2000-07-16, by wenzelm
syntax (symbols) "op o" moved from HOL to Fun;
2000-07-16, by wenzelm
added finite_unit;
2000-07-16, by wenzelm
AST translation rules no longer require constant head on LHS;
2000-07-16, by wenzelm
* tuned AST representation of nested pairs, avoiding bogus output in
2000-07-16, by wenzelm
corrections (cast relation, Prog.ML -> Decl.ML)
2000-07-14, by oheimb
improved add_edges_cyclic;
2000-07-14, by wenzelm
re-structuring MicroJava; added Example; corrected := syntax; simplfied cast
2000-07-14, by oheimb
added (surjective_pairing RS sym) to simpset
2000-07-14, by oheimb
strengthened rtranclD
2000-07-14, by oheimb
added option_map_o_sum_case (also to simpset)
2000-07-14, by oheimb
added sum_case_empty_empty (also to simpset)
2000-07-14, by oheimb
tuned syntax
2000-07-14, by oheimb
added hint on fun_sum
2000-07-14, by oheimb
added fun_upd2_simproc
2000-07-14, by oheimb
re-added subset_empty to simpset
2000-07-14, by oheimb
used bounded quantification in definition of guarantees and other minor
2000-07-14, by paulson
moved sublist from UNITY/AllocBase to List
2000-07-14, by paulson
AddIffs
2000-07-14, by paulson
parent should be Main
2000-07-14, by paulson
changed the quotient syntax from / to //
2000-07-14, by paulson
tuned cycle_msg;
2000-07-13, by wenzelm
updated;
2000-07-13, by wenzelm
HOL: the disjoint sum is now "<+>" instead of "Plus";
2000-07-13, by wenzelm
adapted PureThy.add_defs_i;
2000-07-13, by wenzelm
defs (overloaded);
2000-07-13, by wenzelm
tuned;
2000-07-13, by wenzelm
added read_xnum;
2000-07-13, by wenzelm
fix(_i): admit internal variables;
2000-07-13, by wenzelm
use ProofContext.bind_skolem;
2000-07-13, by wenzelm
defs: (overloaded) option;
2000-07-13, by wenzelm
eq_prop: strip_assums_concl;
2000-07-13, by wenzelm
tuned exceptions;
2000-07-13, by wenzelm
const_deps: unit Graph.T;
2000-07-13, by wenzelm
add_term_consts: ins_string;
2000-07-13, by wenzelm
add_defs(_i): overloaded option;
2000-07-13, by wenzelm
adapted PureThy.add_defs;
2000-07-13, by wenzelm
fixed comment;
2000-07-13, by wenzelm
adapted PureThy.add_defs_i;
2000-07-13, by wenzelm
use Syntax.read_xnum;
2000-07-13, by wenzelm
fixed simplified_cases;
2000-07-13, by wenzelm
fixed name: UN_empty3;
2000-07-13, by wenzelm
replaced infix Plus by <+>;
2000-07-13, by wenzelm
removed duplicate Compl_atMost;
2000-07-13, by wenzelm
fixed compose decl;
2000-07-13, by wenzelm
defs: (overloaded) option;
2000-07-13, by wenzelm
method cases/induct: (opaque) option;
2000-07-13, by wenzelm
defs (overloaded);
2000-07-13, by wenzelm
removed now-redundant proof steps
2000-07-13, by paulson
added an important default rule
2000-07-13, by paulson
fixed a failing proof
2000-07-13, by paulson
le_refl_iff as default rule
2000-07-13, by paulson
removed needless premises
2000-07-13, by paulson
AddIffs now available for FOL, ZF
2000-07-13, by paulson
added simp_case_tac;
2000-07-13, by wenzelm
use InductMethod.simp_case_tac;
2000-07-13, by wenzelm
tuned;
2000-07-13, by wenzelm
export thesisN separately;
2000-07-13, by wenzelm
prep rhs in original context;
2000-07-13, by wenzelm
RuleCases.make opaq;
2000-07-13, by wenzelm
bind_skolem;
2000-07-13, by wenzelm
invoke_case: bind_skolem;
2000-07-13, by wenzelm
"_i" arguments now expected to have skolems already internalized;
2000-07-13, by wenzelm
make: opaq flag;
2000-07-13, by wenzelm
added internal, dest_internal;
2000-07-13, by wenzelm
infix 'OF' is a version of 'MRS' with more appropriate argument order;
2000-07-12, by wenzelm
about.html -> logics.html
2000-07-12, by kleing
munich webserver is now sunbroy51
2000-07-12, by kleing
about -> logics, better access to online libraries
2000-07-12, by kleing
removal of (harmless) circular definitions
2000-07-10, by paulson
Tuned proof.
2000-07-09, by berghofe
Defs are now checked for circularity (if not overloaded).
2000-07-08, by nipkow
inter_sort: keep normal!
2000-07-07, by wenzelm
Tightened up check of types in constant defs.
2000-07-07, by nipkow
added type classes to constant's type
2000-07-07, by nipkow
skp; le;
2000-07-07, by bauerg
added dependency caveat
2000-07-07, by oheimb
added dependency caveat
2000-07-07, by oheimb
added IMP/Examples.ML dependence
2000-07-07, by oheimb
tuned msgs;
2000-07-06, by wenzelm
allow comment in more commands;
2000-07-06, by wenzelm
Isabelle99-1;
2000-07-06, by wenzelm
ADD -> IAdd
2000-07-06, by kleing
Removed some junk thms.
2000-07-06, by nipkow
added zabs to arith_tac
2000-07-06, by nipkow
Deleted list_case thms no subsumed by case_tac
2000-07-06, by nipkow
Now two split thms for same constant at different types is allowed.
2000-07-06, by nipkow
removal of batch style, and tidying
2000-07-06, by paulson
removal of batch style, and tidying
2000-07-06, by paulson
removal of batch style, and tidying
2000-07-06, by paulson
removal of batch style, and tidying
2000-07-06, by paulson
removed sorry;
2000-07-06, by bauerg
removed sorry;
2000-07-06, by bauerg
new ADD instruction
2000-07-06, by kleing
removal of batch style, and tidying
2000-07-06, by paulson
fixed typos reported by Jeremy Dawson
2000-07-06, by paulson
added;
2000-07-06, by bauerg
completed TYPES version of HahnBanach;
2000-07-06, by bauerg
*** empty log message ***
2000-07-06, by nipkow
Compatibility file for Moscow ML 2.00;
2000-07-06, by wenzelm
run Moscow ML 2.00 --- does not handle saved images (yet!?);
2000-07-06, by wenzelm
Moscow ML 2.00 or later (experimental!);
2000-07-06, by wenzelm
more tidying. also generalized some tactics to prove "Type A" and
2000-07-05, by paulson
disambiguated := ; added Examples (factorial)
2000-07-05, by oheimb
removed batch proofs
2000-07-05, by paulson
less
more
|
(0)
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip