mueller [Wed, 30 Apr 1997 11:24:14 +0200] rev 3072
Old ABP files now running under the IOA meta theory based on HOLCF;
mueller [Wed, 30 Apr 1997 11:20:15 +0200] rev 3071
New meta theory for IOA based on HOLCF.
wenzelm [Wed, 30 Apr 1997 11:11:57 +0200] rev 3070
improved display of non-ASCII chars;
wenzelm [Tue, 29 Apr 1997 17:44:26 +0200] rev 3069
fixed enc_start;
wenzelm [Tue, 29 Apr 1997 17:38:02 +0200] rev 3068
deactivated new symbols (not yet printable on xterm, emacs);
wenzelm [Tue, 29 Apr 1997 17:23:53 +0200] rev 3067
renamed \<choice> to \<orelse>;
wenzelm [Tue, 29 Apr 1997 17:14:06 +0200] rev 3066
added \<orelse> symbols syntax for case;
wenzelm [Tue, 29 Apr 1997 17:13:41 +0200] rev 3065
added \<langle>, \<rangle> symbols syntax;
wenzelm [Tue, 29 Apr 1997 16:39:13 +0200] rev 3064
added new chars;
wenzelm [Tue, 29 Apr 1997 16:38:16 +0200] rev 3063
is_blank: added space2 (160);
wenzelm [Fri, 25 Apr 1997 18:11:22 +0200] rev 3062
improved DVI_VIEWER default;
wenzelm [Fri, 25 Apr 1997 17:50:55 +0200] rev 3061
improved tmp comment;
wenzelm [Fri, 25 Apr 1997 17:28:43 +0200] rev 3060
removed -norc;
slotosch [Fri, 25 Apr 1997 15:33:19 +0200] rev 3059
used explcite tactics in instances (since ax_per_trans "loops")
slotosch [Fri, 25 Apr 1997 15:31:51 +0200] rev 3058
changed Domain->Dom for SML/NJ
wenzelm [Fri, 25 Apr 1997 15:24:07 +0200] rev 3057
removed -c option;
wenzelm [Fri, 25 Apr 1997 15:18:58 +0200] rev 3056
removed -c option;
wenzelm [Fri, 25 Apr 1997 15:10:52 +0200] rev 3055
removed COPYDB flag;
wenzelm [Fri, 25 Apr 1997 15:08:52 +0200] rev 3054
removed -c option;
wenzelm [Fri, 25 Apr 1997 15:08:25 +0200] rev 3053
obsolete;
wenzelm [Fri, 25 Apr 1997 15:06:21 +0200] rev 3052
no longer forces default;
wenzelm [Fri, 25 Apr 1997 14:12:33 +0200] rev 3051
misc tuning;
oheimb [Fri, 25 Apr 1997 11:11:52 +0200] rev 3050
removed one blank at end of line 37
wenzelm [Thu, 24 Apr 1997 19:47:53 +0200] rev 3049
refer to SOME, NONE on top-level;
wenzelm [Thu, 24 Apr 1997 19:46:24 +0200] rev 3048
adapted for 1.09.27 (and later);
wenzelm [Thu, 24 Apr 1997 19:46:05 +0200] rev 3047
open General (type option is in Option in the newer versions, but always
the top-level);
wenzelm [Thu, 24 Apr 1997 19:41:00 +0200] rev 3046
adapted to SML/NJ 1.09.27;
minor cleanup;
nipkow [Thu, 24 Apr 1997 19:08:32 +0200] rev 3045
Added 'induct_tac'
nipkow [Thu, 24 Apr 1997 18:51:14 +0200] rev 3044
Updates because nat_ind_tac no longer appends "1" to the ind.var.
wenzelm [Thu, 24 Apr 1997 18:44:32 +0200] rev 3043
removed space;
nipkow [Thu, 24 Apr 1997 18:38:30 +0200] rev 3042
induct_tac
mueller [Thu, 24 Apr 1997 18:07:35 +0200] rev 3041
expandshort
nipkow [Thu, 24 Apr 1997 18:06:46 +0200] rev 3040
Introduced a generic "induct_tac" which picks up the right induction scheme
automatically. Also changed nat_ind_tac, which does no longer append a "1" to
the name of the induction variable. This caused some changes...
nipkow [Thu, 24 Apr 1997 18:03:23 +0200] rev 3039
get_thydata accesses the second component of the data field. This component
used to be empty until set at the end of loading an ML file. Now the second
component is already set when the thy file has ben read.
mueller [Thu, 24 Apr 1997 18:00:22 +0200] rev 3038
Main changes are:
- Lemmas for blift and plift are deleted
- added split_tac for If (via If2, as If does not begin with a constant)
- added new lemmata relating TT, FF and booleans:
Def_bool1, Def_bool2, Def_bool3,Def_bool4
They are added to !simpset, but should not cause difficulties
- added lemma andalso_or relating | on booleans and andalso on truth values
- deleted If_and_if and andalso from !simpset: Pay attention, may kill your proofs!
- added adm lemmas for (f x)~=TT and (f x)~=FF.
nipkow [Thu, 24 Apr 1997 17:59:55 +0200] rev 3037
rename_params_rule used to check if the new name clashed with a free name in
the whole goal state. Now checks only the subgoal concerned.
mueller [Thu, 24 Apr 1997 17:51:27 +0200] rev 3036
deleted definitions for blift and plift
mueller [Thu, 24 Apr 1997 17:50:34 +0200] rev 3035
Complete Redesign of Theory, main points are:
- Extension of the continuity prover:
* Lemmas about continuity of flift1 and flift2 are generalized
* Lemmas about continuity of mixed definitions of HOL and LCF terms generalized
Pay attention: Sometimes proofs are shorter now!
- a number of new lemmas concerning flift1, flift2, Def and Undef,
Def_less_is_eq (Def x << y = (Def x = y)) and lemmas characterizing flift1 and flift2
are added to !simpset
Pay attention: Sometimes proofs are shorter now!
- added tactic def_tac for eliminating x~=UU in assumptions
mueller [Thu, 24 Apr 1997 17:40:30 +0200] rev 3034
added liftpair definition
mueller [Thu, 24 Apr 1997 17:38:33 +0200] rev 3033
only in comments
mueller [Thu, 24 Apr 1997 17:35:47 +0200] rev 3032
minor changes due to more powerful continuity check in Lift3.ML
mueller [Thu, 24 Apr 1997 17:04:07 +0200] rev 3031
added some comments;
paulson [Thu, 24 Apr 1997 11:21:46 +0200] rev 3030
Addition of printed tracing. Also some tidying
paulson [Thu, 24 Apr 1997 11:20:56 +0200] rev 3029
A bit of tidying
oheimb [Thu, 24 Apr 1997 10:40:01 +0200] rev 3028
added dependencies on ax_ops/*.ML and domain/*.ML
oheimb [Thu, 24 Apr 1997 10:39:00 +0200] rev 3027
changed priority of '%': now no parenteses needed for '[...] == %x. [...]'
slotosch [Thu, 24 Apr 1997 09:34:59 +0200] rev 3026
moved antisym_less_inverse,box_less from Porder.ML to Porder0.ML
nipkow [Wed, 23 Apr 1997 13:23:05 +0200] rev 3025
Added NatDef
paulson [Wed, 23 Apr 1997 11:20:18 +0200] rev 3024
Necessary inclusion of depth bound into blast_tac call
paulson [Wed, 23 Apr 1997 11:18:29 +0200] rev 3023
Ran expandshort
paulson [Wed, 23 Apr 1997 11:12:10 +0200] rev 3022
Unfortunately, the \\< syntax does not always accept the beginning of a line
paulson [Wed, 23 Apr 1997 11:11:38 +0200] rev 3021
Loop detection: before expanding a haz formula, see whether it is a duplicate
and, if so, delete it.
Recursion detection: transitivity and similar rules, when applied, put the
new formulae at the end of a branch and not at the front (in effect).
paulson [Wed, 23 Apr 1997 11:05:52 +0200] rev 3020
Made a proof search more deterministic
paulson [Wed, 23 Apr 1997 11:05:18 +0200] rev 3019
Improved indentation of #34
paulson [Wed, 23 Apr 1997 11:02:19 +0200] rev 3018
Ran expandshort
paulson [Wed, 23 Apr 1997 11:00:48 +0200] rev 3017
Fixed typos in comment
paulson [Wed, 23 Apr 1997 10:54:22 +0200] rev 3016
Conversion to use blast_tac
paulson [Wed, 23 Apr 1997 10:52:49 +0200] rev 3015
Ran expandshort
paulson [Wed, 23 Apr 1997 10:49:01 +0200] rev 3014
Moved diamond_trancl (which is independent of the rest) to the top
paulson [Wed, 23 Apr 1997 10:47:36 +0200] rev 3013
Ran expandshort
wenzelm [Wed, 23 Apr 1997 10:08:51 +0200] rev 3012
simprocs called with eta contracted subterm;
nipkow [Wed, 23 Apr 1997 09:14:56 +0200] rev 3011
Tidied up.
wenzelm [Tue, 22 Apr 1997 18:05:42 +0200] rev 3010
fixed bash-2.0 problem;
wenzelm [Tue, 22 Apr 1997 11:49:55 +0200] rev 3009
improved fontserver example;
paulson [Tue, 22 Apr 1997 11:45:22 +0200] rev 3008
Ran expandshort
wenzelm [Tue, 22 Apr 1997 11:37:12 +0200] rev 3007
removed -norc;
wenzelm [Tue, 22 Apr 1997 11:25:45 +0200] rev 3006
tuned;
nipkow [Mon, 21 Apr 1997 13:49:40 +0200] rev 3005
Modified credits.
paulson [Mon, 21 Apr 1997 12:16:29 +0200] rev 3004
New elimination rule for "unique existence"
paulson [Mon, 21 Apr 1997 12:16:04 +0200] rev 3003
New introduction rule for "unique existence"
paulson [Mon, 21 Apr 1997 11:19:28 +0200] rev 3002
Reorganized under headings. Also documented Blast_tac and LFilter
paulson [Mon, 21 Apr 1997 10:38:46 +0200] rev 3001
Tidied up the indentation
paulson [Mon, 21 Apr 1997 10:16:41 +0200] rev 3000
Moved blast_tac demo from ZF/func.ML to ZF/ex/misc.ML
paulson [Mon, 21 Apr 1997 10:16:01 +0200] rev 2999
Penalty for branching instantiations reduced from log3 to log4.
Now allows a branch to close by unifying an OConst with a Const.
paulson [Mon, 21 Apr 1997 10:15:00 +0200] rev 2998
New blast_tac demo
paulson [Mon, 21 Apr 1997 10:14:31 +0200] rev 2997
Without the type constraint, the inner equality was NOT a biconditional...
paulson [Mon, 21 Apr 1997 10:13:47 +0200] rev 2996
Now faster without calling Blast.depth_tac
paulson [Mon, 21 Apr 1997 10:12:40 +0200] rev 2995
Disabled the attempts for mutual induction to work so that single induction
involving sum types can work
nipkow [Fri, 18 Apr 1997 17:33:26 +0200] rev 2994
Tuple patterns are allowed now in `case'
nipkow [Fri, 18 Apr 1997 16:54:52 +0200] rev 2993
*** empty log message ***
wenzelm [Fri, 18 Apr 1997 12:01:12 +0200] rev 2992
print_goals: fixed show_sorts semantics;
wenzelm [Fri, 18 Apr 1997 11:58:38 +0200] rev 2991
tuned check_has_sort;
fixed norm_typ: also does norm_sort;
wenzelm [Fri, 18 Apr 1997 11:57:51 +0200] rev 2990
removed least_sort;
added of_sort;
wenzelm [Fri, 18 Apr 1997 11:55:14 +0200] rev 2989
tuned err msg;
paulson [Fri, 18 Apr 1997 11:54:54 +0200] rev 2988
Renamed sign constructors to eliminate clash with the Plus infix of Sum.thy
paulson [Fri, 18 Apr 1997 11:53:55 +0200] rev 2987
Now loads theory LList indirectly: via LFilter
paulson [Fri, 18 Apr 1997 11:53:16 +0200] rev 2986
Now uses some "case" syntax (but could use more)
paulson [Fri, 18 Apr 1997 11:52:44 +0200] rev 2985
New monotonicity theorems
paulson [Fri, 18 Apr 1997 11:52:19 +0200] rev 2984
New theory: a corecursive filter functional
paulson [Fri, 18 Apr 1997 11:48:16 +0200] rev 2983
Removed needless parentheses from translation
paulson [Fri, 18 Apr 1997 11:47:36 +0200] rev 2982
ex/LFilter is a new theory (and dependency)
paulson [Fri, 18 Apr 1997 11:47:11 +0200] rev 2981
Automatic update
wenzelm [Thu, 17 Apr 1997 19:05:01 +0200] rev 2980
tuned error msgs;
wenzelm [Thu, 17 Apr 1997 18:46:58 +0200] rev 2979
improved type check error messages;
wenzelm [Thu, 17 Apr 1997 18:45:43 +0200] rev 2978
renamed set_ap to setmp;
paulson [Thu, 17 Apr 1997 18:17:23 +0200] rev 2977
Automatic updates
paulson [Thu, 17 Apr 1997 18:16:12 +0200] rev 2976
Removed the \date{} command in order to put the date of typesetting on the
title page
paulson [Thu, 17 Apr 1997 18:10:49 +0200] rev 2975
Corrected the informal description of coinductive definition
paulson [Thu, 17 Apr 1997 18:10:12 +0200] rev 2974
Corrected the informal description of coinductive definition in sections 1
and 4.3, introducing the notion of "consistent with" a set of rules.
Final version for Milner Festschrift?
nipkow [Thu, 17 Apr 1997 17:54:21 +0200] rev 2973
Added ability to have case expressions involving tuples. (via translation)
wenzelm [Thu, 17 Apr 1997 14:41:56 +0200] rev 2972
tuned;
wenzelm [Thu, 17 Apr 1997 14:41:26 +0200] rev 2971
*** empty log message ***
wenzelm [Thu, 17 Apr 1997 14:41:08 +0200] rev 2970
added fixencoding note;
wenzelm [Thu, 17 Apr 1997 10:40:26 +0200] rev 2969
fixed ISAMODE_HOME;
wenzelm [Thu, 17 Apr 1997 10:30:57 +0200] rev 2968
eliminated PLATFORM;
wenzelm [Wed, 16 Apr 1997 18:53:36 +0200] rev 2967
removed lceil, rceil, lfloor, rfloor;
wenzelm [Wed, 16 Apr 1997 18:51:03 +0200] rev 2966
fixed perl path (for sunbroys);
wenzelm [Wed, 16 Apr 1997 18:46:01 +0200] rev 2965
improved translations for subset symbols syntax: constraints;
wenzelm [Wed, 16 Apr 1997 18:25:46 +0200] rev 2964
moved classes / sorts to sorts.ML;
moved (and reimplemented) type inference to type_infer.ML;
cleaned up type unification;
misc cleanup and tuning;
wenzelm [Wed, 16 Apr 1997 18:23:25 +0200] rev 2963
renamed subclass to classrel;
tune type checking error msgs;
wenzelm [Wed, 16 Apr 1997 18:22:10 +0200] rev 2962
Sorts.str_of_sort;
wenzelm [Wed, 16 Apr 1997 18:21:00 +0200] rev 2961
Sorts.str_of_arity;
wenzelm [Wed, 16 Apr 1997 18:17:38 +0200] rev 2960
added sorts.ML, type_infer.ML;
wenzelm [Wed, 16 Apr 1997 18:16:45 +0200] rev 2959
tuned type of eq_ix, mem_ix;
wenzelm [Wed, 16 Apr 1997 18:16:02 +0200] rev 2958
improved inc, dec;
added set_ap;
wenzelm [Wed, 16 Apr 1997 18:15:32 +0200] rev 2957
Type inference (isolated from type.ML, completely reimplemented).
wenzelm [Wed, 16 Apr 1997 18:14:43 +0200] rev 2956
Type classes and sorts (isolated from type.ML).
wenzelm [Wed, 16 Apr 1997 18:13:12 +0200] rev 2955
improved;
paulson [Tue, 15 Apr 1997 10:23:38 +0200] rev 2954
Partially converted to call blast_tac
paulson [Tue, 15 Apr 1997 10:23:17 +0200] rev 2953
Addition of blast_tac benchmark
paulson [Tue, 15 Apr 1997 10:22:50 +0200] rev 2952
Changed penalty from log2 to log3
paulson [Tue, 15 Apr 1997 10:19:14 +0200] rev 2951
An extra call to blast_tac (illustrating a need for type instantiation)
paulson [Tue, 15 Apr 1997 10:18:01 +0200] rev 2950
Now puts basic rewrites for lappend & lmap into the simpset
paulson [Tue, 15 Apr 1997 10:17:15 +0200] rev 2949
Removed "AddSDs [Scons_inject];" because
(a) IT WAS WRONG (should have been AddSEs)
(b) It was redundant (due to the AddIffs [...,Scons_Scons_eq])
paulson [Tue, 15 Apr 1997 10:15:09 +0200] rev 2948
Moved expand_case_tac from Auth/Message.ML to simpdata.ML
wenzelm [Mon, 14 Apr 1997 10:28:21 +0200] rev 2947
no longer includes ~/.emacs;
wenzelm [Sun, 13 Apr 1997 19:16:25 +0200] rev 2946
fixed file name;
wenzelm [Sun, 13 Apr 1997 19:15:07 +0200] rev 2945
GENERATED TEXT;
wenzelm [Sun, 13 Apr 1997 19:12:37 +0200] rev 2944
tuned format;
wenzelm [Sun, 13 Apr 1997 19:11:32 +0200] rev 2943
GENERATED TEXT;
wenzelm [Sun, 13 Apr 1997 19:10:54 +0200] rev 2942
GENERATED TEXT;
wenzelm [Sun, 13 Apr 1997 19:10:27 +0200] rev 2941
fixencoding - fix references to isabelle font encoding;
wenzelm [Sat, 12 Apr 1997 20:02:06 +0200] rev 2940
tuned comments;
wenzelm [Sat, 12 Apr 1997 20:01:38 +0200] rev 2939
misc improvement;
wenzelm [Sat, 12 Apr 1997 20:00:11 +0200] rev 2938
Setup GNU Emacs for Isabelle environment.
wenzelm [Sat, 12 Apr 1997 19:59:44 +0200] rev 2937
tuned;
wenzelm [Fri, 11 Apr 1997 17:30:15 +0200] rev 2936
fixed { ... } shell syntax to accomodate bash 2.x;
paulson [Fri, 11 Apr 1997 15:21:36 +0200] rev 2935
Yet more fast_tac->blast_tac, and other tidying
wenzelm [Fri, 11 Apr 1997 11:33:51 +0200] rev 2934
tuned error msg;
paulson [Thu, 10 Apr 1997 18:07:27 +0200] rev 2933
Updated discussion and references for inductive definitions
nipkow [Thu, 10 Apr 1997 14:26:01 +0200] rev 2932
Deleted stupid proof at the end not needed anywhere.
nipkow [Thu, 10 Apr 1997 12:21:21 +0200] rev 2931
Mod because of "Turned Addsimps into AddIffs for datatype laws."
nipkow [Thu, 10 Apr 1997 12:20:55 +0200] rev 2930
Turned Addsimps into AddIffs for datatype laws.
paulson [Thu, 10 Apr 1997 10:55:37 +0200] rev 2929
Changed some fast_tac to blast_tac
nipkow [Thu, 10 Apr 1997 09:08:05 +0200] rev 2928
Added trace output and replaced fast_tac set_cs by Fast_tac.
oheimb [Wed, 09 Apr 1997 15:56:53 +0200] rev 2927
replaced 'addwrapper' and 'addWrapper' by correct 'compwrapper' and 'compWrapper'
nipkow [Wed, 09 Apr 1997 15:26:32 +0200] rev 2926
Thorough update.
paulson [Wed, 09 Apr 1997 12:37:44 +0200] rev 2925
Using Blast_tac
paulson [Wed, 09 Apr 1997 12:36:52 +0200] rev 2924
Control over excessive branching by applying a log2 penalty
Incorporation of debugging features
Allows backtracking over haz rules if alternatives exist
Subsitution for equality may more a rule from the haz to the safe part
paulson [Wed, 09 Apr 1997 12:34:28 +0200] rev 2923
Explicit depth bounds seem necessary
paulson [Wed, 09 Apr 1997 12:32:04 +0200] rev 2922
Using Blast_tac
paulson [Wed, 09 Apr 1997 12:31:11 +0200] rev 2921
Dependency on Provers/nat_transitive
nipkow [Tue, 08 Apr 1997 12:03:59 +0200] rev 2920
Couldn't solve n < n+1 because of missing -1
nipkow [Tue, 08 Apr 1997 10:48:42 +0200] rev 2919
Dep. on Provers/nat_transitive
wenzelm [Mon, 07 Apr 1997 14:53:08 +0200] rev 2918
added -t (run tests) option;
wenzelm [Fri, 04 Apr 1997 19:11:19 +0200] rev 2917
added -g, -h options;
replaced ISABELLE_HTML by ISABELLE_USEDIR_OPTIONS;
wenzelm [Fri, 04 Apr 1997 19:10:22 +0200] rev 2916
tuned xdvi invocation;
wenzelm [Fri, 04 Apr 1997 19:09:21 +0200] rev 2915
replaced ISABELLE_HTML by ISABELLE_USEDIR_OPTIONS;
wenzelm [Fri, 04 Apr 1997 19:08:35 +0200] rev 2914
improved messages;
wenzelm [Fri, 04 Apr 1997 19:07:54 +0200] rev 2913
fixed diagnostic output of print modes;
nipkow [Fri, 04 Apr 1997 16:33:28 +0200] rev 2912
moved inj and surj from Set to Fun and Inv -> inv.
nipkow [Fri, 04 Apr 1997 16:27:39 +0200] rev 2911
Inv -> inv
slotosch [Fri, 04 Apr 1997 16:16:35 +0200] rev 2910
*** empty log message ***
slotosch [Fri, 04 Apr 1997 16:04:28 +0200] rev 2909
Added Example Quot
CVS ----------------------------------------------------------------------
slotosch [Fri, 04 Apr 1997 16:03:48 +0200] rev 2908
Start Example
nipkow [Fri, 04 Apr 1997 16:03:44 +0200] rev 2907
inv -> inverse
slotosch [Fri, 04 Apr 1997 16:03:11 +0200] rev 2906
Example for higher order quotients: Fractionals
slotosch [Fri, 04 Apr 1997 16:02:12 +0200] rev 2905
(higher-order) quotient constructor quot, based on PER
slotosch [Fri, 04 Apr 1997 16:01:14 +0200] rev 2904
(partial) equivalecne relations. classes er<per
nipkow [Fri, 04 Apr 1997 14:48:40 +0200] rev 2903
Inv -> inv
wenzelm [Fri, 04 Apr 1997 14:47:26 +0200] rev 2902
added -b option (batch mode);
nipkow [Fri, 04 Apr 1997 14:05:12 +0200] rev 2901
renamed variable 'inv'
wenzelm [Fri, 04 Apr 1997 14:01:18 +0200] rev 2900
added Quot examples;
wenzelm [Fri, 04 Apr 1997 13:57:40 +0200] rev 2899
*** empty log message ***
wenzelm [Fri, 04 Apr 1997 13:56:11 +0200] rev 2898
Higher-order quotients.
paulson [Fri, 04 Apr 1997 12:21:28 +0200] rev 2897
Now calls blast_tac
paulson [Fri, 04 Apr 1997 11:33:51 +0200] rev 2896
Another blast_tac call
paulson [Fri, 04 Apr 1997 11:32:44 +0200] rev 2895
Simplified a proof
paulson [Fri, 04 Apr 1997 11:28:28 +0200] rev 2894
Re-organization of the order of haz rules
paulson [Fri, 04 Apr 1997 11:27:02 +0200] rev 2893
Calls Blast_tac. Tidied some proofs
paulson [Fri, 04 Apr 1997 11:20:31 +0200] rev 2892
Calls Blast_tac. Tidied some proofs
paulson [Fri, 04 Apr 1997 11:18:52 +0200] rev 2891
Calls Blast_tac
paulson [Fri, 04 Apr 1997 11:18:19 +0200] rev 2890
Adds image_eqI instead of imageI, as the former is more general
paulson [Fri, 04 Apr 1997 11:17:05 +0200] rev 2889
Added blast.ML as a dependency
paulson [Fri, 04 Apr 1997 11:16:44 +0200] rev 2888
Now calls Blast_tac and has some hard examples (Halting Problem
nipkow [Thu, 03 Apr 1997 19:32:03 +0200] rev 2887
Only layout mods.
nipkow [Thu, 03 Apr 1997 19:29:53 +0200] rev 2886
Now: unit = {True}
paulson [Thu, 03 Apr 1997 10:36:54 +0200] rev 2885
Two extra commands shorten the proof time by 800 seconds...
paulson [Thu, 03 Apr 1997 10:33:33 +0200] rev 2884
More List and ListPair utilities
paulson [Thu, 03 Apr 1997 10:32:34 +0200] rev 2883
Now exports declConsts!
Temporarily erased target signature to aid debugging
paulson [Thu, 03 Apr 1997 10:30:23 +0200] rev 2882
Declares overloading for if-and-only-if
paulson [Thu, 03 Apr 1997 10:29:57 +0200] rev 2881
Declares overloading for set-theoretic constants
nipkow [Thu, 03 Apr 1997 09:46:42 +0200] rev 2880
Removed (Unit) in Prod.
Added test for ancestor Nat in datatype.
wenzelm [Wed, 02 Apr 1997 19:12:26 +0200] rev 2879
misc improvements;
wenzelm [Wed, 02 Apr 1997 17:28:27 +0200] rev 2878
changed signature of dummy goal from proto_pure to pure;
paulson [Wed, 02 Apr 1997 15:39:44 +0200] rev 2877
Converted to call blast_tac.
Proves theorems in ZF.thy to make that theory usable again
paulson [Wed, 02 Apr 1997 15:37:35 +0200] rev 2876
Uses ZF.thy again, to make that theory usable
paulson [Wed, 02 Apr 1997 15:36:32 +0200] rev 2875
Mostly converted to blast_tac
paulson [Wed, 02 Apr 1997 15:30:44 +0200] rev 2874
Datatype declarations now require theory Datatype--NOT in quotes
paulson [Wed, 02 Apr 1997 15:29:48 +0200] rev 2873
Converted back from upair.thy to ZF.thy
paulson [Wed, 02 Apr 1997 15:28:42 +0200] rev 2872
Moved definitions (binary intersection, etc.) from upair.thy back to ZF.thy
paulson [Wed, 02 Apr 1997 15:26:52 +0200] rev 2871
Now checks for existence of theory Inductive (Fixedpt was too small)
paulson [Wed, 02 Apr 1997 15:25:35 +0200] rev 2870
Now a non-trivial theory so that require_thy can find it
paulson [Wed, 02 Apr 1997 15:24:42 +0200] rev 2869
DEEPEN now takes an upper bound for terminating searches
paulson [Wed, 02 Apr 1997 15:23:33 +0200] rev 2868
New DEEPEN allows giving an upper bound for deepen_tac
paulson [Wed, 02 Apr 1997 15:19:40 +0200] rev 2867
Now builds blast_tac
paulson [Wed, 02 Apr 1997 15:18:21 +0200] rev 2866
Now loads blast.ML
paulson [Wed, 02 Apr 1997 15:14:37 +0200] rev 2865
ZF.thy is again usable
wenzelm [Wed, 02 Apr 1997 11:59:02 +0200] rev 2864
The isabelle-0 encoding table.
paulson [Wed, 02 Apr 1997 11:33:14 +0200] rev 2863
Made the error message more explicit
paulson [Wed, 02 Apr 1997 11:32:48 +0200] rev 2862
Now declares Basis Library version of type option
Also function mapPartial
paulson [Wed, 02 Apr 1997 11:30:48 +0200] rev 2861
Replaced Best_tac by the one rule needed for the proof
paulson [Wed, 02 Apr 1997 11:30:03 +0200] rev 2860
Installation of blast_tac
paulson [Wed, 02 Apr 1997 11:27:47 +0200] rev 2859
Now tests for essential ancestors (Lfp or Gfp)
paulson [Wed, 02 Apr 1997 11:25:04 +0200] rev 2858
Re-ordering of rules to assist blast_tac
Powerset rules must not be the most recent
paulson [Wed, 02 Apr 1997 11:23:31 +0200] rev 2857
Now loads blast_tac
paulson [Wed, 02 Apr 1997 11:19:46 +0200] rev 2856
Reorganization of how classical rules are installed
paulson [Wed, 02 Apr 1997 11:16:40 +0200] rev 2855
Now calls require_thy to ensure ancestors are present
paulson [Wed, 02 Apr 1997 11:15:46 +0200] rev 2854
Implementation of blast_tac: fast tableau prover
wenzelm [Tue, 01 Apr 1997 18:26:09 +0200] rev 2853
replaced by usedir;
wenzelm [Tue, 01 Apr 1997 12:54:40 +0200] rev 2852
eliminated references to old 8bit fonts;
wenzelm [Tue, 01 Apr 1997 12:44:12 +0200] rev 2851
improved messages;
wenzelm [Tue, 01 Apr 1997 11:16:06 +0200] rev 2850
removed useless symbol font syntax;
wenzelm [Tue, 01 Apr 1997 09:28:56 +0200] rev 2849
fixed -s option;
wenzelm [Mon, 31 Mar 1997 14:42:13 +0200] rev 2848
simple_ast_of: fixed handling of loose Bounds;
nipkow [Sun, 30 Mar 1997 13:40:38 +0200] rev 2847
Replaced (s,t) : id by s=t.
nipkow [Thu, 27 Mar 1997 17:46:24 +0100] rev 2846
Optimized proofs.
paulson [Thu, 27 Mar 1997 10:08:31 +0100] rev 2845
Changes made necessary by the new ex1 rules
paulson [Thu, 27 Mar 1997 10:07:11 +0100] rev 2844
Now uses the alternative (safe!) rules for ex1
paulson [Thu, 27 Mar 1997 10:06:36 +0100] rev 2843
Updated comment
nipkow [Wed, 26 Mar 1997 18:51:57 +0100] rev 2842
Cleaned up a little.
nipkow [Wed, 26 Mar 1997 17:58:48 +0100] rev 2841
Added "discrete" CPOs and modified IMP to use those rather than "lift"
slotosch [Wed, 26 Mar 1997 13:44:05 +0100] rev 2840
generalized theorems and class instances for Cprod.
Now "*"::(cpo,cpo)cpo and "*"::(pcpo,pcpo)pcpo
slotosch [Tue, 25 Mar 1997 11:19:09 +0100] rev 2839
changed some theorems from pcpo to cpo
slotosch [Tue, 25 Mar 1997 11:13:12 +0100] rev 2838
changed continuous functions from pcpo to cpo (including instances)
paulson [Tue, 25 Mar 1997 10:43:01 +0100] rev 2837
Trivial renamings (for consistency with CSFW papers)
paulson [Tue, 25 Mar 1997 10:41:44 +0100] rev 2836
Toby's better treatment of eta-contraction
paulson [Mon, 24 Mar 1997 10:28:23 +0100] rev 2835
Deleted needless parentheses
paulson [Mon, 24 Mar 1997 10:27:28 +0100] rev 2834
Deleted unnecessary rules
wenzelm [Thu, 20 Mar 1997 19:12:20 +0100] rev 2833
fixed font names;