wenzelm [Thu, 03 Aug 2006 15:03:10 +0200] rev 20323
removed OldGoals.legacy flag (always warn);
added warning for legacy ML scripts;
wenzelm [Thu, 03 Aug 2006 15:03:09 +0200] rev 20322
removed OldGoals.legacy flag (always warn);
wenzelm [Thu, 03 Aug 2006 15:03:08 +0200] rev 20321
tuned;
wenzelm [Thu, 03 Aug 2006 15:03:07 +0200] rev 20320
removed True_implies (cf. True_implies_equals);
wenzelm [Thu, 03 Aug 2006 15:03:05 +0200] rev 20319
Generic reflection and reification (by Amine Chaieb).
ballarin [Thu, 03 Aug 2006 14:57:26 +0200] rev 20318
Restructured algebra library, added ideals and quotient rings.
ballarin [Thu, 03 Aug 2006 14:53:57 +0200] rev 20317
Updated comments.
wenzelm [Thu, 03 Aug 2006 14:53:35 +0200] rev 20316
updated;
wenzelm [Wed, 02 Aug 2006 23:09:49 +0200] rev 20315
tuned proofs;
wenzelm [Wed, 02 Aug 2006 22:27:08 +0200] rev 20314
lemma da_good_approx: adapted induction (was exploting lifted obtain result);
wenzelm [Wed, 02 Aug 2006 22:27:07 +0200] rev 20313
renamed Syntax.indexname to Syntax.read_indexname;
added read_int (not Int.fromString, which admits ~ syntax of ML);
wenzelm [Wed, 02 Aug 2006 22:27:06 +0200] rev 20312
tuned;
wenzelm [Wed, 02 Aug 2006 22:27:05 +0200] rev 20311
moved debug option to proof_display.ML (again);
normalized Proof.context/method type aliases;
wenzelm [Wed, 02 Aug 2006 22:27:04 +0200] rev 20310
normalized Proof.context/method type aliases;
simplified Assumption/ProofContext.export;
prems_limit: < 0 means no output;
added debug option (back from proof_display.ML);
wenzelm [Wed, 02 Aug 2006 22:27:03 +0200] rev 20309
simplified Assumption/ProofContext.export;
simplified end_block;
wenzelm [Wed, 02 Aug 2006 22:27:02 +0200] rev 20308
added tactical result;
simplified obtain_export: no Seq.seq, no lifting of result prems;
tuned;
wenzelm [Wed, 02 Aug 2006 22:27:01 +0200] rev 20307
removed obsolete Drule.frees/vars_of etc.;
simplified Assumption/ProofContext.export;
wenzelm [Wed, 02 Aug 2006 22:27:00 +0200] rev 20306
normalized Proof.context/method type aliases;
simplified Assumption/ProofContext.export;
wenzelm [Wed, 02 Aug 2006 22:26:59 +0200] rev 20305
simplified Proof.end_block;
wenzelm [Wed, 02 Aug 2006 22:26:58 +0200] rev 20304
removed obsolete Drule.frees/vars_of etc.;
tuned;
wenzelm [Wed, 02 Aug 2006 22:26:57 +0200] rev 20303
normalized Proof.context/method type aliases;
added declare/export/import_prf;
added focus_subgoal: reset/declare goal schematics;
wenzelm [Wed, 02 Aug 2006 22:26:56 +0200] rev 20302
renamed Syntax.indexname to Syntax.read_indexname;
wenzelm [Wed, 02 Aug 2006 22:26:55 +0200] rev 20301
Variable.focus_subgoal;
wenzelm [Wed, 02 Aug 2006 22:26:54 +0200] rev 20300
replaced maxidx_of_proof by maxidx_proof;
wenzelm [Wed, 02 Aug 2006 22:26:53 +0200] rev 20299
prems-limit: int_option;
wenzelm [Wed, 02 Aug 2006 22:26:52 +0200] rev 20298
removed obsolete frees/vars_of etc.;
removed obsolete freeze_all etc.;
added norm_hhf_cterm;
tuned fold_terms;
renamed Syntax.indexname to Syntax.read_indexname;
wenzelm [Wed, 02 Aug 2006 22:26:51 +0200] rev 20297
fake predeclaration of type Proof.context;
wenzelm [Wed, 02 Aug 2006 22:26:50 +0200] rev 20296
simplified export: no Seq.seq;
normalized Proof.context/method type aliases;
wenzelm [Wed, 02 Aug 2006 22:26:49 +0200] rev 20295
use proper RecdefPackage.get_hints;
tuned;
wenzelm [Wed, 02 Aug 2006 22:26:48 +0200] rev 20294
removed obsolete Drule.frees/vars_of;
renamed thm_vars to thm_varnames;